From 2a63a519aeeb2e2a368bdf098e6f9a76a5641bb5 Mon Sep 17 00:00:00 2001 From: Kim Morrison Date: Tue, 22 Oct 2024 10:28:05 +1100 Subject: [PATCH 1/3] chore: use Array.modify instead of modifyOp --- src/Lean/Elab/StructInst.lean | 2 +- tests/lean/run/structInst4.lean | 2 +- 2 files changed, 2 insertions(+), 2 deletions(-) diff --git a/src/Lean/Elab/StructInst.lean b/src/Lean/Elab/StructInst.lean index ca64cd377749..b0e484e8806c 100644 --- a/src/Lean/Elab/StructInst.lean +++ b/src/Lean/Elab/StructInst.lean @@ -184,7 +184,7 @@ private def elabModifyOp (stx modifyOp : Syntax) (sources : Array ExplicitSource let lval := modifyOp[0][0] let idx := lval[1] let self := sources[0]!.stx - let stxNew ← `($(self).modifyOp (idx := $idx) (fun s => $val)) + let stxNew ← `($(self).modify (i := $idx) (fun s => $val)) trace[Elab.struct.modifyOp] "{stx}\n===>\n{stxNew}" withMacroExpansion stx stxNew <| elabTerm stxNew expectedType? let rest := modifyOp[0][1] diff --git a/tests/lean/run/structInst4.lean b/tests/lean/run/structInst4.lean index cde1f3d5e319..38306fb841c6 100644 --- a/tests/lean/run/structInst4.lean +++ b/tests/lean/run/structInst4.lean @@ -7,7 +7,7 @@ structure Foo := (x : Array ((Nat × Nat) × Bool) := #[]) (y : Nat := 0) -#check (b).modifyOp (idx := 1) (fun s => 2) +#check (b).modify (i := 1) (fun s => 2) #check { b with [1] := 2 } From 538b7f2af93cb93cd507f5e5b72ea1efed8ce623 Mon Sep 17 00:00:00 2001 From: Kim Morrison Date: Tue, 22 Oct 2024 10:34:20 +1100 Subject: [PATCH 2/3] chore: update stage0 --- stage0/src/kernel/declaration.cpp | 13 +- stage0/src/kernel/declaration.h | 2 +- stage0/src/kernel/expr.cpp | 17 +- stage0/src/kernel/expr.h | 34 +- stage0/src/kernel/inductive.h | 4 +- stage0/stdlib/Init.c | 6 +- stage0/stdlib/Init/Data/Array.c | 6 +- stage0/stdlib/Init/Data/Array/Basic.c | 803 +- stage0/stdlib/Init/Data/Array/DecidableEq.c | 10 +- stage0/stdlib/Init/Data/Array/GetLit.c | 100 +- stage0/stdlib/Init/Data/Array/Lemmas.c | 101 +- stage0/stdlib/Init/Data/Array/MapIdx.c | 90 + stage0/stdlib/Init/Data/Hashable.c | 21 + stage0/stdlib/Init/Data/List/Basic.c | 53 +- stage0/stdlib/Init/Data/List/Impl.c | 34 +- stage0/stdlib/Init/Data/List/Nat.c | 6 +- stage0/stdlib/Init/Data/List/Nat/BEq.c | 94 + stage0/stdlib/Init/Data/Prod.c | 34 + stage0/stdlib/Init/Data/String/Basic.c | 22 +- stage0/stdlib/Init/Data/Sum.c | 265 +- stage0/stdlib/Init/Data/Sum/Basic.c | 676 + stage0/stdlib/Init/Data/Sum/Lemmas.c | 103 + stage0/stdlib/Init/Data/UInt/Lemmas.c | 680 +- stage0/stdlib/Init/NotationExtra.c | 1939 +- stage0/stdlib/Init/Tactics.c | 107 +- stage0/stdlib/Init/While.c | 1980 ++ stage0/stdlib/Lake/Build/Common.c | 4 +- stage0/stdlib/Lake/Build/Facets.c | 218 +- stage0/stdlib/Lake/Build/Index.c | 10 +- stage0/stdlib/Lake/Build/Key.c | 216 +- stage0/stdlib/Lake/CLI/Init.c | 300 +- stage0/stdlib/Lake/CLI/Main.c | 8 +- stage0/stdlib/Lake/Config/Opaque.c | 16 +- stage0/stdlib/Lake/Config/TargetConfig.c | 62 +- stage0/stdlib/Lake/Load/Lean/Elab.c | 4 +- stage0/stdlib/Lake/Util/Log.c | 4 +- stage0/stdlib/Lean.c | 6 +- stage0/stdlib/Lean/Compiler/IR/Basic.c | 2 +- .../Lean/Compiler/IR/ElimDeadBranches.c | 16 +- stage0/stdlib/Lean/Compiler/IR/PushProj.c | 66 +- .../Lean/Compiler/LCNF/ElimDeadBranches.c | 14 +- stage0/stdlib/Lean/Data/Lsp/Basic.c | 86 +- stage0/stdlib/Lean/Data/Lsp/Capabilities.c | 22 +- stage0/stdlib/Lean/Data/Lsp/Client.c | 8 +- stage0/stdlib/Lean/Data/Lsp/CodeActions.c | 20 +- stage0/stdlib/Lean/Data/Lsp/Diagnostics.c | 10 +- stage0/stdlib/Lean/Data/Lsp/Extra.c | 38 +- stage0/stdlib/Lean/Data/Lsp/InitShutdown.c | 20 +- stage0/stdlib/Lean/Data/Lsp/Internal.c | 14 +- .../stdlib/Lean/Data/Lsp/LanguageFeatures.c | 72 +- stage0/stdlib/Lean/Data/Lsp/TextSync.c | 18 +- stage0/stdlib/Lean/Data/Lsp/Window.c | 22 +- stage0/stdlib/Lean/Data/Lsp/Workspace.c | 26 +- stage0/stdlib/Lean/Data/Position.c | 6 +- stage0/stdlib/Lean/Data/Trie.c | 6 +- stage0/stdlib/Lean/Declaration.c | 62 +- stage0/stdlib/Lean/Elab/BuiltinCommand.c | 2065 +- stage0/stdlib/Lean/Elab/BuiltinEvalCommand.c | 28 +- stage0/stdlib/Lean/Elab/BuiltinNotation.c | 1097 +- stage0/stdlib/Lean/Elab/Command.c | 1737 +- stage0/stdlib/Lean/Elab/ComputedFields.c | 226 +- stage0/stdlib/Lean/Elab/DeclModifiers.c | 669 +- stage0/stdlib/Lean/Elab/Declaration.c | 3174 +-- stage0/stdlib/Lean/Elab/DeclarationRange.c | 520 +- stage0/stdlib/Lean/Elab/DefView.c | 28 +- stage0/stdlib/Lean/Elab/Deriving/FromToJson.c | 252 +- stage0/stdlib/Lean/Elab/Frontend.c | 906 +- stage0/stdlib/Lean/Elab/Inductive.c | 48 +- stage0/stdlib/Lean/Elab/LetRec.c | 556 +- stage0/stdlib/Lean/Elab/MutualDef.c | 3598 ++-- stage0/stdlib/Lean/Elab/ParseImportsFast.c | 8 +- stage0/stdlib/Lean/Elab/PreDefinition/Basic.c | 70 +- stage0/stdlib/Lean/Elab/PreDefinition/Main.c | 6 +- .../Elab/PreDefinition/Structural/BRecOn.c | 849 +- .../PreDefinition/Structural/FindRecArg.c | 63 +- .../Lean/Elab/PreDefinition/Structural/Main.c | 532 +- .../PreDefinition/Structural/SmartUnfolding.c | 45 +- .../Lean/Elab/PreDefinition/WF/GuessLex.c | 303 +- .../stdlib/Lean/Elab/PreDefinition/WF/Main.c | 4 +- stage0/stdlib/Lean/Elab/Quotation.c | 89 +- stage0/stdlib/Lean/Elab/StructInst.c | 1301 +- stage0/stdlib/Lean/Elab/Structure.c | 1562 +- stage0/stdlib/Lean/Elab/Syntax.c | 12 +- .../Frontend/BVDecide/ReifiedBVExpr.c | 5711 +++--- .../Frontend/BVDecide/ReifiedBVLogical.c | 3419 ++-- .../Frontend/BVDecide/ReifiedBVPred.c | 3185 +-- .../Frontend/BVDecide/SatAtBVLogical.c | 8 +- .../stdlib/Lean/Elab/Tactic/BuiltinTactic.c | 3746 ++-- stage0/stdlib/Lean/Elab/Tactic/Conv/Pattern.c | 32 +- stage0/stdlib/Lean/Elab/Tactic/Ext.c | 2998 ++- stage0/stdlib/Lean/Elab/Tactic/Induction.c | 733 +- stage0/stdlib/Lean/Elab/Tactic/SolveByElim.c | 12 +- stage0/stdlib/Lean/Elab/Term.c | 754 +- stage0/stdlib/Lean/Language/Basic.c | 129 +- stage0/stdlib/Lean/Language/Lean/Types.c | 7 +- stage0/stdlib/Lean/LazyInitExtension.c | 322 - .../Lean/Linter/ConstructorAsVariable.c | 1222 +- stage0/stdlib/Lean/Linter/UnusedVariables.c | 16434 +++++++++------- stage0/stdlib/Lean/Linter/Util.c | 361 +- stage0/stdlib/Lean/Message.c | 14 +- stage0/stdlib/Lean/Meta/FunInfo.c | 12 +- stage0/stdlib/Lean/Meta/IndPredBelow.c | 1287 +- stage0/stdlib/Lean/Meta/InferType.c | 160 +- .../stdlib/Lean/Meta/Match/CaseArraySizes.c | 18 +- stage0/stdlib/Lean/Meta/Match/Match.c | 583 +- stage0/stdlib/Lean/Meta/Tactic/AC/Main.c | 4171 ++-- stage0/stdlib/Lean/Meta/Tactic/Backtrack.c | 6 +- stage0/stdlib/Lean/Meta/Tactic/Cases.c | 12 +- stage0/stdlib/Lean/Meta/Tactic/FunInd.c | 626 +- .../Lean/Meta/Tactic/LinearArith/Nat/Simp.c | 3119 +-- stage0/stdlib/Lean/Meta/Tactic/SplitIf.c | 1463 +- stage0/stdlib/Lean/Meta/WHNF.c | 11 +- stage0/stdlib/Lean/Parser/Command.c | 923 +- stage0/stdlib/Lean/Parser/Extra.c | 1145 +- .../Lean/PrettyPrinter/Delaborator/Builtins.c | 3598 +--- stage0/stdlib/Lean/Server/CodeActions/Basic.c | 28 +- stage0/stdlib/Lean/Server/Completion.c | 320 +- .../stdlib/Lean/Server/CompletionItemData.c | 4 +- .../Lean/Server/FileWorker/RequestHandling.c | 4 +- .../Lean/Server/FileWorker/WidgetRequests.c | 14 +- stage0/stdlib/Lean/Server/InfoUtils.c | 1060 +- stage0/stdlib/Lean/Server/References.c | 863 +- stage0/stdlib/Lean/Server/Rpc/Basic.c | 6 +- stage0/stdlib/Lean/Server/Watchdog.c | 4 +- stage0/stdlib/Lean/SubExpr.c | 4 +- stage0/stdlib/Lean/Util/FileSetupInfo.c | 4 +- stage0/stdlib/Lean/Util/Paths.c | 6 +- stage0/stdlib/Lean/Util/Profiler.c | 44 +- stage0/stdlib/Lean/Util/Recognizers.c | 3345 ++++ stage0/stdlib/Lean/Widget/Diff.c | 12 +- stage0/stdlib/Lean/Widget/InteractiveCode.c | 4 +- .../Lean/Widget/InteractiveDiagnostic.c | 4 +- stage0/stdlib/Lean/Widget/InteractiveGoal.c | 10 +- stage0/stdlib/Lean/Widget/Types.c | 4 +- stage0/stdlib/Lean/Widget/UserWidget.c | 14 +- .../stdlib/Std/Data/DHashMap/Internal/Defs.c | 18 +- stage0/stdlib/Std/Sat/AIG.c | 6 +- stage0/stdlib/Std/Sat/AIG/Basic.c | 6 +- stage0/stdlib/Std/Sat/AIG/CNF.c | 6 +- stage0/stdlib/Std/Sat/AIG/Cached.c | 6 +- stage0/stdlib/Std/Sat/AIG/CachedGates.c | 6 +- stage0/stdlib/Std/Sat/AIG/CachedGatesLemmas.c | 6 +- stage0/stdlib/Std/Sat/AIG/CachedLemmas.c | 6 +- stage0/stdlib/Std/Sat/AIG/If.c | 6 +- stage0/stdlib/Std/Sat/AIG/LawfulOperator.c | 6 +- stage0/stdlib/Std/Sat/AIG/LawfulVecOperator.c | 6 +- stage0/stdlib/Std/Sat/AIG/Lemmas.c | 6 +- stage0/stdlib/Std/Sat/AIG/RefVec.c | 6 +- stage0/stdlib/Std/Sat/AIG/RefVecOperator.c | 6 +- .../stdlib/Std/Sat/AIG/RefVecOperator/Fold.c | 6 +- .../stdlib/Std/Sat/AIG/RefVecOperator/Map.c | 6 +- .../stdlib/Std/Sat/AIG/RefVecOperator/Zip.c | 6 +- stage0/stdlib/Std/Sat/AIG/Relabel.c | 6 +- stage0/stdlib/Std/Sat/AIG/RelabelNat.c | 6 +- .../Bitblast/BVExpr/Circuit/Impl/Expr.c | 6 +- .../Tactic/BVDecide/LRAT/Internal/Clause.c | 42 - 156 files changed, 49294 insertions(+), 41179 deletions(-) create mode 100644 stage0/stdlib/Init/Data/Array/MapIdx.c create mode 100644 stage0/stdlib/Init/Data/List/Nat/BEq.c create mode 100644 stage0/stdlib/Init/Data/Sum/Basic.c create mode 100644 stage0/stdlib/Init/Data/Sum/Lemmas.c create mode 100644 stage0/stdlib/Init/While.c delete mode 100644 stage0/stdlib/Lean/LazyInitExtension.c diff --git a/stage0/src/kernel/declaration.cpp b/stage0/src/kernel/declaration.cpp index 489a134c1258..492d3942c88b 100644 --- a/stage0/src/kernel/declaration.cpp +++ b/stage0/src/kernel/declaration.cpp @@ -126,7 +126,6 @@ constructor_val::constructor_val(name const & n, names const & lparams, expr con object_ref(lean_mk_constructor_val(n.to_obj_arg(), lparams.to_obj_arg(), type.to_obj_arg(), induct.to_obj_arg(), nat(cidx).to_obj_arg(), nat(nparams).to_obj_arg(), nat(nfields).to_obj_arg(), is_unsafe)) { } - bool constructor_val::is_unsafe() const { return lean_constructor_val_is_unsafe(to_obj_arg()); } extern "C" object * lean_mk_recursor_val(object * n, object * lparams, object * type, object * all, @@ -143,6 +142,18 @@ recursor_val::recursor_val(name const & n, names const & lparams, expr const & t nat(nminors).to_obj_arg(), rules.to_obj_arg(), k, is_unsafe)) { } +name const & recursor_val::get_major_induct() const { + unsigned int n = get_major_idx(); + expr const * t = &(to_constant_val().get_type()); + for (unsigned int i = 0; i < n; i++) { + t = &(binding_body(*t)); + } + t = &(binding_domain(*t)); + t = &(get_app_fn(*t)); + return const_name(*t); +} + + bool recursor_val::is_k() const { return lean_recursor_k(to_obj_arg()); } bool recursor_val::is_unsafe() const { return lean_recursor_is_unsafe(to_obj_arg()); } diff --git a/stage0/src/kernel/declaration.h b/stage0/src/kernel/declaration.h index 9b636ae0a8f6..398d4e1f8967 100644 --- a/stage0/src/kernel/declaration.h +++ b/stage0/src/kernel/declaration.h @@ -370,7 +370,7 @@ class recursor_val : public object_ref { recursor_val & operator=(recursor_val && other) { object_ref::operator=(std::move(other)); return *this; } constant_val const & to_constant_val() const { return static_cast(cnstr_get_ref(*this, 0)); } name const & get_name() const { return to_constant_val().get_name(); } - name const & get_induct() const { return get_name().get_prefix(); } + name const & get_major_induct() const; names const & get_all() const { return static_cast(cnstr_get_ref(*this, 1)); } unsigned get_nparams() const { return static_cast(cnstr_get_ref(*this, 2)).get_small_value(); } unsigned get_nindices() const { return static_cast(cnstr_get_ref(*this, 3)).get_small_value(); } diff --git a/stage0/src/kernel/expr.cpp b/stage0/src/kernel/expr.cpp index 983764623727..957809c2e3aa 100644 --- a/stage0/src/kernel/expr.cpp +++ b/stage0/src/kernel/expr.cpp @@ -79,21 +79,22 @@ extern "C" object * lean_lit_type(obj_arg e); expr lit_type(literal const & lit) { return expr(lean_lit_type(lit.to_obj_arg())); } extern "C" uint64_t lean_expr_hash(obj_arg e); -unsigned hash(expr const & e) { - object * o = e.raw(); - unsigned r = static_cast(lean_ctor_get_uint64(o, lean_ctor_num_objs(o)*sizeof(object*))); - lean_assert(r == lean_expr_hash(e.to_obj_arg())); - return r; +unsigned hash_core(expr const & e) { + return lean_expr_hash(e.to_obj_arg()); } extern "C" uint8 lean_expr_has_fvar(obj_arg e); -bool has_fvar(expr const & e) { return lean_expr_has_fvar(e.to_obj_arg()); } +bool has_fvar_core(expr const & e) { + return lean_expr_has_fvar(e.to_obj_arg()); +} extern "C" uint8 lean_expr_has_expr_mvar(obj_arg e); -bool has_expr_mvar(expr const & e) { return lean_expr_has_expr_mvar(e.to_obj_arg()); } +bool has_expr_mvar_core(expr const & e) { + return lean_expr_has_expr_mvar(e.to_obj_arg()); +} extern "C" uint8 lean_expr_has_level_mvar(obj_arg e); -bool has_univ_mvar(expr const & e) { return lean_expr_has_level_mvar(e.to_obj_arg()); } +bool has_univ_mvar_core(expr const & e) { return lean_expr_has_level_mvar(e.to_obj_arg()); } extern "C" uint8 lean_expr_has_level_param(obj_arg e); bool has_univ_param(expr const & e) { return lean_expr_has_level_param(e.to_obj_arg()); } diff --git a/stage0/src/kernel/expr.h b/stage0/src/kernel/expr.h index d1771e73a366..c110ebd26c32 100644 --- a/stage0/src/kernel/expr.h +++ b/stage0/src/kernel/expr.h @@ -123,11 +123,37 @@ inline bool is_eqp(optional const & a, optional const & b) { return static_cast(a) == static_cast(b) && (!a || is_eqp(*a, *b)); } -unsigned hash(expr const & e); -bool has_expr_mvar(expr const & e); -bool has_univ_mvar(expr const & e); +inline uint64_t get_data(expr const & e) { + return lean_ctor_get_uint64(e.raw(), lean_ctor_num_objs(e.raw())*sizeof(object*)); +} +/* This is the implementation in Lean */ +unsigned hash_core(expr const & e); +inline unsigned hash(expr const & e) { + unsigned r = static_cast(get_data(e)); + lean_assert(r == hash_core(e)); + return r; +} +/* This is the implementation in Lean */ +bool has_expr_mvar_core(expr const & e); +inline bool has_expr_mvar(expr const & e) { + bool r = ((get_data(e) >> 41) & 1) == 1; + lean_assert(r == has_expr_mvar_core(e)); // ensure the C++ implementation matches the Lean one. + return r; +} +bool has_univ_mvar_core(expr const & e); +inline bool has_univ_mvar(expr const & e) { + bool r = ((get_data(e) >> 42) & 1) == 1; + lean_assert(r == has_univ_mvar_core(e)); // ensure the C++ implementation matches the Lean one. + return r; +} inline bool has_mvar(expr const & e) { return has_expr_mvar(e) || has_univ_mvar(e); } -bool has_fvar(expr const & e); +/* This is the implementation in Lean */ +bool has_fvar_core(expr const & e); +inline bool has_fvar(expr const & e) { + bool r = ((get_data(e) >> 40) & 1) == 1; + lean_assert(r == has_fvar_core(e)); // ensure the C++ implementation matches the Lean one. + return r; +} bool has_univ_param(expr const & e); unsigned get_loose_bvar_range(expr const & e); diff --git a/stage0/src/kernel/inductive.h b/stage0/src/kernel/inductive.h index dd6b2671b2bf..a7b2864624ac 100644 --- a/stage0/src/kernel/inductive.h +++ b/stage0/src/kernel/inductive.h @@ -33,7 +33,7 @@ inline expr to_cnstr_when_K(environment const & env, recursor_val const & rval, lean_assert(rval.is_k()); expr app_type = whnf(infer_type(e)); expr const & app_type_I = get_app_fn(app_type); - if (!is_constant(app_type_I) || const_name(app_type_I) != rval.get_induct()) return e; // type incorrect + if (!is_constant(app_type_I) || const_name(app_type_I) != rval.get_major_induct()) return e; // type incorrect if (has_expr_mvar(app_type)) { buffer app_type_args; get_app_args(app_type, app_type_args); @@ -94,7 +94,7 @@ inline optional inductive_reduce_rec(environment const & env, expr const & else if (is_string_lit(major)) major = string_lit_to_constructor(major); else - major = to_cnstr_when_structure(env, rec_val.get_induct(), major, whnf, infer_type); + major = to_cnstr_when_structure(env, rec_val.get_major_induct(), major, whnf, infer_type); optional rule = get_rec_rule_for(rec_val, major); if (!rule) return none_expr(); buffer major_args; diff --git a/stage0/stdlib/Init.c b/stage0/stdlib/Init.c index 09ae651f8920..3b6237764369 100644 --- a/stage0/stdlib/Init.c +++ b/stage0/stdlib/Init.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init -// Imports: Init.Prelude Init.Notation Init.Tactics Init.TacticsExtra Init.ByCases Init.RCases Init.Core Init.Control Init.Data.Basic Init.WF Init.WFTactics Init.Data Init.System Init.Util Init.Dynamic Init.ShareCommon Init.MetaTypes Init.Meta Init.NotationExtra Init.SimpLemmas Init.PropLemmas Init.Hints Init.Conv Init.Guard Init.Simproc Init.SizeOfLemmas Init.BinderPredicates Init.Ext Init.Omega Init.MacroTrace Init.Grind +// Imports: Init.Prelude Init.Notation Init.Tactics Init.TacticsExtra Init.ByCases Init.RCases Init.Core Init.Control Init.Data.Basic Init.WF Init.WFTactics Init.Data Init.System Init.Util Init.Dynamic Init.ShareCommon Init.MetaTypes Init.Meta Init.NotationExtra Init.SimpLemmas Init.PropLemmas Init.Hints Init.Conv Init.Guard Init.Simproc Init.SizeOfLemmas Init.BinderPredicates Init.Ext Init.Omega Init.MacroTrace Init.Grind Init.While #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -44,6 +44,7 @@ lean_object* initialize_Init_Ext(uint8_t builtin, lean_object*); lean_object* initialize_Init_Omega(uint8_t builtin, lean_object*); lean_object* initialize_Init_MacroTrace(uint8_t builtin, lean_object*); lean_object* initialize_Init_Grind(uint8_t builtin, lean_object*); +lean_object* initialize_Init_While(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init(uint8_t builtin, lean_object* w) { lean_object * res; @@ -142,6 +143,9 @@ lean_dec_ref(res); res = initialize_Init_Grind(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_While(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/Data/Array.c b/stage0/stdlib/Init/Data/Array.c index a906ba7df467..2dc8f1febdc8 100644 --- a/stage0/stdlib/Init/Data/Array.c +++ b/stage0/stdlib/Init/Data/Array.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Data.Array -// Imports: Init.Data.Array.Basic Init.Data.Array.QSort Init.Data.Array.BinSearch Init.Data.Array.InsertionSort Init.Data.Array.DecidableEq Init.Data.Array.Mem Init.Data.Array.Attach Init.Data.Array.BasicAux Init.Data.Array.Lemmas Init.Data.Array.TakeDrop Init.Data.Array.Bootstrap Init.Data.Array.GetLit +// Imports: Init.Data.Array.Basic Init.Data.Array.QSort Init.Data.Array.BinSearch Init.Data.Array.InsertionSort Init.Data.Array.DecidableEq Init.Data.Array.Mem Init.Data.Array.Attach Init.Data.Array.BasicAux Init.Data.Array.Lemmas Init.Data.Array.TakeDrop Init.Data.Array.Bootstrap Init.Data.Array.GetLit Init.Data.Array.MapIdx #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -25,6 +25,7 @@ lean_object* initialize_Init_Data_Array_Lemmas(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Array_TakeDrop(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Array_Bootstrap(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Array_GetLit(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_Array_MapIdx(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_Data_Array(uint8_t builtin, lean_object* w) { lean_object * res; @@ -66,6 +67,9 @@ lean_dec_ref(res); res = initialize_Init_Data_Array_GetLit(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_Data_Array_MapIdx(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/Data/Array/Basic.c b/stage0/stdlib/Init/Data/Array/Basic.c index ef545f538a83..b435267eb096 100644 --- a/stage0/stdlib/Init/Data/Array/Basic.c +++ b/stage0/stdlib/Init/Data/Array/Basic.c @@ -18,11 +18,14 @@ LEAN_EXPORT lean_object* l_Array_filterM___rarg(lean_object*, lean_object*, lean LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Array_findRevM_x3f___spec__1___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_concatMapM(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_takeWhile(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, 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__5; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_reduceOption___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Array_isPrefixOf(lean_object*); LEAN_EXPORT lean_object* l_Nat_foldTR_loop___at_Array_range___spec__1___at_Array_range___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_foldl___spec__1___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__15; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_zipWithIndex___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findRev_x3f___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrM_fold___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_instAppend(lean_object*); @@ -38,6 +41,7 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_contains___spec__1(le static lean_object* l_Array_instRepr___rarg___closed__5; static lean_object* l_term_x23_x5b___x2c_x5d___closed__14; LEAN_EXPORT lean_object* l_Array_foldlM_loop___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_data(lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeM_x3f___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_eraseReps___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_insertAt_loop___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -47,8 +51,8 @@ static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_ LEAN_EXPORT lean_object* l_Array_findSome_x21___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_modifyMUnsafe___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatten___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapFinIdx___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_find_x3f___spec__1(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findM_x3f___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, 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_forIn_loop___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -89,6 +93,7 @@ LEAN_EXPORT lean_object* l_Array_allDiff___rarg___boxed(lean_object*, lean_objec lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_toListAppend___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_flatten___rarg___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Array_flatMap___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_filterMap___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -110,6 +115,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findSomeM_x3f___spe LEAN_EXPORT lean_object* l_Array_instGetElemUSizeLtNatToNatSize(lean_object*); LEAN_EXPORT lean_object* l_panic___at_Array_swapAt_x21___spec__1___rarg(lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_reduceOption___spec__2___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_forM___spec__1___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_getIdx_x3f(lean_object*); @@ -122,7 +128,8 @@ LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Array_contains___spec__1___rarg( 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*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_foldr___spec__2___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Nat_foldTR_loop___at_Array_range___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyM_loop___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Array_findRev_x3f___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -131,6 +138,7 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_toListAppend___spe LEAN_EXPORT lean_object* l_Array_unzip(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findSomeM_x3f___spec__1___rarg___lambda__2(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_forIn_loop___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findIdxM_x3f___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findIdxM_x3f___spec__1___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -152,6 +160,7 @@ LEAN_EXPORT lean_object* l_Array_mkArray___boxed(lean_object*, lean_object*, lea LEAN_EXPORT lean_object* l_Array_swapAt(lean_object*); LEAN_EXPORT lean_object* l_Array_zipWithAux(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyM_loop(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_filterMapM___at_Array_reduceOption___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeM_x3f___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_any___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findIdxM_x3f___spec__1(lean_object*, lean_object*); @@ -169,6 +178,7 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec_ static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__18; LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_find_x3f___rarg___closed__2; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_reduceOption___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forRevM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_split___spec__1___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__1; @@ -182,7 +192,6 @@ LEAN_EXPORT lean_object* l_Array_isEqv(lean_object*); LEAN_EXPORT lean_object* l_Array_mapIdx(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_forM___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_unzip___rarg___closed__1; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrM_fold(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_modify(lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_loop___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -196,12 +205,13 @@ LEAN_EXPORT lean_object* l_Array_swapAt_x21___rarg(lean_object*, lean_object*, l LEAN_EXPORT lean_object* l_Array_mapIdx___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_isEmpty(lean_object*); LEAN_EXPORT lean_object* l_Array_mapM_map___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_zipWithIndex___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_singleton(lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeM_x3f___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_flatMap(lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Array_map(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findRev_x3f___rarg___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_concatMapM___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_allM___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*); @@ -213,11 +223,14 @@ LEAN_EXPORT lean_object* l_Array_instToString(lean_object*); LEAN_EXPORT lean_object* l_Array_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_all___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findIdxM_x3f___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_data___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Array_findSomeRev_x3f___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findIdxM_x3f___spec__1___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_any(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Array_map___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_Format_joinSep___at_Array_instRepr___spec__1___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__2(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_findSome_x3f___rarg(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_elem___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlM_loop___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -247,7 +260,6 @@ LEAN_EXPORT lean_object* l_Array_ofFn___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_allM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyM_loop___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_mapIdx___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Array_findSomeRev_x3f___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_indexOf_x3f___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findIdxM_x3f___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -267,18 +279,21 @@ LEAN_EXPORT lean_object* l_Array_indexOfAux(lean_object*); LEAN_EXPORT lean_object* l_Array_insertAt_x21(lean_object*); static lean_object* l_Array_instGetElemUSizeLtNatToNatSize___closed__1; LEAN_EXPORT lean_object* l_Array_back_x3f___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdx___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_partition___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSome_x21___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapFinIdx___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findIdxM_x3f___spec__1___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filterM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Array_findRevM_x3f___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_back_x3f___rarg___boxed(lean_object*); lean_object* lean_array_pop(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__2(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__19; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_allM___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_findSome_x21___rarg___closed__3; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMap___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMap___spec__1___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Nat_foldTR_loop___at_Array_range___spec__1___at_Array_range___spec__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_ofFn_go(lean_object*); @@ -326,17 +341,18 @@ LEAN_EXPORT lean_object* l_Array_filterMapM___rarg___boxed(lean_object*, lean_ob LEAN_EXPORT lean_object* l_Array_zipWith___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_foldr___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_toListAppend___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdx(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_mapIdx___spec__1(lean_object*, 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_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*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg___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_zipWithAux___at_Array_zip___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_findIdxM_x3f___rarg___closed__1; static lean_object* l_term_x23_x5b___x2c_x5d___closed__1; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findRevM_x3f___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_toListAppend___spec__2___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_filter(lean_object*); @@ -360,6 +376,7 @@ LEAN_EXPORT lean_object* l_Array_reverse_loop(lean_object*); static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__11; LEAN_EXPORT lean_object* l_Array_foldl___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_allM___spec__2___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_zipWithIndex___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_filterM___spec__1___rarg___lambda__2(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_insertAt(lean_object*); LEAN_EXPORT lean_object* l_Array_eraseIdx___rarg(lean_object*, lean_object*); @@ -372,7 +389,6 @@ LEAN_EXPORT lean_object* l_Array_get_x3f(lean_object*); LEAN_EXPORT lean_object* l_Array_insertAt_loop(lean_object*); 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*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_zipWithIndex___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_instInhabited(lean_object*); LEAN_EXPORT lean_object* l_Array_getEvenElems___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -387,10 +403,10 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___rarg___lambda__1(size_t, lean_ static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__10; LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_pop___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdx___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Array_instRepr___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Array_erase(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_reduceOption___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_getEvenElems___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -399,6 +415,7 @@ static lean_object* l_term_x23_x5b___x2c_x5d___closed__16; static lean_object* l_term_x23_x5b___x2c_x5d___closed__2; static lean_object* l_term_x23_x5b___x2c_x5d___closed__13; 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_forInUnsafe_loop___at_Array_findM_x3f___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, 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; @@ -417,6 +434,7 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_foldr___spec__1(le LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, 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_forM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdx___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filterMapM___at_Array_filterMap___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_any___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -425,6 +443,7 @@ LEAN_EXPORT lean_object* l_Array_filter___rarg___boxed(lean_object*, lean_object LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold(lean_object*, lean_object*, lean_object*); lean_object* l_Array_appendCore___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filterMap___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapFinIdx___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_allM___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__8; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findM_x3f___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -450,6 +469,8 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findIdxM_x3f___spec 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*); static lean_object* l_Array_instAppend___closed__1; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findSome_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlM_loop___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Array_findRevM_x3f___spec__1___rarg___lambda__1(lean_object*, lean_object*, uint8_t); @@ -464,6 +485,7 @@ LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Array_findRevM_x3f__ LEAN_EXPORT lean_object* l_Array_instRepr___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Array_map___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_shrink___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMap___spec__1___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_filterM___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_takeWhile_go___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_instForIn(lean_object*, lean_object*, lean_object*); @@ -498,9 +520,10 @@ LEAN_EXPORT lean_object* l_Array_insertAt_x21___rarg(lean_object*, lean_object*, static lean_object* l_Array_instRepr___rarg___closed__6; LEAN_EXPORT lean_object* l_Array_toListAppend(lean_object*); LEAN_EXPORT lean_object* l_Array_shrink_loop(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_foldr___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_isPrefixOfAux___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_flatMapM___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__17; LEAN_EXPORT lean_object* l_Array_getEvenElems___rarg(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_allDiffAuxAux(lean_object*); @@ -539,13 +562,18 @@ LEAN_EXPORT lean_object* l_Array_map___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_isPrefixOfAux(lean_object*); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_any___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_flatMap___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Array_instRepr___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_instRepr___rarg___closed__7; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_split___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMap___spec__1___rarg___boxed(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_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; 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*); @@ -556,13 +584,16 @@ LEAN_EXPORT lean_object* l_Array_swapAt___rarg___boxed(lean_object*, lean_object LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_toListImpl___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Array_findRev_x3f___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_all___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_all___spec__1___rarg___boxed(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__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_insertAt___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_zipWithIndex___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop(lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_shrink___rarg___boxed(lean_object*, lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__3; LEAN_EXPORT lean_object* l_Array_indexOfAux___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -584,8 +615,9 @@ LEAN_EXPORT lean_object* l_Array_instRepr(lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__9; LEAN_EXPORT lean_object* l_Array_findIdx_x3f___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_swap___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_zipWithIndex___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdx___spec__1(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_forIn_loop(lean_object*, lean_object*, 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_allM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -606,14 +638,18 @@ lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__8; lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Array_any___spec__1___rarg(lean_object*, lean_object*, size_t, size_t); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_mapIdx___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_allM(lean_object*, lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__18; LEAN_EXPORT lean_object* l_Array_findSomeM_x3f___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdx___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapIdx___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_popWhile___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_filterM___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_term_x23_x5b___x2c_x5d; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_reduceOption(lean_object*); +LEAN_EXPORT lean_object* l_Array_filterMapM___at_Array_reduceOption___spec__1___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forRevM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_allM___spec__1___rarg___lambda__1(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_anyMUnsafe(lean_object*, lean_object*); @@ -634,6 +670,7 @@ LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___rarg(lean_object*, lean 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*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_find_x3f(lean_object*); LEAN_EXPORT lean_object* l_Array_get_x3f___rarg(lean_object*, lean_object*); static lean_object* _init_l_term_x23_x5b___x2c_x5d___closed__1() { @@ -1095,6 +1132,22 @@ return x_34; } } } +LEAN_EXPORT lean_object* l_Array_data___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_array_to_list(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_data(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_data___rarg), 1, 0); +return x_2; +} +} LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__List_toArrayAux_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { @@ -1791,7 +1844,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(220u); +x_13 = lean_unsigned_to_nat(242u); 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); @@ -2924,18 +2977,18 @@ lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___rarg___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_Array_mapFinIdxM_map___rarg___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; lean_object* x_10; lean_object* x_11; x_8 = lean_unsigned_to_nat(1u); x_9 = lean_nat_add(x_1, x_8); x_10 = lean_array_push(x_2, x_7); -x_11 = l_Array_mapIdxM_map___rarg(x_3, x_4, x_5, x_6, x_9, lean_box(0), x_10); +x_11 = l_Array_mapFinIdxM_map___rarg(x_3, x_4, x_5, x_6, x_9, lean_box(0), x_10); return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___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_EXPORT lean_object* l_Array_mapFinIdxM_map___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: { lean_object* x_8; uint8_t x_9; @@ -2952,7 +3005,7 @@ x_13 = lean_array_fget(x_2, x_5); lean_inc(x_3); lean_inc(x_5); x_14 = lean_apply_2(x_3, x_5, x_13); -x_15 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___rarg___lambda__1___boxed), 7, 6); +x_15 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___rarg___lambda__1___boxed), 7, 6); lean_closure_set(x_15, 0, x_5); lean_closure_set(x_15, 1, x_7); lean_closure_set(x_15, 2, x_1); @@ -2979,33 +3032,118 @@ return x_19; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___rarg___boxed), 7, 0); +x_4 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___rarg___boxed), 7, 0); return x_4; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___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_EXPORT lean_object* l_Array_mapFinIdxM_map___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) { _start: { lean_object* x_8; -x_8 = l_Array_mapIdxM_map___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Array_mapFinIdxM_map___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___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_mapFinIdxM_map___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: { lean_object* x_8; -x_8 = l_Array_mapIdxM_map___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Array_mapFinIdxM_map___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_4); return x_8; } } +LEAN_EXPORT lean_object* l_Array_mapFinIdxM___rarg(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; +x_4 = lean_array_get_size(x_2); +x_5 = lean_mk_empty_array_with_capacity(x_4); +x_6 = lean_unsigned_to_nat(0u); +x_7 = l_Array_mapFinIdxM_map___rarg(x_1, x_2, x_3, x_4, x_6, lean_box(0), x_5); +lean_dec(x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_alloc_closure((void*)(l_Array_mapFinIdxM___rarg), 3, 0); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg___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; lean_object* x_11; lean_object* x_12; +x_9 = lean_unsigned_to_nat(1u); +x_10 = lean_nat_add(x_1, x_9); +x_11 = lean_array_push(x_2, x_8); +x_12 = l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg(x_3, x_4, x_5, x_6, x_7, x_10, lean_box(0), x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___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, lean_object* x_8) { +_start: +{ +lean_object* x_9; uint8_t x_10; +x_9 = lean_unsigned_to_nat(0u); +x_10 = lean_nat_dec_eq(x_5, 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; lean_object* x_17; +x_11 = lean_unsigned_to_nat(1u); +x_12 = lean_nat_sub(x_5, x_11); +x_13 = lean_ctor_get(x_1, 1); +lean_inc(x_13); +x_14 = lean_array_fget(x_4, x_6); +lean_inc(x_3); +lean_inc(x_6); +x_15 = lean_apply_2(x_3, x_6, x_14); +x_16 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg___lambda__1___boxed), 8, 7); +lean_closure_set(x_16, 0, x_6); +lean_closure_set(x_16, 1, x_8); +lean_closure_set(x_16, 2, x_1); +lean_closure_set(x_16, 3, x_2); +lean_closure_set(x_16, 4, x_3); +lean_closure_set(x_16, 5, x_4); +lean_closure_set(x_16, 6, x_12); +x_17 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_15, x_16); +return x_17; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_18 = lean_ctor_get(x_1, 0); +lean_inc(x_18); +lean_dec(x_1); +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +lean_dec(x_18); +x_20 = lean_apply_2(x_19, lean_box(0), x_8); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg___boxed), 8, 0); +return x_4; +} +} LEAN_EXPORT lean_object* l_Array_mapIdxM___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -3013,7 +3151,8 @@ lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_4 = lean_array_get_size(x_2); x_5 = lean_mk_empty_array_with_capacity(x_4); x_6 = lean_unsigned_to_nat(0u); -x_7 = l_Array_mapIdxM_map___rarg(x_1, x_2, x_3, x_4, x_6, lean_box(0), x_5); +lean_inc(x_2); +x_7 = l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg(x_1, x_2, x_3, x_2, x_4, x_6, lean_box(0), x_5); lean_dec(x_4); return x_7; } @@ -3026,6 +3165,25 @@ x_4 = lean_alloc_closure((void*)(l_Array_mapIdxM___rarg), 3, 0); return x_4; } } +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___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: +{ +lean_object* x_9; +x_9 = l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg___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_1); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___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) { +_start: +{ +lean_object* x_9; +x_9 = l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_5); +return x_9; +} +} LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Array_findSomeM_x3f___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -5532,7 +5690,87 @@ x_7 = l_Array_mapMUnsafe_map___at_Array_map___spec__1___rarg(x_1, x_5, x_6, x_4) return x_7; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_mapIdx___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) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapFinIdx___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) { +_start: +{ +lean_object* x_8; uint8_t x_9; +x_8 = lean_unsigned_to_nat(0u); +x_9 = lean_nat_dec_eq(x_4, x_8); +if (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; +x_10 = lean_unsigned_to_nat(1u); +x_11 = lean_nat_sub(x_4, x_10); +lean_dec(x_4); +x_12 = lean_array_fget(x_3, x_5); +lean_inc(x_2); +lean_inc(x_5); +x_13 = lean_apply_2(x_2, x_5, x_12); +x_14 = lean_nat_add(x_5, x_10); +lean_dec(x_5); +x_15 = lean_array_push(x_7, x_13); +x_4 = x_11; +x_5 = x_14; +x_6 = lean_box(0); +x_7 = x_15; +goto _start; +} +else +{ +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapFinIdx___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Array_mapFinIdx___spec__1___rarg___boxed), 7, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdx___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; +x_3 = lean_array_get_size(x_1); +x_4 = lean_mk_empty_array_with_capacity(x_3); +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Array_mapFinIdxM_map___at_Array_mapFinIdx___spec__1___rarg(x_1, x_2, x_1, x_3, x_5, lean_box(0), x_4); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdx(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Array_mapFinIdx___rarg___boxed), 2, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapFinIdx___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) { +_start: +{ +lean_object* x_8; +x_8 = l_Array_mapFinIdxM_map___at_Array_mapFinIdx___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_3); +lean_dec(x_1); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdx___rarg___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Array_mapFinIdx___rarg(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdx___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) { _start: { lean_object* x_8; uint8_t x_9; @@ -5566,11 +5804,11 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_mapIdx___spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdx___spec__1(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Array_mapIdx___spec__1___rarg___boxed), 7, 0); +x_3 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Array_mapIdx___spec__1___rarg___boxed), 7, 0); return x_3; } } @@ -5581,7 +5819,7 @@ lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_3 = lean_array_get_size(x_1); x_4 = lean_mk_empty_array_with_capacity(x_3); x_5 = lean_unsigned_to_nat(0u); -x_6 = l_Array_mapIdxM_map___at_Array_mapIdx___spec__1___rarg(x_1, x_2, x_1, x_3, x_5, lean_box(0), x_4); +x_6 = l_Array_mapFinIdxM_map___at_Array_mapIdx___spec__1___rarg(x_1, x_2, x_1, x_3, x_5, lean_box(0), x_4); return x_6; } } @@ -5593,11 +5831,11 @@ x_3 = lean_alloc_closure((void*)(l_Array_mapIdx___rarg___boxed), 2, 0); return x_3; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_mapIdx___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdx___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) { _start: { lean_object* x_8; -x_8 = l_Array_mapIdxM_map___at_Array_mapIdx___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Array_mapFinIdxM_map___at_Array_mapIdx___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_3); lean_dec(x_1); return x_8; @@ -5612,7 +5850,7 @@ lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_zipWithIndex___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_zipWithIndex___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: { lean_object* x_7; uint8_t x_8; @@ -5646,11 +5884,11 @@ return x_6; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_zipWithIndex___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_zipWithIndex___spec__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Array_zipWithIndex___spec__1___rarg___boxed), 6, 0); +x_2 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Array_zipWithIndex___spec__1___rarg___boxed), 6, 0); return x_2; } } @@ -5661,7 +5899,7 @@ lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_2 = lean_array_get_size(x_1); x_3 = lean_mk_empty_array_with_capacity(x_2); x_4 = lean_unsigned_to_nat(0u); -x_5 = l_Array_mapIdxM_map___at_Array_zipWithIndex___spec__1___rarg(x_1, x_1, x_2, x_4, lean_box(0), x_3); +x_5 = l_Array_mapFinIdxM_map___at_Array_zipWithIndex___spec__1___rarg(x_1, x_1, x_2, x_4, lean_box(0), x_3); return x_5; } } @@ -5673,11 +5911,11 @@ x_2 = lean_alloc_closure((void*)(l_Array_zipWithIndex___rarg___boxed), 1, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Array_zipWithIndex___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_zipWithIndex___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) { _start: { lean_object* x_7; -x_7 = l_Array_mapIdxM_map___at_Array_zipWithIndex___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Array_mapFinIdxM_map___at_Array_zipWithIndex___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_2); lean_dec(x_1); return x_7; @@ -6074,7 +6312,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(538u); +x_3 = lean_unsigned_to_nat(570u); 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); @@ -7544,7 +7782,7 @@ x_2 = l_Array_instHAppendList___closed__1; return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___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; @@ -7559,17 +7797,17 @@ x_7 = lean_apply_2(x_5, lean_box(0), x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__2(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__2(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { _start: { size_t x_7; size_t x_8; lean_object* x_9; x_7 = 1; x_8 = lean_usize_add(x_1, x_7); -x_9 = l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg(x_2, x_3, x_4, x_8, x_5, x_6); +x_9 = l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg(x_2, x_3, x_4, x_8, x_5, x_6); return x_9; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg(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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { _start: { uint8_t x_7; @@ -7583,14 +7821,14 @@ x_9 = lean_array_uget(x_3, x_4); lean_inc(x_2); x_10 = lean_apply_1(x_2, x_9); lean_inc(x_1); -x_11 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1___boxed), 3, 2); +x_11 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__1___boxed), 3, 2); lean_closure_set(x_11, 0, x_1); lean_closure_set(x_11, 1, x_6); lean_inc(x_8); x_12 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_10, x_11); x_13 = lean_box_usize(x_4); x_14 = lean_box_usize(x_5); -x_15 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__2___boxed), 6, 5); +x_15 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__2___boxed), 6, 5); lean_closure_set(x_15, 0, x_13); lean_closure_set(x_15, 1, x_1); lean_closure_set(x_15, 2, x_2); @@ -7615,15 +7853,15 @@ return x_19; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___boxed), 6, 0); +x_4 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___boxed), 6, 0); return x_4; } } -LEAN_EXPORT lean_object* l_Array_concatMapM___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_flatMapM___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; @@ -7673,30 +7911,30 @@ x_16 = 0; x_17 = lean_usize_of_nat(x_4); lean_dec(x_4); x_18 = l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__18; -x_19 = l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg(x_1, x_2, x_3, x_16, x_17, x_18); +x_19 = l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg(x_1, x_2, x_3, x_16, x_17, x_18); return x_19; } } } } -LEAN_EXPORT lean_object* l_Array_concatMapM(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_flatMapM(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = lean_alloc_closure((void*)(l_Array_concatMapM___rarg), 3, 0); +x_4 = lean_alloc_closure((void*)(l_Array_flatMapM___rarg), 3, 0); return x_4; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1(x_1, x_2, x_3); +x_4 = l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__1(x_1, x_2, x_3); lean_dec(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___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) { _start: { size_t x_7; size_t x_8; lean_object* x_9; @@ -7704,11 +7942,11 @@ x_7 = lean_unbox_usize(x_1); lean_dec(x_1); x_8 = lean_unbox_usize(x_5); lean_dec(x_5); -x_9 = l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__2(x_7, x_2, x_3, x_4, x_8, x_6); +x_9 = l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__2(x_7, x_2, x_3, x_4, x_8, x_6); return x_9; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMapM___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) { _start: { size_t x_7; size_t x_8; lean_object* x_9; @@ -7716,57 +7954,313 @@ x_7 = lean_unbox_usize(x_4); lean_dec(x_4); x_8 = lean_unbox_usize(x_5); lean_dec(x_5); -x_9 = l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg(x_1, x_2, x_3, x_7, x_8, x_6); +x_9 = l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg(x_1, x_2, x_3, x_7, x_8, x_6); return x_9; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMap___spec__1___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { _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; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg(x_2, x_3, x_4, x_8, x_5, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { +_start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; -x_7 = lean_array_uget(x_2, x_3); +uint8_t x_7; +x_7 = lean_usize_dec_eq(x_4, x_5); +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; +x_8 = lean_ctor_get(x_1, 1); +lean_inc(x_8); +x_9 = lean_array_uget(x_3, x_4); +lean_inc(x_2); +x_10 = lean_apply_1(x_2, x_9); lean_inc(x_1); -x_8 = lean_apply_1(x_1, x_7); -x_9 = l_Array_append___rarg(x_5, x_8); -lean_dec(x_8); -x_10 = 1; -x_11 = lean_usize_add(x_3, x_10); -x_3 = x_11; -x_5 = x_9; -goto _start; +x_11 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_flatMapM___spec__1___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_11, 0, x_1); +lean_closure_set(x_11, 1, x_6); +lean_inc(x_8); +x_12 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_10, x_11); +x_13 = lean_box_usize(x_4); +x_14 = lean_box_usize(x_5); +x_15 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_15, 0, x_13); +lean_closure_set(x_15, 1, x_1); +lean_closure_set(x_15, 2, x_2); +lean_closure_set(x_15, 3, x_3); +lean_closure_set(x_15, 4, x_14); +x_16 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_12, x_15); +return x_16; } else { +lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_dec(x_3); +lean_dec(x_2); +x_17 = lean_ctor_get(x_1, 0); +lean_inc(x_17); lean_dec(x_1); -return x_5; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_19 = lean_apply_2(x_18, lean_box(0), x_6); +return x_19; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMap___spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_concatMap___spec__1___rarg___boxed), 5, 0); -return x_3; +lean_object* x_4; +x_4 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___boxed), 6, 0); +return x_4; } } -LEAN_EXPORT lean_object* l_Array_concatMap___rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_concatMapM___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_3; lean_object* x_4; uint8_t x_5; -x_3 = lean_array_get_size(x_2); -x_4 = lean_unsigned_to_nat(0u); -x_5 = lean_nat_dec_lt(x_4, x_3); -if (x_5 == 0) +lean_object* x_4; lean_object* x_5; uint8_t x_6; +x_4 = lean_array_get_size(x_3); +x_5 = lean_unsigned_to_nat(0u); +x_6 = lean_nat_dec_lt(x_5, x_4); +if (x_6 == 0) { -lean_object* x_6; +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_4); lean_dec(x_3); +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); lean_dec(x_1); -x_6 = l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__18; +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__18; +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +uint8_t x_11; +x_11 = lean_nat_dec_le(x_4, x_4); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +lean_dec(x_1); +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__18; +x_15 = lean_apply_2(x_13, lean_box(0), x_14); +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_4); +lean_dec(x_4); +x_18 = l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__18; +x_19 = l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg(x_1, x_2, x_3, x_16, x_17, x_18); +return x_19; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_concatMapM(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_alloc_closure((void*)(l_Array_concatMapM___rarg), 3, 0); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___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) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMapM___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) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_foldlMUnsafe_fold___at_Array_concatMapM___spec__1___rarg(x_1, x_2, x_3, x_7, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMap___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) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; +x_7 = lean_array_uget(x_2, x_3); +lean_inc(x_1); +x_8 = lean_apply_1(x_1, x_7); +x_9 = l_Array_append___rarg(x_5, x_8); +lean_dec(x_8); +x_10 = 1; +x_11 = lean_usize_add(x_3, x_10); +x_3 = x_11; +x_5 = x_9; +goto _start; +} +else +{ +lean_dec(x_1); +return x_5; +} +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMap___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_flatMap___spec__1___rarg___boxed), 5, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_flatMap___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_array_get_size(x_2); +x_4 = lean_unsigned_to_nat(0u); +x_5 = lean_nat_dec_lt(x_4, x_3); +if (x_5 == 0) +{ +lean_object* x_6; +lean_dec(x_3); +lean_dec(x_1); +x_6 = l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__18; +return x_6; +} +else +{ +uint8_t x_7; +x_7 = lean_nat_dec_le(x_3, x_3); +if (x_7 == 0) +{ +lean_object* x_8; +lean_dec(x_3); +lean_dec(x_1); +x_8 = l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__18; +return x_8; +} +else +{ +size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; +x_9 = 0; +x_10 = lean_usize_of_nat(x_3); +lean_dec(x_3); +x_11 = l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__18; +x_12 = l_Array_foldlMUnsafe_fold___at_Array_flatMap___spec__1___rarg(x_1, x_2, x_9, x_10, x_11); +return x_12; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_flatMap(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Array_flatMap___rarg___boxed), 2, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_flatMap___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_foldlMUnsafe_fold___at_Array_flatMap___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_flatMap___rarg___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Array_flatMap___rarg(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMap___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) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; +x_7 = lean_array_uget(x_2, x_3); +lean_inc(x_1); +x_8 = lean_apply_1(x_1, x_7); +x_9 = l_Array_append___rarg(x_5, x_8); +lean_dec(x_8); +x_10 = 1; +x_11 = lean_usize_add(x_3, x_10); +x_3 = x_11; +x_5 = x_9; +goto _start; +} +else +{ +lean_dec(x_1); +return x_5; +} +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_concatMap___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_concatMap___spec__1___rarg___boxed), 5, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_concatMap___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_array_get_size(x_2); +x_4 = lean_unsigned_to_nat(0u); +x_5 = lean_nat_dec_lt(x_4, x_3); +if (x_5 == 0) +{ +lean_object* x_6; +lean_dec(x_3); +lean_dec(x_1); +x_6 = l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__18; return x_6; } else @@ -9174,7 +9668,7 @@ static lean_object* _init_l_Array_insertAt_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_insertAt_x21___rarg___closed__1; -x_3 = lean_unsigned_to_nat(764u); +x_3 = lean_unsigned_to_nat(800u); x_4 = lean_unsigned_to_nat(7u); x_5 = l_Array_insertAt_x21___rarg___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -9814,6 +10308,143 @@ lean_dec(x_1); return x_3; } } +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_reduceOption___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; 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; lean_object* x_11; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_array_push(x_4, x_10); +x_2 = x_8; +x_4 = x_11; +goto _start; +} +} +else +{ +return x_4; +} +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_reduceOption___spec__2(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Array_reduceOption___spec__2___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_filterMapM___at_Array_reduceOption___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_nat_dec_lt(x_2, x_3); +if (x_4 == 0) +{ +lean_object* x_5; +x_5 = l_Array_filter___rarg___closed__1; +return x_5; +} +else +{ +lean_object* x_6; uint8_t x_7; +x_6 = lean_array_get_size(x_1); +x_7 = lean_nat_dec_le(x_3, x_6); +lean_dec(x_6); +if (x_7 == 0) +{ +lean_object* x_8; +x_8 = l_Array_filter___rarg___closed__1; +return x_8; +} +else +{ +size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_usize_of_nat(x_2); +x_10 = lean_usize_of_nat(x_3); +x_11 = l_Array_filter___rarg___closed__1; +x_12 = l_Array_foldlMUnsafe_fold___at_Array_reduceOption___spec__2___rarg(x_1, x_9, x_10, x_11); +return x_12; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_filterMapM___at_Array_reduceOption___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_filterMapM___at_Array_reduceOption___spec__1___rarg___boxed), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_reduceOption___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_2 = lean_array_get_size(x_1); +x_3 = lean_unsigned_to_nat(0u); +x_4 = l_Array_filterMapM___at_Array_reduceOption___spec__1___rarg(x_1, x_3, x_2); +lean_dec(x_2); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_reduceOption(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_reduceOption___rarg___boxed), 1, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_reduceOption___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_Array_reduceOption___spec__2___rarg(x_1, x_5, x_6, x_4); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_filterMapM___at_Array_reduceOption___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Array_filterMapM___at_Array_reduceOption___spec__1___rarg(x_1, x_2, x_3); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_reduceOption___rarg___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Array_reduceOption___rarg(x_1); +lean_dec(x_1); +return x_2; +} +} LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_eraseReps___spec__1___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { _start: { diff --git a/stage0/stdlib/Init/Data/Array/DecidableEq.c b/stage0/stdlib/Init/Data/Array/DecidableEq.c index 2ddc56fdb3bc..d0515e31b318 100644 --- a/stage0/stdlib/Init/Data/Array/DecidableEq.c +++ b/stage0/stdlib/Init/Data/Array/DecidableEq.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Data.Array.DecidableEq -// Imports: Init.Data.Array.Basic Init.Data.BEq Init.ByCases +// Imports: Init.Data.Array.Basic Init.Data.BEq Init.Data.Nat.Lemmas Init.Data.List.Nat.BEq Init.ByCases #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -187,6 +187,8 @@ return x_5; } lean_object* initialize_Init_Data_Array_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_BEq(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_Nat_Lemmas(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_List_Nat_BEq(uint8_t builtin, lean_object*); lean_object* initialize_Init_ByCases(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_Data_Array_DecidableEq(uint8_t builtin, lean_object* w) { @@ -199,6 +201,12 @@ lean_dec_ref(res); res = initialize_Init_Data_BEq(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_Data_Nat_Lemmas(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Init_Data_List_Nat_BEq(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); res = initialize_Init_ByCases(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/Array/GetLit.c b/stage0/stdlib/Init/Data/Array/GetLit.c index 03fb16fcacd4..6da8fc3d154d 100644 --- a/stage0/stdlib/Init/Data/Array/GetLit.c +++ b/stage0/stdlib/Init/Data/Array/GetLit.c @@ -145,56 +145,6 @@ lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter___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; uint8_t x_7; -x_6 = lean_unsigned_to_nat(0u); -x_7 = lean_nat_dec_eq(x_1, x_6); -if (x_7 == 0) -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; -lean_dec(x_4); -x_8 = lean_unsigned_to_nat(1u); -x_9 = lean_nat_sub(x_1, x_8); -x_10 = lean_apply_3(x_5, x_9, lean_box(0), x_3); -return x_10; -} -else -{ -lean_object* x_11; -lean_dec(x_5); -x_11 = lean_apply_2(x_4, lean_box(0), x_3); -return x_11; -} -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_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_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter___rarg___boxed), 5, 0); -return x_4; -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_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) { -_start: -{ -lean_object* x_6; -x_6 = l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter___rarg(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_1); -return x_6; -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter(x_1, x_2, x_3); -lean_dec(x_2); -return x_4; -} -} LEAN_EXPORT lean_object* l___private_Init_Data_Array_GetLit_0__List_take_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -254,6 +204,56 @@ lean_dec(x_1); return x_6; } } +LEAN_EXPORT lean_object* l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter___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; uint8_t x_7; +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_nat_dec_eq(x_1, x_6); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_4); +x_8 = lean_unsigned_to_nat(1u); +x_9 = lean_nat_sub(x_1, x_8); +x_10 = lean_apply_3(x_5, x_9, lean_box(0), x_3); +return x_10; +} +else +{ +lean_object* x_11; +lean_dec(x_5); +x_11 = lean_apply_2(x_4, lean_box(0), x_3); +return x_11; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_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_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter___rarg___boxed), 5, 0); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_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) { +_start: +{ +lean_object* x_6; +x_6 = l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter___rarg(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Init_Data_Array_GetLit_0__Array_toListLitAux_match__1_splitter(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} lean_object* initialize_Init_Data_Array_Basic(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_Data_Array_GetLit(uint8_t builtin, lean_object* w) { diff --git a/stage0/stdlib/Init/Data/Array/Lemmas.c b/stage0/stdlib/Init/Data/Array/Lemmas.c index 6c9aa1689e37..5dc5fba49771 100644 --- a/stage0/stdlib/Init/Data/Array/Lemmas.c +++ b/stage0/stdlib/Init/Data/Array/Lemmas.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Data.Array.Lemmas -// Imports: Init.Data.Nat.Lemmas Init.Data.List.Impl Init.Data.List.Monadic Init.Data.List.Range Init.Data.Array.Mem Init.TacticsExtra +// Imports: Init.Data.Nat.Lemmas Init.Data.List.Impl Init.Data.List.Monadic Init.Data.List.Range Init.Data.List.Nat.TakeDrop Init.Data.Array.Mem Init.TacticsExtra #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -17,10 +17,10 @@ LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_findSomeRev LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_findSomeRevM_x3f_find_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_toListRev___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_foldlM_loop_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_toListRev___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_instDecidableMemOfDecidableEq___spec__2(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_isEqvAux_match__1_splitter___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__GetElem_x3f_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__List_anyM_match__1_splitter___rarg(uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_instDecidableMemOfDecidableEq___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -45,13 +45,12 @@ LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_findSomeRev LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_toListRev___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__List_anyM_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_foldlM_loop_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Array_instDecidableMemOfDecidableEq___spec__2___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t); lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__List_anyM_match__1_splitter(lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__GetElem_x3f_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_appendCore_loop_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Array_instDecidableMemOfDecidableEq___rarg___boxed(lean_object*, lean_object*, lean_object*); @@ -59,10 +58,47 @@ lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Nat_fold_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_instDecidableMemOfDecidableEq___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_toListRev(lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter___rarg___boxed(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_EXPORT uint8_t l_Array_contains___at_Array_instDecidableMemOfDecidableEq___spec__1___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__GetElem_x3f_match__1_splitter(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__GetElem_x3f_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_2); +lean_inc(x_3); +return x_3; +} +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_2, x_4); +return x_5; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__GetElem_x3f_match__1_splitter(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Array_Lemmas_0__GetElem_x3f_match__1_splitter___rarg___boxed), 3, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__GetElem_x3f_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_Data_Array_Lemmas_0__GetElem_x3f_match__1_splitter___rarg(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_toListRev___spec__1___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { @@ -290,57 +326,6 @@ lean_dec(x_2); return x_4; } } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; uint8_t x_6; -x_5 = lean_unsigned_to_nat(0u); -x_6 = lean_nat_dec_eq(x_1, x_5); -if (x_6 == 0) -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; -lean_dec(x_3); -x_7 = lean_unsigned_to_nat(1u); -x_8 = lean_nat_sub(x_1, x_7); -x_9 = lean_apply_2(x_4, x_8, lean_box(0)); -return x_9; -} -else -{ -lean_object* x_10; -lean_dec(x_4); -x_10 = lean_apply_1(x_3, lean_box(0)); -return x_10; -} -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_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_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter___rarg___boxed), 4, 0); -return x_5; -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter___rarg___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_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter___rarg(x_1, x_2, x_3, x_4); -lean_dec(x_1); -return x_5; -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_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_Init_Data_Array_Lemmas_0__Array_mapIdxM_map_match__1_splitter(x_1, x_2, x_3, x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_5; -} -} LEAN_EXPORT lean_object* l___private_Init_Data_Array_Lemmas_0__Array_findSomeRevM_x3f_find_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -628,6 +613,7 @@ lean_object* initialize_Init_Data_Nat_Lemmas(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_List_Impl(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_List_Monadic(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_List_Range(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_List_Nat_TakeDrop(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Array_Mem(uint8_t builtin, lean_object*); lean_object* initialize_Init_TacticsExtra(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -647,6 +633,9 @@ lean_dec_ref(res); res = initialize_Init_Data_List_Range(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_Data_List_Nat_TakeDrop(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); res = initialize_Init_Data_Array_Mem(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/Array/MapIdx.c b/stage0/stdlib/Init/Data/Array/MapIdx.c new file mode 100644 index 000000000000..9f2d423744f9 --- /dev/null +++ b/stage0/stdlib/Init/Data/Array/MapIdx.c @@ -0,0 +1,90 @@ +// Lean compiler output +// Module: Init.Data.Array.MapIdx +// Imports: Init.Data.Array.Lemmas Init.Data.List.MapIdx +#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___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter(lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +lean_object* lean_nat_sub(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; uint8_t x_6; +x_5 = lean_unsigned_to_nat(0u); +x_6 = lean_nat_dec_eq(x_1, x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_dec(x_3); +x_7 = lean_unsigned_to_nat(1u); +x_8 = lean_nat_sub(x_1, x_7); +x_9 = lean_apply_2(x_4, x_8, lean_box(0)); +return x_9; +} +else +{ +lean_object* x_10; +lean_dec(x_4); +x_10 = lean_apply_1(x_3, lean_box(0)); +return x_10; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_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_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter___rarg___boxed), 4, 0); +return x_5; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter___rarg___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_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter___rarg(x_1, x_2, x_3, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_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_Init_Data_Array_MapIdx_0__Array_mapFinIdxM_map_match__1_splitter(x_1, x_2, x_3, x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_5; +} +} +lean_object* initialize_Init_Data_Array_Lemmas(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_List_MapIdx(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Init_Data_Array_MapIdx(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_Data_Array_Lemmas(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Init_Data_List_MapIdx(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/Init/Data/Hashable.c b/stage0/stdlib/Init/Data/Hashable.c index b212dceca9e0..2387afa1676f 100644 --- a/stage0/stdlib/Init/Data/Hashable.c +++ b/stage0/stdlib/Init/Data/Hashable.c @@ -20,6 +20,7 @@ uint64_t lean_uint64_of_nat(lean_object*); uint64_t lean_uint64_mix_hash(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_instHashableProd(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); +LEAN_EXPORT lean_object* l_instHashableChar___boxed(lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_instHashableList___spec__1(lean_object*); LEAN_EXPORT lean_object* l_hash64___boxed(lean_object*); LEAN_EXPORT lean_object* l_instHashableInt___boxed(lean_object*); @@ -57,6 +58,7 @@ LEAN_EXPORT lean_object* l_instHashable___boxed(lean_object*, lean_object*); uint8_t lean_int_dec_lt(lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); +LEAN_EXPORT uint64_t l_instHashableChar(uint32_t); LEAN_EXPORT lean_object* l_instHashableOption(lean_object*); LEAN_EXPORT uint64_t l_hash64(uint64_t); static lean_object* l_instHashableInt___closed__1; @@ -524,6 +526,25 @@ lean_dec(x_1); return x_2; } } +LEAN_EXPORT uint64_t l_instHashableChar(uint32_t x_1) { +_start: +{ +uint64_t x_2; +x_2 = lean_uint32_to_uint64(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_instHashableChar___boxed(lean_object* x_1) { +_start: +{ +uint32_t x_2; uint64_t x_3; lean_object* x_4; +x_2 = lean_unbox_uint32(x_1); +lean_dec(x_1); +x_3 = l_instHashableChar(x_2); +x_4 = lean_box_uint64(x_3); +return x_4; +} +} static lean_object* _init_l_instHashableInt___closed__1() { _start: { diff --git a/stage0/stdlib/Init/Data/List/Basic.c b/stage0/stdlib/Init/Data/List/Basic.c index 46a7d0004e88..16d73503850b 100644 --- a/stage0/stdlib/Init/Data/List/Basic.c +++ b/stage0/stdlib/Init/Data/List/Basic.c @@ -44,7 +44,7 @@ LEAN_EXPORT lean_object* l_List_enum___rarg(lean_object*); LEAN_EXPORT lean_object* l_List_join(lean_object*); LEAN_EXPORT lean_object* l_List_min_x3f(lean_object*); LEAN_EXPORT lean_object* l_List_zipWith(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_pure(lean_object*); +LEAN_EXPORT lean_object* l_List_pure(lean_object*, lean_object*); static lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x3c_x3a_x2b____1___closed__4; LEAN_EXPORT lean_object* l_List_mapTR_loop(lean_object*, lean_object*); static lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x3c_x2b____1___closed__1; @@ -120,6 +120,7 @@ static lean_object* l_List_term___x3c_x2b_____closed__9; static lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x7e____1___closed__4; LEAN_EXPORT lean_object* l_List_instHasSubset(lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMap___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List___aux__Init__Data__List__Basic______unexpand__List__Perm__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_bind(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_find_x3f(lean_object*); @@ -267,6 +268,7 @@ LEAN_EXPORT lean_object* l_List_instDecidableRelSubsetOfDecidableEq(lean_object* LEAN_EXPORT lean_object* l_List_removeAll___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x3c_x2b____1___closed__6; +LEAN_EXPORT lean_object* l_List_singleton(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_replicateTR_loop_match__1_splitter(lean_object*, lean_object*); lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_unzip(lean_object*, lean_object*); @@ -326,6 +328,7 @@ static lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List_ LEAN_EXPORT lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x3c_x2b____1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_instLEOfLT___boxed(lean_object*, lean_object*); static lean_object* l_List_term___x3c_x2b_____closed__11; +LEAN_EXPORT lean_object* l_List_singleton___rarg(lean_object*); static lean_object* l_List_term___x3c_x3a_x2b_____closed__2; LEAN_EXPORT lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x3c_x3a_x2b____1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_tail_x3f___rarg(lean_object*); @@ -427,7 +430,7 @@ LEAN_EXPORT lean_object* l_List___aux__Init__Data__List__Basic______macroRules__ LEAN_EXPORT lean_object* l_List___aux__Init__Data__List__Basic______unexpand__List__Sublist__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_dropWhile___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_instDecidableMemOfLawfulBEq(lean_object*); -LEAN_EXPORT lean_object* l_List_pure___rarg(lean_object*); +LEAN_EXPORT lean_object* l_List_pure___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR(lean_object*, lean_object*); static lean_object* l_List___aux__Init__Data__List__Basic______macroRules__List__term___x3c_x3a_x2b_x3a____1___closed__4; static lean_object* l_List_term___x3c_x3a_x2b_____closed__4; @@ -474,6 +477,7 @@ LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_beq_match__1_s LEAN_EXPORT lean_object* l_List_map___at_List_zipWithAll___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Basic_0__List_iotaTR_go_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMap(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldr___at_List_sum___spec__1(lean_object*); LEAN_EXPORT lean_object* l_List_unzipTR(lean_object*, lean_object*); static lean_object* l_List_term___x3c_x2b_____closed__6; @@ -1936,7 +1940,7 @@ x_2 = lean_alloc_closure((void*)(l_List_join___rarg), 1, 0); return x_2; } } -LEAN_EXPORT lean_object* l_List_pure___rarg(lean_object* x_1) { +LEAN_EXPORT lean_object* l_List_singleton___rarg(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -1947,15 +1951,31 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_List_pure(lean_object* x_1) { +LEAN_EXPORT lean_object* l_List_singleton(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_List_pure___rarg), 1, 0); +x_2 = lean_alloc_closure((void*)(l_List_singleton___rarg), 1, 0); return x_2; } } -LEAN_EXPORT lean_object* l_List_bind___rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_pure___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_apply_1(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_List_pure(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_List_pure___rarg), 2, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_List_flatMap___rarg(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; @@ -1964,11 +1984,11 @@ x_4 = l_List_flatten___rarg(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_List_bind(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMap(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_List_bind___rarg), 2, 0); +x_3 = lean_alloc_closure((void*)(l_List_flatMap___rarg), 2, 0); return x_3; } } @@ -2011,6 +2031,23 @@ lean_dec(x_2); return x_4; } } +LEAN_EXPORT lean_object* l_List_bind___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; +x_3 = l_List_map___rarg(x_2, x_1); +x_4 = l_List_flatten___rarg(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_List_bind(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_List_bind___rarg), 2, 0); +return x_3; +} +} LEAN_EXPORT lean_object* l_List_replicate___rarg(lean_object* x_1, lean_object* x_2) { _start: { diff --git a/stage0/stdlib/Init/Data/List/Impl.c b/stage0/stdlib/Init/Data/List/Impl.c index a0928ff7ead1..65357e62c067 100644 --- a/stage0/stdlib/Init/Data/List/Impl.c +++ b/stage0/stdlib/Init/Data/List/Impl.c @@ -20,7 +20,6 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_setTR_go___spec__1_ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_enumFromTR___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_enumFromTR___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_eraseIdxTR_go___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_setTR_go___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_eraseTR(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_eraseIdxTR_go___spec__2___rarg(lean_object*, size_t, size_t, lean_object*); @@ -37,6 +36,7 @@ LEAN_EXPORT lean_object* l_List_erasePTR___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_eraseIdx_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_zipWithTR_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); +LEAN_EXPORT lean_object* l_List_flatMapTR_go(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_enumFromTR(lean_object*); LEAN_EXPORT lean_object* l_List_takeTR_go___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterMapTR_go(lean_object*, lean_object*); @@ -44,7 +44,6 @@ LEAN_EXPORT lean_object* l_List_replaceTR_go___rarg(lean_object*, lean_object*, LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_intercalateTR_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_setTR_go(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_setTR_go_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at_List_flattenTR___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_intercalateTR_go___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_takeWhileTR___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_eraseTR_go___spec__2___rarg(lean_object*, size_t, size_t, lean_object*); @@ -52,7 +51,6 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_enumFromTR___spec__ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_intercalateTR_go___spec__2___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_List_takeTR(lean_object*); LEAN_EXPORT lean_object* l_List_eraseTR_go(lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_setTR_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_setTR_go___spec__2___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_List_replaceTR(lean_object*); @@ -60,13 +58,11 @@ LEAN_EXPORT lean_object* l_List_dropLastTR___rarg(lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_List_intercalateTR(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_filterMapTR_go_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_intercalateTR_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterMapTR(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_eraseTR_go___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_intercalateTR_go_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_intercalateTR_go___spec__2(lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_eraseTR_go___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_enumFromTR___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); lean_object* lean_array_pop(lean_object*); @@ -75,7 +71,6 @@ lean_object* lean_array_to_list(lean_object*); LEAN_EXPORT lean_object* l_List_foldrTR(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_setTR_go___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_eraseIdxTR_go(lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at_List_flattenTR___spec__1(lean_object*); LEAN_EXPORT lean_object* l_List_flattenTR(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_intercalateTR_go___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_filterMap_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); @@ -84,6 +79,7 @@ LEAN_EXPORT lean_object* l_List_eraseIdxTR(lean_object*); LEAN_EXPORT lean_object* l_List_erasePTR(lean_object*); LEAN_EXPORT lean_object* l_List_filterMapTR_go___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_enumFromTR___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_enumFromTR___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_filter_match__1_splitter___rarg(uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_eraseIdxTR_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -98,6 +94,7 @@ LEAN_EXPORT lean_object* l_List_erasePTR_go(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_intercalateTR_go_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_takeTR_go(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_takeWhileTR_go_match__1_splitter(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_eraseTR_go___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_enumFromTR___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_eraseTR_go___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -110,6 +107,7 @@ LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_filterMapTR_go_ LEAN_EXPORT lean_object* l_List_zipWithTR_go(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterMapTR___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_replace_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_List_flattenTR___spec__1___rarg(lean_object*, lean_object*); extern lean_object* l_Id_instMonad; LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_filterMapTR_go_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_flattenTR___rarg(lean_object*); @@ -135,6 +133,8 @@ LEAN_EXPORT lean_object* l_List_eraseIdxTR_go___rarg___boxed(lean_object*, lean_ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_eraseIdxTR_go___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_takeWhileTR_go(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_getLast_x3f_match__1_splitter(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_List_flattenTR___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_zipWithTR_go_match__1_splitter(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Impl_0__List_filter_match__1_splitter(lean_object*); @@ -715,7 +715,7 @@ x_3 = lean_alloc_closure((void*)(l_List_foldrTR___rarg), 3, 0); return x_3; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_2) == 0) @@ -742,32 +742,32 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_bindTR_go(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_List_bindTR_go___rarg), 3, 0); +x_3 = lean_alloc_closure((void*)(l_List_flatMapTR_go___rarg), 3, 0); return x_3; } } -LEAN_EXPORT lean_object* l_List_bindTR___rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR___rarg(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; x_3 = l_List_setTR___rarg___closed__1; -x_4 = l_List_bindTR_go___rarg(x_2, x_1, x_3); +x_4 = l_List_flatMapTR_go___rarg(x_2, x_1, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_List_bindTR(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_List_bindTR___rarg), 2, 0); +x_3 = lean_alloc_closure((void*)(l_List_flatMapTR___rarg), 2, 0); return x_3; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at_List_flattenTR___spec__1___rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_List_flattenTR___spec__1___rarg(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -791,11 +791,11 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at_List_flattenTR___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_List_flattenTR___spec__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_List_bindTR_go___at_List_flattenTR___spec__1___rarg), 2, 0); +x_2 = lean_alloc_closure((void*)(l_List_flatMapTR_go___at_List_flattenTR___spec__1___rarg), 2, 0); return x_2; } } @@ -804,7 +804,7 @@ LEAN_EXPORT lean_object* l_List_flattenTR___rarg(lean_object* x_1) { { lean_object* x_2; lean_object* x_3; x_2 = l_List_setTR___rarg___closed__1; -x_3 = l_List_bindTR_go___at_List_flattenTR___spec__1___rarg(x_1, x_2); +x_3 = l_List_flatMapTR_go___at_List_flattenTR___spec__1___rarg(x_1, x_2); return x_3; } } diff --git a/stage0/stdlib/Init/Data/List/Nat.c b/stage0/stdlib/Init/Data/List/Nat.c index c1510a26117e..b9df07d73e7e 100644 --- a/stage0/stdlib/Init/Data/List/Nat.c +++ b/stage0/stdlib/Init/Data/List/Nat.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Data.List.Nat -// Imports: Init.Data.List.Nat.Basic Init.Data.List.Nat.Pairwise Init.Data.List.Nat.Range Init.Data.List.Nat.Sublist Init.Data.List.Nat.TakeDrop Init.Data.List.Nat.Count Init.Data.List.Nat.Erase Init.Data.List.Nat.Find +// Imports: Init.Data.List.Nat.Basic Init.Data.List.Nat.Pairwise Init.Data.List.Nat.Range Init.Data.List.Nat.Sublist Init.Data.List.Nat.TakeDrop Init.Data.List.Nat.Count Init.Data.List.Nat.Erase Init.Data.List.Nat.Find Init.Data.List.Nat.BEq #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -21,6 +21,7 @@ lean_object* initialize_Init_Data_List_Nat_TakeDrop(uint8_t builtin, lean_object lean_object* initialize_Init_Data_List_Nat_Count(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_List_Nat_Erase(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_List_Nat_Find(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_List_Nat_BEq(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_Data_List_Nat(uint8_t builtin, lean_object* w) { lean_object * res; @@ -50,6 +51,9 @@ lean_dec_ref(res); res = initialize_Init_Data_List_Nat_Find(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_Data_List_Nat_BEq(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/Data/List/Nat/BEq.c b/stage0/stdlib/Init/Data/List/Nat/BEq.c new file mode 100644 index 000000000000..bc217a32439d --- /dev/null +++ b/stage0/stdlib/Init/Data/List/Nat/BEq.c @@ -0,0 +1,94 @@ +// Lean compiler output +// Module: Init.Data.List.Nat.BEq +// Imports: Init.Data.Nat.Lemmas Init.Data.List.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___private_Init_Data_List_Nat_BEq_0__List_isEqv_match__1_splitter(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_List_Nat_BEq_0__List_isEqv_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_List_Nat_BEq_0__List_isEqv_match__1_splitter___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: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_dec(x_5); +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_7; +lean_dec(x_6); +x_7 = lean_apply_1(x_4, x_3); +return x_7; +} +else +{ +lean_object* x_8; +lean_dec(x_4); +x_8 = lean_apply_5(x_6, x_1, x_2, x_3, lean_box(0), lean_box(0)); +return x_8; +} +} +else +{ +lean_dec(x_4); +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_9; +lean_dec(x_5); +x_9 = lean_apply_5(x_6, x_1, x_2, x_3, lean_box(0), lean_box(0)); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_10 = lean_ctor_get(x_1, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +lean_dec(x_1); +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_apply_5(x_5, x_10, x_11, x_12, x_13, x_3); +return x_14; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_List_Nat_BEq_0__List_isEqv_match__1_splitter(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Init_Data_List_Nat_BEq_0__List_isEqv_match__1_splitter___rarg), 6, 0); +return x_3; +} +} +lean_object* initialize_Init_Data_Nat_Lemmas(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_List_Basic(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Init_Data_List_Nat_BEq(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_Data_Nat_Lemmas(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Init_Data_List_Basic(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/Init/Data/Prod.c b/stage0/stdlib/Init/Data/Prod.c index fbc2f9481307..067ec63bf32c 100644 --- a/stage0/stdlib/Init/Data/Prod.c +++ b/stage0/stdlib/Init/Data/Prod.c @@ -13,6 +13,40 @@ #ifdef __cplusplus extern "C" { #endif +LEAN_EXPORT lean_object* l_Prod_swap___rarg___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Prod_swap___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Prod_swap(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Prod_swap___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_2 = lean_ctor_get(x_1, 1); +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +lean_inc(x_2); +x_4 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Prod_swap(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Prod_swap___rarg___boxed), 1, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Prod_swap___rarg___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Prod_swap___rarg(x_1); +lean_dec(x_1); +return x_2; +} +} lean_object* initialize_Init_SimpLemmas(uint8_t builtin, lean_object*); lean_object* initialize_Init_NotationExtra(uint8_t builtin, lean_object*); static bool _G_initialized = false; diff --git a/stage0/stdlib/Init/Data/String/Basic.c b/stage0/stdlib/Init/Data/String/Basic.c index 6a968c286229..0f7ed93ad292 100644 --- a/stage0/stdlib/Init/Data/String/Basic.c +++ b/stage0/stdlib/Init/Data/String/Basic.c @@ -6878,29 +6878,39 @@ return x_6; LEAN_EXPORT lean_object* l_String_dropPrefix_x3f(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_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; x_3 = lean_string_utf8_byte_size(x_1); x_4 = lean_unsigned_to_nat(0u); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_1); lean_ctor_set(x_5, 1, x_4); lean_ctor_set(x_5, 2, x_3); -x_6 = l_Substring_dropPrefix_x3f(x_5, x_2); -return x_6; +x_6 = lean_string_utf8_byte_size(x_2); +x_7 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_7, 0, x_2); +lean_ctor_set(x_7, 1, x_4); +lean_ctor_set(x_7, 2, x_6); +x_8 = l_Substring_dropPrefix_x3f(x_5, x_7); +return x_8; } } LEAN_EXPORT lean_object* l_String_dropSuffix_x3f(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_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; x_3 = lean_string_utf8_byte_size(x_1); x_4 = lean_unsigned_to_nat(0u); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_1); lean_ctor_set(x_5, 1, x_4); lean_ctor_set(x_5, 2, x_3); -x_6 = l_Substring_dropSuffix_x3f(x_5, x_2); -return x_6; +x_6 = lean_string_utf8_byte_size(x_2); +x_7 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_7, 0, x_2); +lean_ctor_set(x_7, 1, x_4); +lean_ctor_set(x_7, 2, x_6); +x_8 = l_Substring_dropSuffix_x3f(x_5, x_7); +return x_8; } } LEAN_EXPORT lean_object* l_String_stripPrefix(lean_object* x_1, lean_object* x_2) { diff --git a/stage0/stdlib/Init/Data/Sum.c b/stage0/stdlib/Init/Data/Sum.c index a7f39344c8b0..b8a0e444fc3a 100644 --- a/stage0/stdlib/Init/Data/Sum.c +++ b/stage0/stdlib/Init/Data/Sum.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Data.Sum -// Imports: Init.Core +// Imports: Init.Data.Sum.Basic Init.Data.Sum.Lemmas #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -13,268 +13,17 @@ #ifdef __cplusplus extern "C" { #endif -LEAN_EXPORT lean_object* l_Sum_getRight_x3f(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_decEqSum____x40_Init_Data_Sum___hyg_4____rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Sum_getLeft_x3f(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Sum_getRight_x3f___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Sum_instDecidableEq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_decEqSum____x40_Init_Data_Sum___hyg_4_(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Sum_getLeft_x3f___rarg(lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242_(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Sum_instBEq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Sum_instBEq___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Sum_instDecidableEq___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_decEqSum____x40_Init_Data_Sum___hyg_4____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -if (lean_obj_tag(x_3) == 0) -{ -lean_dec(x_2); -if (lean_obj_tag(x_4) == 0) -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_5 = lean_ctor_get(x_3, 0); -lean_inc(x_5); -lean_dec(x_3); -x_6 = lean_ctor_get(x_4, 0); -lean_inc(x_6); -lean_dec(x_4); -x_7 = lean_apply_2(x_1, x_5, x_6); -return x_7; -} -else -{ -uint8_t x_8; lean_object* x_9; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_8 = 0; -x_9 = lean_box(x_8); -return x_9; -} -} -else -{ -lean_dec(x_1); -if (lean_obj_tag(x_4) == 0) -{ -uint8_t x_10; lean_object* x_11; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_10 = 0; -x_11 = lean_box(x_10); -return x_11; -} -else -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_3, 0); -lean_inc(x_12); -lean_dec(x_3); -x_13 = lean_ctor_get(x_4, 0); -lean_inc(x_13); -lean_dec(x_4); -x_14 = lean_apply_2(x_2, x_12, x_13); -return x_14; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_decEqSum____x40_Init_Data_Sum___hyg_4_(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Sum_0__Sum_decEqSum____x40_Init_Data_Sum___hyg_4____rarg), 4, 0); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Sum_instDecidableEq___rarg(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_Init_Data_Sum_0__Sum_decEqSum____x40_Init_Data_Sum___hyg_4____rarg(x_1, x_2, x_3, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Sum_instDecidableEq(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Sum_instDecidableEq___rarg), 4, 0); -return x_3; -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -if (lean_obj_tag(x_3) == 0) -{ -lean_dec(x_2); -if (lean_obj_tag(x_4) == 0) -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_5 = lean_ctor_get(x_3, 0); -lean_inc(x_5); -lean_dec(x_3); -x_6 = lean_ctor_get(x_4, 0); -lean_inc(x_6); -lean_dec(x_4); -x_7 = lean_apply_2(x_1, x_5, x_6); -return x_7; -} -else -{ -uint8_t x_8; lean_object* x_9; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_8 = 0; -x_9 = lean_box(x_8); -return x_9; -} -} -else -{ -lean_dec(x_1); -if (lean_obj_tag(x_4) == 0) -{ -uint8_t x_10; lean_object* x_11; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_10 = 0; -x_11 = lean_box(x_10); -return x_11; -} -else -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_3, 0); -lean_inc(x_12); -lean_dec(x_3); -x_13 = lean_ctor_get(x_4, 0); -lean_inc(x_13); -lean_dec(x_4); -x_14 = lean_apply_2(x_2, x_12, x_13); -return x_14; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242_(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____rarg), 4, 0); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Sum_instBEq___rarg(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____rarg), 4, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Sum_instBEq(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Sum_instBEq___rarg), 2, 0); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Sum_getLeft_x3f___rarg(lean_object* x_1) { -_start: -{ -if (lean_obj_tag(x_1) == 0) -{ -uint8_t x_2; -x_2 = !lean_is_exclusive(x_1); -if (x_2 == 0) -{ -lean_ctor_set_tag(x_1, 1); -return x_1; -} -else -{ -lean_object* x_3; lean_object* x_4; -x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); -lean_dec(x_1); -x_4 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_4, 0, x_3); -return x_4; -} -} -else -{ -lean_object* x_5; -lean_dec(x_1); -x_5 = lean_box(0); -return x_5; -} -} -} -LEAN_EXPORT lean_object* l_Sum_getLeft_x3f(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Sum_getLeft_x3f___rarg), 1, 0); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Sum_getRight_x3f___rarg(lean_object* x_1) { -_start: -{ -if (lean_obj_tag(x_1) == 0) -{ -lean_object* x_2; -lean_dec(x_1); -x_2 = lean_box(0); -return x_2; -} -else -{ -uint8_t x_3; -x_3 = !lean_is_exclusive(x_1); -if (x_3 == 0) -{ -return x_1; -} -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_alloc_ctor(1, 1, 0); -lean_ctor_set(x_5, 0, x_4); -return x_5; -} -} -} -} -LEAN_EXPORT lean_object* l_Sum_getRight_x3f(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Sum_getRight_x3f___rarg), 1, 0); -return x_3; -} -} -lean_object* initialize_Init_Core(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_Sum_Basic(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_Sum_Lemmas(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_Data_Sum(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()); +res = initialize_Init_Data_Sum_Basic(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Init_Data_Sum_Lemmas(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)); diff --git a/stage0/stdlib/Init/Data/Sum/Basic.c b/stage0/stdlib/Init/Data/Sum/Basic.c new file mode 100644 index 000000000000..60e8434ccdb1 --- /dev/null +++ b/stage0/stdlib/Init/Data/Sum/Basic.c @@ -0,0 +1,676 @@ +// Lean compiler output +// Module: Init.Data.Sum.Basic +// Imports: Init.PropLemmas +#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___private_Init_Data_Sum_Basic_0__Sum_decEqSum____x40_Init_Data_Sum_Basic___hyg_5_(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_isRight(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_swap(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_getRight_x3f(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_map___rarg___lambda__1(lean_object*); +LEAN_EXPORT lean_object* l_Sum_map(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_getRight___rarg___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_getLeft(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_getLeft_x3f(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_map___rarg___lambda__2(lean_object*); +LEAN_EXPORT lean_object* l_Sum_getRight_x3f___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Sum_instDecidableLiftRel(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_instDecidableEq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_isLeft___rarg___boxed(lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243_(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_getRight(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_map___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_swap___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Sum_elim___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_getLeft_x3f___rarg(lean_object*); +static lean_object* l_Sum_map___rarg___closed__1; +LEAN_EXPORT uint8_t l_Sum_isLeft___rarg(lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_decEqSum____x40_Init_Data_Sum_Basic___hyg_5____rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_instDecidableLiftRel___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_isRight___rarg___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Sum_getLeft___rarg___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_instDecidableRelSumLex___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_instDecidableRelSumLex(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_isLeft(lean_object*, lean_object*); +lean_object* l_Function_comp___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_instBEq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_instBEq___rarg(lean_object*, lean_object*); +static lean_object* l_Sum_map___rarg___closed__2; +LEAN_EXPORT uint8_t l_Sum_isRight___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Sum_instDecidableEq___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_getRight___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_elim(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Sum_getLeft___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_decEqSum____x40_Init_Data_Sum_Basic___hyg_5____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_dec(x_2); +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_ctor_get(x_4, 0); +lean_inc(x_6); +lean_dec(x_4); +x_7 = lean_apply_2(x_1, x_5, x_6); +return x_7; +} +else +{ +uint8_t x_8; lean_object* x_9; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_8 = 0; +x_9 = lean_box(x_8); +return x_9; +} +} +else +{ +lean_dec(x_1); +if (lean_obj_tag(x_4) == 0) +{ +uint8_t x_10; lean_object* x_11; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_10 = 0; +x_11 = lean_box(x_10); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_3, 0); +lean_inc(x_12); +lean_dec(x_3); +x_13 = lean_ctor_get(x_4, 0); +lean_inc(x_13); +lean_dec(x_4); +x_14 = lean_apply_2(x_2, x_12, x_13); +return x_14; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_decEqSum____x40_Init_Data_Sum_Basic___hyg_5_(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Sum_Basic_0__Sum_decEqSum____x40_Init_Data_Sum_Basic___hyg_5____rarg), 4, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_instDecidableEq___rarg(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_Init_Data_Sum_Basic_0__Sum_decEqSum____x40_Init_Data_Sum_Basic___hyg_5____rarg(x_1, x_2, x_3, x_4); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Sum_instDecidableEq(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Sum_instDecidableEq___rarg), 4, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_dec(x_2); +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_ctor_get(x_4, 0); +lean_inc(x_6); +lean_dec(x_4); +x_7 = lean_apply_2(x_1, x_5, x_6); +return x_7; +} +else +{ +uint8_t x_8; lean_object* x_9; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_8 = 0; +x_9 = lean_box(x_8); +return x_9; +} +} +else +{ +lean_dec(x_1); +if (lean_obj_tag(x_4) == 0) +{ +uint8_t x_10; lean_object* x_11; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_10 = 0; +x_11 = lean_box(x_10); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_3, 0); +lean_inc(x_12); +lean_dec(x_3); +x_13 = lean_ctor_get(x_4, 0); +lean_inc(x_13); +lean_dec(x_4); +x_14 = lean_apply_2(x_2, x_12, x_13); +return x_14; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243_(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____rarg), 4, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_instBEq___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____rarg), 4, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_instBEq(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Sum_instBEq___rarg), 2, 0); +return x_3; +} +} +LEAN_EXPORT uint8_t l_Sum_isLeft___rarg(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +uint8_t x_2; +x_2 = 1; +return x_2; +} +else +{ +uint8_t x_3; +x_3 = 0; +return x_3; +} +} +} +LEAN_EXPORT lean_object* l_Sum_isLeft(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Sum_isLeft___rarg___boxed), 1, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_isLeft___rarg___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l_Sum_isLeft___rarg(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT uint8_t l_Sum_isRight___rarg(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +uint8_t x_2; +x_2 = 0; +return x_2; +} +else +{ +uint8_t x_3; +x_3 = 1; +return x_3; +} +} +} +LEAN_EXPORT lean_object* l_Sum_isRight(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Sum_isRight___rarg___boxed), 1, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_isRight___rarg___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l_Sum_isRight___rarg(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_getLeft___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_getLeft(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Sum_getLeft___rarg___boxed), 2, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_getLeft___rarg___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Sum_getLeft___rarg(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_getRight___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_getRight(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Sum_getRight___rarg___boxed), 2, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_getRight___rarg___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Sum_getRight___rarg(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_getLeft_x3f___rarg(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +uint8_t x_2; +x_2 = !lean_is_exclusive(x_1); +if (x_2 == 0) +{ +lean_ctor_set_tag(x_1, 1); +return x_1; +} +else +{ +lean_object* x_3; lean_object* x_4; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +lean_dec(x_1); +x_4 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_4, 0, x_3); +return x_4; +} +} +else +{ +lean_object* x_5; +lean_dec(x_1); +x_5 = lean_box(0); +return x_5; +} +} +} +LEAN_EXPORT lean_object* l_Sum_getLeft_x3f(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Sum_getLeft_x3f___rarg), 1, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_getRight_x3f___rarg(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_2; +lean_dec(x_1); +x_2 = lean_box(0); +return x_2; +} +else +{ +uint8_t x_3; +x_3 = !lean_is_exclusive(x_1); +if (x_3 == 0) +{ +return x_1; +} +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_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_4); +return x_5; +} +} +} +} +LEAN_EXPORT lean_object* l_Sum_getRight_x3f(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Sum_getRight_x3f___rarg), 1, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_elim___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_object* x_5; +lean_dec(x_2); +x_4 = lean_ctor_get(x_3, 0); +lean_inc(x_4); +lean_dec(x_3); +x_5 = lean_apply_1(x_1, x_4); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_1); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_dec(x_3); +x_7 = lean_apply_1(x_2, x_6); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l_Sum_elim(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_alloc_closure((void*)(l_Sum_elim___rarg), 3, 0); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Sum_map___rarg___lambda__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Sum_map___rarg___lambda__2(lean_object* x_1) { +_start: +{ +lean_object* x_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_Sum_map___rarg___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Sum_map___rarg___lambda__1), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Sum_map___rarg___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Sum_map___rarg___lambda__2), 1, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Sum_map___rarg(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; +x_4 = l_Sum_map___rarg___closed__1; +x_5 = lean_alloc_closure((void*)(l_Function_comp___rarg), 3, 2); +lean_closure_set(x_5, 0, x_4); +lean_closure_set(x_5, 1, x_1); +x_6 = l_Sum_map___rarg___closed__2; +x_7 = lean_alloc_closure((void*)(l_Function_comp___rarg), 3, 2); +lean_closure_set(x_7, 0, x_6); +lean_closure_set(x_7, 1, x_2); +x_8 = l_Sum_elim___rarg(x_5, x_7, x_3); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Sum_map(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_Sum_map___rarg), 3, 0); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Sum_swap___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_2 = l_Sum_map___rarg___closed__2; +x_3 = l_Sum_map___rarg___closed__1; +x_4 = l_Sum_elim___rarg(x_2, x_3, x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Sum_swap(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Sum_swap___rarg), 1, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Sum_instDecidableLiftRel___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_dec(x_2); +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_ctor_get(x_4, 0); +lean_inc(x_6); +lean_dec(x_4); +x_7 = lean_apply_2(x_1, x_5, x_6); +return x_7; +} +else +{ +uint8_t x_8; lean_object* x_9; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_8 = 0; +x_9 = lean_box(x_8); +return x_9; +} +} +else +{ +lean_dec(x_1); +if (lean_obj_tag(x_4) == 0) +{ +uint8_t x_10; lean_object* x_11; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_10 = 0; +x_11 = lean_box(x_10); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_3, 0); +lean_inc(x_12); +lean_dec(x_3); +x_13 = lean_ctor_get(x_4, 0); +lean_inc(x_13); +lean_dec(x_4); +x_14 = lean_apply_2(x_2, x_12, x_13); +return x_14; +} +} +} +} +LEAN_EXPORT lean_object* l_Sum_instDecidableLiftRel(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_closure((void*)(l_Sum_instDecidableLiftRel___rarg), 4, 0); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Sum_instDecidableRelSumLex___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_dec(x_2); +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_ctor_get(x_4, 0); +lean_inc(x_6); +lean_dec(x_4); +x_7 = lean_apply_2(x_1, x_5, x_6); +return x_7; +} +else +{ +uint8_t x_8; lean_object* x_9; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_8 = 1; +x_9 = lean_box(x_8); +return x_9; +} +} +else +{ +lean_dec(x_1); +if (lean_obj_tag(x_4) == 0) +{ +uint8_t x_10; lean_object* x_11; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_10 = 0; +x_11 = lean_box(x_10); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_3, 0); +lean_inc(x_12); +lean_dec(x_3); +x_13 = lean_ctor_get(x_4, 0); +lean_inc(x_13); +lean_dec(x_4); +x_14 = lean_apply_2(x_2, x_12, x_13); +return x_14; +} +} +} +} +LEAN_EXPORT lean_object* l_Sum_instDecidableRelSumLex(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_Sum_instDecidableRelSumLex___rarg), 4, 0); +return x_5; +} +} +lean_object* initialize_Init_PropLemmas(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Init_Data_Sum_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_PropLemmas(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Sum_map___rarg___closed__1 = _init_l_Sum_map___rarg___closed__1(); +lean_mark_persistent(l_Sum_map___rarg___closed__1); +l_Sum_map___rarg___closed__2 = _init_l_Sum_map___rarg___closed__2(); +lean_mark_persistent(l_Sum_map___rarg___closed__2); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Init/Data/Sum/Lemmas.c b/stage0/stdlib/Init/Data/Sum/Lemmas.c new file mode 100644 index 000000000000..5bd791f44fd4 --- /dev/null +++ b/stage0/stdlib/Init/Data/Sum/Lemmas.c @@ -0,0 +1,103 @@ +// Lean compiler output +// Module: Init.Data.Sum.Lemmas +// Imports: Init.Data.Sum.Basic Init.Ext +#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___private_Init_Data_Sum_Lemmas_0__Sum_getRight_x3f_match__1_splitter(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Lemmas_0__Sum_isLeft_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Lemmas_0__Sum_getRight_x3f_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Lemmas_0__Sum_isLeft_match__1_splitter(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Lemmas_0__Sum_isLeft_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_object* x_4; lean_object* x_5; +lean_dec(x_3); +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_apply_1(x_2, x_4); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_2); +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_apply_1(x_3, x_6); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Lemmas_0__Sum_isLeft_match__1_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_Init_Data_Sum_Lemmas_0__Sum_isLeft_match__1_splitter___rarg), 3, 0); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Lemmas_0__Sum_getRight_x3f_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_object* x_4; lean_object* x_5; +lean_dec(x_2); +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; +} +else +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_3); +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_apply_1(x_2, x_6); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Lemmas_0__Sum_getRight_x3f_match__1_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_Init_Data_Sum_Lemmas_0__Sum_getRight_x3f_match__1_splitter___rarg), 3, 0); +return x_4; +} +} +lean_object* initialize_Init_Data_Sum_Basic(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Ext(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Init_Data_Sum_Lemmas(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_Data_Sum_Basic(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Init_Ext(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/Init/Data/UInt/Lemmas.c b/stage0/stdlib/Init/Data/UInt/Lemmas.c index 227d1f866b53..7f700bb493ec 100644 --- a/stage0/stdlib/Init/Data/UInt/Lemmas.c +++ b/stage0/stdlib/Init/Data/UInt/Lemmas.c @@ -82,6 +82,7 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__179; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__356; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__442; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__515; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__353; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__24; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__190; @@ -99,9 +100,11 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__504; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__189; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__192; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__524; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__134; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__46; static lean_object* l_commandDeclare__uint__theorems_____closed__9; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__518; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__202; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__368; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__309; @@ -227,7 +230,9 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__100; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__425; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__108; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__512; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__341; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__507; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__80; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__416; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__473; @@ -241,6 +246,7 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__62; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__54; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__453; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__522; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__175; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__278; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__333; @@ -252,6 +258,7 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__139; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__355; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__43; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__510; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__437; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__66; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__57; @@ -293,6 +300,7 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__237; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__424; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__17; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__511; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__338; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__29; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__115; @@ -300,10 +308,12 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__432; static lean_object* l_commandDeclare__uint__theorems_____closed__6; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__509; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__295; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__55; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__495; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__77; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__505; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__114; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__307; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__92; @@ -341,8 +351,10 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__489; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__409; LEAN_EXPORT lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1(lean_object*, lean_object*, lean_object*); +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__519; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__185; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__394; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__506; static lean_object* l_commandDeclare__uint__theorems_____closed__2; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__397; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__301; @@ -409,12 +421,14 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__75; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__222; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__516; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__122; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__212; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__73; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__328; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__176; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__369; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__513; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__188; lean_object* l_Lean_Syntax_node7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__344; @@ -444,6 +458,7 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__131; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__106; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__438; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__525; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__161; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__476; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__314; @@ -453,8 +468,10 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__229; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__197; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__474; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__521; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__383; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__388; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__520; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__444; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__121; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__457; @@ -488,7 +505,9 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__27; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__198; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__195; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__523; lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__514; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__402; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__396; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__289; @@ -508,9 +527,11 @@ static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDe static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__349; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__155; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__332; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__517; LEAN_EXPORT uint8_t l_UInt8_instInhabited; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__20; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__249; +static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__508; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__299; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__231; static lean_object* l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__311; @@ -5251,18 +5272,208 @@ static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__com _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("end", 3, 3); +x_1 = lean_mk_string_unchecked("val_ofNat", 9, 9); return x_1; } } static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__504() { _start: { +lean_object* x_1; lean_object* x_2; +x_1 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__503; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__505() { +_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__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__503; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__506() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("noindex", 7, 7); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__507() { +_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__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__3; +x_2 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__4; +x_3 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__15; +x_4 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__506; +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__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__508() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("no_index", 8, 8); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__509() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("OfNat.ofNat", 11, 11); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__510() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__509; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__511() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("OfNat", 5, 5); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__512() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__511; +x_2 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__168; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__513() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("toBitVec_ofNat", 14, 14); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__514() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__513; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__515() { +_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__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__513; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__516() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__90; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__517() { +_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__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__90; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__518() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("BitVec.ofNat", 12, 12); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__519() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__518; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__520() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__249; +x_2 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__168; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__521() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mk_ofNat", 8, 8); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__522() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__521; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__523() { +_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__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__521; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__524() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("end", 3, 3); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__525() { +_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__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__3; x_2 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__4; x_3 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__5; -x_4 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__503; +x_4 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__524; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -5286,7 +5497,7 @@ return x_7; } else { -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_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; 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; 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; lean_object* x_463; lean_object* x_464; 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; 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; 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; lean_object* x_487; lean_object* x_488; lean_object* x_489; 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; 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; lean_object* x_504; lean_object* x_505; 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; lean_object* x_513; lean_object* x_514; lean_object* x_515; 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; 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; lean_object* x_530; lean_object* x_531; lean_object* x_532; lean_object* x_533; lean_object* x_534; lean_object* x_535; 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; lean_object* x_544; lean_object* x_545; lean_object* x_546; lean_object* x_547; lean_object* x_548; lean_object* x_549; lean_object* x_550; lean_object* x_551; lean_object* x_552; lean_object* x_553; lean_object* x_554; lean_object* x_555; lean_object* x_556; lean_object* x_557; lean_object* x_558; lean_object* x_559; lean_object* x_560; lean_object* x_561; lean_object* x_562; 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; 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; 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; 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; 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; lean_object* x_599; lean_object* x_600; lean_object* x_601; lean_object* x_602; lean_object* x_603; lean_object* x_604; lean_object* x_605; 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; lean_object* x_613; lean_object* x_614; lean_object* x_615; 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; lean_object* x_623; 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; lean_object* x_631; lean_object* x_632; 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; lean_object* x_640; lean_object* x_641; 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; lean_object* x_649; lean_object* x_650; lean_object* x_651; lean_object* x_652; lean_object* x_653; 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; lean_object* x_661; 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; lean_object* x_669; lean_object* x_670; lean_object* x_671; lean_object* x_672; lean_object* x_673; lean_object* x_674; lean_object* x_675; lean_object* x_676; 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_object* x_683; lean_object* x_684; lean_object* x_685; lean_object* x_686; lean_object* x_687; lean_object* x_688; 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_object* x_696; lean_object* x_697; lean_object* x_698; lean_object* x_699; lean_object* x_700; 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_object* x_707; lean_object* x_708; lean_object* x_709; lean_object* x_710; lean_object* x_711; lean_object* x_712; 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; lean_object* x_720; 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; lean_object* x_728; 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_object* x_735; lean_object* x_736; lean_object* x_737; lean_object* x_738; lean_object* x_739; 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; lean_object* x_747; lean_object* x_748; lean_object* x_749; lean_object* x_750; 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; lean_object* x_758; 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; lean_object* x_766; lean_object* x_767; lean_object* x_768; lean_object* x_769; lean_object* x_770; lean_object* x_771; lean_object* x_772; lean_object* x_773; lean_object* x_774; lean_object* x_775; lean_object* x_776; lean_object* x_777; lean_object* x_778; lean_object* x_779; lean_object* x_780; lean_object* x_781; lean_object* x_782; lean_object* x_783; lean_object* x_784; lean_object* x_785; lean_object* x_786; lean_object* x_787; lean_object* x_788; lean_object* x_789; lean_object* x_790; lean_object* x_791; lean_object* x_792; lean_object* x_793; lean_object* x_794; lean_object* x_795; lean_object* x_796; 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; lean_object* x_804; lean_object* x_805; lean_object* x_806; lean_object* x_807; 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_object* x_814; lean_object* x_815; 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; lean_object* x_823; 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; lean_object* x_831; lean_object* x_832; 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; lean_object* x_840; lean_object* x_841; 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; lean_object* x_849; lean_object* x_850; lean_object* x_851; lean_object* x_852; lean_object* x_853; 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; lean_object* x_861; 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; 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; lean_object* x_876; lean_object* x_877; lean_object* x_878; lean_object* x_879; lean_object* x_880; lean_object* x_881; lean_object* x_882; lean_object* x_883; 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; 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; 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; 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; lean_object* x_912; lean_object* x_913; lean_object* x_914; lean_object* x_915; lean_object* x_916; lean_object* x_917; lean_object* x_918; lean_object* x_919; 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; 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; lean_object* x_934; lean_object* x_935; lean_object* x_936; lean_object* x_937; lean_object* x_938; lean_object* x_939; lean_object* x_940; 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; lean_object* x_948; lean_object* x_949; lean_object* x_950; lean_object* x_951; 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; lean_object* x_959; lean_object* x_960; lean_object* x_961; lean_object* x_962; 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; lean_object* x_970; 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; lean_object* x_978; lean_object* x_979; lean_object* x_980; lean_object* x_981; lean_object* x_982; lean_object* x_983; lean_object* x_984; lean_object* x_985; lean_object* x_986; lean_object* x_987; lean_object* x_988; lean_object* x_989; lean_object* x_990; lean_object* x_991; 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; 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; lean_object* x_1006; lean_object* x_1007; lean_object* x_1008; lean_object* x_1009; lean_object* x_1010; lean_object* x_1011; lean_object* x_1012; 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; lean_object* x_1020; lean_object* x_1021; lean_object* x_1022; lean_object* x_1023; lean_object* x_1024; lean_object* x_1025; lean_object* x_1026; lean_object* x_1027; lean_object* x_1028; lean_object* x_1029; lean_object* x_1030; lean_object* x_1031; lean_object* x_1032; lean_object* x_1033; 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; 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; 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; lean_object* x_1055; lean_object* x_1056; lean_object* x_1057; lean_object* x_1058; lean_object* x_1059; lean_object* x_1060; lean_object* x_1061; lean_object* x_1062; lean_object* x_1063; lean_object* x_1064; lean_object* x_1065; lean_object* x_1066; lean_object* x_1067; 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; lean_object* x_1075; lean_object* x_1076; lean_object* x_1077; lean_object* x_1078; lean_object* x_1079; lean_object* x_1080; lean_object* x_1081; lean_object* x_1082; lean_object* x_1083; lean_object* x_1084; lean_object* x_1085; lean_object* x_1086; lean_object* x_1087; lean_object* x_1088; lean_object* x_1089; lean_object* x_1090; lean_object* x_1091; lean_object* x_1092; lean_object* x_1093; lean_object* x_1094; lean_object* x_1095; lean_object* x_1096; lean_object* x_1097; lean_object* x_1098; lean_object* x_1099; lean_object* x_1100; lean_object* x_1101; lean_object* x_1102; lean_object* x_1103; lean_object* x_1104; lean_object* x_1105; lean_object* x_1106; lean_object* x_1107; lean_object* x_1108; lean_object* x_1109; lean_object* x_1110; lean_object* x_1111; lean_object* x_1112; lean_object* x_1113; lean_object* x_1114; lean_object* x_1115; lean_object* x_1116; lean_object* x_1117; lean_object* x_1118; lean_object* x_1119; lean_object* x_1120; lean_object* x_1121; lean_object* x_1122; lean_object* x_1123; lean_object* x_1124; lean_object* x_1125; lean_object* x_1126; lean_object* x_1127; lean_object* x_1128; lean_object* x_1129; lean_object* x_1130; lean_object* x_1131; lean_object* x_1132; lean_object* x_1133; lean_object* x_1134; lean_object* x_1135; lean_object* x_1136; lean_object* x_1137; lean_object* x_1138; lean_object* x_1139; lean_object* x_1140; lean_object* x_1141; lean_object* x_1142; lean_object* x_1143; lean_object* x_1144; lean_object* x_1145; lean_object* x_1146; lean_object* x_1147; lean_object* x_1148; lean_object* x_1149; lean_object* x_1150; lean_object* x_1151; lean_object* x_1152; lean_object* x_1153; lean_object* x_1154; lean_object* x_1155; lean_object* x_1156; lean_object* x_1157; lean_object* x_1158; lean_object* x_1159; lean_object* x_1160; lean_object* x_1161; lean_object* x_1162; lean_object* x_1163; lean_object* x_1164; lean_object* x_1165; lean_object* x_1166; lean_object* x_1167; lean_object* x_1168; lean_object* x_1169; lean_object* x_1170; lean_object* x_1171; lean_object* x_1172; lean_object* x_1173; +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_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; 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; 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; lean_object* x_463; lean_object* x_464; 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; 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; 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; lean_object* x_487; lean_object* x_488; lean_object* x_489; 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; 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; lean_object* x_504; lean_object* x_505; 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; lean_object* x_513; lean_object* x_514; lean_object* x_515; 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; 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; lean_object* x_530; lean_object* x_531; lean_object* x_532; lean_object* x_533; lean_object* x_534; lean_object* x_535; 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; lean_object* x_544; lean_object* x_545; lean_object* x_546; lean_object* x_547; lean_object* x_548; lean_object* x_549; lean_object* x_550; lean_object* x_551; lean_object* x_552; lean_object* x_553; lean_object* x_554; lean_object* x_555; lean_object* x_556; lean_object* x_557; lean_object* x_558; lean_object* x_559; lean_object* x_560; lean_object* x_561; lean_object* x_562; 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; 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; 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; 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; 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; lean_object* x_599; lean_object* x_600; lean_object* x_601; lean_object* x_602; lean_object* x_603; lean_object* x_604; lean_object* x_605; 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; lean_object* x_613; lean_object* x_614; lean_object* x_615; 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; lean_object* x_623; 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; lean_object* x_631; lean_object* x_632; 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; lean_object* x_640; lean_object* x_641; 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; lean_object* x_649; lean_object* x_650; lean_object* x_651; lean_object* x_652; lean_object* x_653; 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; lean_object* x_661; 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; lean_object* x_669; lean_object* x_670; lean_object* x_671; lean_object* x_672; lean_object* x_673; lean_object* x_674; lean_object* x_675; lean_object* x_676; 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_object* x_683; lean_object* x_684; lean_object* x_685; lean_object* x_686; lean_object* x_687; lean_object* x_688; 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_object* x_696; lean_object* x_697; lean_object* x_698; lean_object* x_699; lean_object* x_700; 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_object* x_707; lean_object* x_708; lean_object* x_709; lean_object* x_710; lean_object* x_711; lean_object* x_712; 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; lean_object* x_720; 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; lean_object* x_728; 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_object* x_735; lean_object* x_736; lean_object* x_737; lean_object* x_738; lean_object* x_739; 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; lean_object* x_747; lean_object* x_748; lean_object* x_749; lean_object* x_750; 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; lean_object* x_758; 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; lean_object* x_766; lean_object* x_767; lean_object* x_768; lean_object* x_769; lean_object* x_770; lean_object* x_771; lean_object* x_772; lean_object* x_773; lean_object* x_774; lean_object* x_775; lean_object* x_776; lean_object* x_777; lean_object* x_778; lean_object* x_779; lean_object* x_780; lean_object* x_781; lean_object* x_782; lean_object* x_783; lean_object* x_784; lean_object* x_785; lean_object* x_786; lean_object* x_787; lean_object* x_788; lean_object* x_789; lean_object* x_790; lean_object* x_791; lean_object* x_792; lean_object* x_793; lean_object* x_794; lean_object* x_795; lean_object* x_796; 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; lean_object* x_804; lean_object* x_805; lean_object* x_806; lean_object* x_807; 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_object* x_814; lean_object* x_815; 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; lean_object* x_823; 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; lean_object* x_831; lean_object* x_832; 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; lean_object* x_840; lean_object* x_841; 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; lean_object* x_849; lean_object* x_850; lean_object* x_851; lean_object* x_852; lean_object* x_853; 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; lean_object* x_861; 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; 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; lean_object* x_876; lean_object* x_877; lean_object* x_878; lean_object* x_879; lean_object* x_880; lean_object* x_881; lean_object* x_882; lean_object* x_883; 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; 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; 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; 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; lean_object* x_912; lean_object* x_913; lean_object* x_914; lean_object* x_915; lean_object* x_916; lean_object* x_917; lean_object* x_918; lean_object* x_919; 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; 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; lean_object* x_934; lean_object* x_935; lean_object* x_936; lean_object* x_937; lean_object* x_938; lean_object* x_939; lean_object* x_940; 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; lean_object* x_948; lean_object* x_949; lean_object* x_950; lean_object* x_951; 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; lean_object* x_959; lean_object* x_960; lean_object* x_961; lean_object* x_962; 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; lean_object* x_970; 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; lean_object* x_978; lean_object* x_979; lean_object* x_980; lean_object* x_981; lean_object* x_982; lean_object* x_983; lean_object* x_984; lean_object* x_985; lean_object* x_986; lean_object* x_987; lean_object* x_988; lean_object* x_989; lean_object* x_990; lean_object* x_991; 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; 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; lean_object* x_1006; lean_object* x_1007; lean_object* x_1008; lean_object* x_1009; lean_object* x_1010; lean_object* x_1011; lean_object* x_1012; 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; lean_object* x_1020; lean_object* x_1021; lean_object* x_1022; lean_object* x_1023; lean_object* x_1024; lean_object* x_1025; lean_object* x_1026; lean_object* x_1027; lean_object* x_1028; lean_object* x_1029; lean_object* x_1030; lean_object* x_1031; lean_object* x_1032; lean_object* x_1033; 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; 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; 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; lean_object* x_1055; lean_object* x_1056; lean_object* x_1057; lean_object* x_1058; lean_object* x_1059; lean_object* x_1060; lean_object* x_1061; lean_object* x_1062; lean_object* x_1063; lean_object* x_1064; lean_object* x_1065; lean_object* x_1066; lean_object* x_1067; 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; lean_object* x_1075; lean_object* x_1076; lean_object* x_1077; lean_object* x_1078; lean_object* x_1079; lean_object* x_1080; lean_object* x_1081; lean_object* x_1082; lean_object* x_1083; lean_object* x_1084; lean_object* x_1085; lean_object* x_1086; lean_object* x_1087; lean_object* x_1088; lean_object* x_1089; lean_object* x_1090; lean_object* x_1091; lean_object* x_1092; lean_object* x_1093; lean_object* x_1094; lean_object* x_1095; lean_object* x_1096; lean_object* x_1097; lean_object* x_1098; lean_object* x_1099; lean_object* x_1100; lean_object* x_1101; lean_object* x_1102; lean_object* x_1103; lean_object* x_1104; lean_object* x_1105; lean_object* x_1106; lean_object* x_1107; lean_object* x_1108; lean_object* x_1109; lean_object* x_1110; lean_object* x_1111; lean_object* x_1112; lean_object* x_1113; lean_object* x_1114; lean_object* x_1115; lean_object* x_1116; lean_object* x_1117; lean_object* x_1118; lean_object* x_1119; lean_object* x_1120; lean_object* x_1121; lean_object* x_1122; lean_object* x_1123; lean_object* x_1124; lean_object* x_1125; lean_object* x_1126; lean_object* x_1127; lean_object* x_1128; lean_object* x_1129; lean_object* x_1130; lean_object* x_1131; lean_object* x_1132; lean_object* x_1133; lean_object* x_1134; lean_object* x_1135; lean_object* x_1136; lean_object* x_1137; lean_object* x_1138; lean_object* x_1139; lean_object* x_1140; lean_object* x_1141; lean_object* x_1142; lean_object* x_1143; lean_object* x_1144; lean_object* x_1145; lean_object* x_1146; lean_object* x_1147; lean_object* x_1148; lean_object* x_1149; lean_object* x_1150; lean_object* x_1151; lean_object* x_1152; lean_object* x_1153; lean_object* x_1154; lean_object* x_1155; lean_object* x_1156; lean_object* x_1157; lean_object* x_1158; lean_object* x_1159; lean_object* x_1160; lean_object* x_1161; lean_object* x_1162; lean_object* x_1163; lean_object* x_1164; lean_object* x_1165; lean_object* x_1166; lean_object* x_1167; lean_object* x_1168; lean_object* x_1169; lean_object* x_1170; lean_object* x_1171; lean_object* x_1172; lean_object* x_1173; lean_object* x_1174; lean_object* x_1175; lean_object* x_1176; lean_object* x_1177; lean_object* x_1178; lean_object* x_1179; lean_object* x_1180; lean_object* x_1181; lean_object* x_1182; lean_object* x_1183; lean_object* x_1184; lean_object* x_1185; lean_object* x_1186; lean_object* x_1187; lean_object* x_1188; lean_object* x_1189; lean_object* x_1190; lean_object* x_1191; lean_object* x_1192; lean_object* x_1193; lean_object* x_1194; lean_object* x_1195; lean_object* x_1196; lean_object* x_1197; lean_object* x_1198; lean_object* x_1199; lean_object* x_1200; lean_object* x_1201; lean_object* x_1202; lean_object* x_1203; lean_object* x_1204; lean_object* x_1205; lean_object* x_1206; lean_object* x_1207; lean_object* x_1208; lean_object* x_1209; lean_object* x_1210; lean_object* x_1211; lean_object* x_1212; lean_object* x_1213; lean_object* x_1214; lean_object* x_1215; lean_object* x_1216; lean_object* x_1217; lean_object* x_1218; lean_object* x_1219; lean_object* x_1220; lean_object* x_1221; lean_object* x_1222; lean_object* x_1223; lean_object* x_1224; lean_object* x_1225; lean_object* x_1226; lean_object* x_1227; lean_object* x_1228; lean_object* x_1229; x_8 = lean_unsigned_to_nat(1u); x_9 = l_Lean_Syntax_getArg(x_1, x_8); lean_dec(x_1); @@ -5878,6 +6089,7 @@ lean_ctor_set(x_223, 3, x_28); lean_inc(x_135); lean_inc(x_12); x_224 = l_Lean_Syntax_node1(x_12, x_17, x_135); +lean_inc(x_223); lean_inc(x_12); x_225 = l_Lean_Syntax_node2(x_12, x_33, x_223, x_224); lean_inc(x_120); @@ -5951,6 +6163,7 @@ x_251 = l_Lean_Syntax_node1(x_12, x_250, x_249); lean_inc(x_64); lean_inc(x_12); x_252 = l_Lean_Syntax_node4(x_12, x_96, x_64, x_213, x_230, x_251); +lean_inc(x_209); lean_inc(x_12); x_253 = l_Lean_Syntax_node2(x_12, x_61, x_209, x_252); x_254 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__146; @@ -6141,6 +6354,7 @@ lean_inc(x_12); x_317 = l_Lean_Syntax_node5(x_12, x_126, x_71, x_314, x_316, x_19, x_73); lean_inc(x_12); x_318 = l_Lean_Syntax_node2(x_12, x_17, x_310, x_317); +lean_inc(x_309); lean_inc(x_280); lean_inc(x_12); x_319 = l_Lean_Syntax_node2(x_12, x_33, x_280, x_309); @@ -6160,6 +6374,7 @@ lean_inc(x_323); lean_inc(x_285); lean_inc(x_12); x_324 = l_Lean_Syntax_node3(x_12, x_289, x_320, x_285, x_323); +lean_inc(x_308); lean_inc(x_77); lean_inc(x_12); x_325 = l_Lean_Syntax_node3(x_12, x_85, x_324, x_77, x_308); @@ -7078,6 +7293,7 @@ lean_ctor_set(x_640, 0, x_12); lean_ctor_set(x_640, 1, x_638); lean_ctor_set(x_640, 2, x_639); lean_ctor_set(x_640, 3, x_28); +lean_inc(x_640); lean_inc_n(x_19, 2); lean_inc(x_12); x_641 = l_Lean_Syntax_node3(x_12, x_404, x_19, x_19, x_640); @@ -7650,6 +7866,7 @@ lean_inc(x_831); lean_inc(x_12); x_832 = l_Lean_Syntax_node1(x_12, x_17, x_831); lean_inc(x_265); +lean_inc(x_263); lean_inc(x_832); lean_inc(x_259); lean_inc(x_12); @@ -7812,6 +8029,7 @@ lean_ctor_set(x_889, 0, x_12); lean_ctor_set(x_889, 1, x_887); lean_ctor_set(x_889, 2, x_888); lean_ctor_set(x_889, 3, x_28); +lean_inc(x_236); lean_inc(x_12); x_890 = l_Lean_Syntax_node2(x_12, x_17, x_236, x_859); lean_inc(x_889); @@ -8030,6 +8248,8 @@ x_972 = l_Lean_Syntax_node1(x_12, x_971, x_873); lean_inc(x_972); lean_inc(x_12); x_973 = l_Lean_Syntax_node3(x_12, x_169, x_972, x_168, x_972); +lean_inc(x_73); +lean_inc(x_71); lean_inc(x_12); x_974 = l_Lean_Syntax_node3(x_12, x_282, x_71, x_973, x_73); lean_inc_n(x_19, 2); @@ -8459,144 +8679,302 @@ lean_inc(x_12); x_1123 = l_Lean_Syntax_node2(x_12, x_68, x_1122, x_19); lean_inc(x_12); x_1124 = l_Lean_Syntax_node2(x_12, x_33, x_280, x_107); +lean_inc(x_77); lean_inc(x_12); x_1125 = l_Lean_Syntax_node3(x_12, x_85, x_1124, x_77, x_105); +lean_inc(x_27); lean_inc(x_12); x_1126 = l_Lean_Syntax_node2(x_12, x_35, x_27, x_1125); +lean_inc(x_19); lean_inc(x_12); x_1127 = l_Lean_Syntax_node2(x_12, x_37, x_19, x_1126); +lean_inc(x_95); +lean_inc(x_64); lean_inc(x_12); x_1128 = l_Lean_Syntax_node4(x_12, x_96, x_64, x_1123, x_1127, x_95); lean_inc(x_12); x_1129 = l_Lean_Syntax_node2(x_12, x_61, x_391, x_1128); -x_1130 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__503; -lean_inc(x_12); -x_1131 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_1131, 0, x_12); -lean_ctor_set(x_1131, 1, x_1130); -x_1132 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__504; -lean_inc(x_12); -x_1133 = l_Lean_Syntax_node2(x_12, x_1132, x_1131, x_32); -x_1134 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1134, 0, x_1133); -lean_ctor_set(x_1134, 1, x_28); -x_1135 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1135, 0, x_1129); -lean_ctor_set(x_1135, 1, x_1134); -x_1136 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1136, 0, x_1119); -lean_ctor_set(x_1136, 1, x_1135); -x_1137 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1137, 0, x_1101); +x_1130 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__504; +x_1131 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__505; +lean_inc(x_12); +x_1132 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_1132, 0, x_12); +lean_ctor_set(x_1132, 1, x_1130); +lean_ctor_set(x_1132, 2, x_1131); +lean_ctor_set(x_1132, 3, x_28); +lean_inc(x_19); +lean_inc(x_12); +x_1133 = l_Lean_Syntax_node2(x_12, x_68, x_1132, x_19); +lean_inc(x_73); +lean_inc(x_19); +lean_inc(x_309); +lean_inc(x_71); +lean_inc(x_12); +x_1134 = l_Lean_Syntax_node5(x_12, x_126, x_71, x_309, x_263, x_19, x_73); +lean_inc(x_12); +x_1135 = l_Lean_Syntax_node1(x_12, x_17, x_1134); +x_1136 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__508; +lean_inc(x_12); +x_1137 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_1137, 0, x_12); lean_ctor_set(x_1137, 1, x_1136); -x_1138 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1138, 0, x_1074); -lean_ctor_set(x_1138, 1, x_1137); -x_1139 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1139, 0, x_925); -lean_ctor_set(x_1139, 1, x_1138); -x_1140 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1140, 0, x_821); -lean_ctor_set(x_1140, 1, x_1139); -x_1141 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1141, 0, x_808); -lean_ctor_set(x_1141, 1, x_1140); -x_1142 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1142, 0, x_791); -lean_ctor_set(x_1142, 1, x_1141); -x_1143 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1143, 0, x_770); -lean_ctor_set(x_1143, 1, x_1142); -x_1144 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1144, 0, x_747); -lean_ctor_set(x_1144, 1, x_1143); -x_1145 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1145, 0, x_731); -lean_ctor_set(x_1145, 1, x_1144); -x_1146 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1146, 0, x_691); -lean_ctor_set(x_1146, 1, x_1145); -x_1147 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1147, 0, x_653); -lean_ctor_set(x_1147, 1, x_1146); -x_1148 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1148, 0, x_587); -lean_ctor_set(x_1148, 1, x_1147); -x_1149 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1149, 0, x_555); -lean_ctor_set(x_1149, 1, x_1148); -x_1150 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1150, 0, x_536); -lean_ctor_set(x_1150, 1, x_1149); -x_1151 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1151, 0, x_522); -lean_ctor_set(x_1151, 1, x_1150); -x_1152 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1152, 0, x_500); -lean_ctor_set(x_1152, 1, x_1151); -x_1153 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1153, 0, x_484); -lean_ctor_set(x_1153, 1, x_1152); -x_1154 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1154, 0, x_461); -lean_ctor_set(x_1154, 1, x_1153); -x_1155 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1155, 0, x_445); -lean_ctor_set(x_1155, 1, x_1154); -x_1156 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1156, 0, x_428); -lean_ctor_set(x_1156, 1, x_1155); -x_1157 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1157, 0, x_417); -lean_ctor_set(x_1157, 1, x_1156); -x_1158 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1158, 0, x_385); -lean_ctor_set(x_1158, 1, x_1157); -x_1159 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1159, 0, x_374); -lean_ctor_set(x_1159, 1, x_1158); -x_1160 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1160, 0, x_352); -lean_ctor_set(x_1160, 1, x_1159); -x_1161 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1161, 0, x_301); -lean_ctor_set(x_1161, 1, x_1160); -x_1162 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1162, 0, x_253); -lean_ctor_set(x_1162, 1, x_1161); -x_1163 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1163, 0, x_194); -lean_ctor_set(x_1163, 1, x_1162); -x_1164 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1164, 0, x_178); -lean_ctor_set(x_1164, 1, x_1163); -x_1165 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1165, 0, x_162); -lean_ctor_set(x_1165, 1, x_1164); -x_1166 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1166, 0, x_146); -lean_ctor_set(x_1166, 1, x_1165); -x_1167 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1167, 0, x_113); -lean_ctor_set(x_1167, 1, x_1166); -x_1168 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1168, 0, x_98); -lean_ctor_set(x_1168, 1, x_1167); -x_1169 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1169, 0, x_62); -lean_ctor_set(x_1169, 1, x_1168); -x_1170 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1170, 0, x_16); -lean_ctor_set(x_1170, 1, x_1169); -x_1171 = lean_array_mk(x_1170); -x_1172 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_1172, 0, x_12); -lean_ctor_set(x_1172, 1, x_17); -lean_ctor_set(x_1172, 2, x_1171); -x_1173 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_1173, 0, x_1172); -lean_ctor_set(x_1173, 1, x_3); -return x_1173; +x_1138 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__510; +x_1139 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__512; +lean_inc(x_12); +x_1140 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_1140, 0, x_12); +lean_ctor_set(x_1140, 1, x_1138); +lean_ctor_set(x_1140, 2, x_1139); +lean_ctor_set(x_1140, 3, x_28); +lean_inc(x_12); +x_1141 = l_Lean_Syntax_node2(x_12, x_33, x_1140, x_309); +lean_inc(x_73); +lean_inc(x_1141); +lean_inc(x_71); +lean_inc(x_12); +x_1142 = l_Lean_Syntax_node3(x_12, x_282, x_71, x_1141, x_73); +x_1143 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__507; +lean_inc(x_12); +x_1144 = l_Lean_Syntax_node2(x_12, x_1143, x_1137, x_1142); +lean_inc(x_73); +lean_inc(x_71); +lean_inc(x_12); +x_1145 = l_Lean_Syntax_node3(x_12, x_282, x_71, x_1144, x_73); +lean_inc(x_12); +x_1146 = l_Lean_Syntax_node1(x_12, x_17, x_1145); +lean_inc(x_1146); +lean_inc(x_12); +x_1147 = l_Lean_Syntax_node2(x_12, x_33, x_640, x_1146); +lean_inc(x_1141); +lean_inc(x_77); +lean_inc(x_12); +x_1148 = l_Lean_Syntax_node3(x_12, x_85, x_1147, x_77, x_1141); +lean_inc(x_27); +lean_inc(x_12); +x_1149 = l_Lean_Syntax_node2(x_12, x_35, x_27, x_1148); +lean_inc(x_1135); +lean_inc(x_12); +x_1150 = l_Lean_Syntax_node2(x_12, x_37, x_1135, x_1149); +lean_inc(x_95); +lean_inc(x_64); +lean_inc(x_12); +x_1151 = l_Lean_Syntax_node4(x_12, x_96, x_64, x_1133, x_1150, x_95); +lean_inc(x_209); +lean_inc(x_12); +x_1152 = l_Lean_Syntax_node2(x_12, x_61, x_209, x_1151); +x_1153 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__514; +x_1154 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__515; +lean_inc(x_12); +x_1155 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_1155, 0, x_12); +lean_ctor_set(x_1155, 1, x_1153); +lean_ctor_set(x_1155, 2, x_1154); +lean_ctor_set(x_1155, 3, x_28); +lean_inc(x_19); +lean_inc(x_12); +x_1156 = l_Lean_Syntax_node2(x_12, x_68, x_1155, x_19); +x_1157 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__516; +x_1158 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__517; +lean_inc(x_12); +x_1159 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_1159, 0, x_12); +lean_ctor_set(x_1159, 1, x_1157); +lean_ctor_set(x_1159, 2, x_1158); +lean_ctor_set(x_1159, 3, x_28); +lean_inc(x_12); +x_1160 = l_Lean_Syntax_node2(x_12, x_33, x_1159, x_1146); +x_1161 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__519; +x_1162 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__520; +lean_inc(x_12); +x_1163 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_1163, 0, x_12); +lean_ctor_set(x_1163, 1, x_1161); +lean_ctor_set(x_1163, 2, x_1162); +lean_ctor_set(x_1163, 3, x_28); +lean_inc(x_12); +x_1164 = l_Lean_Syntax_node2(x_12, x_17, x_236, x_308); +lean_inc(x_12); +x_1165 = l_Lean_Syntax_node2(x_12, x_33, x_1163, x_1164); +lean_inc(x_1165); +lean_inc(x_77); +lean_inc(x_12); +x_1166 = l_Lean_Syntax_node3(x_12, x_85, x_1160, x_77, x_1165); +lean_inc(x_27); +lean_inc(x_12); +x_1167 = l_Lean_Syntax_node2(x_12, x_35, x_27, x_1166); +lean_inc(x_1135); +lean_inc(x_12); +x_1168 = l_Lean_Syntax_node2(x_12, x_37, x_1135, x_1167); +lean_inc(x_95); +lean_inc(x_64); +lean_inc(x_12); +x_1169 = l_Lean_Syntax_node4(x_12, x_96, x_64, x_1156, x_1168, x_95); +lean_inc(x_209); +lean_inc(x_12); +x_1170 = l_Lean_Syntax_node2(x_12, x_61, x_209, x_1169); +x_1171 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__522; +x_1172 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__523; +lean_inc(x_12); +x_1173 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_1173, 0, x_12); +lean_ctor_set(x_1173, 1, x_1171); +lean_ctor_set(x_1173, 2, x_1172); +lean_ctor_set(x_1173, 3, x_28); +lean_inc(x_12); +x_1174 = l_Lean_Syntax_node2(x_12, x_68, x_1173, x_19); +lean_inc(x_12); +x_1175 = l_Lean_Syntax_node3(x_12, x_282, x_71, x_1165, x_73); +lean_inc(x_12); +x_1176 = l_Lean_Syntax_node1(x_12, x_17, x_1175); +lean_inc(x_12); +x_1177 = l_Lean_Syntax_node2(x_12, x_33, x_223, x_1176); +lean_inc(x_12); +x_1178 = l_Lean_Syntax_node3(x_12, x_85, x_1177, x_77, x_1141); +lean_inc(x_12); +x_1179 = l_Lean_Syntax_node2(x_12, x_35, x_27, x_1178); +lean_inc(x_12); +x_1180 = l_Lean_Syntax_node2(x_12, x_37, x_1135, x_1179); +lean_inc(x_12); +x_1181 = l_Lean_Syntax_node4(x_12, x_96, x_64, x_1174, x_1180, x_95); +lean_inc(x_12); +x_1182 = l_Lean_Syntax_node2(x_12, x_61, x_209, x_1181); +x_1183 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__524; +lean_inc(x_12); +x_1184 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_1184, 0, x_12); +lean_ctor_set(x_1184, 1, x_1183); +x_1185 = l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__525; +lean_inc(x_12); +x_1186 = l_Lean_Syntax_node2(x_12, x_1185, x_1184, x_32); +x_1187 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1187, 0, x_1186); +lean_ctor_set(x_1187, 1, x_28); +x_1188 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1188, 0, x_1182); +lean_ctor_set(x_1188, 1, x_1187); +x_1189 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1189, 0, x_1170); +lean_ctor_set(x_1189, 1, x_1188); +x_1190 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1190, 0, x_1152); +lean_ctor_set(x_1190, 1, x_1189); +x_1191 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1191, 0, x_1129); +lean_ctor_set(x_1191, 1, x_1190); +x_1192 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1192, 0, x_1119); +lean_ctor_set(x_1192, 1, x_1191); +x_1193 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1193, 0, x_1101); +lean_ctor_set(x_1193, 1, x_1192); +x_1194 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1194, 0, x_1074); +lean_ctor_set(x_1194, 1, x_1193); +x_1195 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1195, 0, x_925); +lean_ctor_set(x_1195, 1, x_1194); +x_1196 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1196, 0, x_821); +lean_ctor_set(x_1196, 1, x_1195); +x_1197 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1197, 0, x_808); +lean_ctor_set(x_1197, 1, x_1196); +x_1198 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1198, 0, x_791); +lean_ctor_set(x_1198, 1, x_1197); +x_1199 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1199, 0, x_770); +lean_ctor_set(x_1199, 1, x_1198); +x_1200 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1200, 0, x_747); +lean_ctor_set(x_1200, 1, x_1199); +x_1201 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1201, 0, x_731); +lean_ctor_set(x_1201, 1, x_1200); +x_1202 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1202, 0, x_691); +lean_ctor_set(x_1202, 1, x_1201); +x_1203 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1203, 0, x_653); +lean_ctor_set(x_1203, 1, x_1202); +x_1204 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1204, 0, x_587); +lean_ctor_set(x_1204, 1, x_1203); +x_1205 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1205, 0, x_555); +lean_ctor_set(x_1205, 1, x_1204); +x_1206 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1206, 0, x_536); +lean_ctor_set(x_1206, 1, x_1205); +x_1207 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1207, 0, x_522); +lean_ctor_set(x_1207, 1, x_1206); +x_1208 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1208, 0, x_500); +lean_ctor_set(x_1208, 1, x_1207); +x_1209 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1209, 0, x_484); +lean_ctor_set(x_1209, 1, x_1208); +x_1210 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1210, 0, x_461); +lean_ctor_set(x_1210, 1, x_1209); +x_1211 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1211, 0, x_445); +lean_ctor_set(x_1211, 1, x_1210); +x_1212 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1212, 0, x_428); +lean_ctor_set(x_1212, 1, x_1211); +x_1213 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1213, 0, x_417); +lean_ctor_set(x_1213, 1, x_1212); +x_1214 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1214, 0, x_385); +lean_ctor_set(x_1214, 1, x_1213); +x_1215 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1215, 0, x_374); +lean_ctor_set(x_1215, 1, x_1214); +x_1216 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1216, 0, x_352); +lean_ctor_set(x_1216, 1, x_1215); +x_1217 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1217, 0, x_301); +lean_ctor_set(x_1217, 1, x_1216); +x_1218 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1218, 0, x_253); +lean_ctor_set(x_1218, 1, x_1217); +x_1219 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1219, 0, x_194); +lean_ctor_set(x_1219, 1, x_1218); +x_1220 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1220, 0, x_178); +lean_ctor_set(x_1220, 1, x_1219); +x_1221 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1221, 0, x_162); +lean_ctor_set(x_1221, 1, x_1220); +x_1222 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1222, 0, x_146); +lean_ctor_set(x_1222, 1, x_1221); +x_1223 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1223, 0, x_113); +lean_ctor_set(x_1223, 1, x_1222); +x_1224 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1224, 0, x_98); +lean_ctor_set(x_1224, 1, x_1223); +x_1225 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1225, 0, x_62); +lean_ctor_set(x_1225, 1, x_1224); +x_1226 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1226, 0, x_16); +lean_ctor_set(x_1226, 1, x_1225); +x_1227 = lean_array_mk(x_1226); +x_1228 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1228, 0, x_12); +lean_ctor_set(x_1228, 1, x_17); +lean_ctor_set(x_1228, 2, x_1227); +x_1229 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1229, 0, x_1228); +lean_ctor_set(x_1229, 1, x_3); +return x_1229; } } } @@ -9702,6 +10080,48 @@ l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorem lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__503); l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__504 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__504(); lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__504); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__505 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__505(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__505); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__506 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__506(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__506); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__507 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__507(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__507); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__508 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__508(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__508); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__509 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__509(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__509); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__510 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__510(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__510); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__511 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__511(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__511); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__512 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__512(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__512); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__513 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__513(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__513); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__514 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__514(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__514); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__515 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__515(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__515); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__516 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__516(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__516); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__517 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__517(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__517); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__518 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__518(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__518); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__519 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__519(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__519); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__520 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__520(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__520); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__521 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__521(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__521); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__522 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__522(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__522); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__523 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__523(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__523); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__524 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__524(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__524); +l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__525 = _init_l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__525(); +lean_mark_persistent(l___aux__Init__Data__UInt__Lemmas______macroRules__commandDeclare__uint__theorems____1___closed__525); l_UInt8_instInhabited = _init_l_UInt8_instInhabited(); l_UInt16_instInhabited = _init_l_UInt16_instInhabited(); l_UInt32_instInhabited = _init_l_UInt32_instInhabited(); diff --git a/stage0/stdlib/Init/NotationExtra.c b/stage0/stdlib/Init/NotationExtra.c index a056ecb62ac3..c9d8435f5e69 100644 --- a/stage0/stdlib/Init/NotationExtra.c +++ b/stage0/stdlib/Init/NotationExtra.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.NotationExtra -// Imports: Init.Data.ToString.Basic Init.Data.Array.Subarray Init.Conv Init.Meta +// Imports: Init.Data.ToString.Basic Init.Data.Array.Subarray Init.Conv Init.Meta Init.While #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -18,7 +18,6 @@ static lean_object* l_Lean_unbracketedExplicitBinders___closed__11; static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___closed__14; static lean_object* l_termExists___x2c_____closed__4; static lean_object* l_term_u2203___x2c_____closed__6; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5; static lean_object* l_unexpandEqNDRec___closed__2; static lean_object* l_Lean_unbracketedExplicitBinders___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_classAbbrev; @@ -30,8 +29,6 @@ static lean_object* l_term_x7b___x7d___closed__6; LEAN_EXPORT lean_object* l_unexpandMkArray5(lean_object*, lean_object*, lean_object*); static lean_object* l_term___xd7____1___closed__2; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__11; -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__3; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__15; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__26; static lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1___closed__2; LEAN_EXPORT lean_object* l_unexpandMkArray3___boxed(lean_object*, lean_object*, lean_object*); @@ -44,8 +41,6 @@ static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__ static lean_object* l_Lean_unbracketedExplicitBinders___closed__3; LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__convCalc____1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___closed__8; -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__10; -LEAN_EXPORT lean_object* l_Lean_Loop_toCtorIdx___boxed(lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1___closed__5; LEAN_EXPORT lean_object* l_unexpandEqNDRec(lean_object*, lean_object*, lean_object*); static lean_object* l_termExists___x2c_____closed__7; @@ -97,7 +92,6 @@ LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b_ LEAN_EXPORT lean_object* l_termExists___x2c__; static lean_object* l_term___xd7____1___closed__8; static lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1___lambda__1___closed__4; -static lean_object* l_Lean_doElemRepeat____Until_____closed__8; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__9; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__13; @@ -109,21 +103,18 @@ static lean_object* l_Lean_calcFirstStep___closed__7; static lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__4___closed__2; static lean_object* l___aux__Init__NotationExtra______macroRules__term_u03a3___x2c____1___closed__2; LEAN_EXPORT lean_object* l_unexpandSigma(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__1; static lean_object* l_term___xd7_x27____1___closed__5; lean_object* l_Lean_Syntax_getId(lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__57; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); static lean_object* l_termExists___x2c_____closed__2; static lean_object* l_Lean_calcSteps___closed__4; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__6; LEAN_EXPORT lean_object* l_unexpandMkArray6(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___closed__1; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__41; static lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1___lambda__2___closed__3; LEAN_EXPORT lean_object* l_unexpandListNil___rarg___boxed(lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2; lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_unexpandIte___closed__1; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__26; @@ -163,7 +154,6 @@ static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b__ static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__11; LEAN_EXPORT lean_object* l_Lean_expandExplicitBindersAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Loop_forIn___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__16; lean_object* l_Lean_Syntax_TSepArray_getElems___rarg(lean_object*); static lean_object* l_Lean_unifConstraint___closed__3; @@ -176,14 +166,11 @@ static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__48; LEAN_EXPORT lean_object* l_unexpandListCons___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_term_u03a3___x2c_____closed__2; -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_classAbbrev___closed__20; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__30; LEAN_EXPORT lean_object* l_Lean_unifConstraintElem; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__17; static lean_object* l_unexpandGetElem_x3f___closed__3; static lean_object* l_unexpandGetElem_x3f___closed__2; -static lean_object* l_Lean_doElemRepeat_____closed__1; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__31; static lean_object* l_Lean_unbracketedExplicitBinders___closed__5; static lean_object* l_Lean_cdotTk___closed__1; @@ -203,13 +190,11 @@ static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___spec__4(size_t, size_t, lean_object*); static lean_object* l_Lean_bracketedExplicitBinders___closed__13; LEAN_EXPORT lean_object* l_Lean_expandExplicitBindersAux_loop___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_doElemRepeat____Until_____closed__5; static lean_object* l_term_u03a3_x27___x2c_____closed__4; 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_unexpandGetElem_x21(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; static lean_object* l_Lean_unifConstraintElem___closed__6; static lean_object* l_Lean_Parser_Command_classAbbrev___closed__27; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__40; @@ -220,13 +205,11 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__com static lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__4___closed__4; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__17; static lean_object* l_term___xd7_x27____1___closed__6; -LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_unexpandListToArray___closed__2; static lean_object* l_tacticFunext_________closed__3; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__27; static lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1___lambda__1___closed__1; static lean_object* l_Lean_unifConstraint___closed__16; -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__2; static lean_object* l_Lean_Parser_Command_classAbbrev___closed__2; LEAN_EXPORT lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2__; static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__8; @@ -239,7 +222,6 @@ static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__ LEAN_EXPORT lean_object* l_unexpandProdMk___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Term__letI__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*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1___lambda__1___closed__7; -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__14; static lean_object* l_term___xd7____1___closed__4; static lean_object* l_term_u03a3___x2c_____closed__8; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__12; @@ -247,7 +229,6 @@ static lean_object* l_term_u03a3_x27___x2c_____closed__6; static lean_object* l_Lean_cdotTk___closed__8; static lean_object* l_Lean_explicitBinders___closed__5; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__5; -LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit(lean_object*, lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__1; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__7; @@ -266,10 +247,8 @@ static lean_object* l_term_u2203___x2c_____closed__2; LEAN_EXPORT lean_object* l_unexpandExists___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term___xd7____1__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_doElemRepeat____Until__; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__53; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__3(size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_unexpandExists___closed__3; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__19; static lean_object* l_termExists___x2c_____closed__5; @@ -281,21 +260,17 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__com static lean_object* l_unexpandExists___closed__1; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__39; static lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___spec__3___closed__1; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__1; static lean_object* l_tacticFunext_________closed__8; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__46; static lean_object* l_Lean_term__Matches___x7c___closed__9; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__46; -lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___spec__1___boxed(lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___closed__6; LEAN_EXPORT lean_object* l_unexpandSubtype(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__28; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9; size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_expandExplicitBinders___spec__1(lean_object*, size_t, size_t); static lean_object* l_Lean_cdotTk___closed__3; -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___closed__15; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__1; static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__13; @@ -314,18 +289,13 @@ static lean_object* l_Lean_bracketedExplicitBinders___closed__12; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__termExists___x2c____1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__28; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Term__haveI__1___closed__4; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8; -static lean_object* l_Lean_doElemRepeat_____closed__8; static lean_object* l_Lean_Parser_Command_classAbbrev___closed__30; static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__7; static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___closed__12; static lean_object* l_Lean_calcSteps___closed__12; -static lean_object* l_Lean_doElemRepeat_____closed__2; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__11; static lean_object* l_tacticFunext_________closed__6; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Term__haveI__1___closed__9; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__14; LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_unexpandSubtype___closed__2; @@ -394,15 +364,12 @@ static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__9; lean_object* l_Lean_Syntax_getKind(lean_object*); static lean_object* l_Lean_unbracketedExplicitBinders___closed__17; static lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1___lambda__2___closed__8; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__16; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__12; static lean_object* l_term_x7b___x7d___closed__8; lean_object* l_Lean_mkCIdentFrom(lean_object*, lean_object*, uint8_t); static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__11; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__20; static lean_object* l_Lean_Parser_Command_classAbbrev___closed__10; static lean_object* l_Lean_unifConstraintElem___closed__11; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__3___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__14; static lean_object* l_unexpandListNil___rarg___closed__3; @@ -414,13 +381,11 @@ LEAN_EXPORT lean_object* l_unexpandUnit___boxed(lean_object*); static lean_object* l_unexpandSubtype___closed__5; lean_object* l_outOfBounds___rarg(lean_object*); static lean_object* l_Lean_calcTactic___closed__2; -LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___rarg(lean_object*); LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_unexpandGetElem_x3f(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___lambda__1(lean_object*); static lean_object* l_Lean_solveTactic___closed__11; static lean_object* l_Lean_cdot___closed__6; -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__13; static lean_object* l_term_x7b___x7d___closed__1; static lean_object* l_Lean_bracketedExplicitBinders___closed__2; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__16; @@ -431,7 +396,6 @@ static lean_object* l_Lean_term__Matches___x7c___closed__10; static lean_object* l_Lean_calcSteps___closed__16; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__59; lean_object* l_Lean_Syntax_getOptional_x3f(lean_object*); -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__8; static lean_object* l_Lean_calcStep___closed__1; static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___closed__3; lean_object* l_Lean_Syntax_node3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -440,12 +404,8 @@ static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__ static lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__4___closed__7; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__47; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__9; static lean_object* l_Lean_calcSteps___closed__3; static lean_object* l_Lean_Parser_Command_classAbbrev___closed__22; -LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___rarg___lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_doElemRepeat____Until_____closed__4; -static lean_object* l_Lean_doElemWhile__Do_____closed__2; LEAN_EXPORT lean_object* l_Lean_insertUnexpander(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_unexpandIte___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__convCalc____1(lean_object*, lean_object*, lean_object*); @@ -459,7 +419,6 @@ static lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d LEAN_EXPORT lean_object* l_Lean_expandBrackedBindersAux_loop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_cdot___closed__5; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term___xd7_x27____1__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___closed__2; static lean_object* l_Lean_cdotTk___closed__11; static lean_object* l_unexpandEqNDRec___closed__1; @@ -471,25 +430,19 @@ static lean_object* l_Lean_explicitBinders___closed__6; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_solveTactic___closed__8; static lean_object* l_Lean_bracketedExplicitBinders___closed__15; -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_solveTactic___closed__18; LEAN_EXPORT lean_object* l_Lean_calcTactic; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__1; static lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__4___closed__9; static lean_object* l_Lean_calcSteps___closed__13; static lean_object* l_Lean_unbracketedExplicitBinders___closed__8; -static lean_object* l_Lean_doElemRepeat____Until_____closed__6; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__23; LEAN_EXPORT lean_object* l_unexpandUnit(lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__19; lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__9; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__8; LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__2; lean_object* l_Lean_extractMacroScopes(lean_object*); -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_u2203___x2c____1___closed__1; static lean_object* l_term_u03a3___x2c_____closed__5; static lean_object* l_term_u03a3___x2c_____closed__3; @@ -506,7 +459,6 @@ uint8_t lean_name_eq(lean_object*, lean_object*); static lean_object* l_term___xd7____1___closed__3; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__16; -static lean_object* l_Lean_doElemWhile__Do_____closed__1; static lean_object* l_Lean_unifConstraintElem___closed__9; static lean_object* l_Lean_calcFirstStep___closed__3; lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); @@ -519,7 +471,6 @@ static lean_object* l_term___xd7_x27____1___closed__1; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); static lean_object* l_Lean_unbracketedExplicitBinders___closed__14; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Term__haveI__1___lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_unexpandSubtype___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1___closed__6; static lean_object* l_unexpandListNil___rarg___closed__2; @@ -536,7 +487,6 @@ static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_ uint8_t l_Lean_Syntax_isIdent(lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__3; static lean_object* l_Lean_unifConstraintElem___closed__5; -static lean_object* l_Lean_doElemRepeat_____closed__6; static lean_object* l_Lean_solveTactic___closed__12; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__21; static lean_object* l_Lean_term__Matches___x7c___closed__3; @@ -544,7 +494,6 @@ static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___spec__4___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_unexpandMkArray1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_term___xd7_x27____1___closed__2; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6; static lean_object* l_Lean_bracketedExplicitBinders___closed__17; LEAN_EXPORT lean_object* l_unexpandArrayEmpty___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_cdotTk; @@ -579,17 +528,14 @@ static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_ static lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1___closed__4; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__49; LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop(lean_object*, lean_object*); static lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__4___closed__3; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Term__haveI__1___closed__6; static lean_object* l_term___xd7_x27____1___closed__7; static lean_object* l_term_u03a3_x27___x2c_____closed__2; static lean_object* l_Lean_unifConstraint___closed__13; -LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__32; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__7; static lean_object* l_Lean_term__Matches___x7c___closed__6; -static lean_object* l_Lean_doElemRepeat____Until_____closed__7; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__13; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__42; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__19; @@ -610,7 +556,6 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__com static lean_object* l_Lean_Parser_Command_classAbbrev___closed__9; static lean_object* l_Lean_calcSteps___closed__15; LEAN_EXPORT lean_object* l_term_u2203___x2c__; -static lean_object* l_Lean_doElemRepeat_____closed__5; static lean_object* l_Lean_bracketedExplicitBinders___closed__5; LEAN_EXPORT lean_object* l_Lean_calcSteps; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__50; @@ -647,13 +592,11 @@ static lean_object* l_Lean_Parser_Command_classAbbrev___closed__15; static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__18; static lean_object* l_tacticFunext_________closed__12; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__12; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__23; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_unifConstraint___closed__14; static lean_object* l_Lean_calcFirstStep___closed__6; -static lean_object* l_Lean_doElemRepeat____Until_____closed__3; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term___xd7____1__1(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1___lambda__2___closed__5; static lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1___closed__6; @@ -662,7 +605,6 @@ static lean_object* l_unexpandGetElem_x21___closed__1; static lean_object* l_term_x7b___x7d___closed__2; static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__4; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__6; -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__4; static lean_object* l_Lean_calc___closed__5; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_unexpandListCons(lean_object*, lean_object*, lean_object*); @@ -679,7 +621,6 @@ lean_object* l_Lean_Syntax_SepArray_ofElems(lean_object*, lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__2; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_singletonUnexpander___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__6; LEAN_EXPORT lean_object* l_unexpandProdMk(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_calcStep; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__12; @@ -688,11 +629,9 @@ static lean_object* l_term___xd7_x27____1___closed__4; static lean_object* l_Lean_bracketedExplicitBinders___closed__16; LEAN_EXPORT lean_object* l_term___xd7____1; static lean_object* l_unexpandUnit___rarg___closed__1; -static lean_object* l_Lean_doElemRepeat____Until_____closed__2; LEAN_EXPORT lean_object* l_Lean_expandExplicitBinders___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__8; static lean_object* l_Lean_calcStep___closed__6; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__5; static lean_object* l_Lean_unifConstraint___closed__2; LEAN_EXPORT lean_object* l_unexpandEqRec___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_calcStep___closed__4; @@ -700,8 +639,6 @@ lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_unexpandGetElem___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_expandBrackedBindersAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Term__haveI__1___closed__8; -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3; static lean_object* l_unexpandGetElem_x21___closed__2; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Term__haveI__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*); static lean_object* l_Lean_Parser_Command_classAbbrev___closed__12; @@ -718,13 +655,10 @@ lean_object* l_Lean_mkSepArray(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_unexpandMkArray0___boxed(lean_object*); static lean_object* l_Lean_cdotTk___closed__5; -LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_bracketedExplicitBinders___closed__18; static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__17; -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_calcTactic___closed__4; extern lean_object* l_Lean_binderIdent; -static lean_object* l_Lean_doElemWhile__Do_____closed__3; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__convCalc____1___closed__4; LEAN_EXPORT lean_object* l_Lean_expandExplicitBinders(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_cdotTk___closed__4; @@ -740,7 +674,6 @@ LEAN_EXPORT lean_object* l_unexpandUnit___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_unexpandMkArray0___rarg(lean_object*, lean_object*); static lean_object* l_Lean_unifConstraintElem___closed__4; static lean_object* l_unexpandGetElem_x21___closed__3; -static lean_object* l_Lean_doElemWhile__Do_____closed__6; LEAN_EXPORT lean_object* l_unexpandSigma___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_term_u03a3_x27___x2c_____closed__3; static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__5; @@ -752,24 +685,15 @@ lean_object* lean_nat_sub(lean_object*, lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__45; lean_object* l_Array_mkArray1___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_expandExplicitBinders___spec__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__12; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__22; static lean_object* l_Lean_unbracketedExplicitBinders___closed__23; LEAN_EXPORT lean_object* l_Lean_unbracketedExplicitBinders; -static lean_object* l_Lean_doElemWhile__Do_____closed__5; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__49; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__22; -static lean_object* l_Lean_doElemRepeat_____closed__7; -LEAN_EXPORT lean_object* l_Lean_Loop_toCtorIdx(lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__convCalc____1___closed__9; static lean_object* l_Lean_unbracketedExplicitBinders___closed__21; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__10; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__25; -LEAN_EXPORT lean_object* l_Lean_doElemRepeat__; -LEAN_EXPORT lean_object* l_Lean_Loop_forIn___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Term__haveI__1___closed__7; -static lean_object* l_Lean_doElemRepeat_____closed__3; static lean_object* l_Lean_unbracketedExplicitBinders___closed__10; static lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1___lambda__2___closed__9; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__8; @@ -780,7 +704,6 @@ lean_object* l_Array_ofSubarray___rarg(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___spec__3___closed__2; static lean_object* l_tacticFunext_________closed__10; static lean_object* l_Lean_Parser_Command_classAbbrev___closed__29; -static lean_object* l_Lean_doElemRepeat____Until_____closed__1; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__48; LEAN_EXPORT lean_object* l_unexpandListNil___rarg(lean_object*, lean_object*); static lean_object* l_Lean_calcFirstStep___closed__11; @@ -788,15 +711,12 @@ LEAN_EXPORT lean_object* l_unexpandGetElem(lean_object*, lean_object*, lean_obje LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term___xd7_x27____1__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_solveTactic___closed__17; LEAN_EXPORT lean_object* l_Lean_insertUnexpander___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__7; static lean_object* l_unexpandListCons___closed__3; size_t lean_usize_sub(size_t, size_t); static lean_object* l_Lean_unbracketedExplicitBinders___closed__15; lean_object* lean_array_mk(lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_u03a3___x2c____1___closed__1; -LEAN_EXPORT lean_object* l_Lean_doElemWhile___x3a__Do__; static lean_object* l_Array_forInUnsafe_loop___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___spec__5___closed__1; -LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_unexpandListToArray___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_tacticFunext_________closed__2; static lean_object* l_Lean_calcSteps___closed__9; @@ -807,7 +727,6 @@ LEAN_EXPORT lean_object* l_unexpandListNil___boxed(lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__33; LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__1(lean_object*); static lean_object* l_Lean_bracketedExplicitBinders___closed__6; -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__5; LEAN_EXPORT lean_object* l_unexpandTSyntax___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__27; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___closed__5; @@ -824,7 +743,6 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__com static lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1___closed__2; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__3; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__9; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1; extern lean_object* l_Lean_instInhabitedSyntax; LEAN_EXPORT lean_object* l_unexpandArrayEmpty___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_expandExplicitBindersAux_loop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -837,11 +755,9 @@ static lean_object* l_Lean_term__Matches___x7c___closed__1; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__41; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_x7b___x7d__1___lambda__1___closed__2; -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__9; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Term__haveI__1___lambda__1___closed__3; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__8; static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___closed__9; -LEAN_EXPORT lean_object* l_Lean_doElemWhile__Do__; static lean_object* l_Lean_solveTactic___closed__10; LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_unifConstraint___closed__11; @@ -850,17 +766,14 @@ static lean_object* l_term_x7b___x7d___closed__5; static lean_object* l_term___xd7____1___closed__1; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__18; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__6; -static lean_object* l_Lean_doElemRepeat_____closed__4; LEAN_EXPORT lean_object* l_unexpandPSigma(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_unbracketedExplicitBinders___closed__9; -static lean_object* l_Lean_doElemRepeat_____closed__9; lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1(lean_object*, size_t, size_t, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1___closed__4; lean_object* lean_array_get_size(lean_object*); static lean_object* l_Lean_convCalc_____closed__1; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term_u03a3___x2c____1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__7; static lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__4___closed__5; static lean_object* l_unexpandIte___closed__4; static lean_object* l_Lean_unbracketedExplicitBinders___closed__22; @@ -886,10 +799,8 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__com LEAN_EXPORT lean_object* l_Lean_expandBrackedBinders___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_u03a3_x27___x2c____1___closed__2; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__38; -static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__15; static lean_object* l_Lean_solveTactic___closed__6; static lean_object* l_Lean_bracketedExplicitBinders___closed__10; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__3; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__1; LEAN_EXPORT lean_object* l_tacticFunext______; static lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__13; @@ -899,7 +810,6 @@ static lean_object* l_Lean_term__Matches___x7c___closed__5; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__54; LEAN_EXPORT lean_object* l_unexpandMkArray4(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___spec__7(lean_object*, size_t, size_t, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__13; LEAN_EXPORT lean_object* l_Lean_cdot; LEAN_EXPORT lean_object* l_unexpandExists(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__45; @@ -914,14 +824,11 @@ static lean_object* l___aux__Init__NotationExtra______macroRules__term_u2203___x static lean_object* l_Lean_term__Matches___x7c___closed__2; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); static lean_object* l_term_u03a3_x27___x2c_____closed__7; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__11; static lean_object* l_unexpandGetElem_x3f___closed__1; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10; LEAN_EXPORT lean_object* l_unexpandMkArray8(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__term_u03a3_x27___x2c____1___closed__1; static lean_object* l_Lean_cdot___closed__4; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command____Unif__hint________Where___x7c___x2d_u22a2____1___lambda__2___closed__16; -static lean_object* l_Lean_doElemWhile__Do_____closed__4; static lean_object* l_Lean_unifConstraint___closed__8; static lean_object* l_Lean_solveTactic___closed__4; static lean_object* l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__20; @@ -936,7 +843,6 @@ static lean_object* l_Lean_calcSteps___closed__7; static lean_object* l_unexpandPSigma___closed__1; static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__15; static lean_object* l_Lean_Parser_Command_classAbbrev___closed__14; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__4; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext________1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_calcSteps___closed__14; @@ -945,7 +851,6 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__sol static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__29; static lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__4___closed__1; static lean_object* l_Lean_solveTactic___closed__14; -LEAN_EXPORT lean_object* l_Lean_Loop_forIn(lean_object*, lean_object*); static lean_object* l_Lean_bracketedExplicitBinders___closed__8; static lean_object* _init_l_Lean_unbracketedExplicitBinders___closed__1() { _start: @@ -7593,12 +7498,10 @@ if (x_10 == 0) { lean_object* x_11; uint8_t x_12; x_11 = lean_unsigned_to_nat(2u); -lean_inc(x_9); x_12 = l_Lean_Syntax_matchesNull(x_9, x_11); if (x_12 == 0) { lean_object* x_13; lean_object* x_14; -lean_dec(x_9); x_13 = lean_box(0); x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_13); @@ -7607,90 +7510,39 @@ return x_14; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_15 = lean_unsigned_to_nat(0u); -x_16 = l_Lean_Syntax_getArg(x_9, x_15); -x_17 = l_Lean_expandExplicitBindersAux_loop___closed__12; -x_18 = l_Lean_Syntax_isOfKind(x_16, x_17); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; -lean_dec(x_9); -x_19 = lean_box(0); -x_20 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_3); -return x_20; -} -else -{ -lean_object* x_21; uint8_t x_22; -x_21 = l_Lean_Syntax_getArg(x_9, x_8); -lean_dec(x_9); -x_22 = l_Lean_Syntax_isOfKind(x_21, x_17); -if (x_22 == 0) -{ -lean_object* x_23; lean_object* x_24; -x_23 = lean_box(0); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_23); -lean_ctor_set(x_24, 1, x_3); -return x_24; -} -else -{ -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; -x_25 = 0; -x_26 = l_Lean_SourceInfo_fromRef(x_2, x_25); -x_27 = l_unexpandSorryAx___closed__1; -lean_inc(x_26); -x_28 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -x_29 = l_unexpandSorryAx___closed__2; -x_30 = l_Lean_Syntax_node1(x_26, x_29, x_28); -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_31, 1, x_3); -return x_31; -} -} +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; +x_15 = 0; +x_16 = l_Lean_SourceInfo_fromRef(x_2, x_15); +x_17 = l_unexpandSorryAx___closed__1; +lean_inc(x_16); +x_18 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +x_19 = l_unexpandSorryAx___closed__2; +x_20 = l_Lean_Syntax_node1(x_16, x_19, 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_3); +return x_21; } } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_32 = lean_unsigned_to_nat(0u); -x_33 = l_Lean_Syntax_getArg(x_9, x_32); +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_dec(x_9); -x_34 = l_Lean_expandExplicitBindersAux_loop___closed__12; -x_35 = l_Lean_Syntax_isOfKind(x_33, x_34); -if (x_35 == 0) -{ -lean_object* x_36; lean_object* x_37; -x_36 = lean_box(0); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_3); -return x_37; -} -else -{ -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; -x_38 = 0; -x_39 = l_Lean_SourceInfo_fromRef(x_2, x_38); -x_40 = l_unexpandSorryAx___closed__1; -lean_inc(x_39); -x_41 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_41, 0, x_39); -lean_ctor_set(x_41, 1, x_40); -x_42 = l_unexpandSorryAx___closed__2; -x_43 = l_Lean_Syntax_node1(x_39, x_42, x_41); -x_44 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_3); -return x_44; -} +x_22 = 0; +x_23 = l_Lean_SourceInfo_fromRef(x_2, x_22); +x_24 = l_unexpandSorryAx___closed__1; +lean_inc(x_23); +x_25 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +x_26 = l_unexpandSorryAx___closed__2; +x_27 = l_Lean_Syntax_node1(x_23, x_26, x_25); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_3); +return x_28; } } } @@ -15456,1555 +15308,224 @@ lean_dec(x_2); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Loop_toCtorIdx(lean_object* x_1) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__1() { _start: { -lean_object* x_2; -x_2 = lean_unsigned_to_nat(0u); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("term_Matches_|", 14, 14); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Loop_toCtorIdx___boxed(lean_object* x_1) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__2() { _start: { -lean_object* x_2; -x_2 = l_Lean_Loop_toCtorIdx(x_1); -lean_dec(x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_unbracketedExplicitBinders___closed__1; +x_2 = l_Lean_term__Matches___x7c___closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___rarg(lean_object* x_1) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__3() { _start: { -lean_inc(x_1); +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" matches ", 9, 9); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__4() { _start: { -lean_object* x_5; -x_5 = lean_alloc_closure((void*)(l_Lean_Loop_noConfusion___rarg___boxed), 1, 0); -return x_5; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_term__Matches___x7c___closed__3; +x_2 = lean_alloc_ctor(5, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___rarg___boxed(lean_object* x_1) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__5() { _start: { -lean_object* x_2; -x_2 = l_Lean_Loop_noConfusion___rarg(x_1); -lean_dec(x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_unbracketedExplicitBinders___closed__18; +x_2 = lean_unsigned_to_nat(51u); +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; } } -LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__6() { _start: { -lean_object* x_5; -x_5 = l_Lean_Loop_noConfusion(x_1, x_2, x_3, x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_5; +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" | ", 3, 3); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__7() { _start: { -if (lean_obj_tag(x_3) == 0) -{ -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -lean_dec(x_2); -x_4 = lean_ctor_get(x_3, 0); -lean_inc(x_4); -lean_dec(x_3); -x_5 = lean_ctor_get(x_1, 0); -lean_inc(x_5); -lean_dec(x_1); -x_6 = lean_ctor_get(x_5, 1); -lean_inc(x_6); -lean_dec(x_5); -x_7 = lean_apply_2(x_6, lean_box(0), x_4); -return x_7; -} -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 = l_Lean_Loop_forIn_loop___rarg(x_1, x_2, x_8); -return x_9; -} +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_term__Matches___x7c___closed__6; +x_2 = lean_alloc_ctor(5, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__8() { _start: { -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_1, 1); -lean_inc(x_4); -x_5 = lean_box(0); -lean_inc(x_2); -x_6 = lean_apply_2(x_2, x_5, x_3); -x_7 = lean_alloc_closure((void*)(l_Lean_Loop_forIn_loop___rarg___lambda__1), 3, 2); -lean_closure_set(x_7, 0, x_1); -lean_closure_set(x_7, 1, x_2); -x_8 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_6, x_7); -return x_8; +lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; +x_1 = l_Lean_term__Matches___x7c___closed__5; +x_2 = l_Lean_term__Matches___x7c___closed__6; +x_3 = l_Lean_term__Matches___x7c___closed__7; +x_4 = 0; +x_5 = lean_alloc_ctor(11, 3, 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_uint8(x_5, sizeof(void*)*3, x_4); +return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__9() { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Loop_forIn_loop___rarg), 3, 0); -return x_3; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_unbracketedExplicitBinders___closed__5; +x_2 = l_Lean_term__Matches___x7c___closed__4; +x_3 = l_Lean_term__Matches___x7c___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); +lean_ctor_set(x_4, 2, x_3); +return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Loop_forIn___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l_Lean_term__Matches___x7c___closed__10() { _start: { -lean_object* x_5; -x_5 = l_Lean_Loop_forIn_loop___rarg(x_1, x_4, x_3); +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_term__Matches___x7c___closed__2; +x_2 = lean_unsigned_to_nat(50u); +x_3 = lean_unsigned_to_nat(51u); +x_4 = l_Lean_term__Matches___x7c___closed__9; +x_5 = lean_alloc_ctor(4, 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; } } -LEAN_EXPORT lean_object* l_Lean_Loop_forIn(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_term__Matches___x7c() { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Loop_forIn___rarg___boxed), 4, 0); -return x_3; +lean_object* x_1; +x_1 = l_Lean_term__Matches___x7c___closed__10; +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Loop_forIn___rarg___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_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___spec__1(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { _start: { -lean_object* x_5; -x_5 = l_Lean_Loop_forIn___rarg(x_1, x_2, x_3, x_4); +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ lean_dec(x_2); +lean_dec(x_1); return x_5; } -} -LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +else { -lean_object* x_5; -x_5 = l_Lean_Loop_forIn_loop___rarg(x_1, x_4, x_3); -return x_5; -} +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; +x_7 = lean_array_uget(x_5, x_4); +x_8 = lean_unsigned_to_nat(0u); +x_9 = lean_array_uset(x_5, x_4, x_8); +lean_inc(x_2); +lean_inc(x_1); +x_10 = l_Lean_Syntax_node1(x_1, x_2, x_7); +x_11 = 1; +x_12 = lean_usize_add(x_4, x_11); +x_13 = lean_array_uset(x_9, x_4, x_10); +x_4 = x_12; +x_5 = x_13; +goto _start; } -LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_instForInLoopUnit___rarg___boxed), 4, 0); -return x_3; } } -LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__1() { _start: { -lean_object* x_5; -x_5 = l_Lean_instForInLoopUnit___rarg(x_1, x_2, x_3, x_4); -lean_dec(x_2); +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_unbracketedExplicitBinders___closed__1; +x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; +x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; +x_4 = l___aux__Init__NotationExtra______macroRules__tacticFunext________1___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_doElemRepeat_____closed__1() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("doElemRepeat_", 13, 13); +x_1 = lean_mk_string_unchecked("match", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_doElemRepeat_____closed__2() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__3() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_doElemRepeat_____closed__1; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; +x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; +x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; +x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___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_doElemRepeat_____closed__3() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__4() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("repeat ", 7, 7); +x_1 = lean_mk_string_unchecked("matchDiscr", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_doElemRepeat_____closed__4() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__5() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_doElemRepeat_____closed__3; -x_2 = lean_alloc_ctor(5, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_unbracketedExplicitBinders___closed__1; +x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; +x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; +x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__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_doElemRepeat_____closed__5() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__6() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("doSeq", 5, 5); +x_1 = lean_mk_string_unchecked("with", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_doElemRepeat_____closed__6() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__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_doElemRepeat_____closed__5; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("matchAlts", 9, 9); +return x_1; } } -static lean_object* _init_l_Lean_doElemRepeat_____closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_doElemRepeat_____closed__6; -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_doElemRepeat_____closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemRepeat_____closed__4; -x_3 = l_Lean_doElemRepeat_____closed__7; -x_4 = lean_alloc_ctor(2, 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_doElemRepeat_____closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_doElemRepeat_____closed__2; -x_2 = lean_unsigned_to_nat(1022u); -x_3 = l_Lean_doElemRepeat_____closed__8; -x_4 = lean_alloc_ctor(3, 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_doElemRepeat__() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_doElemRepeat_____closed__9; -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doFor", 5, 5); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____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_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____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___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("for", 3, 3); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doForDecl", 9, 9); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____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_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____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___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("in", 2, 2); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Loop.mk", 7, 7); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__7; -x_2 = l_String_toSubstring_x27(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__9() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Loop", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__9; -x_2 = l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__15; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__9; -x_3 = l___aux__Init__NotationExtra______macroRules__Lean__Parser__Command__classAbbrev__1___lambda__3___closed__15; -x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____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___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__11; -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___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__13() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__11; -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___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__14() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__13; -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___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__15() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__13; -x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__14; -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_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__16() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__12; -x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__15; -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_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__17() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("do", 2, 2); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1(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_doElemRepeat_____closed__2; -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_2); -lean_dec(x_1); -x_6 = lean_box(1); -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; lean_object* x_10; uint8_t 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; -x_8 = lean_unsigned_to_nat(1u); -x_9 = l_Lean_Syntax_getArg(x_1, x_8); -lean_dec(x_1); -x_10 = lean_ctor_get(x_2, 5); -lean_inc(x_10); -x_11 = 0; -x_12 = l_Lean_SourceInfo_fromRef(x_10, x_11); -lean_dec(x_10); -x_13 = lean_ctor_get(x_2, 2); -lean_inc(x_13); -x_14 = lean_ctor_get(x_2, 1); -lean_inc(x_14); -lean_dec(x_2); -x_15 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__3; -lean_inc(x_12); -x_16 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_16, 0, x_12); -lean_ctor_set(x_16, 1, x_15); -x_17 = l_Lean_expandExplicitBindersAux_loop___closed__6; -x_18 = l_Lean_expandExplicitBindersAux_loop___closed__14; -lean_inc(x_12); -x_19 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_19, 0, x_12); -lean_ctor_set(x_19, 1, x_17); -lean_ctor_set(x_19, 2, x_18); -x_20 = l_Lean_expandExplicitBindersAux_loop___closed__13; -lean_inc(x_12); -x_21 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_21, 0, x_12); -lean_ctor_set(x_21, 1, x_20); -x_22 = l_Lean_expandExplicitBindersAux_loop___closed__12; -lean_inc(x_12); -x_23 = l_Lean_Syntax_node1(x_12, x_22, x_21); -x_24 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__6; -lean_inc(x_12); -x_25 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_25, 0, x_12); -lean_ctor_set(x_25, 1, x_24); -x_26 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__10; -x_27 = l_Lean_addMacroScope(x_14, x_26, x_13); -x_28 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__8; -x_29 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__16; -lean_inc(x_12); -x_30 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_30, 0, x_12); -lean_ctor_set(x_30, 1, x_28); -lean_ctor_set(x_30, 2, x_27); -lean_ctor_set(x_30, 3, x_29); -x_31 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__5; -lean_inc(x_12); -x_32 = l_Lean_Syntax_node4(x_12, x_31, x_19, x_23, x_25, x_30); -lean_inc(x_12); -x_33 = l_Lean_Syntax_node1(x_12, x_17, x_32); -x_34 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__17; -lean_inc(x_12); -x_35 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_35, 0, x_12); -lean_ctor_set(x_35, 1, x_34); -x_36 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__2; -x_37 = l_Lean_Syntax_node4(x_12, x_36, x_16, x_33, x_35, x_9); -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_37); -lean_ctor_set(x_38, 1, x_3); -return x_38; -} -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doElemWhile_:_Do_", 17, 17); -return x_1; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_doElemWhile___x3a__Do_____closed__1; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("while ", 6, 6); -return x_1; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_doElemWhile___x3a__Do_____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_Lean_doElemWhile___x3a__Do_____closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemWhile___x3a__Do_____closed__4; -x_3 = l_Lean_command____Unif__hint________Where___x7c___x2d_u22a2_____closed__16; -x_4 = lean_alloc_ctor(2, 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_doElemWhile___x3a__Do_____closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemWhile___x3a__Do_____closed__5; -x_3 = l_Lean_unbracketedExplicitBinders___closed__16; -x_4 = lean_alloc_ctor(2, 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_doElemWhile___x3a__Do_____closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("termBeforeDo", 12, 12); -return x_1; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_doElemWhile___x3a__Do_____closed__7; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_doElemWhile___x3a__Do_____closed__8; -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_doElemWhile___x3a__Do_____closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemWhile___x3a__Do_____closed__6; -x_3 = l_Lean_doElemWhile___x3a__Do_____closed__9; -x_4 = lean_alloc_ctor(2, 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_doElemWhile___x3a__Do_____closed__11() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" do ", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__12() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_doElemWhile___x3a__Do_____closed__11; -x_2 = lean_alloc_ctor(5, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__13() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemWhile___x3a__Do_____closed__10; -x_3 = l_Lean_doElemWhile___x3a__Do_____closed__12; -x_4 = lean_alloc_ctor(2, 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_doElemWhile___x3a__Do_____closed__14() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemWhile___x3a__Do_____closed__13; -x_3 = l_Lean_doElemRepeat_____closed__7; -x_4 = lean_alloc_ctor(2, 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_doElemWhile___x3a__Do_____closed__15() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_doElemWhile___x3a__Do_____closed__2; -x_2 = lean_unsigned_to_nat(1022u); -x_3 = l_Lean_doElemWhile___x3a__Do_____closed__14; -x_4 = lean_alloc_ctor(3, 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_doElemWhile___x3a__Do__() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_doElemWhile___x3a__Do_____closed__15; -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doSeqIndent", 11, 11); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____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_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____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___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doSeqItem", 9, 9); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___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_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___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___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doIf", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___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_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___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___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doIfProp", 8, 8); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___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_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doBreak", 7, 7); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___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_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___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___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("break", 5, 5); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1(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_doElemWhile___x3a__Do_____closed__2; -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(1); -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; lean_object* x_10; lean_object* x_11; lean_object* x_12; 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; 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; -x_8 = lean_unsigned_to_nat(1u); -x_9 = l_Lean_Syntax_getArg(x_1, x_8); -x_10 = lean_unsigned_to_nat(3u); -x_11 = l_Lean_Syntax_getArg(x_1, x_10); -x_12 = lean_unsigned_to_nat(5u); -x_13 = l_Lean_Syntax_getArg(x_1, x_12); -lean_dec(x_1); -x_14 = lean_ctor_get(x_2, 5); -x_15 = 0; -x_16 = l_Lean_SourceInfo_fromRef(x_14, x_15); -x_17 = l___aux__Init__NotationExtra______macroRules__tacticFunext________1___closed__4; -lean_inc(x_16); -x_18 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_18, 0, x_16); -lean_ctor_set(x_18, 1, x_17); -x_19 = l_unexpandIte___closed__3; -lean_inc(x_16); -x_20 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_20, 0, x_16); -lean_ctor_set(x_20, 1, x_19); -x_21 = l_Lean_expandExplicitBindersAux_loop___closed__18; -lean_inc(x_16); -x_22 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_22, 0, x_16); -lean_ctor_set(x_22, 1, x_21); -x_23 = l_Lean_expandExplicitBindersAux_loop___closed__6; -lean_inc(x_16); -x_24 = l_Lean_Syntax_node2(x_16, x_23, x_9, x_22); -x_25 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8; -lean_inc(x_16); -x_26 = l_Lean_Syntax_node2(x_16, x_25, x_24, x_11); -x_27 = l_unexpandIte___closed__4; -lean_inc(x_16); -x_28 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_28, 0, x_16); -lean_ctor_set(x_28, 1, x_27); -x_29 = l_Lean_expandExplicitBindersAux_loop___closed__14; -lean_inc(x_16); -x_30 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_30, 0, x_16); -lean_ctor_set(x_30, 1, x_23); -lean_ctor_set(x_30, 2, x_29); -x_31 = l_unexpandIte___closed__5; -lean_inc(x_16); -x_32 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_32, 0, x_16); -lean_ctor_set(x_32, 1, x_31); -x_33 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; -lean_inc(x_16); -x_34 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_34, 0, x_16); -lean_ctor_set(x_34, 1, x_33); -x_35 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10; -lean_inc(x_16); -x_36 = l_Lean_Syntax_node1(x_16, x_35, x_34); -x_37 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4; -lean_inc(x_30); -lean_inc(x_16); -x_38 = l_Lean_Syntax_node2(x_16, x_37, x_36, x_30); -lean_inc(x_16); -x_39 = l_Lean_Syntax_node1(x_16, x_23, x_38); -x_40 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2; -lean_inc(x_16); -x_41 = l_Lean_Syntax_node1(x_16, x_40, x_39); -lean_inc(x_16); -x_42 = l_Lean_Syntax_node2(x_16, x_23, x_32, x_41); -x_43 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6; -lean_inc(x_30); -lean_inc(x_16); -x_44 = l_Lean_Syntax_node6(x_16, x_43, x_20, x_26, x_28, x_13, x_30, x_42); -lean_inc(x_16); -x_45 = l_Lean_Syntax_node2(x_16, x_37, x_44, x_30); -lean_inc(x_16); -x_46 = l_Lean_Syntax_node1(x_16, x_23, x_45); -lean_inc(x_16); -x_47 = l_Lean_Syntax_node1(x_16, x_40, x_46); -x_48 = l_Lean_doElemRepeat_____closed__2; -x_49 = l_Lean_Syntax_node2(x_16, x_48, x_18, 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_3); -return x_50; -} -} -} -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1(x_1, x_2, x_3); -lean_dec(x_2); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doElemWhile_Do_", 15, 15); -return x_1; -} -} -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_doElemWhile__Do_____closed__1; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemWhile___x3a__Do_____closed__4; -x_3 = l_Lean_doElemWhile___x3a__Do_____closed__9; -x_4 = lean_alloc_ctor(2, 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_doElemWhile__Do_____closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemWhile__Do_____closed__3; -x_3 = l_Lean_doElemWhile___x3a__Do_____closed__12; -x_4 = lean_alloc_ctor(2, 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_doElemWhile__Do_____closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemWhile__Do_____closed__4; -x_3 = l_Lean_doElemRepeat_____closed__7; -x_4 = lean_alloc_ctor(2, 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_doElemWhile__Do_____closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_doElemWhile__Do_____closed__2; -x_2 = lean_unsigned_to_nat(1022u); -x_3 = l_Lean_doElemWhile__Do_____closed__5; -x_4 = lean_alloc_ctor(3, 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_doElemWhile__Do__() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_doElemWhile__Do_____closed__6; -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1(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_doElemWhile__Do_____closed__2; -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(1); -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; 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; -x_8 = lean_unsigned_to_nat(1u); -x_9 = l_Lean_Syntax_getArg(x_1, x_8); -x_10 = lean_unsigned_to_nat(3u); -x_11 = l_Lean_Syntax_getArg(x_1, x_10); -lean_dec(x_1); -x_12 = lean_ctor_get(x_2, 5); -x_13 = 0; -x_14 = l_Lean_SourceInfo_fromRef(x_12, x_13); -x_15 = l___aux__Init__NotationExtra______macroRules__tacticFunext________1___closed__4; -lean_inc(x_14); -x_16 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_16, 0, x_14); -lean_ctor_set(x_16, 1, x_15); -x_17 = l_unexpandIte___closed__3; -lean_inc(x_14); -x_18 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_18, 0, x_14); -lean_ctor_set(x_18, 1, x_17); -x_19 = l_Lean_expandExplicitBindersAux_loop___closed__6; -x_20 = l_Lean_expandExplicitBindersAux_loop___closed__14; -lean_inc(x_14); -x_21 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_21, 0, x_14); -lean_ctor_set(x_21, 1, x_19); -lean_ctor_set(x_21, 2, x_20); -x_22 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8; -lean_inc(x_21); -lean_inc(x_14); -x_23 = l_Lean_Syntax_node2(x_14, x_22, x_21, x_9); -x_24 = l_unexpandIte___closed__4; -lean_inc(x_14); -x_25 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_25, 0, x_14); -lean_ctor_set(x_25, 1, x_24); -x_26 = l_unexpandIte___closed__5; -lean_inc(x_14); -x_27 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_27, 0, x_14); -lean_ctor_set(x_27, 1, x_26); -x_28 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; -lean_inc(x_14); -x_29 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_29, 0, x_14); -lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10; -lean_inc(x_14); -x_31 = l_Lean_Syntax_node1(x_14, x_30, x_29); -x_32 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4; -lean_inc(x_21); -lean_inc(x_14); -x_33 = l_Lean_Syntax_node2(x_14, x_32, x_31, x_21); -lean_inc(x_14); -x_34 = l_Lean_Syntax_node1(x_14, x_19, x_33); -x_35 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2; -lean_inc(x_14); -x_36 = l_Lean_Syntax_node1(x_14, x_35, x_34); -lean_inc(x_14); -x_37 = l_Lean_Syntax_node2(x_14, x_19, x_27, x_36); -x_38 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6; -lean_inc(x_21); -lean_inc(x_14); -x_39 = l_Lean_Syntax_node6(x_14, x_38, x_18, x_23, x_25, x_11, x_21, x_37); -lean_inc(x_14); -x_40 = l_Lean_Syntax_node2(x_14, x_32, x_39, x_21); -lean_inc(x_14); -x_41 = l_Lean_Syntax_node1(x_14, x_19, x_40); -lean_inc(x_14); -x_42 = l_Lean_Syntax_node1(x_14, x_35, x_41); -x_43 = l_Lean_doElemRepeat_____closed__2; -x_44 = l_Lean_Syntax_node2(x_14, x_43, x_16, x_42); -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_3); -return x_45; -} -} -} -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1(x_1, x_2, x_3); -lean_dec(x_2); -return x_4; -} -} -static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doElemRepeat__Until_", 20, 20); -return x_1; -} -} -static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_doElemRepeat____Until_____closed__1; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemRepeat_____closed__8; -x_3 = l_Lean_solveTactic___closed__7; -x_4 = lean_alloc_ctor(2, 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_doElemRepeat____Until_____closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("until ", 6, 6); -return x_1; -} -} -static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_doElemRepeat____Until_____closed__4; -x_2 = lean_alloc_ctor(5, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemRepeat____Until_____closed__3; -x_3 = l_Lean_doElemRepeat____Until_____closed__5; -x_4 = lean_alloc_ctor(2, 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_doElemRepeat____Until_____closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_doElemRepeat____Until_____closed__6; -x_3 = l_Lean_unbracketedExplicitBinders___closed__19; -x_4 = lean_alloc_ctor(2, 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_doElemRepeat____Until_____closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_doElemRepeat____Until_____closed__2; -x_2 = lean_unsigned_to_nat(1022u); -x_3 = l_Lean_doElemRepeat____Until_____closed__7; -x_4 = lean_alloc_ctor(3, 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_doElemRepeat____Until__() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_doElemRepeat____Until_____closed__8; -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("doNested", 8, 8); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____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_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__1; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1(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_doElemRepeat____Until_____closed__2; -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(1); -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; 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; -x_8 = lean_unsigned_to_nat(1u); -x_9 = l_Lean_Syntax_getArg(x_1, x_8); -x_10 = lean_unsigned_to_nat(3u); -x_11 = l_Lean_Syntax_getArg(x_1, x_10); -lean_dec(x_1); -x_12 = lean_ctor_get(x_2, 5); -x_13 = 0; -x_14 = l_Lean_SourceInfo_fromRef(x_12, x_13); -x_15 = l___aux__Init__NotationExtra______macroRules__tacticFunext________1___closed__4; -lean_inc(x_14); -x_16 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_16, 0, x_14); -lean_ctor_set(x_16, 1, x_15); -x_17 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__17; -lean_inc(x_14); -x_18 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_18, 0, x_14); -lean_ctor_set(x_18, 1, x_17); -x_19 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__2; -lean_inc(x_14); -x_20 = l_Lean_Syntax_node2(x_14, x_19, x_18, x_9); -x_21 = l___aux__Init__NotationExtra______macroRules__tacticFunext________1___lambda__2___closed__9; -lean_inc(x_14); -x_22 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_22, 0, x_14); -lean_ctor_set(x_22, 1, x_21); -x_23 = l_Lean_expandExplicitBindersAux_loop___closed__6; -lean_inc(x_14); -x_24 = l_Lean_Syntax_node1(x_14, x_23, x_22); -x_25 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4; -lean_inc(x_14); -x_26 = l_Lean_Syntax_node2(x_14, x_25, x_20, x_24); -x_27 = l_unexpandIte___closed__3; -lean_inc(x_14); -x_28 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_28, 0, x_14); -lean_ctor_set(x_28, 1, x_27); -x_29 = l_Lean_expandExplicitBindersAux_loop___closed__14; -lean_inc(x_14); -x_30 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_30, 0, x_14); -lean_ctor_set(x_30, 1, x_23); -lean_ctor_set(x_30, 2, x_29); -x_31 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8; -lean_inc(x_30); -lean_inc(x_14); -x_32 = l_Lean_Syntax_node2(x_14, x_31, x_30, x_11); -x_33 = l_unexpandIte___closed__4; -lean_inc(x_14); -x_34 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_34, 0, x_14); -lean_ctor_set(x_34, 1, x_33); -x_35 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; -lean_inc(x_14); -x_36 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_36, 0, x_14); -lean_ctor_set(x_36, 1, x_35); -x_37 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10; -lean_inc(x_14); -x_38 = l_Lean_Syntax_node1(x_14, x_37, x_36); -lean_inc(x_30); -lean_inc(x_14); -x_39 = l_Lean_Syntax_node2(x_14, x_25, x_38, x_30); -lean_inc(x_14); -x_40 = l_Lean_Syntax_node1(x_14, x_23, x_39); -x_41 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2; -lean_inc(x_14); -x_42 = l_Lean_Syntax_node1(x_14, x_41, x_40); -x_43 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6; -lean_inc_n(x_30, 2); -lean_inc(x_14); -x_44 = l_Lean_Syntax_node6(x_14, x_43, x_28, x_32, x_34, x_42, x_30, x_30); -lean_inc(x_14); -x_45 = l_Lean_Syntax_node2(x_14, x_25, x_44, x_30); -lean_inc(x_14); -x_46 = l_Lean_Syntax_node2(x_14, x_23, x_26, x_45); -lean_inc(x_14); -x_47 = l_Lean_Syntax_node1(x_14, x_41, x_46); -x_48 = l_Lean_doElemRepeat_____closed__2; -x_49 = l_Lean_Syntax_node2(x_14, x_48, x_16, 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_3); -return x_50; -} -} -} -LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1(x_1, x_2, x_3); -lean_dec(x_2); -return x_4; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("term_Matches_|", 14, 14); -return x_1; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_term__Matches___x7c___closed__1; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" matches ", 9, 9); -return x_1; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_term__Matches___x7c___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_Lean_term__Matches___x7c___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_unbracketedExplicitBinders___closed__18; -x_2 = lean_unsigned_to_nat(51u); -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_Lean_term__Matches___x7c___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" | ", 3, 3); -return x_1; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_term__Matches___x7c___closed__6; -x_2 = lean_alloc_ctor(5, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c___closed__8() { -_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_term__Matches___x7c___closed__5; -x_2 = l_Lean_term__Matches___x7c___closed__6; -x_3 = l_Lean_term__Matches___x7c___closed__7; -x_4 = 0; -x_5 = lean_alloc_ctor(11, 3, 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_uint8(x_5, sizeof(void*)*3, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c___closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_unbracketedExplicitBinders___closed__5; -x_2 = l_Lean_term__Matches___x7c___closed__4; -x_3 = l_Lean_term__Matches___x7c___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); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_term__Matches___x7c___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_term__Matches___x7c___closed__2; -x_2 = lean_unsigned_to_nat(50u); -x_3 = lean_unsigned_to_nat(51u); -x_4 = l_Lean_term__Matches___x7c___closed__9; -x_5 = lean_alloc_ctor(4, 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_Lean_term__Matches___x7c() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_term__Matches___x7c___closed__10; -return x_1; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___spec__1(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_lt(x_4, x_3); -if (x_6 == 0) -{ -lean_dec(x_2); -lean_dec(x_1); -return x_5; -} -else -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; -x_7 = lean_array_uget(x_5, x_4); -x_8 = lean_unsigned_to_nat(0u); -x_9 = lean_array_uset(x_5, x_4, x_8); -lean_inc(x_2); -lean_inc(x_1); -x_10 = l_Lean_Syntax_node1(x_1, x_2, x_7); -x_11 = 1; -x_12 = lean_usize_add(x_4, x_11); -x_13 = lean_array_uset(x_9, x_4, x_10); -x_4 = x_12; -x_5 = x_13; -goto _start; -} -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___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_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l___aux__Init__NotationExtra______macroRules__tacticFunext________1___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___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("match", 5, 5); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___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_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___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___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("matchDiscr", 10, 10); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__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_Lean_unbracketedExplicitBinders___closed__1; -x_2 = l_Lean_expandExplicitBindersAux_loop___closed__1; -x_3 = l_Lean_expandExplicitBindersAux_loop___closed__2; -x_4 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__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___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("with", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("matchAlts", 9, 9); -return x_1; -} -} -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__8() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; @@ -18036,6 +16557,7 @@ lean_object* initialize_Init_Data_ToString_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Array_Subarray(uint8_t builtin, lean_object*); lean_object* initialize_Init_Conv(uint8_t builtin, lean_object*); lean_object* initialize_Init_Meta(uint8_t builtin, lean_object*); +lean_object* initialize_Init_While(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_NotationExtra(uint8_t builtin, lean_object* w) { lean_object * res; @@ -18053,6 +16575,9 @@ lean_dec_ref(res); res = initialize_Init_Meta(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_While(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_unbracketedExplicitBinders___closed__1 = _init_l_Lean_unbracketedExplicitBinders___closed__1(); lean_mark_persistent(l_Lean_unbracketedExplicitBinders___closed__1); l_Lean_unbracketedExplicitBinders___closed__2 = _init_l_Lean_unbracketedExplicitBinders___closed__2(); @@ -19147,150 +17672,6 @@ l_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___closed lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___closed__4); l_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___closed__5 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___closed__5(); lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__solveTactic__1___closed__5); -l_Lean_doElemRepeat_____closed__1 = _init_l_Lean_doElemRepeat_____closed__1(); -lean_mark_persistent(l_Lean_doElemRepeat_____closed__1); -l_Lean_doElemRepeat_____closed__2 = _init_l_Lean_doElemRepeat_____closed__2(); -lean_mark_persistent(l_Lean_doElemRepeat_____closed__2); -l_Lean_doElemRepeat_____closed__3 = _init_l_Lean_doElemRepeat_____closed__3(); -lean_mark_persistent(l_Lean_doElemRepeat_____closed__3); -l_Lean_doElemRepeat_____closed__4 = _init_l_Lean_doElemRepeat_____closed__4(); -lean_mark_persistent(l_Lean_doElemRepeat_____closed__4); -l_Lean_doElemRepeat_____closed__5 = _init_l_Lean_doElemRepeat_____closed__5(); -lean_mark_persistent(l_Lean_doElemRepeat_____closed__5); -l_Lean_doElemRepeat_____closed__6 = _init_l_Lean_doElemRepeat_____closed__6(); -lean_mark_persistent(l_Lean_doElemRepeat_____closed__6); -l_Lean_doElemRepeat_____closed__7 = _init_l_Lean_doElemRepeat_____closed__7(); -lean_mark_persistent(l_Lean_doElemRepeat_____closed__7); -l_Lean_doElemRepeat_____closed__8 = _init_l_Lean_doElemRepeat_____closed__8(); -lean_mark_persistent(l_Lean_doElemRepeat_____closed__8); -l_Lean_doElemRepeat_____closed__9 = _init_l_Lean_doElemRepeat_____closed__9(); -lean_mark_persistent(l_Lean_doElemRepeat_____closed__9); -l_Lean_doElemRepeat__ = _init_l_Lean_doElemRepeat__(); -lean_mark_persistent(l_Lean_doElemRepeat__); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__1 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__1(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__1); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__2 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__2(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__2); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__3 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__3(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__3); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__4 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__4(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__4); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__5 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__5(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__5); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__6 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__6(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__6); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__7 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__7(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__7); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__8 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__8(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__8); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__9 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__9(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__9); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__10 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__10(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__10); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__11 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__11(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__11); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__12 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__12(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__12); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__13 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__13(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__13); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__14 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__14(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__14); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__15 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__15(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__15); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__16 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__16(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__16); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__17 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__17(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__17); -l_Lean_doElemWhile___x3a__Do_____closed__1 = _init_l_Lean_doElemWhile___x3a__Do_____closed__1(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__1); -l_Lean_doElemWhile___x3a__Do_____closed__2 = _init_l_Lean_doElemWhile___x3a__Do_____closed__2(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__2); -l_Lean_doElemWhile___x3a__Do_____closed__3 = _init_l_Lean_doElemWhile___x3a__Do_____closed__3(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__3); -l_Lean_doElemWhile___x3a__Do_____closed__4 = _init_l_Lean_doElemWhile___x3a__Do_____closed__4(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__4); -l_Lean_doElemWhile___x3a__Do_____closed__5 = _init_l_Lean_doElemWhile___x3a__Do_____closed__5(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__5); -l_Lean_doElemWhile___x3a__Do_____closed__6 = _init_l_Lean_doElemWhile___x3a__Do_____closed__6(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__6); -l_Lean_doElemWhile___x3a__Do_____closed__7 = _init_l_Lean_doElemWhile___x3a__Do_____closed__7(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__7); -l_Lean_doElemWhile___x3a__Do_____closed__8 = _init_l_Lean_doElemWhile___x3a__Do_____closed__8(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__8); -l_Lean_doElemWhile___x3a__Do_____closed__9 = _init_l_Lean_doElemWhile___x3a__Do_____closed__9(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__9); -l_Lean_doElemWhile___x3a__Do_____closed__10 = _init_l_Lean_doElemWhile___x3a__Do_____closed__10(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__10); -l_Lean_doElemWhile___x3a__Do_____closed__11 = _init_l_Lean_doElemWhile___x3a__Do_____closed__11(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__11); -l_Lean_doElemWhile___x3a__Do_____closed__12 = _init_l_Lean_doElemWhile___x3a__Do_____closed__12(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__12); -l_Lean_doElemWhile___x3a__Do_____closed__13 = _init_l_Lean_doElemWhile___x3a__Do_____closed__13(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__13); -l_Lean_doElemWhile___x3a__Do_____closed__14 = _init_l_Lean_doElemWhile___x3a__Do_____closed__14(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__14); -l_Lean_doElemWhile___x3a__Do_____closed__15 = _init_l_Lean_doElemWhile___x3a__Do_____closed__15(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__15); -l_Lean_doElemWhile___x3a__Do__ = _init_l_Lean_doElemWhile___x3a__Do__(); -lean_mark_persistent(l_Lean_doElemWhile___x3a__Do__); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11); -l_Lean_doElemWhile__Do_____closed__1 = _init_l_Lean_doElemWhile__Do_____closed__1(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__1); -l_Lean_doElemWhile__Do_____closed__2 = _init_l_Lean_doElemWhile__Do_____closed__2(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__2); -l_Lean_doElemWhile__Do_____closed__3 = _init_l_Lean_doElemWhile__Do_____closed__3(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__3); -l_Lean_doElemWhile__Do_____closed__4 = _init_l_Lean_doElemWhile__Do_____closed__4(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__4); -l_Lean_doElemWhile__Do_____closed__5 = _init_l_Lean_doElemWhile__Do_____closed__5(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__5); -l_Lean_doElemWhile__Do_____closed__6 = _init_l_Lean_doElemWhile__Do_____closed__6(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__6); -l_Lean_doElemWhile__Do__ = _init_l_Lean_doElemWhile__Do__(); -lean_mark_persistent(l_Lean_doElemWhile__Do__); -l_Lean_doElemRepeat____Until_____closed__1 = _init_l_Lean_doElemRepeat____Until_____closed__1(); -lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__1); -l_Lean_doElemRepeat____Until_____closed__2 = _init_l_Lean_doElemRepeat____Until_____closed__2(); -lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__2); -l_Lean_doElemRepeat____Until_____closed__3 = _init_l_Lean_doElemRepeat____Until_____closed__3(); -lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__3); -l_Lean_doElemRepeat____Until_____closed__4 = _init_l_Lean_doElemRepeat____Until_____closed__4(); -lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__4); -l_Lean_doElemRepeat____Until_____closed__5 = _init_l_Lean_doElemRepeat____Until_____closed__5(); -lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__5); -l_Lean_doElemRepeat____Until_____closed__6 = _init_l_Lean_doElemRepeat____Until_____closed__6(); -lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__6); -l_Lean_doElemRepeat____Until_____closed__7 = _init_l_Lean_doElemRepeat____Until_____closed__7(); -lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__7); -l_Lean_doElemRepeat____Until_____closed__8 = _init_l_Lean_doElemRepeat____Until_____closed__8(); -lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__8); -l_Lean_doElemRepeat____Until__ = _init_l_Lean_doElemRepeat____Until__(); -lean_mark_persistent(l_Lean_doElemRepeat____Until__); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__1 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__1(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__1); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__2 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__2(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____Until____1___closed__2); l_Lean_term__Matches___x7c___closed__1 = _init_l_Lean_term__Matches___x7c___closed__1(); lean_mark_persistent(l_Lean_term__Matches___x7c___closed__1); l_Lean_term__Matches___x7c___closed__2 = _init_l_Lean_term__Matches___x7c___closed__2(); diff --git a/stage0/stdlib/Init/Tactics.c b/stage0/stdlib/Init/Tactics.c index cefc8c1aee82..7ddcdaab450e 100644 --- a/stage0/stdlib/Init/Tactics.c +++ b/stage0/stdlib/Init/Tactics.c @@ -4257,64 +4257,67 @@ 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; 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_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; -x_8 = lean_unsigned_to_nat(1u); +lean_object* x_8; lean_object* x_9; 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; 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; 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_8 = lean_unsigned_to_nat(0u); x_9 = l_Lean_Syntax_getArg(x_1, x_8); -x_10 = lean_unsigned_to_nat(2u); +x_10 = lean_unsigned_to_nat(1u); x_11 = l_Lean_Syntax_getArg(x_1, x_10); -x_12 = lean_unsigned_to_nat(3u); +x_12 = lean_unsigned_to_nat(2u); x_13 = l_Lean_Syntax_getArg(x_1, x_12); +x_14 = lean_unsigned_to_nat(3u); +x_15 = l_Lean_Syntax_getArg(x_1, x_14); lean_dec(x_1); -x_14 = l_Lean_Syntax_getArgs(x_9); +x_16 = l_Lean_Syntax_getArgs(x_11); +lean_dec(x_11); +x_17 = lean_ctor_get(x_2, 5); +x_18 = l_Lean_replaceRef(x_13, x_17); +x_19 = 0; +x_20 = l_Lean_SourceInfo_fromRef(x_18, x_19); +lean_dec(x_18); +x_21 = 1; +x_22 = l_Lean_SourceInfo_fromRef(x_9, x_21); lean_dec(x_9); -x_15 = lean_ctor_get(x_2, 5); -x_16 = l_Lean_replaceRef(x_11, x_15); -x_17 = 0; -x_18 = l_Lean_SourceInfo_fromRef(x_16, x_17); +x_23 = l_Lean_Parser_Tactic_case___closed__1; +x_24 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +x_25 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticExfalso__1___closed__16; +lean_inc(x_20); +x_26 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_26, 0, x_20); +lean_ctor_set(x_26, 1, x_25); +x_27 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__5; +lean_inc(x_20); +x_28 = l_Lean_Syntax_node1(x_20, x_27, x_26); +x_29 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__2; +lean_inc(x_20); +x_30 = l_Lean_Syntax_node1(x_20, x_29, x_28); +x_31 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__6; +x_32 = l_Array_appendCore___rarg(x_31, x_16); lean_dec(x_16); -x_19 = l_Lean_Parser_Tactic_case___closed__1; -lean_inc(x_18); -x_20 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set(x_20, 1, x_19); -x_21 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticExfalso__1___closed__16; -lean_inc(x_18); -x_22 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_22, 0, x_18); -lean_ctor_set(x_22, 1, x_21); -x_23 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__5; -lean_inc(x_18); -x_24 = l_Lean_Syntax_node1(x_18, x_23, x_22); -x_25 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__2; -lean_inc(x_18); -x_26 = l_Lean_Syntax_node1(x_18, x_25, x_24); -x_27 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__6; -x_28 = l_Array_appendCore___rarg(x_27, x_14); -lean_dec(x_14); -x_29 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticExfalso__1___closed__12; -lean_inc(x_18); -x_30 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_30, 0, x_18); -lean_ctor_set(x_30, 1, x_29); -lean_ctor_set(x_30, 2, x_28); -x_31 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__4; -lean_inc(x_18); -x_32 = l_Lean_Syntax_node2(x_18, x_31, x_26, x_30); -lean_inc(x_18); -x_33 = l_Lean_Syntax_node1(x_18, x_29, x_32); -x_34 = 1; -x_35 = l_Lean_SourceInfo_fromRef(x_11, x_34); -lean_dec(x_11); -x_36 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__7; -x_37 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -x_38 = l_Lean_Parser_Tactic_case___closed__2; -x_39 = l_Lean_Syntax_node4(x_18, x_38, x_20, x_33, x_37, x_13); -x_40 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_3); -return x_40; +x_33 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticExfalso__1___closed__12; +lean_inc(x_20); +x_34 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_34, 0, x_20); +lean_ctor_set(x_34, 1, x_33); +lean_ctor_set(x_34, 2, x_32); +x_35 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__4; +lean_inc(x_20); +x_36 = l_Lean_Syntax_node2(x_20, x_35, x_30, x_34); +lean_inc(x_20); +x_37 = l_Lean_Syntax_node1(x_20, x_33, x_36); +x_38 = l_Lean_SourceInfo_fromRef(x_13, x_21); +lean_dec(x_13); +x_39 = l_Lean_Parser_Tactic___aux__Init__Tactics______macroRules__Lean__Parser__Tactic__tacticNext___x3d_x3e____1___closed__7; +x_40 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +x_41 = l_Lean_Parser_Tactic_case___closed__2; +x_42 = l_Lean_Syntax_node4(x_20, x_41, x_24, x_37, x_40, x_15); +x_43 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_43, 1, x_3); +return x_43; } } } diff --git a/stage0/stdlib/Init/While.c b/stage0/stdlib/Init/While.c new file mode 100644 index 000000000000..cbdb412116c6 --- /dev/null +++ b/stage0/stdlib/Init/While.c @@ -0,0 +1,1980 @@ +// Lean compiler output +// Module: Init.While +// Imports: Init.Core +#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_doElemWhile___x3a__Do_____closed__3; +static lean_object* l_Lean_doElemRepeat____Until_____closed__10; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__10; +LEAN_EXPORT lean_object* l_Lean_Loop_toCtorIdx___boxed(lean_object*); +lean_object* lean_mk_empty_array_with_capacity(lean_object*); +static lean_object* l_Lean_doElemRepeat_____closed__11; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__8; +static lean_object* l_Lean_doElemRepeat____Until_____closed__11; +static lean_object* l_Lean_doElemRepeat_____closed__12; +static lean_object* l_Lean_doElemRepeat____Until_____closed__8; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__3; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__1; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4; +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat____Until_____closed__12; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8; +LEAN_EXPORT lean_object* l_Lean_Loop_forIn___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat_____closed__1; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; +static lean_object* l_Lean_doElemRepeat____Until_____closed__5; +uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__2; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__11; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__23; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__14; +LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit(lean_object*, lean_object*); +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__13; +LEAN_EXPORT lean_object* l_Lean_doElemRepeat____Until__; +static lean_object* l_Lean_doElemRepeat____Until_____closed__9; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__14; +lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat_____closed__8; +static lean_object* l_Lean_doElemRepeat_____closed__2; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__18; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__11; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__9; +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile__Do____1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__18; +lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); +lean_object* l_Lean_Syntax_node6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat_____closed__10; +LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___rarg(lean_object*); +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__13; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__25; +static lean_object* l_Lean_doElemRepeat____Until_____closed__15; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__8; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__17; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__22; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat____Until_____closed__4; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5; +static lean_object* l_Lean_doElemRepeat____Until_____closed__17; +static lean_object* l_Lean_doElemWhile__Do_____closed__2; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__17; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__6; +static lean_object* l_Lean_doElemRepeat____Until_____closed__6; +lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__16; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__19; +lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +static lean_object* l_Lean_doElemWhile__Do_____closed__1; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2; +lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__2; +lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat____Until_____closed__16; +LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___rarg___boxed(lean_object*); +static lean_object* l_Lean_doElemRepeat_____closed__6; +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile__Do____1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9; +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat____Until_____closed__7; +lean_object* l_Lean_Syntax_node4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat_____closed__5; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__7; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1; +static lean_object* l_Lean_doElemRepeat____Until_____closed__3; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__19; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__4; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__21; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__6; +static lean_object* l_Lean_doElemRepeat____Until_____closed__2; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__15; +lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__4; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__20; +lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemWhile__Do_____closed__3; +static lean_object* l_Lean_doElemWhile__Do_____closed__6; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__12; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__16; +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__12; +static lean_object* l_Lean_doElemWhile__Do_____closed__5; +static lean_object* l_Lean_doElemRepeat_____closed__7; +LEAN_EXPORT lean_object* l_Lean_Loop_toCtorIdx(lean_object*); +LEAN_EXPORT lean_object* l_Lean_doElemRepeat__; +LEAN_EXPORT lean_object* l_Lean_Loop_forIn___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat_____closed__3; +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat____Until_____closed__1; +LEAN_EXPORT lean_object* l_Lean_doElemWhile___x3a__Do__; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__15; +LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__3; +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__10; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__16; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__1; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__5; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__5; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__20; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__13; +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemRepeat____Until_____closed__13; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__9; +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_doElemWhile__Do__; +static lean_object* l_Lean_doElemRepeat_____closed__4; +static lean_object* l_Lean_doElemRepeat_____closed__9; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__7; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__24; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__15; +lean_object* l_String_toSubstring_x27(lean_object*); +static lean_object* l_Lean_doElemWhile__Do_____closed__4; +static lean_object* l_Lean_doElemRepeat____Until_____closed__14; +static lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__14; +LEAN_EXPORT lean_object* l_Lean_Loop_forIn(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Loop_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_Loop_toCtorIdx___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_Loop_toCtorIdx(x_1); +lean_dec(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___rarg(lean_object* x_1) { +_start: +{ +lean_inc(x_1); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_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_Loop_noConfusion___rarg___boxed), 1, 0); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_noConfusion___rarg___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_Loop_noConfusion___rarg(x_1); +lean_dec(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_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_Loop_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_Loop_forIn_loop___rarg___lambda__1(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_object* x_5; lean_object* x_6; lean_object* x_7; +lean_dec(x_2); +x_4 = lean_ctor_get(x_3, 0); +lean_inc(x_4); +lean_dec(x_3); +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_apply_2(x_6, lean_box(0), x_4); +return x_7; +} +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 = l_Lean_Loop_forIn_loop___rarg(x_1, x_2, x_8); +return x_9; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___rarg(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; +x_4 = lean_ctor_get(x_1, 1); +lean_inc(x_4); +x_5 = lean_box(0); +lean_inc(x_2); +x_6 = lean_apply_2(x_2, x_5, x_3); +x_7 = lean_alloc_closure((void*)(l_Lean_Loop_forIn_loop___rarg___lambda__1), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +x_8 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_6, x_7); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Lean_Loop_forIn_loop___rarg), 3, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_forIn___rarg(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_Loop_forIn_loop___rarg(x_1, x_4, x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_forIn(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Lean_Loop_forIn___rarg___boxed), 4, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_forIn___rarg___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_Loop_forIn___rarg(x_1, x_2, x_3, x_4); +lean_dec(x_2); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit___rarg(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_Loop_forIn_loop___rarg(x_1, x_4, x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Lean_instForInLoopUnit___rarg___boxed), 4, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit___rarg___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_instForInLoopUnit___rarg(x_1, x_2, x_3, x_4); +lean_dec(x_2); +return x_5; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____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_doElemRepeat_____closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doElemRepeat_", 13, 13); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean_doElemRepeat_____closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("andthen", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_doElemRepeat_____closed__4; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("repeat ", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_doElemRepeat_____closed__6; +x_2 = lean_alloc_ctor(5, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doSeq", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_doElemRepeat_____closed__8; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemRepeat_____closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_doElemRepeat_____closed__9; +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_doElemRepeat_____closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemRepeat_____closed__7; +x_3 = l_Lean_doElemRepeat_____closed__10; +x_4 = lean_alloc_ctor(2, 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_doElemRepeat_____closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__3; +x_2 = lean_unsigned_to_nat(1022u); +x_3 = l_Lean_doElemRepeat_____closed__11; +x_4 = lean_alloc_ctor(3, 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_doElemRepeat__() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_doElemRepeat_____closed__12; +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Parser", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Term", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doFor", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___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_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___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___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("for", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("null", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____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___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__6; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doForDecl", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___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_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___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___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__10() { +_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___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__11() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("hole", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___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_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___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___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__13() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("_", 1, 1); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__14() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("in", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__15() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Loop.mk", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__15; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__17() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Loop", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__18() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mk", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__19() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__17; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__18; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__20() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__17; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__18; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____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___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__20; +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___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__22() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__20; +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___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__23() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__22; +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___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__24() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__21; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__23; +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_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__25() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("do", 2, 2); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1(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_doElemRepeat_____closed__3; +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_2); +lean_dec(x_1); +x_6 = lean_box(1); +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; lean_object* x_10; uint8_t 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; +x_8 = lean_unsigned_to_nat(1u); +x_9 = l_Lean_Syntax_getArg(x_1, x_8); +lean_dec(x_1); +x_10 = lean_ctor_get(x_2, 5); +lean_inc(x_10); +x_11 = 0; +x_12 = l_Lean_SourceInfo_fromRef(x_10, x_11); +lean_dec(x_10); +x_13 = lean_ctor_get(x_2, 2); +lean_inc(x_13); +x_14 = lean_ctor_get(x_2, 1); +lean_inc(x_14); +lean_dec(x_2); +x_15 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__5; +lean_inc(x_12); +x_16 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_16, 0, x_12); +lean_ctor_set(x_16, 1, x_15); +x_17 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__7; +x_18 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__10; +lean_inc(x_12); +x_19 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_19, 0, x_12); +lean_ctor_set(x_19, 1, x_17); +lean_ctor_set(x_19, 2, x_18); +x_20 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__13; +lean_inc(x_12); +x_21 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_21, 0, x_12); +lean_ctor_set(x_21, 1, x_20); +x_22 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__12; +lean_inc(x_12); +x_23 = l_Lean_Syntax_node1(x_12, x_22, x_21); +x_24 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__14; +lean_inc(x_12); +x_25 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_25, 0, x_12); +lean_ctor_set(x_25, 1, x_24); +x_26 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__19; +x_27 = l_Lean_addMacroScope(x_14, x_26, x_13); +x_28 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__16; +x_29 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__24; +lean_inc(x_12); +x_30 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_30, 0, x_12); +lean_ctor_set(x_30, 1, x_28); +lean_ctor_set(x_30, 2, x_27); +lean_ctor_set(x_30, 3, x_29); +x_31 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__9; +lean_inc(x_12); +x_32 = l_Lean_Syntax_node4(x_12, x_31, x_19, x_23, x_25, x_30); +lean_inc(x_12); +x_33 = l_Lean_Syntax_node1(x_12, x_17, x_32); +x_34 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__25; +lean_inc(x_12); +x_35 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_35, 0, x_12); +lean_ctor_set(x_35, 1, x_34); +x_36 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__4; +x_37 = l_Lean_Syntax_node4(x_12, x_36, x_16, x_33, x_35, x_9); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_3); +return x_38; +} +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doElemWhile_:_Do_", 17, 17); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("while ", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_doElemWhile___x3a__Do_____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_Lean_doElemWhile___x3a__Do_____closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ident", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__5; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_doElemWhile___x3a__Do_____closed__6; +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_doElemWhile___x3a__Do_____closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__4; +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__7; +x_4 = lean_alloc_ctor(2, 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_doElemWhile___x3a__Do_____closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" : ", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_doElemWhile___x3a__Do_____closed__9; +x_2 = lean_alloc_ctor(5, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__8; +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__10; +x_4 = lean_alloc_ctor(2, 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_doElemWhile___x3a__Do_____closed__12() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("termBeforeDo", 12, 12); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__12; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_doElemWhile___x3a__Do_____closed__13; +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_doElemWhile___x3a__Do_____closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__11; +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__14; +x_4 = lean_alloc_ctor(2, 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_doElemWhile___x3a__Do_____closed__16() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" do ", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__17() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_doElemWhile___x3a__Do_____closed__16; +x_2 = lean_alloc_ctor(5, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__15; +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__17; +x_4 = lean_alloc_ctor(2, 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_doElemWhile___x3a__Do_____closed__19() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__18; +x_3 = l_Lean_doElemRepeat_____closed__10; +x_4 = lean_alloc_ctor(2, 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_doElemWhile___x3a__Do_____closed__20() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemWhile___x3a__Do_____closed__2; +x_2 = lean_unsigned_to_nat(1022u); +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__19; +x_4 = lean_alloc_ctor(3, 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_doElemWhile___x3a__Do__() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_doElemWhile___x3a__Do_____closed__20; +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("repeat", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doSeqIndent", 11, 11); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___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_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___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___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doSeqItem", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____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_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____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___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doIf", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___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_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___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___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("if", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doIfProp", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___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_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___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___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(":", 1, 1); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("then", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__13() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("else", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__14() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doBreak", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___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_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___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___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__16() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("break", 5, 5); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1(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_doElemWhile___x3a__Do_____closed__2; +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(1); +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; lean_object* x_10; lean_object* x_11; lean_object* x_12; 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; 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; +x_8 = lean_unsigned_to_nat(1u); +x_9 = l_Lean_Syntax_getArg(x_1, x_8); +x_10 = lean_unsigned_to_nat(3u); +x_11 = l_Lean_Syntax_getArg(x_1, x_10); +x_12 = lean_unsigned_to_nat(5u); +x_13 = l_Lean_Syntax_getArg(x_1, x_12); +lean_dec(x_1); +x_14 = lean_ctor_get(x_2, 5); +x_15 = 0; +x_16 = l_Lean_SourceInfo_fromRef(x_14, x_15); +x_17 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1; +lean_inc(x_16); +x_18 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +x_19 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8; +lean_inc(x_16); +x_20 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_20, 0, x_16); +lean_ctor_set(x_20, 1, x_19); +x_21 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; +lean_inc(x_16); +x_22 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_22, 0, x_16); +lean_ctor_set(x_22, 1, x_21); +x_23 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__7; +lean_inc(x_16); +x_24 = l_Lean_Syntax_node2(x_16, x_23, x_9, x_22); +x_25 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10; +lean_inc(x_16); +x_26 = l_Lean_Syntax_node2(x_16, x_25, x_24, x_11); +x_27 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12; +lean_inc(x_16); +x_28 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_28, 0, x_16); +lean_ctor_set(x_28, 1, x_27); +x_29 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__10; +lean_inc(x_16); +x_30 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_30, 0, x_16); +lean_ctor_set(x_30, 1, x_23); +lean_ctor_set(x_30, 2, x_29); +x_31 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__13; +lean_inc(x_16); +x_32 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_32, 0, x_16); +lean_ctor_set(x_32, 1, x_31); +x_33 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__16; +lean_inc(x_16); +x_34 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_34, 0, x_16); +lean_ctor_set(x_34, 1, x_33); +x_35 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__15; +lean_inc(x_16); +x_36 = l_Lean_Syntax_node1(x_16, x_35, x_34); +x_37 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5; +lean_inc(x_30); +lean_inc(x_16); +x_38 = l_Lean_Syntax_node2(x_16, x_37, x_36, x_30); +lean_inc(x_16); +x_39 = l_Lean_Syntax_node1(x_16, x_23, x_38); +x_40 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3; +lean_inc(x_16); +x_41 = l_Lean_Syntax_node1(x_16, x_40, x_39); +lean_inc(x_16); +x_42 = l_Lean_Syntax_node2(x_16, x_23, x_32, x_41); +x_43 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; +lean_inc(x_30); +lean_inc(x_16); +x_44 = l_Lean_Syntax_node6(x_16, x_43, x_20, x_26, x_28, x_13, x_30, x_42); +lean_inc(x_16); +x_45 = l_Lean_Syntax_node2(x_16, x_37, x_44, x_30); +lean_inc(x_16); +x_46 = l_Lean_Syntax_node1(x_16, x_23, x_45); +lean_inc(x_16); +x_47 = l_Lean_Syntax_node1(x_16, x_40, x_46); +x_48 = l_Lean_doElemRepeat_____closed__3; +x_49 = l_Lean_Syntax_node2(x_16, x_48, x_18, 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_3); +return x_50; +} +} +} +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemWhile__Do_____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doElemWhile_Do_", 15, 15); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemWhile__Do_____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean_doElemWhile__Do_____closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemWhile__Do_____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__4; +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__14; +x_4 = lean_alloc_ctor(2, 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_doElemWhile__Do_____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemWhile__Do_____closed__3; +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__17; +x_4 = lean_alloc_ctor(2, 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_doElemWhile__Do_____closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemWhile__Do_____closed__4; +x_3 = l_Lean_doElemRepeat_____closed__10; +x_4 = lean_alloc_ctor(2, 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_doElemWhile__Do_____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemWhile__Do_____closed__2; +x_2 = lean_unsigned_to_nat(1022u); +x_3 = l_Lean_doElemWhile__Do_____closed__5; +x_4 = lean_alloc_ctor(3, 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_doElemWhile__Do__() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_doElemWhile__Do_____closed__6; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile__Do____1(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_doElemWhile__Do_____closed__2; +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(1); +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; 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; +x_8 = lean_unsigned_to_nat(1u); +x_9 = l_Lean_Syntax_getArg(x_1, x_8); +x_10 = lean_unsigned_to_nat(3u); +x_11 = l_Lean_Syntax_getArg(x_1, x_10); +lean_dec(x_1); +x_12 = lean_ctor_get(x_2, 5); +x_13 = 0; +x_14 = l_Lean_SourceInfo_fromRef(x_12, x_13); +x_15 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1; +lean_inc(x_14); +x_16 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +x_17 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8; +lean_inc(x_14); +x_18 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_18, 0, x_14); +lean_ctor_set(x_18, 1, x_17); +x_19 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__7; +x_20 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__10; +lean_inc(x_14); +x_21 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_21, 0, x_14); +lean_ctor_set(x_21, 1, x_19); +lean_ctor_set(x_21, 2, x_20); +x_22 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10; +lean_inc(x_21); +lean_inc(x_14); +x_23 = l_Lean_Syntax_node2(x_14, x_22, x_21, x_9); +x_24 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12; +lean_inc(x_14); +x_25 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_25, 0, x_14); +lean_ctor_set(x_25, 1, x_24); +x_26 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__13; +lean_inc(x_14); +x_27 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_27, 0, x_14); +lean_ctor_set(x_27, 1, x_26); +x_28 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__16; +lean_inc(x_14); +x_29 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_29, 0, x_14); +lean_ctor_set(x_29, 1, x_28); +x_30 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__15; +lean_inc(x_14); +x_31 = l_Lean_Syntax_node1(x_14, x_30, x_29); +x_32 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5; +lean_inc(x_21); +lean_inc(x_14); +x_33 = l_Lean_Syntax_node2(x_14, x_32, x_31, x_21); +lean_inc(x_14); +x_34 = l_Lean_Syntax_node1(x_14, x_19, x_33); +x_35 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3; +lean_inc(x_14); +x_36 = l_Lean_Syntax_node1(x_14, x_35, x_34); +lean_inc(x_14); +x_37 = l_Lean_Syntax_node2(x_14, x_19, x_27, x_36); +x_38 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; +lean_inc(x_21); +lean_inc(x_14); +x_39 = l_Lean_Syntax_node6(x_14, x_38, x_18, x_23, x_25, x_11, x_21, x_37); +lean_inc(x_14); +x_40 = l_Lean_Syntax_node2(x_14, x_32, x_39, x_21); +lean_inc(x_14); +x_41 = l_Lean_Syntax_node1(x_14, x_19, x_40); +lean_inc(x_14); +x_42 = l_Lean_Syntax_node1(x_14, x_35, x_41); +x_43 = l_Lean_doElemRepeat_____closed__3; +x_44 = l_Lean_Syntax_node2(x_14, x_43, x_16, x_42); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_3); +return x_45; +} +} +} +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemWhile__Do____1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile__Do____1(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doElemRepeat__Until_", 20, 20); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean_doElemRepeat____Until_____closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ppDedent", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_doElemRepeat____Until_____closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ppLine", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_doElemRepeat____Until_____closed__5; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_doElemRepeat____Until_____closed__6; +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_doElemRepeat____Until_____closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_doElemRepeat____Until_____closed__4; +x_2 = l_Lean_doElemRepeat____Until_____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_Lean_doElemRepeat____Until_____closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemRepeat_____closed__11; +x_3 = l_Lean_doElemRepeat____Until_____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); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__10() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("until ", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_doElemRepeat____Until_____closed__10; +x_2 = lean_alloc_ctor(5, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemRepeat____Until_____closed__9; +x_3 = l_Lean_doElemRepeat____Until_____closed__11; +x_4 = lean_alloc_ctor(2, 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_doElemRepeat____Until_____closed__13() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("term", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_doElemRepeat____Until_____closed__13; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_doElemRepeat____Until_____closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_doElemRepeat____Until_____closed__14; +x_2 = lean_unsigned_to_nat(0u); +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_Lean_doElemRepeat____Until_____closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat_____closed__5; +x_2 = l_Lean_doElemRepeat____Until_____closed__12; +x_3 = l_Lean_doElemRepeat____Until_____closed__15; +x_4 = lean_alloc_ctor(2, 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_doElemRepeat____Until_____closed__17() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemRepeat____Until_____closed__2; +x_2 = lean_unsigned_to_nat(1022u); +x_3 = l_Lean_doElemRepeat____Until_____closed__16; +x_4 = lean_alloc_ctor(3, 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_doElemRepeat____Until__() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_doElemRepeat____Until_____closed__17; +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("doNested", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____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_Lean_doElemRepeat_____closed__1; +x_2 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1; +x_3 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____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___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(";", 1, 1); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1(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_doElemRepeat____Until_____closed__2; +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(1); +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; 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; +x_8 = lean_unsigned_to_nat(1u); +x_9 = l_Lean_Syntax_getArg(x_1, x_8); +x_10 = lean_unsigned_to_nat(3u); +x_11 = l_Lean_Syntax_getArg(x_1, x_10); +lean_dec(x_1); +x_12 = lean_ctor_get(x_2, 5); +x_13 = 0; +x_14 = l_Lean_SourceInfo_fromRef(x_12, x_13); +x_15 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1; +lean_inc(x_14); +x_16 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +x_17 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__25; +lean_inc(x_14); +x_18 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_18, 0, x_14); +lean_ctor_set(x_18, 1, x_17); +x_19 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__2; +lean_inc(x_14); +x_20 = l_Lean_Syntax_node2(x_14, x_19, x_18, x_9); +x_21 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__3; +lean_inc(x_14); +x_22 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_22, 0, x_14); +lean_ctor_set(x_22, 1, x_21); +x_23 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__7; +lean_inc(x_14); +x_24 = l_Lean_Syntax_node1(x_14, x_23, x_22); +x_25 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5; +lean_inc(x_14); +x_26 = l_Lean_Syntax_node2(x_14, x_25, x_20, x_24); +x_27 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8; +lean_inc(x_14); +x_28 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_28, 0, x_14); +lean_ctor_set(x_28, 1, x_27); +x_29 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__10; +lean_inc(x_14); +x_30 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_30, 0, x_14); +lean_ctor_set(x_30, 1, x_23); +lean_ctor_set(x_30, 2, x_29); +x_31 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10; +lean_inc(x_30); +lean_inc(x_14); +x_32 = l_Lean_Syntax_node2(x_14, x_31, x_30, x_11); +x_33 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12; +lean_inc(x_14); +x_34 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_34, 0, x_14); +lean_ctor_set(x_34, 1, x_33); +x_35 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__16; +lean_inc(x_14); +x_36 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_36, 0, x_14); +lean_ctor_set(x_36, 1, x_35); +x_37 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__15; +lean_inc(x_14); +x_38 = l_Lean_Syntax_node1(x_14, x_37, x_36); +lean_inc(x_30); +lean_inc(x_14); +x_39 = l_Lean_Syntax_node2(x_14, x_25, x_38, x_30); +lean_inc(x_14); +x_40 = l_Lean_Syntax_node1(x_14, x_23, x_39); +x_41 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3; +lean_inc(x_14); +x_42 = l_Lean_Syntax_node1(x_14, x_41, x_40); +x_43 = l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; +lean_inc_n(x_30, 2); +lean_inc(x_14); +x_44 = l_Lean_Syntax_node6(x_14, x_43, x_28, x_32, x_34, x_42, x_30, x_30); +lean_inc(x_14); +x_45 = l_Lean_Syntax_node2(x_14, x_25, x_44, x_30); +lean_inc(x_14); +x_46 = l_Lean_Syntax_node2(x_14, x_23, x_26, x_45); +lean_inc(x_14); +x_47 = l_Lean_Syntax_node1(x_14, x_41, x_46); +x_48 = l_Lean_doElemRepeat_____closed__3; +x_49 = l_Lean_Syntax_node2(x_14, x_48, x_16, 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_3); +return x_50; +} +} +} +LEAN_EXPORT lean_object* l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} +lean_object* initialize_Init_Core(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Init_While(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); +l_Lean_doElemRepeat_____closed__1 = _init_l_Lean_doElemRepeat_____closed__1(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__1); +l_Lean_doElemRepeat_____closed__2 = _init_l_Lean_doElemRepeat_____closed__2(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__2); +l_Lean_doElemRepeat_____closed__3 = _init_l_Lean_doElemRepeat_____closed__3(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__3); +l_Lean_doElemRepeat_____closed__4 = _init_l_Lean_doElemRepeat_____closed__4(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__4); +l_Lean_doElemRepeat_____closed__5 = _init_l_Lean_doElemRepeat_____closed__5(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__5); +l_Lean_doElemRepeat_____closed__6 = _init_l_Lean_doElemRepeat_____closed__6(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__6); +l_Lean_doElemRepeat_____closed__7 = _init_l_Lean_doElemRepeat_____closed__7(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__7); +l_Lean_doElemRepeat_____closed__8 = _init_l_Lean_doElemRepeat_____closed__8(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__8); +l_Lean_doElemRepeat_____closed__9 = _init_l_Lean_doElemRepeat_____closed__9(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__9); +l_Lean_doElemRepeat_____closed__10 = _init_l_Lean_doElemRepeat_____closed__10(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__10); +l_Lean_doElemRepeat_____closed__11 = _init_l_Lean_doElemRepeat_____closed__11(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__11); +l_Lean_doElemRepeat_____closed__12 = _init_l_Lean_doElemRepeat_____closed__12(); +lean_mark_persistent(l_Lean_doElemRepeat_____closed__12); +l_Lean_doElemRepeat__ = _init_l_Lean_doElemRepeat__(); +lean_mark_persistent(l_Lean_doElemRepeat__); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__1); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__2); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__3 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__3(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__3); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__4 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__4(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__4); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__5 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__5(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__5); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__6 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__6(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__6); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__7 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__7(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__7); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__8 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__8(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__8); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__9 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__9(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__9); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__10 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__10(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__10); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__11 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__11(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__11); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__12 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__12(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__12); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__13 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__13(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__13); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__14 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__14(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__14); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__15 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__15(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__15); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__16 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__16(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__16); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__17 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__17(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__17); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__18 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__18(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__18); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__19 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__19(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__19); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__20 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__20(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__20); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__21 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__21(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__21); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__22 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__22(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__22); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__23 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__23(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__23); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__24 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__24(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__24); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__25 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__25(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____1___closed__25); +l_Lean_doElemWhile___x3a__Do_____closed__1 = _init_l_Lean_doElemWhile___x3a__Do_____closed__1(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__1); +l_Lean_doElemWhile___x3a__Do_____closed__2 = _init_l_Lean_doElemWhile___x3a__Do_____closed__2(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__2); +l_Lean_doElemWhile___x3a__Do_____closed__3 = _init_l_Lean_doElemWhile___x3a__Do_____closed__3(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__3); +l_Lean_doElemWhile___x3a__Do_____closed__4 = _init_l_Lean_doElemWhile___x3a__Do_____closed__4(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__4); +l_Lean_doElemWhile___x3a__Do_____closed__5 = _init_l_Lean_doElemWhile___x3a__Do_____closed__5(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__5); +l_Lean_doElemWhile___x3a__Do_____closed__6 = _init_l_Lean_doElemWhile___x3a__Do_____closed__6(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__6); +l_Lean_doElemWhile___x3a__Do_____closed__7 = _init_l_Lean_doElemWhile___x3a__Do_____closed__7(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__7); +l_Lean_doElemWhile___x3a__Do_____closed__8 = _init_l_Lean_doElemWhile___x3a__Do_____closed__8(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__8); +l_Lean_doElemWhile___x3a__Do_____closed__9 = _init_l_Lean_doElemWhile___x3a__Do_____closed__9(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__9); +l_Lean_doElemWhile___x3a__Do_____closed__10 = _init_l_Lean_doElemWhile___x3a__Do_____closed__10(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__10); +l_Lean_doElemWhile___x3a__Do_____closed__11 = _init_l_Lean_doElemWhile___x3a__Do_____closed__11(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__11); +l_Lean_doElemWhile___x3a__Do_____closed__12 = _init_l_Lean_doElemWhile___x3a__Do_____closed__12(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__12); +l_Lean_doElemWhile___x3a__Do_____closed__13 = _init_l_Lean_doElemWhile___x3a__Do_____closed__13(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__13); +l_Lean_doElemWhile___x3a__Do_____closed__14 = _init_l_Lean_doElemWhile___x3a__Do_____closed__14(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__14); +l_Lean_doElemWhile___x3a__Do_____closed__15 = _init_l_Lean_doElemWhile___x3a__Do_____closed__15(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__15); +l_Lean_doElemWhile___x3a__Do_____closed__16 = _init_l_Lean_doElemWhile___x3a__Do_____closed__16(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__16); +l_Lean_doElemWhile___x3a__Do_____closed__17 = _init_l_Lean_doElemWhile___x3a__Do_____closed__17(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__17); +l_Lean_doElemWhile___x3a__Do_____closed__18 = _init_l_Lean_doElemWhile___x3a__Do_____closed__18(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__18); +l_Lean_doElemWhile___x3a__Do_____closed__19 = _init_l_Lean_doElemWhile___x3a__Do_____closed__19(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__19); +l_Lean_doElemWhile___x3a__Do_____closed__20 = _init_l_Lean_doElemWhile___x3a__Do_____closed__20(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__20); +l_Lean_doElemWhile___x3a__Do__ = _init_l_Lean_doElemWhile___x3a__Do__(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do__); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__13 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__13(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__13); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__14 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__14(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__14); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__15 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__15(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__15); +l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__16 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__16(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemWhile___x3a__Do____1___closed__16); +l_Lean_doElemWhile__Do_____closed__1 = _init_l_Lean_doElemWhile__Do_____closed__1(); +lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__1); +l_Lean_doElemWhile__Do_____closed__2 = _init_l_Lean_doElemWhile__Do_____closed__2(); +lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__2); +l_Lean_doElemWhile__Do_____closed__3 = _init_l_Lean_doElemWhile__Do_____closed__3(); +lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__3); +l_Lean_doElemWhile__Do_____closed__4 = _init_l_Lean_doElemWhile__Do_____closed__4(); +lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__4); +l_Lean_doElemWhile__Do_____closed__5 = _init_l_Lean_doElemWhile__Do_____closed__5(); +lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__5); +l_Lean_doElemWhile__Do_____closed__6 = _init_l_Lean_doElemWhile__Do_____closed__6(); +lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__6); +l_Lean_doElemWhile__Do__ = _init_l_Lean_doElemWhile__Do__(); +lean_mark_persistent(l_Lean_doElemWhile__Do__); +l_Lean_doElemRepeat____Until_____closed__1 = _init_l_Lean_doElemRepeat____Until_____closed__1(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__1); +l_Lean_doElemRepeat____Until_____closed__2 = _init_l_Lean_doElemRepeat____Until_____closed__2(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__2); +l_Lean_doElemRepeat____Until_____closed__3 = _init_l_Lean_doElemRepeat____Until_____closed__3(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__3); +l_Lean_doElemRepeat____Until_____closed__4 = _init_l_Lean_doElemRepeat____Until_____closed__4(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__4); +l_Lean_doElemRepeat____Until_____closed__5 = _init_l_Lean_doElemRepeat____Until_____closed__5(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__5); +l_Lean_doElemRepeat____Until_____closed__6 = _init_l_Lean_doElemRepeat____Until_____closed__6(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__6); +l_Lean_doElemRepeat____Until_____closed__7 = _init_l_Lean_doElemRepeat____Until_____closed__7(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__7); +l_Lean_doElemRepeat____Until_____closed__8 = _init_l_Lean_doElemRepeat____Until_____closed__8(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__8); +l_Lean_doElemRepeat____Until_____closed__9 = _init_l_Lean_doElemRepeat____Until_____closed__9(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__9); +l_Lean_doElemRepeat____Until_____closed__10 = _init_l_Lean_doElemRepeat____Until_____closed__10(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__10); +l_Lean_doElemRepeat____Until_____closed__11 = _init_l_Lean_doElemRepeat____Until_____closed__11(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__11); +l_Lean_doElemRepeat____Until_____closed__12 = _init_l_Lean_doElemRepeat____Until_____closed__12(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__12); +l_Lean_doElemRepeat____Until_____closed__13 = _init_l_Lean_doElemRepeat____Until_____closed__13(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__13); +l_Lean_doElemRepeat____Until_____closed__14 = _init_l_Lean_doElemRepeat____Until_____closed__14(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__14); +l_Lean_doElemRepeat____Until_____closed__15 = _init_l_Lean_doElemRepeat____Until_____closed__15(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__15); +l_Lean_doElemRepeat____Until_____closed__16 = _init_l_Lean_doElemRepeat____Until_____closed__16(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__16); +l_Lean_doElemRepeat____Until_____closed__17 = _init_l_Lean_doElemRepeat____Until_____closed__17(); +lean_mark_persistent(l_Lean_doElemRepeat____Until_____closed__17); +l_Lean_doElemRepeat____Until__ = _init_l_Lean_doElemRepeat____Until__(); +lean_mark_persistent(l_Lean_doElemRepeat____Until__); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__1 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__1(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__1); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__2 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__2(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__2); +l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__3 = _init_l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__3(); +lean_mark_persistent(l_Lean___aux__Init__While______macroRules__Lean__doElemRepeat____Until____1___closed__3); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lake/Build/Common.c b/stage0/stdlib/Lake/Build/Common.c index d8c313ce6108..71ec0bf8bbec 100644 --- a/stage0/stdlib/Lake/Build/Common.c +++ b/stage0/stdlib/Lake/Build/Common.c @@ -190,6 +190,7 @@ lean_object* l_Array_extract___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Substring_nextn(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_buildFileAfterDep(lean_object*); LEAN_EXPORT lean_object* l_IO_withStderr___at_Lake_buildFileAfterDep___spec__4(lean_object*, lean_object*, lean_object*, 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_Lake_computeDynlibOfShared___lambda__2___closed__7; 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*); LEAN_EXPORT lean_object* l_Lake_computeDynlibOfShared(lean_object*, lean_object*, lean_object*); @@ -219,7 +220,6 @@ lean_object* l_Substring_takeRightWhileAux___at_Substring_trimRight___spec__1(le LEAN_EXPORT lean_object* l_Lake_buildUnlessUpToDate_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_buildO___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_buildLeanSharedLibOfStatic___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_List_bindTR_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_Lake_computeDynlibOfShared___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_computeDynlibOfShared___lambda__2___closed__3; lean_object* l_Array_mapMUnsafe_map___at_Lake_instFromJsonLog___spec__1(size_t, size_t, lean_object*); @@ -393,7 +393,7 @@ x_19 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_19, 0, x_9); lean_ctor_set(x_19, 1, x_18); x_20 = l___private_Lake_Build_Common_0__Lake_toJsonBuildMetadata____x40_Lake_Build_Common___hyg_31____closed__3; -x_21 = l_List_bindTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_19, x_20); +x_21 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_19, x_20); x_22 = l_Lean_Json_mkObj(x_21); return x_22; } diff --git a/stage0/stdlib/Lake/Build/Facets.c b/stage0/stdlib/Lake/Build/Facets.c index 52ad5de8b9f1..7bfd127b6ba6 100644 --- a/stage0/stdlib/Lake/Build/Facets.c +++ b/stage0/stdlib/Lake/Build/Facets.c @@ -15,29 +15,35 @@ extern "C" { #endif static lean_object* l_Lake_Module_cFacet___closed__2; static lean_object* l_Lake_Module_coNoExportFacet___closed__2; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__7; lean_object* l_Lean_Name_reprPrec(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Module_coExportFacet; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__9; static lean_object* l_Lake_Module_ileanFacet___closed__2; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__2; LEAN_EXPORT lean_object* l_Lake_instCoeDepNameModuleFacetOfFamilyOutModuleData___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_Package_reservoirBarrelFacet___closed__1; LEAN_EXPORT lean_object* l_Lake_instReprModuleFacet___boxed(lean_object*, lean_object*); +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__17; static lean_object* l_Lake_ExternLib_staticFacet___closed__2; static lean_object* l_Lake_ExternLib_dynlibFacet___closed__2; static lean_object* l_Lake_Package_gitHubReleaseFacet___closed__1; static lean_object* l_Lake_Module_oFacet___closed__1; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__18; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__2; LEAN_EXPORT lean_object* l_Lake_ExternLib_sharedFacet; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__9; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__15; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__12; LEAN_EXPORT lean_object* l_Lake_Module_cFacet; static lean_object* l_Lake_ExternLib_staticFacet___closed__1; LEAN_EXPORT lean_object* l_Lake_ExternLib_dynlibFacet; static lean_object* l_Lake_Package_extraDepFacet___closed__1; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__13; -LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Module_ileanFacet; static lean_object* l_Lake_Module_leanArtsFacet___closed__1; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__4; static lean_object* l_Lake_Package_gitHubReleaseFacet___closed__2; LEAN_EXPORT lean_object* l_Lake_Module_depsFacet; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__10; LEAN_EXPORT lean_object* l_Lake_LeanLib_extraDepFacet; static lean_object* l_Lake_Module_bcFacet___closed__2; LEAN_EXPORT lean_object* l_Lake_Dynlib_dir_x3f(lean_object*); @@ -45,32 +51,31 @@ static lean_object* l_Lake_Module_ileanFacet___closed__1; LEAN_EXPORT lean_object* l_Lake_Package_gitHubReleaseFacet; LEAN_EXPORT lean_object* l_Lake_Module_coNoExportFacet; static lean_object* l_Lake_instReprModuleFacet___closed__1; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__5; static lean_object* l_Lake_Package_reservoirBarrelFacet___closed__2; lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__11; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__17; LEAN_EXPORT lean_object* l_Lake_LeanExe_exeFacet; -LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___boxed(lean_object*, lean_object*); static lean_object* l_Lake_Module_bcoFacet___closed__1; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__8; static lean_object* l_Lake_Module_oleanFacet___closed__2; static lean_object* l_Lake_LeanLib_staticFacet___closed__1; static lean_object* l_Lake_LeanLib_sharedFacet___closed__2; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__19; +LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____boxed(lean_object*, lean_object*); lean_object* lean_nat_to_int(lean_object*); static lean_object* l_Lake_LeanLib_sharedFacet___closed__1; static lean_object* l_Lake_Package_buildCacheFacet___closed__2; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__14; LEAN_EXPORT lean_object* l_Lake_LeanLib_leanArtsFacet; LEAN_EXPORT lean_object* l_Lake_Module_leanArtsFacet; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__16; +LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66_(lean_object*, lean_object*); +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__11; static lean_object* l_Lake_Module_coExportFacet___closed__2; static lean_object* l_Lake_Module_oleanFacet___closed__1; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__14; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__5; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__13; LEAN_EXPORT lean_object* l_Lake_Module_bcFacet; static lean_object* l_Lake_Package_optReservoirBarrelFacet___closed__1; -LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg(lean_object*, lean_object*); +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__16; lean_object* l_System_FilePath_parent(lean_object*); -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__18; static lean_object* l_Lake_Module_oExportFacet___closed__1; static lean_object* l_Lake_LeanLib_staticExportFacet___closed__1; static lean_object* l_Lake_LeanLib_staticFacet___closed__2; @@ -78,55 +83,50 @@ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_instCoeDepNameModuleFacetOfFamilyOutModuleData(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_Package_buildCacheFacet___closed__1; static lean_object* l_Lake_ExternLib_sharedFacet___closed__1; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__12; static lean_object* l_Lake_LeanExe_exeFacet___closed__1; LEAN_EXPORT lean_object* l_Lake_LeanLib_staticFacet; static lean_object* l_Lake_Module_coFacet___closed__2; LEAN_EXPORT lean_object* l_Lake_Package_buildCacheFacet; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__15; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__10; static lean_object* l_Lake_Package_optBuildCacheFacet___closed__1; static lean_object* l_Lake_Module_depsFacet___closed__2; LEAN_EXPORT lean_object* l_Lake_LeanLib_staticExportFacet; +LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Package_extraDepFacet; lean_object* lean_string_length(lean_object*); static lean_object* l_Lake_Package_optGitHubReleaseFacet___closed__2; static lean_object* l_Lake_Package_optReservoirBarrelFacet___closed__2; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__3; static lean_object* l_Lake_Module_coNoExportFacet___closed__1; static lean_object* l_Lake_Module_leanArtsFacet___closed__2; -LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Package_optGitHubReleaseFacet; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l_Lake_ExternLib_dynlibFacet___closed__1; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__8; LEAN_EXPORT lean_object* l_Lake_Module_coFacet; static lean_object* l_Lake_Module_cFacet___closed__1; LEAN_EXPORT lean_object* l_Lake_Module_bcoFacet; LEAN_EXPORT lean_object* l_Lake_Module_oExportFacet; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__6; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__19; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__1; LEAN_EXPORT lean_object* l_Lake_Package_releaseFacet; static lean_object* l_Lake_Package_optBuildCacheFacet___closed__2; LEAN_EXPORT lean_object* l_Lake_instReprModuleFacet(lean_object*, lean_object*); static lean_object* l_Lake_Module_coFacet___closed__1; static lean_object* l_Lake_Package_extraDepFacet___closed__2; LEAN_EXPORT lean_object* l_Lake_Dynlib_dir_x3f___boxed(lean_object*); -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__6; LEAN_EXPORT lean_object* l_Lake_ExternLib_staticFacet; LEAN_EXPORT lean_object* l_Lake_Module_oNoExportFacet; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__4; LEAN_EXPORT lean_object* l_Lake_Package_reservoirBarrelFacet; LEAN_EXPORT lean_object* l_Lake_Package_optBuildCacheFacet; static lean_object* l_Lake_Package_optGitHubReleaseFacet___closed__1; static lean_object* l_Lake_Module_depsFacet___closed__1; static lean_object* l_Lake_Module_coExportFacet___closed__1; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__1; LEAN_EXPORT lean_object* l_Lake_LeanLib_sharedFacet; +static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__3; LEAN_EXPORT lean_object* l_Lake_Module_oleanFacet; static lean_object* l_Lake_Module_oNoExportFacet___closed__1; LEAN_EXPORT lean_object* l_Lake_Module_oFacet; static lean_object* l_Lake_LeanExe_exeFacet___closed__2; LEAN_EXPORT lean_object* l_Lake_Package_optReleaseFacet; -static lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__7; LEAN_EXPORT lean_object* l_Lake_Package_optReservoirBarrelFacet; static lean_object* l_Lake_Module_bcFacet___closed__1; LEAN_EXPORT lean_object* l_Lake_Dynlib_dir_x3f(lean_object* x_1) { @@ -147,7 +147,7 @@ lean_dec(x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__1() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__1() { _start: { lean_object* x_1; @@ -155,29 +155,29 @@ x_1 = lean_mk_string_unchecked("name", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__2() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__1; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___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_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__3() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__2; +x_2 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___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_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__4() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__4() { _start: { lean_object* x_1; @@ -185,29 +185,29 @@ x_1 = lean_mk_string_unchecked(" := ", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__5() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__4; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___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_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__6() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__3; -x_2 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__5; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__3; +x_2 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___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_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__7() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__7() { _start: { lean_object* x_1; lean_object* x_2; @@ -216,7 +216,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__8() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__8() { _start: { lean_object* x_1; @@ -224,17 +224,17 @@ x_1 = lean_mk_string_unchecked(",", 1, 1); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__9() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__8; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___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_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__10() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__10() { _start: { lean_object* x_1; @@ -242,17 +242,17 @@ x_1 = lean_mk_string_unchecked("data_eq", 7, 7); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__11() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__11() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__10; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___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_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__12() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__12() { _start: { lean_object* x_1; @@ -260,17 +260,17 @@ x_1 = lean_mk_string_unchecked("_", 1, 1); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__13() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__13() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__12; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___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_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__14() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__14() { _start: { lean_object* x_1; @@ -278,35 +278,35 @@ x_1 = lean_mk_string_unchecked("{ ", 2, 2); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__15() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__15() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__14; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__14; x_2 = lean_string_length(x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__16() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__16() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__15; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__15; x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__17() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__17() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__14; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___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_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__18() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__18() { _start: { lean_object* x_1; @@ -314,23 +314,23 @@ x_1 = lean_mk_string_unchecked(" }", 2, 2); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__19() { +static lean_object* _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__19() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__18; +x_1 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__18; 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_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____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; 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; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; x_3 = lean_unsigned_to_nat(0u); x_4 = l_Lean_Name_reprPrec(x_1, x_3); -x_5 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__7; +x_5 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__7; x_6 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_6, 0, x_5); lean_ctor_set(x_6, 1, x_4); @@ -338,11 +338,11 @@ x_7 = 0; x_8 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_8, 0, x_6); lean_ctor_set_uint8(x_8, sizeof(void*)*1, x_7); -x_9 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__6; +x_9 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__6; x_10 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_10, 0, x_9); lean_ctor_set(x_10, 1, x_8); -x_11 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__9; +x_11 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__9; x_12 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_12, 0, x_10); lean_ctor_set(x_12, 1, x_11); @@ -350,27 +350,27 @@ x_13 = lean_box(1); x_14 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_14, 0, x_12); lean_ctor_set(x_14, 1, x_13); -x_15 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__11; +x_15 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__11; x_16 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); -x_17 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__5; +x_17 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__5; x_18 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_18, 0, x_16); lean_ctor_set(x_18, 1, x_17); -x_19 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__13; +x_19 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__13; 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 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__17; +x_21 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__17; x_22 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_22, 0, x_21); lean_ctor_set(x_22, 1, x_20); -x_23 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__19; +x_23 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__19; 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_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__16; +x_25 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__16; x_26 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_26, 0, x_25); lean_ctor_set(x_26, 1, x_24); @@ -380,28 +380,28 @@ lean_ctor_set_uint8(x_27, sizeof(void*)*1, x_7); return x_27; } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66_(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___boxed), 2, 0); +x_3 = lean_alloc_closure((void*)(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___boxed), 2, 0); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg(x_1, x_2); +x_3 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg(x_1, x_2); lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65_(x_1, x_2); +x_3 = l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66_(x_1, x_2); lean_dec(x_2); return x_3; } @@ -410,7 +410,7 @@ static lean_object* _init_l_Lake_instReprModuleFacet___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___boxed), 2, 0); return x_1; } } @@ -1152,44 +1152,44 @@ lean_dec_ref(res); res = initialize_Lake_Build_Data(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__1 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__1(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__1); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__2 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__2(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__2); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__3 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__3(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__3); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__4 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__4(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__4); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__5 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__5(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__5); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__6 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__6(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__6); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__7 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__7(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__7); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__8 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__8(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__8); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__9 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__9(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__9); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__10 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__10(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__10); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__11 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__11(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__11); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__12 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__12(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__12); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__13 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__13(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__13); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__14 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__14(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__14); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__15 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__15(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__15); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__16 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__16(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__16); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__17 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__17(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__17); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__18 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__18(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__18); -l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__19 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__19(); -lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_65____rarg___closed__19); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__1 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__1(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__1); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__2 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__2(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__2); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__3 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__3(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__3); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__4 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__4(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__4); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__5 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__5(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__5); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__6 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__6(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__6); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__7 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__7(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__7); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__8 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__8(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__8); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__9 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__9(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__9); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__10 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__10(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__10); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__11 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__11(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__11); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__12 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__12(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__12); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__13 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__13(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__13); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__14 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__14(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__14); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__15 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__15(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__15); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__16 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__16(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__16); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__17 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__17(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__17); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__18 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__18(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__18); +l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__19 = _init_l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__19(); +lean_mark_persistent(l___private_Lake_Build_Facets_0__Lake_reprModuleFacet____x40_Lake_Build_Facets___hyg_66____rarg___closed__19); l_Lake_instReprModuleFacet___closed__1 = _init_l_Lake_instReprModuleFacet___closed__1(); lean_mark_persistent(l_Lake_instReprModuleFacet___closed__1); l_Lake_Module_depsFacet___closed__1 = _init_l_Lake_Module_depsFacet___closed__1(); diff --git a/stage0/stdlib/Lake/Build/Index.c b/stage0/stdlib/Lake/Build/Index.c index 404039800d43..260b4e3ad000 100644 --- a/stage0/stdlib/Lake/Build/Index.c +++ b/stage0/stdlib/Lake/Build/Index.c @@ -46,7 +46,6 @@ static lean_object* l_Lake_ExternLib_recBuildStatic___closed__4; lean_object* l_Lake_withRegisterJob___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_EquipT_map___at_Lake_ExternLib_recBuildStatic___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_partition_loop___at_Lake_FetchM_run___spec__5___boxed(lean_object*, lean_object*, lean_object*); -uint8_t l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325_(lean_object*, lean_object*); lean_object* l_Lake_Workspace_findLibraryFacetConfig_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_ExternLib_recBuildShared(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_EquipT_map___at_Lake_ExternLib_recBuildStatic___spec__1(lean_object*, lean_object*); @@ -84,6 +83,7 @@ lean_object* lean_array_mk(lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); uint8_t l_Lake_BuildKey_quickCmp(lean_object*, lean_object*); +uint8_t l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_FetchM_run(lean_object*); LEAN_EXPORT lean_object* l_Lake_mkTargetFacetBuild___boxed(lean_object*, lean_object*); lean_object* l_Lake_LeanExe_recBuildExe(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1350,7 +1350,7 @@ 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, 1); -x_6 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325_(x_1, x_4); +x_6 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326_(x_1, x_4); if (x_6 == 0) { x_2 = x_5; @@ -3852,7 +3852,7 @@ x_16 = lean_ctor_get(x_2, 0); x_17 = lean_ctor_get(x_2, 1); x_18 = lean_ctor_get(x_3, 0); x_19 = lean_ctor_get(x_3, 1); -x_20 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325_(x_16, x_1); +x_20 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326_(x_16, x_1); if (x_20 == 0) { lean_ctor_set(x_2, 1, x_18); @@ -3878,7 +3878,7 @@ x_26 = lean_ctor_get(x_3, 1); lean_inc(x_26); lean_inc(x_25); lean_dec(x_3); -x_27 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325_(x_23, x_1); +x_27 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326_(x_23, x_1); if (x_27 == 0) { lean_object* x_28; @@ -3923,7 +3923,7 @@ if (lean_is_exclusive(x_3)) { lean_dec_ref(x_3); x_36 = lean_box(0); } -x_37 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325_(x_32, x_1); +x_37 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326_(x_32, x_1); if (x_37 == 0) { lean_object* x_38; lean_object* x_39; diff --git a/stage0/stdlib/Lake/Build/Key.c b/stage0/stdlib/Lake/Build/Key.c index fd77dd167432..849128964e10 100644 --- a/stage0/stdlib/Lake/Build/Key.c +++ b/stage0/stdlib/Lake/Build/Key.c @@ -13,32 +13,32 @@ #ifdef __cplusplus extern "C" { #endif -LEAN_EXPORT uint64_t l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1274_(lean_object*); lean_object* l_Lean_Name_reprPrec(lean_object*, lean_object*); -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__6; -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1274____boxed(lean_object*); +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_93____rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1275____boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__1_splitter(lean_object*); -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325____boxed(lean_object*, lean_object*); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__2; +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326____boxed(lean_object*, lean_object*); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__9; uint64_t lean_uint64_mix_hash(uint64_t, uint64_t); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__13; lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_92____rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__8; -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__9; -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__14; -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____boxed(lean_object*, lean_object*); -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__12; -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_92_(lean_object*); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__7; +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_93_(lean_object*); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__8; +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__14; LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__4_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__3; LEAN_EXPORT lean_object* l_Lake_BuildKey_quickCmp___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__5_splitter(lean_object*); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__12; static lean_object* l_Lake_instInhabitedBuildKey___closed__1; +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__2_splitter(lean_object*); lean_object* lean_nat_to_int(lean_object*); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__3; LEAN_EXPORT lean_object* l_Lake_instReprBuildKey; -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__1; LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__3_splitter(lean_object*); -LEAN_EXPORT uint8_t l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325_(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____boxed(lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_BuildKey_toSimpleString(lean_object*); LEAN_EXPORT lean_object* l_Lake_BuildKey_toSimpleString_eraseHead(lean_object*); @@ -47,7 +47,10 @@ LEAN_EXPORT lean_object* l_Lake_BuildKey_toString(lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lake_BuildKey_toString___closed__1; -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92_(lean_object*, lean_object*); +LEAN_EXPORT uint64_t l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1275_(lean_object*); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5; +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__6; +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__1; LEAN_EXPORT uint8_t l_Lake_BuildKey_toString___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lake_instInhabitedBuildKey; LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__5_splitter___rarg(lean_object*, lean_object*, lean_object*); @@ -55,31 +58,28 @@ LEAN_EXPORT lean_object* l_Lake_instHashableBuildKey; LEAN_EXPORT lean_object* l_Lake_instDecidableEqBuildKey___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__3_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_BuildKey_instToString(lean_object*); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__10; LEAN_EXPORT lean_object* l_Lake_BuildKey_toString___lambda__1___boxed(lean_object*); static lean_object* l_Lake_BuildKey_toString___closed__3; -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__11; -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__7; +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__11; uint64_t l_Lean_Name_hash___override(lean_object*); +static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4; lean_object* l_Repr_addAppParen(lean_object*, lean_object*); static lean_object* l_Lake_instReprBuildKey___closed__1; -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__10; static lean_object* l_Lake_instHashableBuildKey___closed__1; uint8_t l_Lean_Name_quickCmp(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__1_splitter___rarg(uint8_t, lean_object*, lean_object*); -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4; static lean_object* l_Lake_BuildKey_toString___closed__6; lean_object* lean_string_append(lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lake_BuildKey_quickCmp(lean_object*, lean_object*); -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__13; +LEAN_EXPORT uint8_t l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__4_splitter(lean_object*); LEAN_EXPORT uint8_t l_Lake_instDecidableEqBuildKey(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_BuildKey_quickCmp_match__2_splitter___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_BuildKey_toString___closed__4; -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5; static lean_object* l_Lake_BuildKey_toString___closed__5; static lean_object* l_Lake_BuildKey_toString___closed__2; -static lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__2; static lean_object* _init_l_Lake_instInhabitedBuildKey___closed__1() { _start: { @@ -99,7 +99,7 @@ x_1 = l_Lake_instInhabitedBuildKey___closed__1; return x_1; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__1() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__1() { _start: { lean_object* x_1; @@ -107,21 +107,21 @@ x_1 = lean_mk_string_unchecked("Lake.BuildKey.moduleFacet", 25, 25); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__2() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__1; +x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____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_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__3() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__2; +x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__2; x_2 = lean_box(1); x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -129,7 +129,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4() { _start: { lean_object* x_1; lean_object* x_2; @@ -138,7 +138,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -147,7 +147,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__6() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__6() { _start: { lean_object* x_1; @@ -155,21 +155,21 @@ x_1 = lean_mk_string_unchecked("Lake.BuildKey.packageFacet", 26, 26); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__7() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__6; +x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____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___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__8() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__7; +x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__7; x_2 = lean_box(1); x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -177,7 +177,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__9() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__9() { _start: { lean_object* x_1; @@ -185,21 +185,21 @@ x_1 = lean_mk_string_unchecked("Lake.BuildKey.targetFacet", 25, 25); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__10() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__9; +x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____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___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__11() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__10; +x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__10; x_2 = lean_box(1); x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -207,7 +207,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__12() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__12() { _start: { lean_object* x_1; @@ -215,21 +215,21 @@ x_1 = lean_mk_string_unchecked("Lake.BuildKey.customTarget", 26, 26); return x_1; } } -static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__13() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__13() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__12; +x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____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_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__14() { +static lean_object* _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__13; +x_1 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__13; x_2 = lean_box(1); x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -237,7 +237,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93_(lean_object* x_1, lean_object* x_2) { _start: { switch (lean_obj_tag(x_1)) { @@ -253,7 +253,7 @@ x_5 = lean_ctor_get(x_1, 1); x_6 = lean_unsigned_to_nat(1024u); x_7 = lean_nat_dec_le(x_6, x_2); x_8 = l_Lean_Name_reprPrec(x_4, x_6); -x_9 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__3; +x_9 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__3; lean_ctor_set_tag(x_1, 5); lean_ctor_set(x_1, 1, x_8); lean_ctor_set(x_1, 0, x_9); @@ -268,7 +268,7 @@ lean_ctor_set(x_13, 1, x_12); if (x_7 == 0) { lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; lean_object* x_18; -x_14 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4; +x_14 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4; x_15 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_13); @@ -282,7 +282,7 @@ return x_18; else { lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; -x_19 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5; +x_19 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5; x_20 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_20, 0, x_19); lean_ctor_set(x_20, 1, x_13); @@ -305,7 +305,7 @@ lean_dec(x_1); x_26 = lean_unsigned_to_nat(1024u); x_27 = lean_nat_dec_le(x_26, x_2); x_28 = l_Lean_Name_reprPrec(x_24, x_26); -x_29 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__3; +x_29 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__3; x_30 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_30, 0, x_29); lean_ctor_set(x_30, 1, x_28); @@ -320,7 +320,7 @@ lean_ctor_set(x_34, 1, x_33); if (x_27 == 0) { lean_object* x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; -x_35 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4; +x_35 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4; x_36 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_36, 0, x_35); lean_ctor_set(x_36, 1, x_34); @@ -334,7 +334,7 @@ return x_39; else { lean_object* x_40; lean_object* x_41; uint8_t x_42; lean_object* x_43; lean_object* x_44; -x_40 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5; +x_40 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5; x_41 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_41, 0, x_40); lean_ctor_set(x_41, 1, x_34); @@ -359,7 +359,7 @@ x_47 = lean_ctor_get(x_1, 1); x_48 = lean_unsigned_to_nat(1024u); x_49 = lean_nat_dec_le(x_48, x_2); x_50 = l_Lean_Name_reprPrec(x_46, x_48); -x_51 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__8; +x_51 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__8; lean_ctor_set_tag(x_1, 5); lean_ctor_set(x_1, 1, x_50); lean_ctor_set(x_1, 0, x_51); @@ -374,7 +374,7 @@ lean_ctor_set(x_55, 1, x_54); if (x_49 == 0) { lean_object* x_56; lean_object* x_57; uint8_t x_58; lean_object* x_59; lean_object* x_60; -x_56 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4; +x_56 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4; x_57 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_57, 0, x_56); lean_ctor_set(x_57, 1, x_55); @@ -388,7 +388,7 @@ return x_60; else { lean_object* x_61; lean_object* x_62; uint8_t x_63; lean_object* x_64; lean_object* x_65; -x_61 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5; +x_61 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5; x_62 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_62, 0, x_61); lean_ctor_set(x_62, 1, x_55); @@ -411,7 +411,7 @@ lean_dec(x_1); x_68 = lean_unsigned_to_nat(1024u); x_69 = lean_nat_dec_le(x_68, x_2); x_70 = l_Lean_Name_reprPrec(x_66, x_68); -x_71 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__8; +x_71 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__8; x_72 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_72, 0, x_71); lean_ctor_set(x_72, 1, x_70); @@ -426,7 +426,7 @@ lean_ctor_set(x_76, 1, x_75); if (x_69 == 0) { lean_object* x_77; lean_object* x_78; uint8_t x_79; lean_object* x_80; lean_object* x_81; -x_77 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4; +x_77 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4; x_78 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_78, 0, x_77); lean_ctor_set(x_78, 1, x_76); @@ -440,7 +440,7 @@ return x_81; else { lean_object* x_82; lean_object* x_83; uint8_t x_84; lean_object* x_85; lean_object* x_86; -x_82 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5; +x_82 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5; x_83 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_83, 0, x_82); lean_ctor_set(x_83, 1, x_76); @@ -466,7 +466,7 @@ lean_dec(x_1); x_90 = lean_unsigned_to_nat(1024u); x_91 = lean_nat_dec_le(x_90, x_2); x_92 = l_Lean_Name_reprPrec(x_87, x_90); -x_93 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__11; +x_93 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__11; x_94 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_94, 0, x_93); lean_ctor_set(x_94, 1, x_92); @@ -488,7 +488,7 @@ lean_ctor_set(x_101, 1, x_100); if (x_91 == 0) { lean_object* x_102; lean_object* x_103; uint8_t x_104; lean_object* x_105; lean_object* x_106; -x_102 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4; +x_102 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4; x_103 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_103, 0, x_102); lean_ctor_set(x_103, 1, x_101); @@ -502,7 +502,7 @@ return x_106; else { lean_object* x_107; lean_object* x_108; uint8_t x_109; lean_object* x_110; lean_object* x_111; -x_107 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5; +x_107 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5; x_108 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_108, 0, x_107); lean_ctor_set(x_108, 1, x_101); @@ -526,7 +526,7 @@ x_114 = lean_ctor_get(x_1, 1); x_115 = lean_unsigned_to_nat(1024u); x_116 = lean_nat_dec_le(x_115, x_2); x_117 = l_Lean_Name_reprPrec(x_113, x_115); -x_118 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__14; +x_118 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__14; lean_ctor_set_tag(x_1, 5); lean_ctor_set(x_1, 1, x_117); lean_ctor_set(x_1, 0, x_118); @@ -541,7 +541,7 @@ lean_ctor_set(x_122, 1, x_121); if (x_116 == 0) { lean_object* x_123; lean_object* x_124; uint8_t x_125; lean_object* x_126; lean_object* x_127; -x_123 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4; +x_123 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4; x_124 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_124, 0, x_123); lean_ctor_set(x_124, 1, x_122); @@ -555,7 +555,7 @@ return x_127; else { lean_object* x_128; lean_object* x_129; uint8_t x_130; lean_object* x_131; lean_object* x_132; -x_128 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5; +x_128 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5; x_129 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_129, 0, x_128); lean_ctor_set(x_129, 1, x_122); @@ -578,7 +578,7 @@ lean_dec(x_1); x_135 = lean_unsigned_to_nat(1024u); x_136 = lean_nat_dec_le(x_135, x_2); x_137 = l_Lean_Name_reprPrec(x_133, x_135); -x_138 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__14; +x_138 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__14; x_139 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_139, 0, x_138); lean_ctor_set(x_139, 1, x_137); @@ -593,7 +593,7 @@ lean_ctor_set(x_143, 1, x_142); if (x_136 == 0) { lean_object* x_144; lean_object* x_145; uint8_t x_146; lean_object* x_147; lean_object* x_148; -x_144 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4; +x_144 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4; x_145 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_145, 0, x_144); lean_ctor_set(x_145, 1, x_143); @@ -607,7 +607,7 @@ return x_148; else { lean_object* x_149; lean_object* x_150; uint8_t x_151; lean_object* x_152; lean_object* x_153; -x_149 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5; +x_149 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5; x_150 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_150, 0, x_149); lean_ctor_set(x_150, 1, x_143); @@ -623,11 +623,11 @@ return x_153; } } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92_(x_1, x_2); +x_3 = l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93_(x_1, x_2); lean_dec(x_2); return x_3; } @@ -636,7 +636,7 @@ static lean_object* _init_l_Lake_instReprBuildKey___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____boxed), 2, 0); return x_1; } } @@ -648,7 +648,7 @@ x_1 = l_Lake_instReprBuildKey___closed__1; return x_1; } } -LEAN_EXPORT uint8_t l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326_(lean_object* x_1, lean_object* x_2) { _start: { switch (lean_obj_tag(x_1)) { @@ -788,11 +788,11 @@ return x_38; } } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325_(x_1, x_2); +x_3 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326_(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); @@ -803,7 +803,7 @@ LEAN_EXPORT uint8_t l_Lake_instDecidableEqBuildKey(lean_object* x_1, lean_object _start: { uint8_t x_3; -x_3 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_325_(x_1, x_2); +x_3 = l___private_Lake_Build_Key_0__Lake_decEqBuildKey____x40_Lake_Build_Key___hyg_326_(x_1, x_2); return x_3; } } @@ -818,7 +818,7 @@ x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT uint64_t l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1274_(lean_object* x_1) { +LEAN_EXPORT uint64_t l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1275_(lean_object* x_1) { _start: { switch (lean_obj_tag(x_1)) { @@ -876,11 +876,11 @@ return x_32; } } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1274____boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1275____boxed(lean_object* x_1) { _start: { uint64_t x_2; lean_object* x_3; -x_2 = l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1274_(x_1); +x_2 = l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1275_(x_1); lean_dec(x_1); x_3 = lean_box_uint64(x_2); return x_3; @@ -890,7 +890,7 @@ static lean_object* _init_l_Lake_instHashableBuildKey___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1274____boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lake_Build_Key_0__Lake_hashBuildKey____x40_Lake_Build_Key___hyg_1275____boxed), 1, 0); return x_1; } } @@ -1427,7 +1427,7 @@ lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_92____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___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_93____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { switch (lean_obj_tag(x_1)) { @@ -1492,11 +1492,11 @@ return x_18; } } } -LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_92_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_93_(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_92____rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l___private_Lake_Build_Key_0____private_Lake_Build_Key_0__Lake_reprBuildKey_match__1_splitter____x40_Lake_Build_Key___hyg_93____rarg), 5, 0); return x_2; } } @@ -1681,34 +1681,34 @@ l_Lake_instInhabitedBuildKey___closed__1 = _init_l_Lake_instInhabitedBuildKey___ lean_mark_persistent(l_Lake_instInhabitedBuildKey___closed__1); l_Lake_instInhabitedBuildKey = _init_l_Lake_instInhabitedBuildKey(); lean_mark_persistent(l_Lake_instInhabitedBuildKey); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__1 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__1(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__1); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__2 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__2(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__2); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__3 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__3(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__3); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__4); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__5); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__6 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__6(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__6); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__7 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__7(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__7); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__8 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__8(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__8); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__9 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__9(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__9); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__10 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__10(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__10); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__11 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__11(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__11); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__12 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__12(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__12); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__13 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__13(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__13); -l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__14 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__14(); -lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_92____closed__14); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__1 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__1(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__1); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__2 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__2(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__2); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__3 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__3(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__3); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__4); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__5); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__6 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__6(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__6); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__7 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__7(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__7); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__8 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__8(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__8); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__9 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__9(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__9); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__10 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__10(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__10); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__11 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__11(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__11); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__12 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__12(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__12); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__13 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__13(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__13); +l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__14 = _init_l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__14(); +lean_mark_persistent(l___private_Lake_Build_Key_0__Lake_reprBuildKey____x40_Lake_Build_Key___hyg_93____closed__14); l_Lake_instReprBuildKey___closed__1 = _init_l_Lake_instReprBuildKey___closed__1(); lean_mark_persistent(l_Lake_instReprBuildKey___closed__1); l_Lake_instReprBuildKey = _init_l_Lake_instReprBuildKey(); diff --git a/stage0/stdlib/Lake/CLI/Init.c b/stage0/stdlib/Lake/CLI/Init.c index c970af835dda..7e2e9dd8da67 100644 --- a/stage0/stdlib/Lake/CLI/Init.c +++ b/stage0/stdlib/Lake/CLI/Init.c @@ -18,24 +18,24 @@ LEAN_EXPORT lean_object* l_Lake_defaultExeRoot; lean_object* lean_string_utf8_extract(lean_object*, lean_object*, lean_object*); lean_object* lean_format_pretty(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_mathToolchainUrl___closed__1; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__7; lean_object* l_instBEqOfDecidableEq___rarg(lean_object*, lean_object*, lean_object*); uint32_t lean_string_utf8_get(lean_object*, lean_object*); static lean_object* l_Lake_stdLeanConfigFileContents___closed__3; LEAN_EXPORT lean_object* l_Lake_initPkg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_String_anyAux___at_Lake_validatePkgName___spec__2___closed__4___boxed__const__1; static lean_object* l_Lake_escapeName_x21___closed__1; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__20; lean_object* lean_io_prim_handle_put_str(lean_object*, lean_object*, lean_object*); static lean_object* l_String_anyAux___at_Lake_validatePkgName___spec__2___closed__3; static lean_object* l_Lake_initPkg___lambda__2___closed__11; static lean_object* l_Lake_mainFileName___closed__3; LEAN_EXPORT lean_object* l_Lake_leanActionWorkflowContents; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__5; LEAN_EXPORT lean_object* l_Lake_initPkg(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*); lean_object* l_System_FilePath_join(lean_object*, lean_object*); +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__1; LEAN_EXPORT lean_object* l_Lake_libRootFileContents(lean_object*, lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__1; LEAN_EXPORT lean_object* l_Lake_libRootFileContents___lambda__1___boxed(lean_object*); +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__10; LEAN_EXPORT lean_object* l_Lake_toolchainFileName; static lean_object* l_Lake_validatePkgName___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lake_createLeanActionWorkflow(lean_object*, lean_object*, lean_object*); @@ -43,14 +43,12 @@ static lean_object* l_Lake_mainFileContents___closed__2; static lean_object* l_Lake_defaultExeRoot___closed__1; static lean_object* l_Lake_escapeName_x21___closed__3; static lean_object* l_Lake_createLeanActionWorkflow___closed__7; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__15; LEAN_EXPORT lean_object* l_Lake_InitTemplate_noConfusion___rarg___lambda__1(lean_object*); static lean_object* l_Lake_validatePkgName___lambda__1___closed__4; static lean_object* l_Lake_initPkg___lambda__2___closed__6; LEAN_EXPORT lean_object* l_Lake_validatePkgName___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_createLeanActionWorkflow___closed__4; lean_object* l_String_quote(lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__25; static lean_object* l_Lake_stdTomlConfigFileContents___closed__5; lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); LEAN_EXPORT uint8_t l_String_anyAux___at_Lake_validatePkgName___spec__2(lean_object*, lean_object*, lean_object*); @@ -59,9 +57,9 @@ uint8_t lean_nat_dec_le(lean_object*, lean_object*); static lean_object* l_Lake_initPkg___lambda__1___closed__4; lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_InitTemplate_noConfusion(lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__11; static lean_object* l_Lake_stdTomlConfigFileContents___closed__4; static lean_object* l_Lake_gitignoreContents___closed__5; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__8; static lean_object* l_Lake_createLeanActionWorkflow___lambda__1___closed__2; lean_object* l_instDecidableEqChar___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_escapeName_x21___boxed(lean_object*); @@ -71,69 +69,66 @@ static lean_object* l_Lake_mathToolchainBlobUrl___closed__1; lean_object* l_System_FilePath_withExtension(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lake_libRootFileContents___lambda__1(lean_object*); static lean_object* l_Lake_mainFileName___closed__4; -LEAN_EXPORT lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____boxed(lean_object*, lean_object*); static lean_object* l_Lake_initPkg___lambda__2___closed__4; LEAN_EXPORT lean_object* l_Lake_new___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_instReprInitTemplate; static lean_object* l_Lake_initPkg___lambda__6___closed__2; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__4; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__5; static lean_object* l_Lake_mathTomlConfigFileContents___closed__2; static lean_object* l_Lake_mathLeanConfigFileContents___closed__2; static lean_object* l_Lake_initPkg___lambda__1___closed__9; +LEAN_EXPORT lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415_(uint8_t, lean_object*); static lean_object* l_Lake_validatePkgName___lambda__1___closed__5; static lean_object* l_Lake_InitTemplate_ofString_x3f___closed__4; static lean_object* l_Lake_initPkg___lambda__1___closed__10; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__26; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__24; LEAN_EXPORT lean_object* l_Lake_InitTemplate_ofString_x3f___boxed(lean_object*); lean_object* lean_string_utf8_set(lean_object*, lean_object*, uint32_t); +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__25; extern uint32_t l_Lean_idBeginEscape; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__8; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__12; static lean_object* l_Lake_basicFileContents___closed__1; uint8_t lean_string_dec_eq(lean_object*, lean_object*); static lean_object* l_Lake_createLeanActionWorkflow___closed__5; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__21; static lean_object* l_Lake_InitTemplate_ofString_x3f___closed__3; lean_object* l_System_FilePath_pathExists(lean_object*, lean_object*); static lean_object* l_Lake_libLeanConfigFileContents___closed__2; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__23; lean_object* lean_string_utf8_byte_size(lean_object*); static lean_object* l_Lake_initPkg___lambda__2___closed__3; lean_object* lean_string_push(lean_object*, uint32_t); +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__3; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__20; LEAN_EXPORT uint8_t l_Lake_instInhabitedInitTemplate; LEAN_EXPORT lean_object* l_Lake_mathToolchainUrl; lean_object* l_IO_FS_createDirAll(lean_object*, lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__9; LEAN_EXPORT lean_object* l_String_anyAux___at_Lake_validatePkgName___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_mathTomlConfigFileContents___boxed(lean_object*, lean_object*); static lean_object* l_Lake_initPkg___lambda__2___closed__17; LEAN_EXPORT lean_object* l_Lake_initPkg___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_InitTemplate_ofString_x3f___closed__8; static lean_object* l_Lake_stdTomlConfigFileContents___closed__3; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__6; static lean_object* l_Lake_toolchainFileName___closed__1; LEAN_EXPORT lean_object* l_Lake_initPkg___lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_validatePkgName___lambda__1___closed__7; static lean_object* l_Lake_escapeName_x21___closed__4; static lean_object* l_Lake_exeTomlConfigFileContents___closed__1; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__10; LEAN_EXPORT lean_object* l_Lake_initPkg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_InitTemplate_configFileContents(uint8_t, uint8_t, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414_(uint8_t, lean_object*); lean_object* lean_string_utf8_next(lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_instDecidableEqInitTemplate___boxed(lean_object*, lean_object*); lean_object* l_System_FilePath_isDir(lean_object*, lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__21; LEAN_EXPORT lean_object* l_String_anyAux___at_Lake_validatePkgName___spec__2___closed__3___boxed__const__1; LEAN_EXPORT lean_object* l_Lake_gitignoreContents; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__16; LEAN_EXPORT lean_object* l_Lake_escapeIdent___boxed(lean_object*); lean_object* lean_nat_to_int(lean_object*); static lean_object* l_Lake_validatePkgName___lambda__1___closed__3; static lean_object* l_Lake_initPkg___lambda__2___closed__14; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__3; static lean_object* l_Lake_initPkg___lambda__2___closed__18; static lean_object* l_Lake_createLeanActionWorkflow___closed__3; static lean_object* l_Lake_instReprInitTemplate___closed__1; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__22; static lean_object* l_Lake_validatePkgName___lambda__1___closed__10; LEAN_EXPORT lean_object* l_Lake_dotlessName(lean_object*); static lean_object* l_Lake_initPkg___lambda__2___closed__2; @@ -145,25 +140,26 @@ lean_object* l_Lake_stringToLegalOrSimpleName(lean_object*); LEAN_EXPORT lean_object* l_Lake_readmeFileContents___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lake_initPkg___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_initPkg___lambda__4(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__11; static lean_object* l_Lake_initPkg___closed__2; static lean_object* l_String_anyAux___at_Lake_validatePkgName___spec__2___closed__1; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__19; static lean_object* l_Lake_initPkg___lambda__2___closed__10; LEAN_EXPORT lean_object* l_Lake_InitTemplate_ofNat___boxed(lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__14; lean_object* l_System_FilePath_fileName(lean_object*); static lean_object* l_Lake_gitignoreContents___closed__2; LEAN_EXPORT lean_object* l_Lake_mainFileName; static lean_object* l_Lake_InitTemplate_ofString_x3f___closed__5; static lean_object* l_String_anyAux___at_Lake_validatePkgName___spec__2___closed__2; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__19; uint8_t lean_string_utf8_at_end(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_initPkg___lambda__6(lean_object*, lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_String_fromUTF8_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lake_stdLeanConfigFileContents(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__4; lean_object* l_System_FilePath_addExtension(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_validatePkgName___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_initPkg___lambda__1___closed__6; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__17; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__2; static lean_object* l_Lake_createLeanActionWorkflow___closed__6; static lean_object* l_Lake_validatePkgName___closed__1; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); @@ -188,11 +184,14 @@ static lean_object* l_Lake_initPkg___closed__1; extern lean_object* l_Std_Format_defWidth; LEAN_EXPORT lean_object* l_Lake_basicFileContents; static lean_object* l_Lake_initPkg___lambda__1___closed__1; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__14; static lean_object* l_Lake_initPkg___lambda__2___closed__8; static lean_object* l_Lake_stdLeanConfigFileContents___closed__1; static lean_object* l_Lake_stdTomlConfigFileContents___closed__1; static lean_object* l_Lake_escapeIdent___closed__2; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__15; LEAN_EXPORT lean_object* l_Lake_initPkg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__13; LEAN_EXPORT lean_object* l_Lake_createLeanActionWorkflow___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_mainFileName___closed__1; LEAN_EXPORT lean_object* l_Lake_init___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -227,26 +226,29 @@ static lean_object* l_Lake_validatePkgName___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lake_exeFileContents; static lean_object* l_Lake_createLeanActionWorkflow___closed__2; LEAN_EXPORT lean_object* l_Lake_mathLeanConfigFileContents(lean_object*, lean_object*); +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__18; lean_object* lean_io_realpath(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_validatePkgName(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__6; static lean_object* l_Lake_initPkg___lambda__2___closed__9; LEAN_EXPORT lean_object* l_Lake_stdLeanConfigFileContents___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Repr_addAppParen(lean_object*, lean_object*); static lean_object* l_Lake_gitignoreContents___closed__1; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__9; static lean_object* l_Lake_exeFileContents___closed__1; LEAN_EXPORT lean_object* l_Lake_libRootFileContents___boxed(lean_object*, lean_object*); static lean_object* l_Lake_validatePkgName___lambda__1___closed__6; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__17; static lean_object* l_Lake_libRootFileContents___closed__3; LEAN_EXPORT lean_object* l_Lake_stdTomlConfigFileContents(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_mainFileContents(lean_object*); static lean_object* l_Lake_mathTomlConfigFileContents___closed__1; LEAN_EXPORT lean_object* l_Lake_InitTemplate_ofString_x3f(lean_object*); lean_object* l_Lake_proc(lean_object*, uint8_t, lean_object*, lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__22; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__16; static lean_object* l_Lake_libRootFileContents___closed__1; LEAN_EXPORT lean_object* l_Lake_mathToolchainBlobUrl; LEAN_EXPORT lean_object* l_Lake_init(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__18; static lean_object* l_Lake_initPkg___lambda__2___closed__16; lean_object* l_Lake_toUpperCamelCase(lean_object*); lean_object* lean_array_mk(lean_object*); @@ -255,14 +257,12 @@ LEAN_EXPORT lean_object* l_String_mapAux___at_Lake_dotlessName___spec__1(lean_ob LEAN_EXPORT lean_object* l_Lake_escapeName_x21(lean_object*); LEAN_EXPORT lean_object* l_Lake_libLeanConfigFileContents(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_libTomlConfigFileContents(lean_object*, lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__13; lean_object* l_Lake_Env_toolchain(lean_object*); static lean_object* l_Lake_libRootFileContents___closed__2; static lean_object* l_Lake_mainFileName___closed__5; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__12; LEAN_EXPORT lean_object* l_Lake_readmeFileContents(lean_object*); lean_object* lean_io_error_to_string(lean_object*); -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__26; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__24; extern lean_object* l_Lake_defaultConfigFile; static lean_object* l_Lake_initPkg___lambda__2___closed__15; static lean_object* l_Lake_stdLeanConfigFileContents___closed__4; @@ -272,7 +272,6 @@ static lean_object* l_String_anyAux___at_Lake_validatePkgName___spec__2___closed lean_object* l_IO_FS_writeFile(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_validatePkgName___lambda__1___closed__9; static lean_object* l_Lake_mainFileName___closed__2; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__23; LEAN_EXPORT uint8_t l_Lake_instDecidableEqInitTemplate(uint8_t, uint8_t); lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lake_InitTemplate_ofNat(lean_object*); @@ -285,7 +284,9 @@ static lean_object* l_Lake_libLeanConfigFileContents___closed__1; uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_exeTomlConfigFileContents___boxed(lean_object*, lean_object*); static lean_object* l_Lake_createLeanActionWorkflow___lambda__1___closed__1; +LEAN_EXPORT lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____boxed(lean_object*, lean_object*); static lean_object* l_Lake_initPkg___lambda__1___closed__7; +static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__7; static lean_object* l_Lake_init___closed__1; LEAN_EXPORT lean_object* l_Lake_initPkg___lambda__3(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_gitignoreContents___closed__4; @@ -298,7 +299,6 @@ lean_object* l_instDecidableEqString___boxed(lean_object*, lean_object*); static lean_object* l_Lake_leanActionWorkflowContents___closed__1; LEAN_EXPORT lean_object* l_Lake_InitTemplate_toCtorIdx(uint8_t); static lean_object* l_Lake_defaultExeRoot___closed__2; -static lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__2; extern lean_object* l_Lake_Git_upstreamBranch; LEAN_EXPORT lean_object* l_Lake_createLeanActionWorkflow___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* _init_l_Lake_defaultExeRoot___closed__1() { @@ -931,7 +931,7 @@ static lean_object* _init_l_Lake_mathLeanConfigFileContents___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked(" where\n version := v!\"0.1.0\"\n keywords := #[\"math\"]\n leanOptions := #[\n ⟨`pp.unicode.fun, true⟩ -- pretty-prints `fun a ↦ b`\n ]\n\nrequire \"leanprover-community\" / \"mathlib\"\n\n@[default_target]\nlean_lib ", 213, 207); +x_1 = lean_mk_string_unchecked(" where\n version := v!\"0.1.0\"\n keywords := #[\"math\"]\n leanOptions := #[\n ⟨`pp.unicode.fun, true⟩, -- pretty-prints `fun a ↦ b`\n ⟨`autoImplicit, false⟩\n ]\n\nrequire \"leanprover-community\" / \"mathlib\"\n\n@[default_target]\nlean_lib ", 245, 235); return x_1; } } @@ -986,7 +986,7 @@ static lean_object* _init_l_Lake_mathTomlConfigFileContents___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("]\n\n[leanOptions]\npp.unicode.fun = true # pretty-prints `fun a ↦ b`\n\n[[require]]\nname = \"mathlib\"\nscope = \"leanprover-community\"\n\n[[lean_lib]]\nname = ", 151, 149); +x_1 = lean_mk_string_unchecked("]\n\n[leanOptions]\npp.unicode.fun = true # pretty-prints `fun a ↦ b`\nautoImplicit = false\n\n[[require]]\nname = \"mathlib\"\nscope = \"leanprover-community\"\n\n[[lean_lib]]\nname = ", 172, 170); return x_1; } } @@ -1198,7 +1198,7 @@ x_6 = l_Lake_InitTemplate_noConfusion___rarg(x_4, x_5, x_3); return x_6; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__1() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__1() { _start: { lean_object* x_1; @@ -1206,17 +1206,17 @@ x_1 = lean_mk_string_unchecked("Lake.InitTemplate.std", 21, 21); return x_1; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__2() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__1; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____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_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__3() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__3() { _start: { lean_object* x_1; lean_object* x_2; @@ -1225,23 +1225,23 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__4() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__3; -x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__2; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__3; +x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__2; 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_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__5() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__5() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__4; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__4; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1249,7 +1249,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__6() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__6() { _start: { lean_object* x_1; lean_object* x_2; @@ -1258,23 +1258,23 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__7() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__6; -x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__2; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__6; +x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__2; 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_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__8() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__8() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__7; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__7; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1282,7 +1282,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__9() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__9() { _start: { lean_object* x_1; @@ -1290,33 +1290,33 @@ x_1 = lean_mk_string_unchecked("Lake.InitTemplate.exe", 21, 21); return x_1; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__10() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__9; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____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___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__11() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__3; -x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__10; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__3; +x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__10; 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_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__12() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__12() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__11; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__11; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1324,23 +1324,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__13() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__6; -x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__10; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__6; +x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__10; 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_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__14() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__14() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__13; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__13; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1348,7 +1348,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__15() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__15() { _start: { lean_object* x_1; @@ -1356,33 +1356,33 @@ x_1 = lean_mk_string_unchecked("Lake.InitTemplate.lib", 21, 21); return x_1; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__16() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__16() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__15; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__15; 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_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__17() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__3; -x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__16; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__3; +x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__16; 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_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__18() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__18() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__17; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__17; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1390,23 +1390,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__19() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__6; -x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__16; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__6; +x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__16; 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_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__20() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__20() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__19; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__19; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1414,7 +1414,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__21() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__21() { _start: { lean_object* x_1; @@ -1422,33 +1422,33 @@ x_1 = lean_mk_string_unchecked("Lake.InitTemplate.math", 22, 22); return x_1; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__22() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__22() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__21; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__21; 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_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__23() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__23() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__3; -x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__22; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__3; +x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__22; 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_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__24() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__24() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__23; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__23; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1456,23 +1456,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__25() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__25() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__6; -x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__22; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__6; +x_2 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__22; 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_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__26() { +static lean_object* _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__26() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__25; +x_1 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__25; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -1480,7 +1480,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414_(uint8_t x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415_(uint8_t x_1, lean_object* x_2) { _start: { switch (x_1) { @@ -1492,14 +1492,14 @@ x_4 = lean_nat_dec_le(x_3, x_2); if (x_4 == 0) { lean_object* x_5; lean_object* x_6; -x_5 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__5; +x_5 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__5; x_6 = l_Repr_addAppParen(x_5, x_2); return x_6; } else { lean_object* x_7; lean_object* x_8; -x_7 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__8; +x_7 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__8; x_8 = l_Repr_addAppParen(x_7, x_2); return x_8; } @@ -1512,14 +1512,14 @@ x_10 = lean_nat_dec_le(x_9, x_2); if (x_10 == 0) { lean_object* x_11; lean_object* x_12; -x_11 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__12; +x_11 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__12; x_12 = l_Repr_addAppParen(x_11, x_2); return x_12; } else { lean_object* x_13; lean_object* x_14; -x_13 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__14; +x_13 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__14; x_14 = l_Repr_addAppParen(x_13, x_2); return x_14; } @@ -1532,14 +1532,14 @@ x_16 = lean_nat_dec_le(x_15, x_2); if (x_16 == 0) { lean_object* x_17; lean_object* x_18; -x_17 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__18; +x_17 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__18; x_18 = l_Repr_addAppParen(x_17, x_2); return x_18; } else { lean_object* x_19; lean_object* x_20; -x_19 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__20; +x_19 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__20; x_20 = l_Repr_addAppParen(x_19, x_2); return x_20; } @@ -1552,14 +1552,14 @@ x_22 = lean_nat_dec_le(x_21, x_2); if (x_22 == 0) { lean_object* x_23; lean_object* x_24; -x_23 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__24; +x_23 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__24; x_24 = l_Repr_addAppParen(x_23, x_2); return x_24; } else { lean_object* x_25; lean_object* x_26; -x_25 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__26; +x_25 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__26; x_26 = l_Repr_addAppParen(x_25, x_2); return x_26; } @@ -1567,13 +1567,13 @@ return x_26; } } } -LEAN_EXPORT lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; x_3 = lean_unbox(x_1); lean_dec(x_1); -x_4 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414_(x_3, x_2); +x_4 = l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415_(x_3, x_2); lean_dec(x_2); return x_4; } @@ -1582,7 +1582,7 @@ static lean_object* _init_l_Lake_instReprInitTemplate___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____boxed), 2, 0); return x_1; } } @@ -1891,7 +1891,7 @@ static lean_object* _init_l_Lake_escapeName_x21___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_Lake_escapeName_x21___closed__1; x_2 = l_Lake_escapeName_x21___closed__2; -x_3 = lean_unsigned_to_nat(199u); +x_3 = lean_unsigned_to_nat(202u); x_4 = lean_unsigned_to_nat(23u); x_5 = l_Lake_escapeName_x21___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -1912,7 +1912,7 @@ static lean_object* _init_l_Lake_escapeName_x21___closed__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; x_1 = l_Lake_escapeName_x21___closed__1; x_2 = l_Lake_escapeName_x21___closed__2; -x_3 = lean_unsigned_to_nat(202u); +x_3 = lean_unsigned_to_nat(205u); x_4 = lean_unsigned_to_nat(23u); x_5 = l_Lake_escapeName_x21___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -7002,58 +7002,58 @@ l_Lake_leanActionWorkflowContents = _init_l_Lake_leanActionWorkflowContents(); lean_mark_persistent(l_Lake_leanActionWorkflowContents); l_Lake_InitTemplate_noConfusion___rarg___closed__1 = _init_l_Lake_InitTemplate_noConfusion___rarg___closed__1(); lean_mark_persistent(l_Lake_InitTemplate_noConfusion___rarg___closed__1); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__1 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__1(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__1); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__2 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__2(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__2); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__3 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__3(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__3); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__4 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__4(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__4); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__5 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__5(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__5); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__6 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__6(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__6); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__7 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__7(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__7); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__8 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__8(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__8); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__9 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__9(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__9); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__10 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__10(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__10); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__11 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__11(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__11); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__12 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__12(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__12); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__13 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__13(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__13); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__14 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__14(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__14); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__15 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__15(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__15); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__16 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__16(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__16); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__17 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__17(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__17); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__18 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__18(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__18); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__19 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__19(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__19); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__20 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__20(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__20); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__21 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__21(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__21); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__22 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__22(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__22); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__23 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__23(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__23); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__24 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__24(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__24); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__25 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__25(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__25); -l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__26 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__26(); -lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_414____closed__26); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__1 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__1(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__1); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__2 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__2(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__2); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__3 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__3(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__3); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__4 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__4(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__4); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__5 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__5(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__5); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__6 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__6(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__6); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__7 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__7(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__7); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__8 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__8(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__8); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__9 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__9(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__9); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__10 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__10(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__10); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__11 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__11(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__11); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__12 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__12(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__12); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__13 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__13(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__13); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__14 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__14(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__14); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__15 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__15(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__15); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__16 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__16(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__16); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__17 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__17(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__17); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__18 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__18(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__18); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__19 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__19(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__19); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__20 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__20(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__20); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__21 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__21(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__21); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__22 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__22(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__22); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__23 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__23(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__23); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__24 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__24(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__24); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__25 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__25(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__25); +l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__26 = _init_l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__26(); +lean_mark_persistent(l___private_Lake_CLI_Init_0__Lake_reprInitTemplate____x40_Lake_CLI_Init___hyg_415____closed__26); l_Lake_instReprInitTemplate___closed__1 = _init_l_Lake_instReprInitTemplate___closed__1(); lean_mark_persistent(l_Lake_instReprInitTemplate___closed__1); l_Lake_instReprInitTemplate = _init_l_Lake_instReprInitTemplate(); diff --git a/stage0/stdlib/Lake/CLI/Main.c b/stage0/stdlib/Lake/CLI/Main.c index b8dd418d232b..0194e02b52d6 100644 --- a/stage0/stdlib/Lake/CLI/Main.c +++ b/stage0/stdlib/Lake/CLI/Main.c @@ -241,6 +241,7 @@ lean_object* l_Lake_loadWorkspace(lean_object*, uint8_t, lean_object*, lean_obje LEAN_EXPORT lean_object* l_Lake_lake_serve___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_lake_checkBuild___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_lake_resolveDeps___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); lean_object* lean_io_process_spawn(lean_object*, lean_object*); static lean_object* l_Lake_lakeCli___closed__5; static lean_object* l_Lake_lake_ReservoirConfig_currentSchemaVersion___closed__1; @@ -286,7 +287,6 @@ static lean_object* l_Lake_lakeCli___closed__2; LEAN_EXPORT lean_object* l_Lake_lake_test(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_lake_pack___lambda__2___boxed__const__1; LEAN_EXPORT lean_object* l_Lake_lake_versionTags(lean_object*, lean_object*, lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); uint8_t l_Lake_BuildConfig_showProgress(lean_object*); static lean_object* l_Lake_lakeLongOption___closed__6; LEAN_EXPORT lean_object* l_Lake_lake_script_doc___lambda__1___boxed__const__1; @@ -55937,7 +55937,7 @@ x_81 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_81, 0, x_18); lean_ctor_set(x_81, 1, x_80); x_82 = l_Lake_CliStateM_runLogIO___rarg___closed__1; -x_83 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_81, x_82); +x_83 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_81, x_82); x_84 = l_Lean_Json_mkObj(x_83); return x_84; } @@ -55990,7 +55990,7 @@ x_100 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_100, 0, x_18); lean_ctor_set(x_100, 1, x_99); x_101 = l_Lake_CliStateM_runLogIO___rarg___closed__1; -x_102 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_100, x_101); +x_102 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_100, x_101); x_103 = l_Lean_Json_mkObj(x_102); return x_103; } @@ -56041,7 +56041,7 @@ x_119 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_119, 0, x_18); lean_ctor_set(x_119, 1, x_118); x_120 = l_Lake_CliStateM_runLogIO___rarg___closed__1; -x_121 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_119, x_120); +x_121 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_119, x_120); x_122 = l_Lean_Json_mkObj(x_121); return x_122; } diff --git a/stage0/stdlib/Lake/Config/Opaque.c b/stage0/stdlib/Lake/Config/Opaque.c index 348bedded3f9..97bd749741f3 100644 --- a/stage0/stdlib/Lake/Config/Opaque.c +++ b/stage0/stdlib/Lake/Config/Opaque.c @@ -13,10 +13,10 @@ #ifdef __cplusplus extern "C" { #endif -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_nonemptyType___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_nonemptyType___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_OpaquePackage_nonemptyType; LEAN_EXPORT lean_object* l_Lake_OpaqueWorkspace_nonemptyType; -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_nonemptyType(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_nonemptyType(lean_object*, lean_object*, lean_object*); static lean_object* _init_l_Lake_OpaquePackage_nonemptyType() { _start: { @@ -29,20 +29,20 @@ static lean_object* _init_l_Lake_OpaqueWorkspace_nonemptyType() { return lean_box(0); } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_nonemptyType(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_nonemptyType(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { return lean_box(0); } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_nonemptyType___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_nonemptyType___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_3; -x_3 = l_Lake_OpaqueTargetConfig_nonemptyType(x_1, x_2); +lean_object* x_4; +x_4 = l_Lake_OpaqueTargetConfig_nonemptyType(x_1, x_2, x_3); +lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -return x_3; +return x_4; } } lean_object* initialize_Init(uint8_t builtin, lean_object*); diff --git a/stage0/stdlib/Lake/Config/TargetConfig.c b/stage0/stdlib/Lake/Config/TargetConfig.c index 740ff3e6a224..623c20d43113 100644 --- a/stage0/stdlib/Lake/Config/TargetConfig.c +++ b/stage0/stdlib/Lake/Config/TargetConfig.c @@ -15,55 +15,55 @@ extern "C" { #endif LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_unsafeMk___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_RBNode_dFind___at_Lake_Package_findTargetConfig_x3f___spec__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1___closed__1; +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_unsafeGet___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lake_mkTargetJobConfig(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_unsafeGet___rarg___boxed(lean_object*); -static lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig___closed__1; -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lake_Package_findTargetConfig_x3f___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfigName(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_unsafeMk___rarg___boxed(lean_object*); lean_object* lean_task_pure(lean_object*); LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_unsafeGet(lean_object*, lean_object*); static lean_object* l_Lake_instInhabitedTargetConfig___lambda__2___closed__5; LEAN_EXPORT lean_object* l_Lake_instInhabitedTargetConfig(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_unsafeMk___rarg(lean_object*); LEAN_EXPORT lean_object* l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lake_instInhabitedTargetConfig___lambda__2___boxed(lean_object*); static lean_object* l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1___rarg___closed__1; -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_instInhabitedTargetConfig___boxed(lean_object*, lean_object*); static lean_object* l_Lake_instInhabitedTargetConfig___closed__1; LEAN_EXPORT lean_object* l_Lake_Package_findTargetConfig_x3f(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig___boxed(lean_object*, lean_object*); extern lean_object* l_Task_Priority_default; -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfigName___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_instInhabitedTargetConfig___lambda__2(lean_object*); static lean_object* l_Lake_instInhabitedTargetConfig___lambda__2___closed__4; extern lean_object* l_Lake_BuildTrace_nil; +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig___rarg___boxed(lean_object*); lean_object* l_Lake_EResult_map___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_mkTargetJobConfig___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_RBNode_dFind___at_Lake_Package_findTargetConfig_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfigName___closed__1; LEAN_EXPORT lean_object* l_Lake_instInhabitedTargetConfig___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_instInhabitedTargetConfig___lambda__2___closed__3; static lean_object* l_Lake_instInhabitedTargetConfig___closed__2; static lean_object* l_Lake_instInhabitedTargetConfig___lambda__2___closed__6; static lean_object* l_Lake_instInhabitedTargetConfig___lambda__2___closed__7; LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_unsafeGet___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig(lean_object*, lean_object*); lean_object* lean_task_map(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1___rarg___lambda__1(lean_object*); static lean_object* l_Lake_instInhabitedTargetConfig___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_unsafeMk(lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); uint8_t l_Lean_Name_quickCmp(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig___boxed(lean_object*, lean_object*); static lean_object* l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1___rarg___closed__2; LEAN_EXPORT lean_object* l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lake_instInhabitedTargetConfig___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_instInhabitedTargetConfig___lambda__2___closed__2; +static lean_object* l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig___closed__1; LEAN_EXPORT lean_object* l_Lake_instInhabitedTargetConfig___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: { @@ -370,7 +370,7 @@ lean_dec(x_1); return x_3; } } -static lean_object* _init_l_Lake_OpaqueTargetConfig_instCoeTargetConfig___closed__1() { +static lean_object* _init_l_Lake_OpaqueTargetConfig_instCoeTargetConfigName___closed__1() { _start: { lean_object* x_1; @@ -378,19 +378,19 @@ x_1 = lean_alloc_closure((void*)(l_Lake_OpaqueTargetConfig_unsafeMk___rarg___box return x_1; } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfigName(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lake_OpaqueTargetConfig_instCoeTargetConfig___closed__1; +x_3 = l_Lake_OpaqueTargetConfig_instCoeTargetConfigName___closed__1; return x_3; } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfigName___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lake_OpaqueTargetConfig_instCoeTargetConfig(x_1, x_2); +x_3 = l_Lake_OpaqueTargetConfig_instCoeTargetConfigName(x_1, x_2); lean_dec(x_2); lean_dec(x_1); return x_3; @@ -430,7 +430,7 @@ lean_dec(x_1); return x_3; } } -static lean_object* _init_l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1___closed__1() { +static lean_object* _init_l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig___closed__1() { _start: { lean_object* x_1; @@ -438,53 +438,53 @@ x_1 = lean_alloc_closure((void*)(l_Lake_OpaqueTargetConfig_unsafeGet___rarg___bo return x_1; } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1___closed__1; +x_3 = l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig___closed__1; return x_3; } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1(x_1, x_2); +x_3 = l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig(x_1, x_2); lean_dec(x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig___rarg(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig___rarg(lean_object* x_1) { _start: { lean_inc(x_1); return x_1; } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig___rarg___boxed), 1, 0); +x_3 = lean_alloc_closure((void*)(l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig___rarg___boxed), 1, 0); return x_3; } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig___rarg___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig___rarg___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig___rarg(x_1); +x_2 = l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig___rarg(x_1); lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lake_OpaqueTargetConfig_instInhabitedOfTargetConfig(x_1, x_2); +x_3 = l_Lake_OpaqueTargetConfig_instInhabitedNameOfTargetConfig(x_1, x_2); lean_dec(x_2); lean_dec(x_1); return x_3; @@ -619,10 +619,10 @@ l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1___rarg___closed__1 = _in lean_mark_persistent(l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1___rarg___closed__1); l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1___rarg___closed__2 = _init_l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1___rarg___closed__2(); lean_mark_persistent(l_Functor_discard___at_Lake_mkTargetJobConfig___spec__1___rarg___closed__2); -l_Lake_OpaqueTargetConfig_instCoeTargetConfig___closed__1 = _init_l_Lake_OpaqueTargetConfig_instCoeTargetConfig___closed__1(); -lean_mark_persistent(l_Lake_OpaqueTargetConfig_instCoeTargetConfig___closed__1); -l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1___closed__1 = _init_l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1___closed__1(); -lean_mark_persistent(l_Lake_OpaqueTargetConfig_instCoeTargetConfig__1___closed__1); +l_Lake_OpaqueTargetConfig_instCoeTargetConfigName___closed__1 = _init_l_Lake_OpaqueTargetConfig_instCoeTargetConfigName___closed__1(); +lean_mark_persistent(l_Lake_OpaqueTargetConfig_instCoeTargetConfigName___closed__1); +l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig___closed__1 = _init_l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig___closed__1(); +lean_mark_persistent(l_Lake_OpaqueTargetConfig_instCoeNameTargetConfig___closed__1); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lake/Load/Lean/Elab.c b/stage0/stdlib/Lake/Load/Lean/Elab.c index 450a4790aac7..70976656366a 100644 --- a/stage0/stdlib/Lake/Load/Lean/Elab.c +++ b/stage0/stdlib/Lake/Load/Lean/Elab.c @@ -133,6 +133,7 @@ lean_object* lean_st_mk_ref(lean_object*, lean_object*); lean_object* l_System_FilePath_fileName(lean_object*); static lean_object* l_Lake_importConfigFileCore_lakeExts___closed__34; static lean_object* l_Lake_importConfigFileCore_lakeExts___closed__23; +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static uint64_t l_Lake_importModulesUsingCache___closed__3; static lean_object* l_Lake_importConfigFileCore_lakeExts___closed__18; static lean_object* l_Lake_importConfigFileCore_lakeExts___closed__5; @@ -156,7 +157,6 @@ lean_object* lean_io_prim_handle_mk(lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lake_instFromJsonConfigTrace; lean_object* l_Lean_bignumFromJson_x3f(lean_object*); static lean_object* l___private_Lake_Load_Lean_Elab_0__Lake_fromJsonConfigTrace____x40_Lake_Load_Lean_Elab___hyg_1110____closed__11; -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l_Lake_configModuleName___closed__1; static lean_object* l_Lake_importConfigFileCore_lakeExts___closed__35; static lean_object* l_Lake_importConfigFileCore_lakeExts___closed__41; @@ -4635,7 +4635,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_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_30, x_31); +x_32 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_30, x_31); x_33 = l_Lean_Json_mkObj(x_32); return x_33; } diff --git a/stage0/stdlib/Lake/Util/Log.c b/stage0/stdlib/Lake/Util/Log.c index c3985d845651..06340765de45 100644 --- a/stage0/stdlib/Lake/Util/Log.c +++ b/stage0/stdlib/Lake/Util/Log.c @@ -113,6 +113,7 @@ LEAN_EXPORT lean_object* l_Lake_logWarning(lean_object*); LEAN_EXPORT lean_object* l_Lake_Log_replay___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_MonadLog_ofMonadState(lean_object*); LEAN_EXPORT lean_object* l_Lake_logVerbose___rarg(lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l_Lake_getLogPos___rarg___closed__1; static lean_object* l_Lake_LogLevel_ofString_x3f___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lake_instFromJsonLog___spec__1___boxed(lean_object*, lean_object*, lean_object*); @@ -328,7 +329,6 @@ static lean_object* l_Lake_LogLevel_ofString_x3f___closed__6; LEAN_EXPORT lean_object* l_Lake_ELogT_takeAndRun___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lake_Util_Log_0__Lake_reprLogLevel____x40_Lake_Util_Log___hyg_505____closed__2; lean_object* l_Substring_takeWhileAux___at_Substring_trimLeft___spec__1(lean_object*, lean_object*, lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Log_takeFrom___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_ELogT_replayLog_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_instToStringLogEntry(lean_object*); @@ -3128,7 +3128,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lake_Util_Log_0__Lake_fromJsonLogLevel____x40_Lake_Util_Log___hyg_917____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } diff --git a/stage0/stdlib/Lean.c b/stage0/stdlib/Lean.c index 3688e5cf6c25..eee8e4226bfe 100644 --- a/stage0/stdlib/Lean.c +++ b/stage0/stdlib/Lean.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean -// Imports: Init Lean.Data Lean.Compiler Lean.Environment Lean.Modifiers Lean.ProjFns Lean.Runtime Lean.ResolveName Lean.Attributes Lean.Parser Lean.ReducibilityAttrs Lean.Elab Lean.Class Lean.LocalContext Lean.MetavarContext Lean.AuxRecursor Lean.Meta Lean.Util Lean.Structure Lean.PrettyPrinter Lean.CoreM Lean.ReservedNameAction Lean.InternalExceptionId Lean.Server Lean.ScopedEnvExtension Lean.DocString Lean.DeclarationRange Lean.LazyInitExtension Lean.LoadDynlib Lean.Widget Lean.Log Lean.Linter Lean.SubExpr Lean.LabelAttribute Lean.AddDecl Lean.Replay +// Imports: Init Lean.Data Lean.Compiler Lean.Environment Lean.Modifiers Lean.ProjFns Lean.Runtime Lean.ResolveName Lean.Attributes Lean.Parser Lean.ReducibilityAttrs Lean.Elab Lean.Class Lean.LocalContext Lean.MetavarContext Lean.AuxRecursor Lean.Meta Lean.Util Lean.Structure Lean.PrettyPrinter Lean.CoreM Lean.ReservedNameAction Lean.InternalExceptionId Lean.Server Lean.ScopedEnvExtension Lean.DocString Lean.DeclarationRange Lean.LoadDynlib Lean.Widget Lean.Log Lean.Linter Lean.SubExpr Lean.LabelAttribute Lean.AddDecl Lean.Replay #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -40,7 +40,6 @@ lean_object* initialize_Lean_Server(uint8_t builtin, lean_object*); lean_object* initialize_Lean_ScopedEnvExtension(uint8_t builtin, lean_object*); lean_object* initialize_Lean_DocString(uint8_t builtin, lean_object*); lean_object* initialize_Lean_DeclarationRange(uint8_t builtin, lean_object*); -lean_object* initialize_Lean_LazyInitExtension(uint8_t builtin, lean_object*); lean_object* initialize_Lean_LoadDynlib(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Widget(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Log(uint8_t builtin, lean_object*); @@ -135,9 +134,6 @@ lean_dec_ref(res); res = initialize_Lean_DeclarationRange(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -res = initialize_Lean_LazyInitExtension(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Lean_LoadDynlib(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Lean/Compiler/IR/Basic.c b/stage0/stdlib/Lean/Compiler/IR/Basic.c index b4a4d956d7d3..868d5d2ccd31 100644 --- a/stage0/stdlib/Lean/Compiler/IR/Basic.c +++ b/stage0/stdlib/Lean/Compiler/IR/Basic.c @@ -5244,7 +5244,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(220u); +x_17 = lean_unsigned_to_nat(242u); 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/IR/ElimDeadBranches.c b/stage0/stdlib/Lean/Compiler/IR/ElimDeadBranches.c index e2c938382024..aa583e4f6835 100644 --- a/stage0/stdlib/Lean/Compiler/IR/ElimDeadBranches.c +++ b/stage0/stdlib/Lean/Compiler/IR/ElimDeadBranches.c @@ -161,13 +161,14 @@ LEAN_EXPORT uint8_t l_Lean_IR_UnreachableBranches_Value_toFormat___lambda__1(lea static lean_object* l_Lean_IR_UnreachableBranches_interpFnBody___closed__4; static lean_object* l_List_mapTR_loop___at_Lean_IR_UnreachableBranches_Value_toFormat___spec__1___closed__2; lean_object* l_Lean_IR_LocalContext_getJPParams(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_elimDeadBranches___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_repr___at___private_Lean_Compiler_IR_ElimDeadBranches_0__Lean_IR_UnreachableBranches_reprValue____x40_Lean_Compiler_IR_ElimDeadBranches___hyg_42____spec__4___closed__10; static lean_object* l___private_Lean_Compiler_IR_ElimDeadBranches_0__Lean_IR_UnreachableBranches_reprValue____x40_Lean_Compiler_IR_ElimDeadBranches___hyg_42____closed__4; LEAN_EXPORT lean_object* l_Lean_IR_formatArray___at_Lean_IR_UnreachableBranches_Value_format___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_IR_UnreachableBranches_inferStep(lean_object*, lean_object*); static lean_object* l_List_repr___at___private_Lean_Compiler_IR_ElimDeadBranches_0__Lean_IR_UnreachableBranches_reprValue____x40_Lean_Compiler_IR_ElimDeadBranches___hyg_42____spec__4___closed__7; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_UnreachableBranches_Value_truncate_go___spec__10(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_modifyAux___at_Lean_IR_UnreachableBranches_updateCurrFnSummary___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_IR_UnreachableBranches_Value_toFormat(lean_object*); lean_object* l_Lean_IR_Decl_name(lean_object*); @@ -328,7 +329,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_UnreachableBranches static lean_object* l___private_Lean_Compiler_IR_ElimDeadBranches_0__Lean_IR_UnreachableBranches_reprValue____x40_Lean_Compiler_IR_ElimDeadBranches___hyg_42____closed__12; static lean_object* l_Lean_IR_UnreachableBranches_Value_addChoice___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_UnreachableBranches_Value_truncate_go___spec__5(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_elimDeadBranches___spec__2___boxed(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_Std_Format_joinSep___at___private_Lean_Compiler_IR_ElimDeadBranches_0__Lean_IR_UnreachableBranches_reprValue____x40_Lean_Compiler_IR_ElimDeadBranches___hyg_42____spec__2(lean_object*, lean_object*); @@ -10382,7 +10382,7 @@ return x_6; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_elimDeadBranches___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_elimDeadBranches___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_8; uint8_t x_9; @@ -10483,7 +10483,7 @@ lean_inc(x_9); x_22 = l_Nat_foldTR_loop___at_Lean_IR_elimDeadBranches___spec__1(x_1, x_9, x_20, x_9, x_9, x_5); lean_ctor_set(x_3, 0, x_22); x_23 = lean_mk_empty_array_with_capacity(x_9); -x_24 = l_Array_mapIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(x_1, x_21, x_1, x_9, x_13, lean_box(0), x_23); +x_24 = l_Array_mapFinIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(x_1, x_21, x_1, x_9, x_13, lean_box(0), x_23); lean_dec(x_21); lean_dec(x_1); lean_ctor_set(x_16, 1, x_3); @@ -10505,7 +10505,7 @@ lean_inc(x_9); x_28 = l_Nat_foldTR_loop___at_Lean_IR_elimDeadBranches___spec__1(x_1, x_9, x_26, x_9, x_9, x_5); lean_ctor_set(x_3, 0, x_28); x_29 = lean_mk_empty_array_with_capacity(x_9); -x_30 = l_Array_mapIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(x_1, x_27, x_1, x_9, x_13, lean_box(0), x_29); +x_30 = l_Array_mapFinIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(x_1, x_27, x_1, x_9, x_13, lean_box(0), x_29); lean_dec(x_27); lean_dec(x_1); x_31 = lean_alloc_ctor(0, 2, 0); @@ -10564,7 +10564,7 @@ x_50 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_50, 0, x_49); lean_ctor_set(x_50, 1, x_33); x_51 = lean_mk_empty_array_with_capacity(x_37); -x_52 = l_Array_mapIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(x_1, x_48, x_1, x_37, x_41, lean_box(0), x_51); +x_52 = l_Array_mapFinIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(x_1, x_48, x_1, x_37, x_41, lean_box(0), x_51); lean_dec(x_48); lean_dec(x_1); if (lean_is_scalar(x_46)) { @@ -10589,11 +10589,11 @@ lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_elimDeadBranches___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_elimDeadBranches___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_8; -x_8 = l_Array_mapIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Array_mapFinIdxM_map___at_Lean_IR_elimDeadBranches___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); diff --git a/stage0/stdlib/Lean/Compiler/IR/PushProj.c b/stage0/stdlib/Lean/Compiler/IR/PushProj.c index 45973f1db7ed..a8d4d8f238f7 100644 --- a/stage0/stdlib/Lean/Compiler/IR/PushProj.c +++ b/stage0/stdlib/Lean/Compiler/IR/PushProj.c @@ -13,36 +13,38 @@ #ifdef __cplusplus extern "C" { #endif -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9___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_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6(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_Lean_IR_pushProjs___spec__9(lean_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_IR_pushProjs___spec__7___at_Lean_IR_pushProjs___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5(lean_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_mapFinIdxM_map___at_Lean_IR_pushProjs___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_array_push(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___spec__2___boxed(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_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9___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_IR_instInhabitedFnBody; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__11___at_Lean_IR_pushProjs___spec__12(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__11(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__11___at_Lean_IR_pushProjs___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_IR_FnBody_flatten(lean_object*); lean_object* l_Lean_IR_FnBody_freeIndices(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_reverse___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___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_Array_mapMUnsafe_map___at_Lean_IR_FnBody_pushProj___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_IR_FnBody_pushProj___closed__1; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_IR_Decl_pushProj(lean_object*); lean_object* lean_array_pop(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5___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_IR_pushProjs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_FnBody_pushProj___spec__3(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_FnBody_pushProj___spec__2(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_IR_instInhabitedIndexSet; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___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_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__3(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___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_IR_FnBody_pushProj(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_FnBody_pushProj___spec__1(size_t, size_t, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); @@ -50,8 +52,8 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__7 LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__3___at_Lean_IR_pushProjs___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_IR_FnBody_setBody(lean_object*, lean_object*); lean_object* l_Lean_IR_Decl_updateBody_x21(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10___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_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5(lean_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_IR_FnBody_pushProj___spec__3___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_IR_AltCore_body(lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); @@ -61,24 +63,22 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__7 lean_object* lean_array_mk(lean_object*); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_pushProjs___spec__3___at_Lean_IR_pushProjs___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___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_IR_mkIndexSet(lean_object*); lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); lean_object* l_Lean_IR_FnBody_collectFreeIndices(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_RBNode_findCore___at_Lean_IR_UniqueIds_checkId___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___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_array_get_size(lean_object*); lean_object* l_Lean_IR_reshape(lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); lean_object* l_Lean_IR_Decl_normalizeIds(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_IR_FnBody_pushProj___spec__2___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___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_array_uset(lean_object*, size_t, lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); uint8_t l_Array_isEmpty___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___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_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___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; @@ -262,7 +262,7 @@ return x_10; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___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; uint8_t x_11; @@ -528,7 +528,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___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) { _start: { lean_object* x_11; uint8_t x_12; @@ -712,7 +712,7 @@ return x_10; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___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) { _start: { lean_object* x_10; uint8_t x_11; @@ -978,7 +978,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___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, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___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, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; uint8_t x_12; @@ -1162,7 +1162,7 @@ return x_10; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___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, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___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, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; uint8_t x_11; @@ -1510,7 +1510,7 @@ x_27 = lean_array_get_size(x_2); x_28 = lean_mk_empty_array_with_capacity(x_27); x_29 = lean_unsigned_to_nat(0u); lean_inc(x_8); -x_30 = l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___spec__2(x_2, x_3, x_8, x_25, x_2, x_27, x_29, lean_box(0), x_28); +x_30 = l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___spec__2(x_2, x_3, x_8, x_25, x_2, x_27, x_29, lean_box(0), x_28); lean_dec(x_2); x_31 = lean_array_size(x_3); x_32 = 0; @@ -1549,7 +1549,7 @@ x_40 = lean_array_get_size(x_2); x_41 = lean_mk_empty_array_with_capacity(x_40); x_42 = lean_unsigned_to_nat(0u); lean_inc(x_8); -x_43 = l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6(x_2, x_3, x_8, x_38, x_2, x_40, x_42, lean_box(0), x_41); +x_43 = l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6(x_2, x_3, x_8, x_38, x_2, x_40, x_42, lean_box(0), x_41); lean_dec(x_2); x_44 = lean_array_size(x_3); x_45 = 0; @@ -1588,7 +1588,7 @@ x_53 = lean_array_get_size(x_2); x_54 = lean_mk_empty_array_with_capacity(x_53); x_55 = lean_unsigned_to_nat(0u); lean_inc(x_8); -x_56 = l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10(x_2, x_3, x_8, x_51, x_2, x_53, x_55, lean_box(0), x_54); +x_56 = l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10(x_2, x_3, x_8, x_51, x_2, x_53, x_55, lean_box(0), x_54); lean_dec(x_2); x_57 = lean_array_size(x_3); x_58 = 0; @@ -1831,11 +1831,11 @@ return x_117; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___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_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___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_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___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_6); lean_dec(x_5); lean_dec(x_4); @@ -1844,11 +1844,11 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___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_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__1___at_Lean_IR_pushProjs___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); @@ -1883,11 +1883,11 @@ lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___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) { _start: { lean_object* x_11; -x_11 = l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); @@ -1896,11 +1896,11 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___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) { _start: { lean_object* x_10; -x_10 = l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__5___at_Lean_IR_pushProjs___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); @@ -1935,11 +1935,11 @@ lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___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) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___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: { lean_object* x_11; -x_11 = l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); @@ -1948,11 +1948,11 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___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_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___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) { _start: { lean_object* x_10; -x_10 = l_Array_mapIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Array_mapFinIdxM_map___at_Lean_IR_pushProjs___spec__9___at_Lean_IR_pushProjs___spec__10(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); diff --git a/stage0/stdlib/Lean/Compiler/LCNF/ElimDeadBranches.c b/stage0/stdlib/Lean/Compiler/LCNF/ElimDeadBranches.c index 42308d51761d..97bc8fdbe112 100644 --- a/stage0/stdlib/Lean/Compiler/LCNF/ElimDeadBranches.c +++ b/stage0/stdlib/Lean/Compiler/LCNF/ElimDeadBranches.c @@ -122,6 +122,7 @@ lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_UnreachableBranches_instReprValue___closed__1; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_UnreachableBranches_elimDead_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Environment_addExtraName(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___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_EXPORT lean_object* l_Prod_repr___at_Lean_Compiler_LCNF_UnreachableBranches_elimDead___spec__4___boxed(lean_object*, lean_object*); static lean_object* l_panic___at_Lean_Compiler_LCNF_UnreachableBranches_Value_getLiteral_go___spec__1___closed__5; uint8_t l___private_Lean_Util_Trace_0__Lean_checkTraceOption(lean_object*, lean_object*, lean_object*); @@ -130,7 +131,6 @@ static lean_object* l_List_repr___at___private_Lean_Compiler_LCNF_ElimDeadBranch uint8_t l_List_any___rarg(lean_object*, lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_ElimDeadBranches___hyg_6212____closed__8; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___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_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Compiler_LCNF_UnreachableBranches_getFunctionSummary_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Compiler_LCNF_UnreachableBranches_Value_beq___lambda__1(lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Compiler_LCNF_UnreachableBranches_inferMain___spec__1___closed__2; @@ -221,13 +221,13 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Compiler_LCNF_Unreacha static lean_object* l_Lean_Compiler_LCNF_UnreachableBranches_initFn____x40_Lean_Compiler_LCNF_ElimDeadBranches___hyg_1931____closed__3; static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_ElimDeadBranches___hyg_6212____closed__1; lean_object* l_Lean_MessageData_ofFormat(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___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_Lean_Compiler_LCNF_UnreachableBranches_initFn____x40_Lean_Compiler_LCNF_ElimDeadBranches___hyg_1931____closed__9; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_UnreachableBranches_instInhabitedValue; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Compiler_LCNF_UnreachableBranches_interpCode___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* l_outOfBounds___rarg(lean_object*); LEAN_EXPORT lean_object* l_repr___at_Lean_Compiler_LCNF_UnreachableBranches_elimDead___spec__3(lean_object*); static lean_object* l_Lean_Compiler_LCNF_UnreachableBranches_Value_ofNat_goSmall___closed__2; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___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_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Compiler_LCNF_UnreachableBranches_Value_truncate_go___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_ElimDeadBranches___hyg_6212____closed__15; @@ -18316,7 +18316,7 @@ return x_6; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___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_13; uint8_t x_14; @@ -18575,7 +18575,7 @@ x_35 = lean_ctor_get(x_34, 1); lean_inc(x_35); lean_dec(x_34); x_36 = lean_mk_empty_array_with_capacity(x_10); -x_37 = l_Array_mapIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___spec__3(x_1, x_25, x_1, x_10, x_13, lean_box(0), x_36, x_2, x_3, x_4, x_5, x_35); +x_37 = l_Array_mapFinIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___spec__3(x_1, x_25, x_1, x_10, x_13, lean_box(0), x_36, x_2, x_3, x_4, x_5, x_35); lean_dec(x_25); lean_dec(x_1); return x_37; @@ -18612,7 +18612,7 @@ x_48 = lean_ctor_get(x_47, 1); lean_inc(x_48); lean_dec(x_47); x_49 = lean_mk_empty_array_with_capacity(x_10); -x_50 = l_Array_mapIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___spec__3(x_1, x_25, x_1, x_10, x_13, lean_box(0), x_49, x_2, x_3, x_4, x_5, x_48); +x_50 = l_Array_mapFinIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___spec__3(x_1, x_25, x_1, x_10, x_13, lean_box(0), x_49, x_2, x_3, x_4, x_5, x_48); lean_dec(x_25); lean_dec(x_1); return x_50; @@ -18670,11 +18670,11 @@ lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___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_Array_mapFinIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___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_13; -x_13 = l_Array_mapIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___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 = l_Array_mapFinIdxM_map___at_Lean_Compiler_LCNF_Decl_elimDeadBranches___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_3); lean_dec(x_2); lean_dec(x_1); diff --git a/stage0/stdlib/Lean/Data/Lsp/Basic.c b/stage0/stdlib/Lean/Data/Lsp/Basic.c index 3743cc64aad2..32a9dea6abde 100644 --- a/stage0/stdlib/Lean/Data/Lsp/Basic.c +++ b/stage0/stdlib/Lean/Data/Lsp/Basic.c @@ -392,6 +392,7 @@ static lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonLocation LEAN_EXPORT lean_object* l_Lean_Lsp_instToStringPosition(lean_object*); static lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonDeleteFile____x40_Lean_Data_Lsp_Basic___hyg_3950____closed__3; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonCreateFile; +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_ins___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonWorkspaceEdit____x40_Lean_Data_Lsp_Basic___hyg_4439____spec__3(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_CreateFile_toJsonOptions____x40_Lean_Data_Lsp_Basic___hyg_3022____closed__2; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonLocationLink; @@ -452,7 +453,6 @@ LEAN_EXPORT lean_object* l_Lean_RBNode_foldM___at___private_Lean_Data_Lsp_Basic_ static lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonWorkspaceEdit____x40_Lean_Data_Lsp_Basic___hyg_4439____closed__7; static lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonStaticRegistrationOptions____x40_Lean_Data_Lsp_Basic___hyg_5746____closed__6; static lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonLocationLink____x40_Lean_Data_Lsp_Basic___hyg_1410____closed__7; -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonSnippetString____x40_Lean_Data_Lsp_Basic___hyg_1878____closed__6; LEAN_EXPORT lean_object* l_Lean_RBNode_ins___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonWorkspaceEdit____x40_Lean_Data_Lsp_Basic___hyg_4439____spec__18(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonDeleteFile____x40_Lean_Data_Lsp_Basic___hyg_3904_(lean_object*); @@ -932,7 +932,7 @@ x_1 = l_Lean_Lsp_instBEqCancelParams___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -1034,7 +1034,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_2); x_8 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -1057,7 +1057,7 @@ 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___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } @@ -1081,7 +1081,7 @@ x_24 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_24, 0, x_23); lean_ctor_set(x_24, 1, x_2); x_25 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_26 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_24, x_25); +x_26 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_24, x_25); x_27 = l_Lean_Json_mkObj(x_26); return x_27; } @@ -1104,7 +1104,7 @@ x_33 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_33, 0, x_32); lean_ctor_set(x_33, 1, x_2); x_34 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_35 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_33, x_34); +x_35 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_33, x_34); x_36 = l_Lean_Json_mkObj(x_35); return x_36; } @@ -1114,7 +1114,7 @@ return x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; x_37 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__5; x_38 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_39 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_37, x_38); +x_39 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_37, x_38); x_40 = l_Lean_Json_mkObj(x_39); return x_40; } @@ -1591,7 +1591,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_8); lean_ctor_set(x_16, 1, x_15); x_17 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } @@ -2093,7 +2093,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -2581,7 +2581,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___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -2618,7 +2618,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___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_32 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_30, x_31); +x_32 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_30, x_31); x_33 = l_Lean_Json_mkObj(x_32); return x_33; } @@ -3104,7 +3104,7 @@ x_24 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_24, 0, x_4); lean_ctor_set(x_24, 1, x_23); x_25 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_26 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_24, x_25); +x_26 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_24, x_25); x_27 = l_Lean_Json_mkObj(x_26); return x_27; } @@ -3878,7 +3878,7 @@ x_18 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_18, 0, x_9); lean_ctor_set(x_18, 1, x_17); x_19 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_20 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_18, x_19); +x_20 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_18, x_19); x_21 = l_Lean_Json_mkObj(x_20); return x_21; } @@ -4462,7 +4462,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___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -4782,7 +4782,7 @@ x_22 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_22, 0, x_7); lean_ctor_set(x_22, 1, x_21); x_23 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_24 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_22, x_23); +x_24 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_22, x_23); x_25 = l_Lean_Json_mkObj(x_24); return x_25; } @@ -5818,7 +5818,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___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -6057,7 +6057,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_8); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_14 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -6088,7 +6088,7 @@ x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_22); lean_ctor_set(x_26, 1, x_25); x_27 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_28 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } @@ -6571,7 +6571,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_7); lean_ctor_set(x_17, 1, x_16); x_18 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -7009,7 +7009,7 @@ x_18 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_18, 0, x_9); lean_ctor_set(x_18, 1, x_17); x_19 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_20 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_18, x_19); +x_20 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_18, x_19); x_21 = l_Lean_Json_mkObj(x_20); return x_21; } @@ -7435,7 +7435,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___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -7772,7 +7772,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___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -8123,7 +8123,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_9); lean_ctor_set(x_16, 1, x_15); x_17 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } @@ -8682,7 +8682,7 @@ x_22 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_22, 0, x_10); lean_ctor_set(x_22, 1, x_21); x_23 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_24 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_22, x_23); +x_24 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_22, x_23); x_25 = l_Lean_Json_mkObj(x_24); return x_25; } @@ -9134,7 +9134,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_9); lean_ctor_set(x_16, 1, x_15); x_17 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } @@ -10502,7 +10502,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_4); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -20468,7 +20468,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_4); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_14 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -20837,7 +20837,7 @@ x_27 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_27, 0, x_10); lean_ctor_set(x_27, 1, x_26); x_28 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_29 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_27, x_28); +x_29 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_27, x_28); x_30 = l_Lean_Json_mkObj(x_29); return x_30; } @@ -21289,7 +21289,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -21639,7 +21639,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_4); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -22218,7 +22218,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_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_7 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -22473,7 +22473,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_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_7 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -23147,7 +23147,7 @@ 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___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_13 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_11, x_12); +x_13 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_11, x_12); x_14 = l_Lean_Json_mkObj(x_13); return x_14; } @@ -23159,7 +23159,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_15); lean_ctor_set(x_16, 1, x_9); x_17 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } @@ -23515,7 +23515,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_9); lean_ctor_set(x_15, 1, x_14); x_16 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_17 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -23552,7 +23552,7 @@ x_31 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_31, 0, x_25); lean_ctor_set(x_31, 1, x_30); x_32 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_33 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_31, x_32); +x_33 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_31, x_32); x_34 = l_Lean_Json_mkObj(x_33); return x_34; } @@ -23655,7 +23655,7 @@ x_22 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_22, 0, x_10); lean_ctor_set(x_22, 1, x_21); x_23 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_24 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_22, x_23); +x_24 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_22, x_23); x_25 = l_Lean_Json_mkObj(x_24); return x_25; } @@ -23741,7 +23741,7 @@ x_29 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_29, 0, x_11); lean_ctor_set(x_29, 1, x_28); x_30 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_31 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_29, x_30); +x_31 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_29, x_30); x_32 = l_Lean_Json_mkObj(x_31); return x_32; } @@ -23790,7 +23790,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_8); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_14 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -23821,7 +23821,7 @@ x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_22); lean_ctor_set(x_26, 1, x_25); x_27 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_28 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } @@ -23909,7 +23909,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_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_7 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -24288,7 +24288,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_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_7 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -24495,7 +24495,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___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } diff --git a/stage0/stdlib/Lean/Data/Lsp/Capabilities.c b/stage0/stdlib/Lean/Data/Lsp/Capabilities.c index ee189634c2c9..9cdb88c2fba3 100644 --- a/stage0/stdlib/Lean/Data/Lsp/Capabilities.c +++ b/stage0/stdlib/Lean/Data/Lsp/Capabilities.c @@ -92,6 +92,7 @@ static lean_object* l_Lean_Lsp_instFromJsonWindowClientCapabilities___closed__1; lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeActionOptions____x40_Lean_Data_Lsp_CodeActions___hyg_884_(lean_object*); static lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonWorkspaceClientCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_963____closed__1; LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonServerCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_1460____spec__2(lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_fromJsonWorkspaceEditClientCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_794____closed__7; static lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_fromJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_48____closed__2; static lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_fromJsonChangeAnnotationSupport____x40_Lean_Data_Lsp_Capabilities___hyg_654____closed__6; @@ -216,7 +217,6 @@ LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Capabiliti static lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_fromJsonServerCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_1644____closed__53; static lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_fromJsonServerCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_1644____closed__33; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonCompletionItemCapabilities; -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonTextDocumentClientCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_248____spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonWorkspaceClientCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_963_(lean_object*); static lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_fromJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_48____closed__13; @@ -393,7 +393,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_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_7 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -686,7 +686,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_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_7 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -1166,7 +1166,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_4); lean_ctor_set(x_10, 1, x_9); x_11 = l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_12 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -1838,7 +1838,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___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_9 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -2070,7 +2070,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_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_7 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -2449,7 +2449,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_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_7 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -2719,7 +2719,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_4); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_16 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -3344,7 +3344,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_4); lean_ctor_set(x_10, 1, x_9); x_11 = l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_12 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -3938,7 +3938,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_4); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_16 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -5280,7 +5280,7 @@ x_82 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_82, 0, x_4); lean_ctor_set(x_82, 1, x_81); x_83 = l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonCompletionItemCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_20____closed__2; -x_84 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_82, x_83); +x_84 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_82, x_83); x_85 = l_Lean_Json_mkObj(x_84); return x_85; } diff --git a/stage0/stdlib/Lean/Data/Lsp/Client.c b/stage0/stdlib/Lean/Data/Lsp/Client.c index 2759c97dee51..51a4f39710a6 100644 --- a/stage0/stdlib/Lean/Data/Lsp/Client.c +++ b/stage0/stdlib/Lean/Data/Lsp/Client.c @@ -44,6 +44,7 @@ static lean_object* l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_fromJsonRegistr static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Client_0__Lean_Lsp_fromJsonRegistrationParams____x40_Lean_Data_Lsp_Client___hyg_296____spec__1___closed__1; lean_object* l_Lean_Json_getObjValD(lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_fromJsonRegistration____x40_Lean_Data_Lsp_Client___hyg_100____lambda__1(lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_toJsonRegistration____x40_Lean_Data_Lsp_Client___hyg_34____closed__5; static lean_object* l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_fromJsonRegistrationParams____x40_Lean_Data_Lsp_Client___hyg_296____closed__2; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonRegistration; @@ -52,7 +53,6 @@ static lean_object* l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_fromJsonRegistr LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_fromJsonRegistration____x40_Lean_Data_Lsp_Client___hyg_100_(lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_toJsonRegistrationParams____x40_Lean_Data_Lsp_Client___hyg_258____closed__1; -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_fromJsonRegistration____x40_Lean_Data_Lsp_Client___hyg_100____closed__2; static lean_object* l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_fromJsonRegistration____x40_Lean_Data_Lsp_Client___hyg_100____closed__10; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_Client_0__Lean_Lsp_fromJsonRegistrationParams____x40_Lean_Data_Lsp_Client___hyg_296____spec__2(size_t, size_t, lean_object*); @@ -199,7 +199,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_9); lean_ctor_set(x_16, 1, x_15); x_17 = l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_toJsonRegistration____x40_Lean_Data_Lsp_Client___hyg_34____closed__3; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } @@ -225,7 +225,7 @@ x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_9); lean_ctor_set(x_26, 1, x_25); x_27 = l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_toJsonRegistration____x40_Lean_Data_Lsp_Client___hyg_34____closed__3; -x_28 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } @@ -702,7 +702,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_9); lean_ctor_set(x_10, 1, x_8); x_11 = l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_toJsonRegistration____x40_Lean_Data_Lsp_Client___hyg_34____closed__3; -x_12 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } diff --git a/stage0/stdlib/Lean/Data/Lsp/CodeActions.c b/stage0/stdlib/Lean/Data/Lsp/CodeActions.c index 5f4143d78cec..0d646703d94f 100644 --- a/stage0/stdlib/Lean/Data/Lsp/CodeActions.c +++ b/stage0/stdlib/Lean/Data/Lsp/CodeActions.c @@ -96,6 +96,7 @@ LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Ls static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeActionLiteralSupportValueSet____x40_Lean_Data_Lsp_CodeActions___hyg_1753____closed__3; static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeActionClientCapabilities____x40_Lean_Data_Lsp_CodeActions___hyg_2049____closed__43; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeAction____x40_Lean_Data_Lsp_CodeActions___hyg_1204_(lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeActionDisabled____x40_Lean_Data_Lsp_CodeActions___hyg_698____closed__7; static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeActionClientCapabilities____x40_Lean_Data_Lsp_CodeActions___hyg_2049____closed__9; static lean_object* l_Lean_Lsp_CodeActionTriggerKind_noConfusion___rarg___closed__1; @@ -262,7 +263,6 @@ static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCo static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeActionClientCapabilities____x40_Lean_Data_Lsp_CodeActions___hyg_2049____closed__22; static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeActionClientCapabilities____x40_Lean_Data_Lsp_CodeActions___hyg_2049____closed__12; static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeActionLiteralSupportValueSet____x40_Lean_Data_Lsp_CodeActions___hyg_1753____closed__8; -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeActionOptions____x40_Lean_Data_Lsp_CodeActions___hyg_884____closed__15; static lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeAction____x40_Lean_Data_Lsp_CodeActions___hyg_1204____closed__12; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonCodeActionContext; @@ -1742,7 +1742,7 @@ x_19 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_19, 0, x_10); lean_ctor_set(x_19, 1, x_18); x_20 = l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionContext____x40_Lean_Data_Lsp_CodeActions___hyg_292____closed__1; -x_21 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_19, x_20); +x_21 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_19, x_20); x_22 = l_Lean_Json_mkObj(x_21); return x_22; } @@ -2415,7 +2415,7 @@ x_28 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_28, 0, x_4); lean_ctor_set(x_28, 1, x_27); x_29 = l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionContext____x40_Lean_Data_Lsp_CodeActions___hyg_292____closed__1; -x_30 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_28, x_29); +x_30 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_28, x_29); x_31 = l_Lean_Json_mkObj(x_30); return x_31; } @@ -2614,7 +2614,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___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionContext____x40_Lean_Data_Lsp_CodeActions___hyg_292____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -2725,7 +2725,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_10); lean_ctor_set(x_17, 1, x_16); x_18 = l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionContext____x40_Lean_Data_Lsp_CodeActions___hyg_292____closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -3604,7 +3604,7 @@ x_44 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_44, 0, x_4); lean_ctor_set(x_44, 1, x_43); x_45 = l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionContext____x40_Lean_Data_Lsp_CodeActions___hyg_292____closed__1; -x_46 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_44, x_45); +x_46 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_44, x_45); x_47 = l_Lean_Json_mkObj(x_46); return x_47; } @@ -5806,7 +5806,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_9); lean_ctor_set(x_10, 1, x_8); x_11 = l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionContext____x40_Lean_Data_Lsp_CodeActions___hyg_292____closed__1; -x_12 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -6112,7 +6112,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_9); lean_ctor_set(x_10, 1, x_8); x_11 = l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionContext____x40_Lean_Data_Lsp_CodeActions___hyg_292____closed__1; -x_12 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -6328,7 +6328,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___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionContext____x40_Lean_Data_Lsp_CodeActions___hyg_292____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -7608,7 +7608,7 @@ x_30 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_30, 0, x_4); lean_ctor_set(x_30, 1, x_29); x_31 = l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionContext____x40_Lean_Data_Lsp_CodeActions___hyg_292____closed__1; -x_32 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_30, x_31); +x_32 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_30, x_31); x_33 = l_Lean_Json_mkObj(x_32); return x_33; } diff --git a/stage0/stdlib/Lean/Data/Lsp/Diagnostics.c b/stage0/stdlib/Lean/Data/Lsp/Diagnostics.c index 4556dc51d242..f0faf487387c 100644 --- a/stage0/stdlib/Lean/Data/Lsp/Diagnostics.c +++ b/stage0/stdlib/Lean/Data/Lsp/Diagnostics.c @@ -90,6 +90,7 @@ lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__L static lean_object* l_Lean_Lsp_instToJsonDiagnosticSeverity___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_beqDiagnosticTag____x40_Lean_Data_Lsp_Diagnostics___hyg_625____boxed(lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instFromJsonDiagnosticCode___closed__1; +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_DiagnosticWith_ordUserVisible____x40_Lean_Data_Lsp_Diagnostics___hyg_2053____rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_fromJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_1550____rarg___closed__25; static lean_object* l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_fromJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_1550____rarg___closed__19; @@ -219,7 +220,6 @@ static lean_object* l_Lean_Lsp_instFromJsonDiagnosticSeverity___closed__3; static lean_object* l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_fromJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_1550____rarg___closed__40; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_DiagnosticWith_UserVisible_ofDiagnostic___rarg(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_1452_(lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_ordDiagnosticCode____x40_Lean_Data_Lsp_Diagnostics___hyg_404____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_compareByUserVisible(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonPublishDiagnosticsParams____x40_Lean_Data_Lsp_Diagnostics___hyg_2411____spec__3(size_t, size_t, lean_object*); @@ -1905,7 +1905,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticRelatedInformation____x40_Lean_Data_Lsp_Diagnostics___hyg_901____closed__3; -x_16 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -3548,7 +3548,7 @@ x_43 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_43, 0, x_8); lean_ctor_set(x_43, 1, x_42); x_44 = l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticRelatedInformation____x40_Lean_Data_Lsp_Diagnostics___hyg_901____closed__3; -x_45 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_43, x_44); +x_45 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_43, x_44); x_46 = l_Lean_Json_mkObj(x_45); return x_46; } @@ -6883,7 +6883,7 @@ x_42 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_42, 0, x_7); lean_ctor_set(x_42, 1, x_41); x_43 = l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticRelatedInformation____x40_Lean_Data_Lsp_Diagnostics___hyg_901____closed__3; -x_44 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_42, x_43); +x_44 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_42, x_43); x_45 = l_Lean_Json_mkObj(x_44); return x_45; } @@ -6982,7 +6982,7 @@ x_21 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_21, 0, x_9); lean_ctor_set(x_21, 1, x_20); x_22 = l___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticRelatedInformation____x40_Lean_Data_Lsp_Diagnostics___hyg_901____closed__3; -x_23 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_21, x_22); +x_23 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_21, x_22); x_24 = l_Lean_Json_mkObj(x_23); return x_24; } diff --git a/stage0/stdlib/Lean/Data/Lsp/Extra.c b/stage0/stdlib/Lean/Data/Lsp/Extra.c index 30f8532feeaf..c5828e88b977 100644 --- a/stage0/stdlib/Lean/Data/Lsp/Extra.c +++ b/stage0/stdlib/Lean/Data/Lsp/Extra.c @@ -110,6 +110,7 @@ static lean_object* l_Lean_Lsp_instToJsonPlainTermGoalParams___closed__1; static lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonRpcCallParams____x40_Lean_Data_Lsp_Extra___hyg_2012____closed__6; static lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonPlainTermGoal____x40_Lean_Data_Lsp_Extra___hyg_1584____closed__4; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonLeanFileProgressProcessingInfo____x40_Lean_Data_Lsp_Extra___hyg_814_(lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonRpcConnected____x40_Lean_Data_Lsp_Extra___hyg_1871____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instReprLineRange___closed__1; lean_object* l___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173_(size_t); @@ -272,7 +273,6 @@ static lean_object* l_Lean_Lsp_instFromJsonRpcKeepAliveParams___closed__1; static lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_132____closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonPlainGoal____x40_Lean_Data_Lsp_Extra___hyg_1342____spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonRpcReleaseParams; -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonRpcCallParams____x40_Lean_Data_Lsp_Extra___hyg_2012____closed__15; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____lambda__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonDependencyBuildMode; @@ -1496,7 +1496,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_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_14 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -1811,7 +1811,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___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_17 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -1850,7 +1850,7 @@ x_32 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_32, 0, x_25); lean_ctor_set(x_32, 1, x_31); x_33 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_34 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_32, x_33); +x_34 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_32, x_33); x_35 = l_Lean_Json_mkObj(x_34); return x_35; } @@ -2828,7 +2828,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_7); lean_ctor_set(x_10, 1, x_9); x_11 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_12 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -2840,7 +2840,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_7); lean_ctor_set(x_15, 1, x_14); x_16 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_17 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -3320,7 +3320,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_7); lean_ctor_set(x_17, 1, x_16); x_18 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -3615,7 +3615,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -4117,7 +4117,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_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -4158,7 +4158,7 @@ x_36 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_36, 0, x_27); lean_ctor_set(x_36, 1, x_35); x_37 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_38 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_36, x_37); +x_38 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_36, x_37); x_39 = l_Lean_Json_mkObj(x_38); return x_39; } @@ -4425,7 +4425,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -4709,7 +4709,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___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -4746,7 +4746,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___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_32 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_30, x_31); +x_32 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_30, x_31); x_33 = l_Lean_Json_mkObj(x_32); return x_33; } @@ -4917,7 +4917,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___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -5223,7 +5223,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); x_9 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_10 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_8, x_9); +x_10 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_8, x_9); x_11 = l_Lean_Json_mkObj(x_10); return x_11; } @@ -5949,7 +5949,7 @@ x_36 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_36, 0, x_8); lean_ctor_set(x_36, 1, x_35); x_37 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_38 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_36, x_37); +x_38 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_36, x_37); x_39 = l_Lean_Json_mkObj(x_38); return x_39; } @@ -6503,7 +6503,7 @@ x_24 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_24, 0, x_9); lean_ctor_set(x_24, 1, x_23); x_25 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_26 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_24, x_25); +x_26 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_24, x_25); x_27 = l_Lean_Json_mkObj(x_26); return x_27; } @@ -6773,7 +6773,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___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_17 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -7365,7 +7365,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_8); lean_ctor_set(x_16, 1, x_15); x_17 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonDependencyBuildMode____x40_Lean_Data_Lsp_Extra___hyg_10____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } diff --git a/stage0/stdlib/Lean/Data/Lsp/InitShutdown.c b/stage0/stdlib/Lean/Data/Lsp/InitShutdown.c index f86a5fe5ceb7..267e8d587b9b 100644 --- a/stage0/stdlib/Lean/Data/Lsp/InitShutdown.c +++ b/stage0/stdlib/Lean/Data/Lsp/InitShutdown.c @@ -61,6 +61,7 @@ static lean_object* l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_fromJsonI LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_fromJsonInitializeResult____x40_Lean_Data_Lsp_InitShutdown___hyg_966____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonInitializeParams____x40_Lean_Data_Lsp_InitShutdown___hyg_522____closed__2; static lean_object* l_Lean_Lsp_Trace_noConfusion___rarg___closed__1; +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); static lean_object* l_Lean_Json_getObjValAs_x3f___at_Lean_Lsp_instFromJsonInitializeParams___spec__6___closed__1; lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonVersionedTextDocumentIdentifier____x40_Lean_Data_Lsp_Basic___hyg_2438____spec__1(lean_object*, lean_object*); @@ -129,7 +130,6 @@ lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_fromJsonClientCa LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at_Lean_Lsp_instFromJsonInitializeParams___spec__5___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at_Lean_Lsp_instFromJsonInitializeParams___spec__3___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_fromJsonInitializationOptions____x40_Lean_Data_Lsp_InitShutdown___hyg_342____closed__10; -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; static lean_object* l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_fromJsonServerInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_796____closed__4; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_fromJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_70____lambda__1___boxed(lean_object*); @@ -261,7 +261,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_8); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; -x_14 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -292,7 +292,7 @@ x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_22); lean_ctor_set(x_26, 1, x_25); x_27 = l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; -x_28 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } @@ -949,7 +949,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_4); lean_ctor_set(x_10, 1, x_9); x_11 = l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; -x_12 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -1556,7 +1556,7 @@ x_31 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_31, 0, x_4); lean_ctor_set(x_31, 1, x_30); x_32 = l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; -x_33 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_31, x_32); +x_33 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_31, x_32); x_34 = l_Lean_Json_mkObj(x_33); return x_34; } @@ -1583,7 +1583,7 @@ x_41 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_41, 0, x_4); lean_ctor_set(x_41, 1, x_40); x_42 = l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; -x_43 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_41, x_42); +x_43 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_41, x_42); x_44 = l_Lean_Json_mkObj(x_43); return x_44; } @@ -1610,7 +1610,7 @@ x_51 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_51, 0, x_4); lean_ctor_set(x_51, 1, x_50); x_52 = l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; -x_53 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_51, x_52); +x_53 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_51, x_52); x_54 = l_Lean_Json_mkObj(x_53); return x_54; } @@ -4199,7 +4199,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_8); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; -x_14 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -4230,7 +4230,7 @@ x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_22); lean_ctor_set(x_26, 1, x_25); x_27 = l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; -x_28 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } @@ -4515,7 +4515,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_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonClientInfo____x40_Lean_Data_Lsp_InitShutdown___hyg_28____closed__3; -x_14 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } diff --git a/stage0/stdlib/Lean/Data/Lsp/Internal.c b/stage0/stdlib/Lean/Data/Lsp/Internal.c index 5f2a5fcb6091..df2d810cb271 100644 --- a/stage0/stdlib/Lean/Data/Lsp/Internal.c +++ b/stage0/stdlib/Lean/Data/Lsp/Internal.c @@ -117,6 +117,7 @@ LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonRefInfo(lean_object*); static lean_object* l_Lean_Lsp_instInhabitedRefIdent___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instToJsonModuleRefs___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_RBNode_foldM___at_Lean_Lsp_instFromJsonModuleRefs___spec__6___closed__1; +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_toJsonLeanIleanInfoParams____x40_Lean_Data_Lsp_Internal___hyg_1979____spec__2(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_RefIdent_fromJsonRefIdentJsonRepr____x40_Lean_Data_Lsp_Internal___hyg_268____lambda__1___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Lsp_instToJsonModuleRefs___spec__4(lean_object*, size_t, size_t, lean_object*); @@ -135,7 +136,6 @@ static lean_object* l_Lean_Lsp_instToJsonRefInfo___closed__3; static lean_object* l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_fromJsonLeanStaleDependencyParams____x40_Lean_Data_Lsp_Internal___hyg_2161____closed__4; LEAN_EXPORT lean_object* l_Lean_Lsp_RefIdent_fromJson_x3f(lean_object*); static lean_object* l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_fromJsonLeanIleanInfoParams____x40_Lean_Data_Lsp_Internal___hyg_1873____closed__8; -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_fromJsonLeanIleanInfoParams____x40_Lean_Data_Lsp_Internal___hyg_1873____closed__13; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instFromJsonRefInfo___spec__2___closed__1; static lean_object* l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_fromJsonLeanIleanInfoParams____x40_Lean_Data_Lsp_Internal___hyg_1873____closed__19; @@ -1805,7 +1805,7 @@ x_20 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_20, 0, x_9); lean_ctor_set(x_20, 1, x_19); x_21 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_RefInfo_toJsonParentDecl____x40_Lean_Data_Lsp_Internal___hyg_721____closed__4; -x_22 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); +x_22 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); x_23 = l_Lean_Json_mkObj(x_22); return x_23; } @@ -16575,7 +16575,7 @@ x_20 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_20, 0, x_8); lean_ctor_set(x_20, 1, x_19); x_21 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_RefInfo_toJsonParentDecl____x40_Lean_Data_Lsp_Internal___hyg_721____closed__4; -x_22 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); +x_22 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); x_23 = l_Lean_Json_mkObj(x_22); return x_23; } @@ -16604,7 +16604,7 @@ x_31 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_31, 0, x_8); lean_ctor_set(x_31, 1, x_30); x_32 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_RefInfo_toJsonParentDecl____x40_Lean_Data_Lsp_Internal___hyg_721____closed__4; -x_33 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_31, x_32); +x_33 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_31, x_32); x_34 = l_Lean_Json_mkObj(x_33); return x_34; } @@ -16632,7 +16632,7 @@ x_44 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_44, 0, x_8); lean_ctor_set(x_44, 1, x_43); x_45 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_RefInfo_toJsonParentDecl____x40_Lean_Data_Lsp_Internal___hyg_721____closed__4; -x_46 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_44, x_45); +x_46 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_44, x_45); x_47 = l_Lean_Json_mkObj(x_46); return x_47; } @@ -17035,7 +17035,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_9); lean_ctor_set(x_10, 1, x_8); x_11 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_RefInfo_toJsonParentDecl____x40_Lean_Data_Lsp_Internal___hyg_721____closed__4; -x_12 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -17246,7 +17246,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___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_RefInfo_toJsonParentDecl____x40_Lean_Data_Lsp_Internal___hyg_721____closed__4; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } diff --git a/stage0/stdlib/Lean/Data/Lsp/LanguageFeatures.c b/stage0/stdlib/Lean/Data/Lsp/LanguageFeatures.c index 38505f3c21f4..40b423c9bb62 100644 --- a/stage0/stdlib/Lean/Data/Lsp/LanguageFeatures.c +++ b/stage0/stdlib/Lean/Data/Lsp/LanguageFeatures.c @@ -675,6 +675,7 @@ static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJ static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1756____closed__5; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1756____closed__49; static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__8; +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonDocumentHighlightParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3855____closed__6; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7320____closed__10; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonHoverParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2816_(lean_object*); @@ -789,7 +790,6 @@ static lean_object* l_Lean_Lsp_instToJsonDocumentHighlightKind___closed__3; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonRenameParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_10390____closed__9; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonDocumentSymbol_go(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_348____closed__110; -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonDocumentSymbolAux(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_9149____closed__2; @@ -2272,7 +2272,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_4); lean_ctor_set(x_16, 1, x_15); x_17 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } @@ -5537,7 +5537,7 @@ x_20 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_20, 0, x_9); lean_ctor_set(x_20, 1, x_19); x_21 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_22 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); +x_22 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); x_23 = l_Lean_Json_mkObj(x_22); return x_23; } @@ -7820,7 +7820,7 @@ x_36 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_36, 0, x_14); lean_ctor_set(x_36, 1, x_35); x_37 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_38 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_36, x_37); +x_38 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_36, x_37); x_39 = l_Lean_Json_mkObj(x_38); return x_39; } @@ -8379,7 +8379,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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -8703,7 +8703,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -8768,7 +8768,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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_14 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -9290,7 +9290,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -9544,7 +9544,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -9798,7 +9798,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -10052,7 +10052,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -10251,7 +10251,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___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -10647,7 +10647,7 @@ x_22 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_22, 0, x_8); lean_ctor_set(x_22, 1, x_21); x_23 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_24 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_22, x_23); +x_24 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_22, x_23); x_25 = l_Lean_Json_mkObj(x_24); return x_25; } @@ -10846,7 +10846,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___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -11100,7 +11100,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -11342,7 +11342,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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_14 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -11520,7 +11520,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___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -21351,7 +21351,7 @@ x_35 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_35, 0, x_13); lean_ctor_set(x_35, 1, x_34); x_36 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_37 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_35, x_36); +x_37 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_35, x_36); x_38 = l_Lean_Json_mkObj(x_37); return x_38; } @@ -21733,7 +21733,7 @@ x_34 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_34, 0, x_12); lean_ctor_set(x_34, 1, x_33); x_35 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_36 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_34, x_35); +x_36 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_34, x_35); x_37 = l_Lean_Json_mkObj(x_36); return x_37; } @@ -23360,7 +23360,7 @@ 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 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_35 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_33, x_34); +x_35 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_33, x_34); x_36 = l_Lean_Json_mkObj(x_35); return x_36; } @@ -23627,7 +23627,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -24755,7 +24755,7 @@ x_44 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_44, 0, x_14); lean_ctor_set(x_44, 1, x_43); x_45 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_46 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_44, x_45); +x_46 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_44, x_45); x_47 = l_Lean_Json_mkObj(x_46); return x_47; } @@ -25552,7 +25552,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___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -26052,7 +26052,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_7); lean_ctor_set(x_17, 1, x_16); x_18 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -26262,7 +26262,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___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -26549,7 +26549,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_7); lean_ctor_set(x_17, 1, x_16); x_18 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -31072,7 +31072,7 @@ x_19 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_19, 0, x_10); lean_ctor_set(x_19, 1, x_18); x_20 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_21 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_19, x_20); +x_21 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_19, x_20); x_22 = l_Lean_Json_mkObj(x_21); return x_22; } @@ -31486,7 +31486,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___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_22 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); +x_22 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); x_23 = l_Lean_Json_mkObj(x_22); return x_23; } @@ -31655,7 +31655,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___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -31909,7 +31909,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -32405,7 +32405,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_4); lean_ctor_set(x_15, 1, x_14); x_16 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_17 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -32586,7 +32586,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___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -32859,7 +32859,7 @@ x_20 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_20, 0, x_8); lean_ctor_set(x_20, 1, x_19); x_21 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_22 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); +x_22 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); x_23 = l_Lean_Json_mkObj(x_22); return x_23; } @@ -33067,7 +33067,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___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -33444,7 +33444,7 @@ x_21 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_21, 0, x_8); lean_ctor_set(x_21, 1, x_20); x_22 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_23 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_21, x_22); +x_23 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_21, x_22); x_24 = l_Lean_Json_mkObj(x_23); return x_24; } @@ -33698,7 +33698,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_7); lean_ctor_set(x_14, 1, x_13); x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_189____closed__1; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } diff --git a/stage0/stdlib/Lean/Data/Lsp/TextSync.c b/stage0/stdlib/Lean/Data/Lsp/TextSync.c index b2f2f7517135..f9097fd91fdf 100644 --- a/stage0/stdlib/Lean/Data/Lsp/TextSync.c +++ b/stage0/stdlib/Lean/Data/Lsp/TextSync.c @@ -114,6 +114,7 @@ static lean_object* l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonTextD LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_toJsonDidChangeTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_529_(lean_object*); static lean_object* l_Lean_Lsp_instToJsonDidSaveTextDocumentParams___closed__1; static lean_object* l_Lean_Lsp_instFromJsonTextDocumentSyncKind___closed__3; +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonDidChangeTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_581____spec__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonDidSaveTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_750____closed__11; static lean_object* l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonTextDocumentSyncOptions____x40_Lean_Data_Lsp_TextSync___hyg_1219____closed__19; @@ -127,7 +128,6 @@ static lean_object* l_Lean_Lsp_instFromJsonSaveOptions___closed__1; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonTextDocumentChangeRegistrationOptions____x40_Lean_Data_Lsp_TextSync___hyg_252____spec__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonDidOpenTextDocumentParams___closed__1; static lean_object* l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonTextDocumentSyncOptions____x40_Lean_Data_Lsp_TextSync___hyg_1219____closed__18; -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonSaveOptions____x40_Lean_Data_Lsp_TextSync___hyg_906____closed__6; static lean_object* l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonSaveOptions____x40_Lean_Data_Lsp_TextSync___hyg_906____closed__3; static lean_object* l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonDidCloseTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_1023____closed__4; @@ -556,7 +556,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___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_toJsonDidOpenTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_125____closed__2; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -1616,7 +1616,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_7); lean_ctor_set(x_17, 1, x_16); x_18 = l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_toJsonDidOpenTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_125____closed__2; -x_19 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -2179,7 +2179,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_Data_Lsp_TextSync_0__Lean_Lsp_toJsonDidOpenTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_125____closed__2; -x_14 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -2455,7 +2455,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___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_toJsonDidOpenTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_125____closed__2; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -2655,7 +2655,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___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_toJsonDidOpenTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_125____closed__2; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -3011,7 +3011,7 @@ x_27 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_27, 0, x_11); lean_ctor_set(x_27, 1, x_26); x_28 = l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_toJsonDidOpenTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_125____closed__2; -x_29 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_27, x_28); +x_29 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_27, x_28); x_30 = l_Lean_Json_mkObj(x_29); return x_30; } @@ -3026,7 +3026,7 @@ 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 = l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_toJsonDidOpenTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_125____closed__2; -x_35 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_33, x_34); +x_35 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_33, x_34); x_36 = l_Lean_Json_mkObj(x_35); return x_36; } @@ -3041,7 +3041,7 @@ x_39 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_39, 0, x_11); lean_ctor_set(x_39, 1, x_38); x_40 = l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_toJsonDidOpenTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_125____closed__2; -x_41 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_39, x_40); +x_41 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_39, x_40); x_42 = l_Lean_Json_mkObj(x_41); return x_42; } diff --git a/stage0/stdlib/Lean/Data/Lsp/Window.c b/stage0/stdlib/Lean/Data/Lsp/Window.c index e323c52d2750..f1e8b38c7dde 100644 --- a/stage0/stdlib/Lean/Data/Lsp/Window.c +++ b/stage0/stdlib/Lean/Data/Lsp/Window.c @@ -47,7 +47,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Window_0__fromJsonMessageActi static lean_object* l___private_Lean_Data_Lsp_Window_0__fromJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_134____closed__2; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Window_0__toJsonShowMessageRequestParams____x40_Lean_Data_Lsp_Window___hyg_586_(lean_object*); static lean_object* l_instToJsonMessageType___closed__7; -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_MessageType_toCtorIdx___boxed(lean_object*); static lean_object* l___private_Lean_Data_Lsp_Window_0__fromJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_134____closed__10; lean_object* lean_nat_to_int(lean_object*); @@ -137,6 +136,7 @@ static lean_object* l_instToJsonMessageType___closed__3; static lean_object* l___private_Lean_Data_Lsp_Window_0__fromJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_134____closed__13; static lean_object* l___private_Lean_Data_Lsp_Window_0__fromJsonShowMessageRequestParams____x40_Lean_Data_Lsp_Window___hyg_441____closed__8; static lean_object* l___private_Lean_Data_Lsp_Window_0__fromJsonShowMessageRequestParams____x40_Lean_Data_Lsp_Window___hyg_441____closed__14; +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(lean_object*, lean_object*); lean_object* l_Lean_Json_pretty(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Window_0__fromJsonShowMessageRequestParams____x40_Lean_Data_Lsp_Window___hyg_441____closed__12; static lean_object* l___private_Lean_Data_Lsp_Window_0__fromJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_134____closed__12; @@ -1053,7 +1053,7 @@ x_1 = l_instFromJsonShowMessageParams___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -1211,7 +1211,7 @@ 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___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____closed__1; -x_13 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_11, x_12); +x_13 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_11, x_12); x_14 = l_Lean_Json_mkObj(x_13); return x_14; } @@ -1223,7 +1223,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_15); lean_ctor_set(x_16, 1, x_9); x_17 = l___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } @@ -1235,7 +1235,7 @@ x_21 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_21, 0, x_20); lean_ctor_set(x_21, 1, x_9); x_22 = l___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____closed__1; -x_23 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_21, x_22); +x_23 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_21, x_22); x_24 = l_Lean_Json_mkObj(x_23); return x_24; } @@ -1247,7 +1247,7 @@ x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_25); lean_ctor_set(x_26, 1, x_9); x_27 = l___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____closed__1; -x_28 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } @@ -1456,7 +1456,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___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -2174,7 +2174,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_13); x_16 = l___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____closed__1; -x_17 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -2186,7 +2186,7 @@ x_20 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_20, 0, x_19); lean_ctor_set(x_20, 1, x_13); x_21 = l___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____closed__1; -x_22 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_20, x_21); +x_22 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_20, x_21); x_23 = l_Lean_Json_mkObj(x_22); return x_23; } @@ -2198,7 +2198,7 @@ x_25 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_25, 0, x_24); lean_ctor_set(x_25, 1, x_13); x_26 = l___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____closed__1; -x_27 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_25, x_26); +x_27 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_25, x_26); x_28 = l_Lean_Json_mkObj(x_27); return x_28; } @@ -2210,7 +2210,7 @@ x_30 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_30, 0, x_29); lean_ctor_set(x_30, 1, x_13); x_31 = l___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____closed__1; -x_32 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_30, x_31); +x_32 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Window_0__toJsonShowMessageParams____x40_Lean_Data_Lsp_Window___hyg_240____spec__1(x_30, x_31); x_33 = l_Lean_Json_mkObj(x_32); return x_33; } diff --git a/stage0/stdlib/Lean/Data/Lsp/Workspace.c b/stage0/stdlib/Lean/Data/Lsp/Workspace.c index be035e77ffc9..8d0fdf23353b 100644 --- a/stage0/stdlib/Lean/Data/Lsp/Workspace.c +++ b/stage0/stdlib/Lean/Data/Lsp/Workspace.c @@ -101,6 +101,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonF static lean_object* l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_fromJsonDidChangeWatchedFilesRegistrationOptions____x40_Lean_Data_Lsp_Workspace___hyg_390____closed__5; static lean_object* l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_fromJsonDidChangeWatchedFilesRegistrationOptions____x40_Lean_Data_Lsp_Workspace___hyg_390____closed__2; static lean_object* l_Lean_Lsp_instFromJsonFileChangeType___closed__5; +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_fromJsonDidChangeWatchedFilesRegistrationOptions____x40_Lean_Data_Lsp_Workspace___hyg_390____spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_fromJsonDidChangeWatchedFilesRegistrationOptions____x40_Lean_Data_Lsp_Workspace___hyg_390____spec__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_fromJsonFileEvent____x40_Lean_Data_Lsp_Workspace___hyg_640____closed__3; @@ -117,7 +118,6 @@ LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonFileEvent; static lean_object* l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_fromJsonFileEvent____x40_Lean_Data_Lsp_Workspace___hyg_640____closed__10; static lean_object* l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_fromJsonFileSystemWatcher____x40_Lean_Data_Lsp_Workspace___hyg_205____closed__10; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonDidChangeWatchedFilesRegistrationOptions____x40_Lean_Data_Lsp_Workspace___hyg_457____spec__1(size_t, size_t, lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonFileEvent; static lean_object* l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_fromJsonDidChangeWatchedFilesRegistrationOptions____x40_Lean_Data_Lsp_Workspace___hyg_390____closed__1; static lean_object* l_Lean_Lsp_instToJsonFileSystemWatcher___closed__1; @@ -242,7 +242,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___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -280,7 +280,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___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_32 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_30, x_31); +x_32 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_30, x_31); x_33 = l_Lean_Json_mkObj(x_32); return x_33; } @@ -923,7 +923,7 @@ 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 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_12 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -952,7 +952,7 @@ x_21 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_21, 0, x_8); lean_ctor_set(x_21, 1, x_20); x_22 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_23 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_21, x_22); +x_23 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_21, x_22); x_24 = l_Lean_Json_mkObj(x_23); return x_24; } @@ -979,7 +979,7 @@ x_32 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_32, 0, x_8); lean_ctor_set(x_32, 1, x_31); x_33 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_34 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_32, x_33); +x_34 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_32, x_33); x_35 = l_Lean_Json_mkObj(x_34); return x_35; } @@ -1011,7 +1011,7 @@ 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 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_46 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_44, x_45); +x_46 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_44, x_45); x_47 = l_Lean_Json_mkObj(x_46); return x_47; } @@ -1049,7 +1049,7 @@ x_56 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_56, 0, x_42); lean_ctor_set(x_56, 1, x_55); x_57 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_58 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_56, x_57); +x_58 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_56, x_57); x_59 = l_Lean_Json_mkObj(x_58); return x_59; } @@ -1477,7 +1477,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_9); lean_ctor_set(x_10, 1, x_8); x_11 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_12 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -2419,7 +2419,7 @@ 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 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_12 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } @@ -2431,7 +2431,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___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_17 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -2443,7 +2443,7 @@ x_20 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_20, 0, x_8); lean_ctor_set(x_20, 1, x_19); x_21 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_22 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); +x_22 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); x_23 = l_Lean_Json_mkObj(x_22); return x_23; } @@ -2841,7 +2841,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_9); lean_ctor_set(x_10, 1, x_8); x_11 = l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonWorkspaceFolder____x40_Lean_Data_Lsp_Workspace___hyg_25____closed__3; -x_12 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } diff --git a/stage0/stdlib/Lean/Data/Position.c b/stage0/stdlib/Lean/Data/Position.c index 0e01c7ea27c2..3faad395f081 100644 --- a/stage0/stdlib/Lean/Data/Position.c +++ b/stage0/stdlib/Lean/Data/Position.c @@ -138,8 +138,8 @@ lean_object* lean_array_get_size(lean_object*); static lean_object* l___private_Lean_Data_Position_0__Lean_fromJsonPosition____x40_Lean_Data_Position___hyg_289____closed__3; uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Position_0__Lean_decEqPosition____x40_Lean_Data_Position___hyg_34____boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237_(lean_object*); static lean_object* l_Lean_Position_instToFormat___closed__6; LEAN_EXPORT lean_object* l_Lean_FileMap_toPosition_loop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -488,7 +488,7 @@ x_1 = l_Lean_instReprPosition___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -558,7 +558,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_8); lean_ctor_set(x_16, 1, x_15); x_17 = l___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } diff --git a/stage0/stdlib/Lean/Data/Trie.c b/stage0/stdlib/Lean/Data/Trie.c index 48f8d680db1a..51de47874c7e 100644 --- a/stage0/stdlib/Lean/Data/Trie.c +++ b/stage0/stdlib/Lean/Data/Trie.c @@ -61,6 +61,7 @@ LEAN_EXPORT lean_object* l_Lean_Data_Trie_findPrefix_go___rarg(lean_object*, lea LEAN_EXPORT lean_object* l_Lean_Data_Trie_matchPrefix_loop___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Data_Trie_values_go___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Data_Trie_instEmptyCollection(lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Trie_0__Lean_Data_Trie_toStringAux___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Data_Trie_matchPrefix_loop___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Data_Trie_upsert_loop___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Data_Trie_matchPrefix_loop(lean_object*); @@ -81,7 +82,6 @@ LEAN_EXPORT lean_object* l_ByteArray_findIdx_x3f_loop___at_Lean_Data_Trie_matchP LEAN_EXPORT lean_object* l_Lean_Data_Trie_upsert___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Data_Trie_insert___rarg___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Data_Trie_upsert_loop___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Data_Trie_0__Lean_Data_Trie_toStringAux___spec__1(lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Data_Trie_values_go___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Data_Trie_upsert(lean_object*); @@ -1769,7 +1769,7 @@ lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Data_Trie_0__Lean_Data_Trie_toStringAux___spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Trie_0__Lean_Data_Trie_toStringAux___spec__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -1895,7 +1895,7 @@ x_21 = lean_array_to_list(x_19); x_22 = l___private_Lean_Data_Trie_0__Lean_Data_Trie_toStringAux___rarg___closed__1; x_23 = l_Lean_Data_Trie_values___rarg___closed__1; x_24 = l_List_zipWithTR_go___rarg(x_22, x_20, x_21, x_23); -x_25 = l_List_bindTR_go___at___private_Lean_Data_Trie_0__Lean_Data_Trie_toStringAux___spec__1(x_24, x_23); +x_25 = l_List_flatMapTR_go___at___private_Lean_Data_Trie_0__Lean_Data_Trie_toStringAux___spec__1(x_24, x_23); return x_25; } } diff --git a/stage0/stdlib/Lean/Declaration.c b/stage0/stdlib/Lean/Declaration.c index b05ffad0183b..cfef3ea024ce 100644 --- a/stage0/stdlib/Lean/Declaration.c +++ b/stage0/stdlib/Lean/Declaration.c @@ -38,11 +38,13 @@ LEAN_EXPORT lean_object* l_Lean_ConstantInfo_levelParams(lean_object*); LEAN_EXPORT lean_object* l_Lean_Declaration_foldExprM___at_Lean_Declaration_forExprM___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Declaration_definitionVal_x21___boxed(lean_object*); static lean_object* l___private_Lean_Declaration_0__Lean_reprDefinitionSafety____x40_Lean_Declaration___hyg_685____closed__3; +LEAN_EXPORT lean_object* l_Lean_RecursorVal_getMajorInduct_go(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instBEqConstantVal; LEAN_EXPORT lean_object* l_Lean_mkAxiomValEx___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_instInhabitedRecursorVal___closed__1; static lean_object* l_Lean_instReprDefinitionSafety___closed__1; LEAN_EXPORT lean_object* l_Lean_Declaration_isUnsafeInductiveDeclEx___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_RecursorVal_getMajorInduct(lean_object*); LEAN_EXPORT lean_object* l_Lean_ConstantInfo_inductiveVal_x21(lean_object*); LEAN_EXPORT uint8_t l_List_beq___at___private_Lean_Declaration_0__Lean_beqRecursorVal____x40_Lean_Declaration___hyg_3174____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_instInhabitedDeclaration___closed__1; @@ -123,7 +125,6 @@ LEAN_EXPORT uint8_t l___private_Lean_Declaration_0__Lean_beqDeclaration____x40_L LEAN_EXPORT lean_object* l_Lean_Declaration_foldExprM___at_Lean_Declaration_forExprM___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instBEqInductiveType; static lean_object* l_Lean_ConstantInfo_value_x21___closed__3; -lean_object* l_Lean_Name_getPrefix(lean_object*); LEAN_EXPORT uint8_t l_Lean_ConstantInfo_isCtor(lean_object*); LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Declaration_forExprM___spec__2___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_instInhabitedConstantVal___closed__2; @@ -156,6 +157,7 @@ static lean_object* l___private_Lean_Declaration_0__Lean_reprDefinitionSafety___ LEAN_EXPORT uint8_t l_List_beq___at___private_Lean_Declaration_0__Lean_beqDeclaration____x40_Lean_Declaration___hyg_1774____spec__2(lean_object*, lean_object*); LEAN_EXPORT uint8_t lean_axiom_val_is_unsafe(lean_object*); LEAN_EXPORT uint32_t lean_reducibility_hints_get_height(lean_object*); +lean_object* l_Lean_Expr_constName_x21(lean_object*); static lean_object* l___private_Lean_Declaration_0__Lean_reprDefinitionSafety____x40_Lean_Declaration___hyg_685____closed__18; LEAN_EXPORT lean_object* l_Lean_instInhabitedConstructor; LEAN_EXPORT lean_object* l_Lean_ConstantInfo_numLevelParams___boxed(lean_object*); @@ -182,7 +184,6 @@ LEAN_EXPORT uint8_t l_Lean_instInhabitedDefinitionSafety; static lean_object* l___private_Lean_Declaration_0__Lean_reprDefinitionSafety____x40_Lean_Declaration___hyg_685____closed__7; LEAN_EXPORT lean_object* l_Lean_instBEqDeclaration; LEAN_EXPORT lean_object* l_Lean_DefinitionSafety_noConfusion___rarg(uint8_t, uint8_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_RecursorVal_getInduct(lean_object*); LEAN_EXPORT lean_object* l_Lean_Declaration_foldExprM___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ReducibilityHints_lt___boxed(lean_object*, lean_object*); LEAN_EXPORT uint8_t lean_recursor_k(lean_object*); @@ -205,6 +206,7 @@ static lean_object* l_Lean_instBEqReducibilityHints___closed__1; static lean_object* l_Lean_ReducibilityHints_instOrd___closed__1; LEAN_EXPORT uint8_t lean_is_unsafe_inductive_decl(lean_object*); LEAN_EXPORT lean_object* l_List_beq___at___private_Lean_Declaration_0__Lean_beqConstantVal____x40_Lean_Declaration___hyg_433____spec__1___boxed(lean_object*, lean_object*); +lean_object* l_Lean_Expr_bindingDomain_x21(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Declaration_0__Lean_reprDefinitionSafety____x40_Lean_Declaration___hyg_685_(uint8_t, lean_object*); LEAN_EXPORT uint8_t lean_inductive_val_is_reflexive(lean_object*); LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Declaration_forExprM___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -237,8 +239,10 @@ LEAN_EXPORT lean_object* l___private_Lean_Declaration_0__Lean_beqDefinitionVal__ lean_object* l_Repr_addAppParen(lean_object*, lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_ReducibilityHints_isAbbrev(lean_object*); +lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_InductiveVal_isNested___boxed(lean_object*); static lean_object* l_Lean_instBEqTheoremVal___closed__1; +lean_object* l_Lean_Expr_getAppFn(lean_object*); static lean_object* l___private_Lean_Declaration_0__Lean_reprDefinitionSafety____x40_Lean_Declaration___hyg_685____closed__14; static lean_object* l_Lean_instInhabitedInductiveType___closed__1; LEAN_EXPORT uint8_t l___private_Lean_Declaration_0__Lean_beqRecursorRule____x40_Lean_Declaration___hyg_2988_(lean_object*, lean_object*); @@ -256,7 +260,6 @@ static lean_object* l_Lean_instInhabitedDefinitionVal___closed__1; LEAN_EXPORT lean_object* l_Lean_instInhabitedOpaqueVal; uint8_t lean_uint32_dec_lt(uint32_t, uint32_t); LEAN_EXPORT uint8_t l___private_Lean_Declaration_0__Lean_beqDefinitionSafety____x40_Lean_Declaration___hyg_667_(uint8_t, uint8_t); -LEAN_EXPORT lean_object* l_Lean_RecursorVal_getInduct___boxed(lean_object*); static lean_object* l_Lean_instBEqOpaqueVal___closed__1; LEAN_EXPORT lean_object* l_Lean_instInhabitedDefinitionVal; LEAN_EXPORT uint8_t l___private_Lean_Declaration_0__Lean_beqRecursorVal____x40_Lean_Declaration___hyg_3174_(lean_object*, lean_object*); @@ -267,6 +270,7 @@ LEAN_EXPORT lean_object* l_Lean_RecursorVal_getFirstMinorIdx___boxed(lean_object LEAN_EXPORT lean_object* l_Lean_ConstantInfo_levelParams___boxed(lean_object*); static lean_object* l_Lean_Declaration_definitionVal_x21___closed__3; static lean_object* l_Lean_Declaration_definitionVal_x21___closed__4; +lean_object* l_Lean_Expr_bindingBody_x21(lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Declaration_0__Lean_beqReducibilityHints____x40_Lean_Declaration___hyg_27_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_DefinitionSafety_noConfusion___rarg___lambda__1___boxed(lean_object*); static lean_object* l_Lean_instInhabitedRecursorRule___closed__1; @@ -3888,23 +3892,51 @@ lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_RecursorVal_getInduct(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_RecursorVal_getMajorInduct_go(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = lean_ctor_get(x_1, 0); -x_3 = lean_ctor_get(x_2, 0); -x_4 = l_Lean_Name_getPrefix(x_3); -return x_4; +lean_object* x_3; uint8_t x_4; +x_3 = lean_unsigned_to_nat(0u); +x_4 = lean_nat_dec_eq(x_1, x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_unsigned_to_nat(1u); +x_6 = lean_nat_sub(x_1, x_5); +lean_dec(x_1); +x_7 = l_Lean_Expr_bindingBody_x21(x_2); +lean_dec(x_2); +x_1 = x_6; +x_2 = x_7; +goto _start; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; +lean_dec(x_1); +x_9 = l_Lean_Expr_bindingDomain_x21(x_2); +lean_dec(x_2); +x_10 = l_Lean_Expr_getAppFn(x_9); +lean_dec(x_9); +x_11 = l_Lean_Expr_constName_x21(x_10); +lean_dec(x_10); +return x_11; } } -LEAN_EXPORT lean_object* l_Lean_RecursorVal_getInduct___boxed(lean_object* x_1) { +} +LEAN_EXPORT lean_object* l_Lean_RecursorVal_getMajorInduct(lean_object* x_1) { _start: { -lean_object* x_2; -x_2 = l_Lean_RecursorVal_getInduct(x_1); +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_2 = l_Lean_RecursorVal_getMajorIdx(x_1); +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); lean_dec(x_1); -return x_2; +x_4 = lean_ctor_get(x_3, 2); +lean_inc(x_4); +lean_dec(x_3); +x_5 = l_Lean_RecursorVal_getMajorInduct_go(x_2, x_4); +return x_5; } } LEAN_EXPORT lean_object* l_Lean_QuotKind_toCtorIdx(uint8_t x_1) { @@ -4388,7 +4420,7 @@ static lean_object* _init_l_Lean_ConstantInfo_value_x21___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_Lean_Declaration_definitionVal_x21___closed__1; x_2 = l_Lean_ConstantInfo_value_x21___closed__1; -x_3 = lean_unsigned_to_nat(456u); +x_3 = lean_unsigned_to_nat(461u); x_4 = lean_unsigned_to_nat(33u); x_5 = l_Lean_ConstantInfo_value_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -4547,7 +4579,7 @@ static lean_object* _init_l_Lean_ConstantInfo_inductiveVal_x21___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_Lean_Declaration_definitionVal_x21___closed__1; x_2 = l_Lean_ConstantInfo_inductiveVal_x21___closed__1; -x_3 = lean_unsigned_to_nat(472u); +x_3 = lean_unsigned_to_nat(477u); x_4 = lean_unsigned_to_nat(9u); x_5 = l_Lean_ConstantInfo_inductiveVal_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Elab/BuiltinCommand.c b/stage0/stdlib/Lean/Elab/BuiltinCommand.c index 012a45bc3678..ab58f99a2828 100644 --- a/stage0/stdlib/Lean/Elab/BuiltinCommand.c +++ b/stage0/stdlib/Lean/Elab/BuiltinCommand.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean.Elab.BuiltinCommand -// Imports: Lean.Util.CollectLevelParams Lean.Util.CollectAxioms Lean.Meta.Reduce Lean.Elab.DeclarationRange Lean.Elab.Eval Lean.Elab.Command Lean.Elab.Open Lean.Elab.SetOption +// Imports: Lean.Util.CollectLevelParams Lean.Util.CollectAxioms Lean.Meta.Reduce Lean.Elab.DeclarationRange Lean.Elab.Eval Lean.Elab.Command Lean.Elab.Open Lean.Elab.SetOption Init.System.Platform #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -25,15 +25,19 @@ static lean_object* l_Lean_Elab_Command_elabOmit___closed__1; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); lean_object* lean_string_utf8_extract(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__2; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__24; lean_object* l_Lean_Elab_Term_levelMVarToParam(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*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheckFailure_declRange__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabExport(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___closed__1; LEAN_EXPORT lean_object* l_Lean_Syntax_forArgsM___at_Lean_Elab_Command_elabUniverse___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabUniverse___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabReduce_declRange__1___closed__5; LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabExport___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__1; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__19; static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheck__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAddDeclDoc_declRange__1___closed__7; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Elab_Command_elabOmit___spec__10___boxed(lean_object*, lean_object*); @@ -56,6 +60,7 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCom LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabChoice___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___lambda__1(lean_object*, lean_object*, uint8_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSection__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion___boxed(lean_object*); lean_object* l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_elabOpen___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__4; @@ -63,6 +68,7 @@ lean_object* l_Lean_Elab_addCompletionInfo___at_Lean_withSetOptionIn___spec__2(l LEAN_EXPORT lean_object* l_Lean_getDocStringText___at_Lean_Elab_Command_elabAddDeclDoc___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_hasNoErrorMessages___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabNamespace_declRange__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_elabChoice__1___closed__1; lean_object* l_Array_sequenceMap___at_Lean_Elab_OpenDecl_elabOpenDecl___spec__2(lean_object*, lean_object*); @@ -72,6 +78,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheck_declRange__1___cl lean_object* l_Lean_ScopedEnvExtension_activateScoped___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOpen___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSection_declRange__1___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabOpen___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd_declRange__1___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScope___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -102,6 +109,7 @@ static lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_ty static lean_object* l_Lean_Elab_Command_elabAddDeclDoc___closed__5; static lean_object* l_Lean_Elab_Command_expandInCmd___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOpen___spec__17(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__17; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVariable___lambda__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_Command_elabExit__1___closed__5; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabVariable___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -113,6 +121,7 @@ lean_object* l_Lean_indentD(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__6; static lean_object* l_Lean_Elab_Command_elabExit___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_addConstInfo___at_Lean_Elab_Command_elabOpen___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__30; static lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__2; uint8_t l_Lean_Exception_isInterrupt(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabExit__1___closed__4; @@ -121,11 +130,13 @@ lean_object* l_Lean_Elab_Command_getMainModule___rarg(lean_object*, lean_object* 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*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabEoi__1___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabCheck__1(lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__16; LEAN_EXPORT lean_object* l_Lean_Elab_addConstInfo___at_Lean_Elab_Command_elabExport___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_elabTerm(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_pushScope___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScope___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabReduce_go___lambda__1(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* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__15; lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabImport___rarg___closed__1; static lean_object* l_Lean_Elab_Command_elabOmit___lambda__1___closed__1; @@ -135,6 +146,7 @@ LEAN_EXPORT lean_object* l_Lean_Syntax_forArgsM___at_Lean_Elab_Command_elabUnive size_t lean_uint64_to_usize(uint64_t); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSection__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabNamespace___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__34; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabOpen___spec__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInclude___spec__1___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabOpen___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -147,6 +159,7 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___s lean_object* l_Lean_Syntax_getId(lean_object*); uint8_t l_List_beq___at___private_Lean_Data_OpenDecl_0__Lean_beqOpenDecl____x40_Lean_Data_OpenDecl___hyg_40____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitQuot___boxed(lean_object*); +extern uint8_t l_System_Platform_isOSX; static lean_object* l___regBuiltin_Lean_Elab_Command_expandInCmd__1___closed__4; lean_object* l_Array_findIdx_x3f_loop___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1(lean_object*); @@ -162,6 +175,7 @@ lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*) LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInclude___spec__1___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabExit___boxed(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__3; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__10; uint8_t l_Array_contains___at_Lean_findField_x3f___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCheckFailure___closed__3; static lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___closed__1; @@ -175,6 +189,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_failIfSucceeds___lambda__1(uint8_t, static lean_object* l_Lean_Elab_Command_elabExit___rarg___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabUniverse_declRange__1___closed__3; lean_object* l_Lean_Syntax_getArgs(lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_elabOpen___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen_declRange__1___closed__3; @@ -198,7 +213,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabUniverse__1___closed__3 lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabExport___spec__21(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabImport_declRange__1___closed__3; -lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); static lean_object* l_Lean_Elab_Command_elabReduce_go___lambda__1___closed__1; lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_expandDeclId___spec__8(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_getScopes___rarg(lean_object*, lean_object*); @@ -209,9 +223,12 @@ static lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___closed__7; static lean_object* l_Lean_logWarning___at_Lean_Elab_Command_elabExit___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabReduce_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_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___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*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__14; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__11; lean_object* l_Lean_Expr_fvarId_x21(lean_object*); extern lean_object* l_Lean_instInhabitedException; static lean_object* l___regBuiltin_Lean_Elab_Command_expandInCmd__1___closed__3; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__18; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__5; lean_object* l_Lean_ScopedEnvExtension_pushScope___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabVariable_declRange__1(lean_object*); @@ -236,6 +253,7 @@ lean_object* l_Lean_Syntax_node5(lean_object*, lean_object*, lean_object*, lean_ static lean_object* l___regBuiltin_Lean_Elab_Command_elabReduce_declRange__1___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabExport__1(lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__39; lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabSetOption_declRange__1(lean_object*); static lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__1; @@ -279,6 +297,7 @@ LEAN_EXPORT lean_object* l_Lean_resolveUniqueNamespace___at_Lean_Elab_Command_el static lean_object* l___regBuiltin_Lean_Elab_Command_elabExport_declRange__1___closed__5; LEAN_EXPORT lean_object* l_Lean_activateScoped___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScope___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc_declRange__1___closed__4; +static lean_object* l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__2; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Elab_Command_elabOmit___spec__5___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__20___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -298,6 +317,7 @@ LEAN_EXPORT lean_object* l_Lean_activateScoped___at___private_Lean_Elab_BuiltinC static lean_object* l___regBuiltin_Lean_Elab_Command_elabSection_declRange__1___closed__3; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabModuleDoc___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabImport(lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__26; LEAN_EXPORT lean_object* l_Lean_Syntax_foldArgsM___at_Lean_Elab_Command_elabUniverse___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVariable___lambda__2___boxed(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_mkConstWithLevelParams___spec__1(lean_object*, lean_object*); @@ -315,6 +335,7 @@ static lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___closed__10; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_containsId(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_popScopes___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Command_elabSetOption_declRange__1___closed__3; lean_object* l_Lean_InternalExceptionId_getName(lean_object*, lean_object*); static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabNamespace___spec__1___rarg___closed__2; @@ -322,6 +343,7 @@ extern lean_object* l___private_Lean_DocString_Extension_0__Lean_moduleDocExt; LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScope___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabNonComputableSection_declRange__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabCheck_declRange__1(lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__20; lean_object* l_Lean_MessageData_signature(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSetOption_declRange__1___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAddDeclDoc__1___closed__3; @@ -360,7 +382,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheckFailure_declRange_ static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__9; lean_object* l_Array_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabOpen___spec__2___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabModuleDoc___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabImport__1(lean_object*); static lean_object* l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExport___spec__1___closed__1; static lean_object* l_Lean_Elab_Command_elabSection___closed__3; @@ -404,6 +425,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabEoi_declRange__1___clos lean_object* lean_nat_div(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___closed__4; static lean_object* l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Command_elabExport___spec__18___closed__1; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVariable___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd_declRange__1___closed__5; lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_mkTermContext___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); @@ -420,8 +442,10 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabNonComputableSection_de static lean_object* l___regBuiltin_Lean_Elab_Command_elabNamespace_declRange__1___closed__6; uint64_t l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(lean_object*); lean_object* l_Lean_PersistentEnvExtension_addEntry___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_typelessBinder_x3f___closed__5; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__3; LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Command_elabExport___spec__20___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabReduce__1___closed__3; @@ -434,7 +458,9 @@ lean_object* l_Lean_Elab_Command_getRef(lean_object*, lean_object*, lean_object* LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitQuot(lean_object*); static lean_object* l_Lean_resolveUniqueNamespace___at_Lean_Elab_Command_elabOpen___spec__3___closed__1; static lean_object* l_Lean_Elab_Command_elabExport___closed__1; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__38; static lean_object* l_Lean_Elab_Command_elabNonComputableSection___closed__1; +extern lean_object* l_Lean_versionString; static lean_object* l___regBuiltin_Lean_Elab_Command_elabExport__1___closed__3; lean_object* l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabExport___closed__2; @@ -455,6 +481,7 @@ LEAN_EXPORT lean_object* l_Lean_resolveNamespace___at_Lean_Elab_Command_elabExpo static lean_object* l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabAddDeclDoc__1(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_Command_elabVersion___rarg___lambda__1___closed__28; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabExport___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_outOfBounds___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_findDeclarationRangesCore_x3f___at_Lean_Elab_Command_elabAddDeclDoc___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -469,6 +496,7 @@ static lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveName lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__16(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabExport__1___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabVariable_declRange__1___closed__3; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__29; lean_object* lean_st_ref_get(lean_object*, lean_object*); lean_object* l_Lean_Exception_getRef(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSynth___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -495,8 +523,10 @@ static lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveName static lean_object* l___regBuiltin_Lean_Elab_Command_elabReduce_declRange__1___closed__7; lean_object* lean_array_to_list(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScopes___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__33; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInclude___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___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_Elab_Command_elabVersion___rarg___lambda__1___closed__27; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabUniverse_declRange__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd__1___closed__1; @@ -511,6 +541,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheckFailure_declRange_ LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Command_elabExport___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc_declRange__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabNamespace(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__31; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabExport___spec__23___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_forInUnsafe_loop___at_Lean_Elab_Command_elabOpen___spec__17___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1___closed__1; @@ -522,6 +553,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabChoice__1___closed__4; static lean_object* l_Lean_resolveUniqueNamespace___at_Lean_Elab_Command_elabOpen___spec__3___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabOpen___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_modifyScope(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCheckCore___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_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___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* l_Lean_Elab_realizeGlobalConstNoOverloadWithInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -536,6 +568,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabNamespace_declRange__1_ static lean_object* l___regBuiltin_Lean_Elab_Command_elabExport_declRange__1___closed__1; LEAN_EXPORT lean_object* l_Lean_logWarning___at_Lean_Elab_Command_elabExit___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabExport___spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_List_foldl___at_String_join___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabExit_declRange__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabEoi___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); @@ -580,6 +613,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabExport___lambda__1(lean_object* static lean_object* l___regBuiltin_Lean_Elab_Command_elabSection_declRange__1___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd_declRange__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabReduce___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__36; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Elab_Command_elabOmit___spec__10(lean_object*, lean_object*); lean_object* l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); @@ -590,6 +624,7 @@ LEAN_EXPORT lean_object* l_Lean_pushScope___at___private_Lean_Elab_BuiltinComman LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSection_declRange__1___closed__7; static lean_object* l___regBuiltin_Lean_Elab_Command_elabEoi_declRange__1___closed__5; +extern uint8_t l_System_Platform_isEmscripten; static lean_object* l_Lean_resolveNamespaceCore___at_Lean_Elab_Command_elabExport___spec__3___closed__3; uint8_t l_Lean_Syntax_isIdent(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Command_elabOpen___spec__22(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -604,12 +639,15 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_elabChoice_declRange__1___closed__2; lean_object* l_Lean_Elab_Command_getScope___rarg(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandInCmd__1___closed__2; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__35; lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg(lean_object*, uint8_t, 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_Lean_Elab_Command_elabOmit___spec__6(lean_object*); lean_object* l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2(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_Lean_Syntax_forArgsM___at_Lean_Elab_Command_elabUniverse___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabUniverse(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__5; lean_object* l_Array_eraseIdx___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__22; static lean_object* l_Lean_Elab_Command_elabImport___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSynth_declRange__1___closed__5; @@ -619,12 +657,14 @@ lean_object* l_Lean_Elab_realizeGlobalConstWithInfos(lean_object*, lean_object*, lean_object* l_Lean_KVMap_setBool(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabVariable___spec__4(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_add_alias(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__12; lean_object* l_Lean_Environment_addDecl(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInclude___spec__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabSynth__1___closed__5; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheck__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabReduce(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd_declRange__1___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabVariable_declRange__1___closed__1; @@ -636,6 +676,7 @@ static lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_elabOpen___s LEAN_EXPORT lean_object* l_Lean_popScope___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_popScopes___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCheckCore___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11___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_Command_elabVersion___rarg___lambda__1___closed__32; static lean_object* l___regBuiltin_Lean_Elab_Command_elabExit_declRange__1___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabExport___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Command_elabExport___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -643,6 +684,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Comma lean_object* l_Array_append___rarg(lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageLog_errorsToWarnings(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabModuleDoc___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabVariable__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation(lean_object*, lean_object*, lean_object*, lean_object*); @@ -695,10 +737,12 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabSection_declRange_ static lean_object* l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__7; static lean_object* l___regBuiltin_Lean_Elab_Command_elabChoice_declRange__1___closed__6; lean_object* l_Lean_FileMap_leanPosToLspPos(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__7; static lean_object* l_Lean_Elab_Command_elabCheckFailure___closed__1; static lean_object* l_Lean_Elab_Command_elabCheckCore___closed__2; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOpen___spec__17___lambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_expandInCmd_declRange__1___closed__5; +static lean_object* l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_elabEoi__1___closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___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_resolveNamespace___at_Lean_Elab_Command_elabExport___spec__1___closed__3; @@ -720,11 +764,13 @@ static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___s static lean_object* l___regBuiltin_Lean_Elab_Command_elabSynth_declRange__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCheckCore___lambda__4(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___regBuiltin_Lean_Elab_Command_elabSynth__1___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabVersion__1(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabInitQuot_declRange__1___closed__5; extern lean_object* l_Lean_NameSet_empty; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__12___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScope___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOmit___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_Elab_Command_elabVersion___rarg___lambda__1___closed__21; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabEnd___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___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_Elab_Command_elabVariable(lean_object*, lean_object*, lean_object*, lean_object*); @@ -750,6 +796,7 @@ uint8_t lean_nat_dec_lt(lean_object*, lean_object*); lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_OpenDecl_elabOpenDecl___spec__5(size_t, size_t, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSection_declRange__1___closed__2; LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_elabOpen___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__3; static lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_typelessBinder_x3f___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSynth___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_Command_elabChoice_declRange__1___closed__3; @@ -804,6 +851,7 @@ lean_object* l_Lean_Meta_reduce(lean_object*, uint8_t, uint8_t, uint8_t, lean_ob lean_object* l_Lean_LocalDecl_type(lean_object*); uint64_t lean_uint64_xor(uint64_t, uint64_t); static lean_object* l___regBuiltin_Lean_Elab_Command_elabImport__1___closed__3; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___closed__4; static lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___closed__11; uint8_t l_Lean_Syntax_isNone(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabOpen___spec__2___boxed(lean_object*, lean_object*, lean_object*); @@ -829,18 +877,22 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabVa lean_object* l_Lean_Elab_Command_liftCoreM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabChoice__1(lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__4; LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Command_elabExport___spec__14(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Core_resetMessageLog(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabReduce_go___lambda__2___closed__2; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__23; static lean_object* l___regBuiltin_Lean_Elab_Command_elabNonComputableSection_declRange__1___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen__1___closed__3; LEAN_EXPORT lean_object* l_Lean_setEnv___at_Lean_Elab_Command_elabInitQuot___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabNonComputableSection___closed__2; +lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___spec__4___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen_declRange__1(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabSynth_declRange__1___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabModuleDoc___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabEoi_declRange__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_elabExit_declRange__1___closed__7; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabSection__1(lean_object*); @@ -872,6 +924,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabModuleDoc(lean_object*, lean_ob static lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScopes___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_Elab_Command_elabOpen___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCheckFailure(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___closed__1; static lean_object* l_Lean_Elab_Command_elabAddDeclDoc___closed__6; static lean_object* l_Lean_Elab_Command_elabInclude___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_resolveId___at_Lean_Elab_Command_elabExport___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -920,11 +973,12 @@ static lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_ela static lean_object* l___regBuiltin_Lean_Elab_Command_elabImport_declRange__1___closed__2; static lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___closed__1; static lean_object* l_Lean_Elab_Command_elabCheckCore___lambda__4___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabModuleDoc___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_addOpenDecl___at_Lean_Elab_Command_elabOpen___spec__10(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_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__25; static lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen__1___closed__1; +static uint8_t l_Lean_Elab_Command_elabVersion___rarg___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_elabOpen___spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Command_elabOpen___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -934,6 +988,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen__1(lean_objec lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11(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___regBuiltin_Lean_Elab_Command_elabReduce_declRange__1(lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__37; static lean_object* l___regBuiltin_Lean_Elab_Command_elabEoi_declRange__1___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Command_elabUniverse__1___closed__4; LEAN_EXPORT lean_object* l_Lean_filterFieldList___at_Lean_Elab_Command_elabExport___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -987,13 +1042,17 @@ static lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_ch lean_object* l_List_toString___at_Lean_OpenDecl_instToString___spec__1(lean_object*); static lean_object* l_Lean_Elab_Command_elabReduce___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSetOption(lean_object*, lean_object*, lean_object*, lean_object*); +extern lean_object* l_System_Platform_target; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__4___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabExport___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVariable___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Elab_Command_elabInclude___spec__2(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__40; +extern uint8_t l_System_Platform_isWindows; lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___spec__2(size_t, size_t, lean_object*); lean_object* l_Lean_KernelException_toMessageData(lean_object*, lean_object*); lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Command_expandDeclId___spec__11(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Command_elabCheck_declRange__1___closed__3; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabAddDeclDoc___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabNonComputableSection(lean_object*, lean_object*, lean_object*, lean_object*); @@ -1002,10 +1061,13 @@ LEAN_EXPORT lean_object* l___private_Lean_ResolveName_0__Lean_resolveGlobalConst lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOpen___spec__23(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen_declRange__1___closed__1; lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabChoice__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabOpen__1___closed__2; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__13; +static lean_object* l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__41; lean_object* l_List_filterTR_loop___at_Lean_filterFieldList___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabEnd___closed__2; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__5___closed__3; @@ -1096,237 +1158,146 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabModuleDoc___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabModuleDoc___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_5; uint8_t x_6; lean_object* x_7; lean_object* x_8; -x_5 = lean_ctor_get(x_2, 1); -lean_inc(x_5); -lean_dec(x_2); -x_6 = 0; -x_7 = l_Lean_Syntax_getPos_x3f(x_1, x_6); -x_8 = l_Lean_Syntax_getTailPos_x3f(x_1, x_6); -if (lean_obj_tag(x_7) == 0) +uint8_t x_5; lean_object* x_6; +x_5 = 0; +x_6 = l_Lean_Syntax_getRange_x3f(x_1, x_5); +if (lean_obj_tag(x_6) == 0) { -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = lean_unsigned_to_nat(0u); -lean_inc(x_5); -x_10 = l_Lean_FileMap_toPosition(x_5, x_9); -lean_inc(x_10); -x_11 = l_Lean_FileMap_leanPosToLspPos(x_5, x_10); -if (lean_obj_tag(x_8) == 0) +lean_object* x_7; lean_object* x_8; +lean_dec(x_2); +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_4); +return x_8; +} +else { -uint8_t x_12; -lean_dec(x_5); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +uint8_t x_9; +x_9 = !lean_is_exclusive(x_6); +if (x_9 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_11, 1); -x_14 = lean_ctor_get(x_11, 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; uint8_t x_17; +x_10 = lean_ctor_get(x_6, 0); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +lean_dec(x_2); +x_12 = lean_ctor_get(x_10, 0); +lean_inc(x_12); +lean_inc(x_11); +x_13 = l_Lean_FileMap_toPosition(x_11, x_12); +lean_dec(x_12); +x_14 = lean_ctor_get(x_10, 1); +lean_inc(x_14); +lean_dec(x_10); +lean_inc(x_11); +x_15 = l_Lean_FileMap_toPosition(x_11, x_14); lean_dec(x_14); lean_inc(x_13); -lean_inc(x_10); -x_15 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_15, 0, x_10); -lean_ctor_set(x_15, 1, x_13); -lean_ctor_set(x_15, 2, x_10); -lean_ctor_set(x_15, 3, x_13); -lean_ctor_set(x_11, 1, x_4); -lean_ctor_set(x_11, 0, x_15); -return x_11; -} -else +x_16 = l_Lean_FileMap_leanPosToLspPos(x_11, x_13); +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) { -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_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_18 = lean_ctor_get(x_16, 1); +x_19 = lean_ctor_get(x_16, 0); +lean_dec(x_19); +lean_inc(x_15); +x_20 = l_Lean_FileMap_leanPosToLspPos(x_11, x_15); lean_dec(x_11); -lean_inc(x_16); -lean_inc(x_10); -x_17 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_17, 0, x_10); -lean_ctor_set(x_17, 1, x_16); -lean_ctor_set(x_17, 2, x_10); -lean_ctor_set(x_17, 3, 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_4); -return x_18; -} +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_22, 0, x_13); +lean_ctor_set(x_22, 1, x_18); +lean_ctor_set(x_22, 2, x_15); +lean_ctor_set(x_22, 3, x_21); +lean_ctor_set(x_6, 0, x_22); +lean_ctor_set(x_16, 1, x_4); +lean_ctor_set(x_16, 0, x_6); +return x_16; } else { -uint8_t x_19; -x_19 = !lean_is_exclusive(x_11); -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; -x_20 = lean_ctor_get(x_11, 1); -x_21 = lean_ctor_get(x_11, 0); -lean_dec(x_21); -x_22 = lean_ctor_get(x_8, 0); -lean_inc(x_22); -lean_dec(x_8); -lean_inc(x_5); -x_23 = l_Lean_FileMap_toPosition(x_5, x_22); -lean_dec(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_16, 1); lean_inc(x_23); -x_24 = l_Lean_FileMap_leanPosToLspPos(x_5, x_23); -lean_dec(x_5); +lean_dec(x_16); +lean_inc(x_15); +x_24 = l_Lean_FileMap_leanPosToLspPos(x_11, x_15); +lean_dec(x_11); x_25 = lean_ctor_get(x_24, 1); lean_inc(x_25); lean_dec(x_24); x_26 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_26, 0, x_10); -lean_ctor_set(x_26, 1, x_20); -lean_ctor_set(x_26, 2, x_23); +lean_ctor_set(x_26, 0, x_13); +lean_ctor_set(x_26, 1, x_23); +lean_ctor_set(x_26, 2, x_15); lean_ctor_set(x_26, 3, x_25); -lean_ctor_set(x_11, 1, x_4); -lean_ctor_set(x_11, 0, x_26); -return x_11; +lean_ctor_set(x_6, 0, x_26); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_6); +lean_ctor_set(x_27, 1, x_4); +return x_27; +} } 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_ctor_get(x_11, 1); -lean_inc(x_27); -lean_dec(x_11); -x_28 = lean_ctor_get(x_8, 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; +x_28 = lean_ctor_get(x_6, 0); lean_inc(x_28); -lean_dec(x_8); -lean_inc(x_5); -x_29 = l_Lean_FileMap_toPosition(x_5, x_28); +lean_dec(x_6); +x_29 = lean_ctor_get(x_2, 1); +lean_inc(x_29); +lean_dec(x_2); +x_30 = lean_ctor_get(x_28, 0); +lean_inc(x_30); +lean_inc(x_29); +x_31 = l_Lean_FileMap_toPosition(x_29, x_30); +lean_dec(x_30); +x_32 = lean_ctor_get(x_28, 1); +lean_inc(x_32); lean_dec(x_28); lean_inc(x_29); -x_30 = l_Lean_FileMap_leanPosToLspPos(x_5, x_29); -lean_dec(x_5); -x_31 = lean_ctor_get(x_30, 1); +x_33 = l_Lean_FileMap_toPosition(x_29, x_32); +lean_dec(x_32); lean_inc(x_31); -lean_dec(x_30); -x_32 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_32, 0, x_10); -lean_ctor_set(x_32, 1, x_27); -lean_ctor_set(x_32, 2, x_29); -lean_ctor_set(x_32, 3, 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_4); -return x_33; -} -} -} -else -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_7, 0); -lean_inc(x_34); -lean_dec(x_7); -lean_inc(x_5); -x_35 = l_Lean_FileMap_toPosition(x_5, x_34); -lean_dec(x_34); -lean_inc(x_35); -x_36 = l_Lean_FileMap_leanPosToLspPos(x_5, x_35); -if (lean_obj_tag(x_8) == 0) -{ -uint8_t x_37; -lean_dec(x_5); -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, 1); -x_39 = lean_ctor_get(x_36, 0); -lean_dec(x_39); -lean_inc(x_38); -lean_inc(x_35); -x_40 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_40, 0, x_35); -lean_ctor_set(x_40, 1, x_38); -lean_ctor_set(x_40, 2, x_35); -lean_ctor_set(x_40, 3, x_38); -lean_ctor_set(x_36, 1, x_4); -lean_ctor_set(x_36, 0, x_40); -return x_36; -} -else -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_36, 1); -lean_inc(x_41); -lean_dec(x_36); -lean_inc(x_41); +x_34 = l_Lean_FileMap_leanPosToLspPos(x_29, x_31); +x_35 = lean_ctor_get(x_34, 1); lean_inc(x_35); -x_42 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_42, 0, x_35); -lean_ctor_set(x_42, 1, x_41); -lean_ctor_set(x_42, 2, x_35); -lean_ctor_set(x_42, 3, 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_4); -return x_43; -} -} -else -{ -uint8_t x_44; -x_44 = !lean_is_exclusive(x_36); -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 = lean_ctor_get(x_36, 1); -x_46 = lean_ctor_get(x_36, 0); -lean_dec(x_46); -x_47 = lean_ctor_get(x_8, 0); -lean_inc(x_47); -lean_dec(x_8); -lean_inc(x_5); -x_48 = l_Lean_FileMap_toPosition(x_5, x_47); -lean_dec(x_47); -lean_inc(x_48); -x_49 = l_Lean_FileMap_leanPosToLspPos(x_5, x_48); -lean_dec(x_5); -x_50 = lean_ctor_get(x_49, 1); -lean_inc(x_50); -lean_dec(x_49); -x_51 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_51, 0, x_35); -lean_ctor_set(x_51, 1, x_45); -lean_ctor_set(x_51, 2, x_48); -lean_ctor_set(x_51, 3, x_50); -lean_ctor_set(x_36, 1, x_4); -lean_ctor_set(x_36, 0, x_51); -return x_36; +if (lean_is_exclusive(x_34)) { + lean_ctor_release(x_34, 0); + lean_ctor_release(x_34, 1); + x_36 = x_34; +} else { + lean_dec_ref(x_34); + x_36 = lean_box(0); } -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; -x_52 = lean_ctor_get(x_36, 1); -lean_inc(x_52); -lean_dec(x_36); -x_53 = lean_ctor_get(x_8, 0); -lean_inc(x_53); -lean_dec(x_8); -lean_inc(x_5); -x_54 = l_Lean_FileMap_toPosition(x_5, x_53); -lean_dec(x_53); -lean_inc(x_54); -x_55 = l_Lean_FileMap_leanPosToLspPos(x_5, x_54); -lean_dec(x_5); -x_56 = lean_ctor_get(x_55, 1); -lean_inc(x_56); -lean_dec(x_55); -x_57 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_57, 0, x_35); -lean_ctor_set(x_57, 1, x_52); -lean_ctor_set(x_57, 2, x_54); -lean_ctor_set(x_57, 3, x_56); -x_58 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_58, 0, x_57); -lean_ctor_set(x_58, 1, x_4); -return x_58; +lean_inc(x_33); +x_37 = l_Lean_FileMap_leanPosToLspPos(x_29, x_33); +lean_dec(x_29); +x_38 = lean_ctor_get(x_37, 1); +lean_inc(x_38); +lean_dec(x_37); +x_39 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_39, 0, x_31); +lean_ctor_set(x_39, 1, x_35); +lean_ctor_set(x_39, 2, x_33); +lean_ctor_set(x_39, 3, x_38); +x_40 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_40, 0, x_39); +if (lean_is_scalar(x_36)) { + x_41 = lean_alloc_ctor(0, 2, 0); +} else { + x_41 = x_36; } +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_4); +return x_41; } } } @@ -1381,7 +1352,7 @@ x_5 = lean_unsigned_to_nat(1u); x_6 = l_Lean_Syntax_getArg(x_1, x_5); if (lean_obj_tag(x_6) == 2) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; 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; +lean_object* x_7; lean_object* x_8; 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_7 = lean_ctor_get(x_6, 1); lean_inc(x_7); lean_dec(x_6); @@ -1393,202 +1364,236 @@ x_11 = lean_unsigned_to_nat(0u); x_12 = lean_string_utf8_extract(x_7, x_11, x_10); lean_dec(x_10); lean_dec(x_7); -x_13 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabModuleDoc___spec__2(x_1, x_2, x_3, x_4); +x_13 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabModuleDoc___spec__2(x_1, x_2, x_3, x_4); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); +if (lean_obj_tag(x_14) == 0) +{ +uint8_t x_15; +lean_dec(x_12); +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_16 = lean_st_ref_take(x_3, x_15); -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) +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_18; uint8_t x_19; -x_18 = lean_ctor_get(x_16, 0); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) +lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_21 = lean_ctor_get(x_13, 1); +lean_inc(x_21); +lean_dec(x_13); +x_22 = lean_ctor_get(x_14, 0); +lean_inc(x_22); +lean_dec(x_14); +x_23 = lean_st_ref_take(x_3, x_21); +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) { -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_20 = lean_ctor_get(x_16, 1); -x_21 = lean_ctor_get(x_18, 0); -lean_ctor_set(x_16, 1, x_14); -lean_ctor_set(x_16, 0, x_12); -x_22 = l_Lean_Elab_Command_elabModuleDoc___closed__5; -x_23 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_22, x_21, x_16); -lean_ctor_set(x_18, 0, x_23); -x_24 = lean_st_ref_set(x_3, x_18, x_20); -x_25 = !lean_is_exclusive(x_24); -if (x_25 == 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_26; lean_object* x_27; -x_26 = lean_ctor_get(x_24, 0); -lean_dec(x_26); -x_27 = lean_box(0); -lean_ctor_set(x_24, 0, x_27); -return x_24; +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_23, 1); +x_28 = lean_ctor_get(x_25, 0); +lean_ctor_set(x_23, 1, x_22); +lean_ctor_set(x_23, 0, x_12); +x_29 = l_Lean_Elab_Command_elabModuleDoc___closed__5; +x_30 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_29, x_28, x_23); +lean_ctor_set(x_25, 0, x_30); +x_31 = lean_st_ref_set(x_3, x_25, x_27); +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_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_24, 1); -lean_inc(x_28); -lean_dec(x_24); -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; +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 { -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; -x_31 = lean_ctor_get(x_16, 1); -x_32 = lean_ctor_get(x_18, 0); -x_33 = lean_ctor_get(x_18, 1); -x_34 = lean_ctor_get(x_18, 2); -x_35 = lean_ctor_get(x_18, 3); -x_36 = lean_ctor_get(x_18, 4); -x_37 = lean_ctor_get(x_18, 5); -x_38 = lean_ctor_get(x_18, 6); -x_39 = lean_ctor_get(x_18, 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_dec(x_18); -lean_ctor_set(x_16, 1, x_14); -lean_ctor_set(x_16, 0, x_12); -x_40 = l_Lean_Elab_Command_elabModuleDoc___closed__5; -x_41 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_40, x_32, x_16); -x_42 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_33); -lean_ctor_set(x_42, 2, x_34); -lean_ctor_set(x_42, 3, x_35); -lean_ctor_set(x_42, 4, x_36); -lean_ctor_set(x_42, 5, x_37); -lean_ctor_set(x_42, 6, x_38); -lean_ctor_set(x_42, 7, x_39); -x_43 = lean_st_ref_set(x_3, x_42, x_31); -x_44 = lean_ctor_get(x_43, 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; 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_38 = lean_ctor_get(x_23, 1); +x_39 = lean_ctor_get(x_25, 0); +x_40 = lean_ctor_get(x_25, 1); +x_41 = lean_ctor_get(x_25, 2); +x_42 = lean_ctor_get(x_25, 3); +x_43 = lean_ctor_get(x_25, 4); +x_44 = lean_ctor_get(x_25, 5); +x_45 = lean_ctor_get(x_25, 6); +x_46 = lean_ctor_get(x_25, 7); +lean_inc(x_46); +lean_inc(x_45); lean_inc(x_44); -if (lean_is_exclusive(x_43)) { - lean_ctor_release(x_43, 0); - lean_ctor_release(x_43, 1); - x_45 = x_43; +lean_inc(x_43); +lean_inc(x_42); +lean_inc(x_41); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_25); +lean_ctor_set(x_23, 1, x_22); +lean_ctor_set(x_23, 0, x_12); +x_47 = l_Lean_Elab_Command_elabModuleDoc___closed__5; +x_48 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_47, x_39, x_23); +x_49 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_40); +lean_ctor_set(x_49, 2, x_41); +lean_ctor_set(x_49, 3, x_42); +lean_ctor_set(x_49, 4, x_43); +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_st_ref_set(x_3, x_49, x_38); +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_43); - x_45 = lean_box(0); + lean_dec_ref(x_50); + x_52 = lean_box(0); } -x_46 = lean_box(0); -if (lean_is_scalar(x_45)) { - x_47 = lean_alloc_ctor(0, 2, 0); +x_53 = lean_box(0); +if (lean_is_scalar(x_52)) { + x_54 = lean_alloc_ctor(0, 2, 0); } else { - x_47 = x_45; + x_54 = x_52; } -lean_ctor_set(x_47, 0, x_46); -lean_ctor_set(x_47, 1, x_44); -return x_47; +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_51); +return x_54; } } 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; 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_48 = lean_ctor_get(x_16, 0); -x_49 = lean_ctor_get(x_16, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_16); -x_50 = lean_ctor_get(x_48, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_48, 1); -lean_inc(x_51); -x_52 = lean_ctor_get(x_48, 2); -lean_inc(x_52); -x_53 = lean_ctor_get(x_48, 3); -lean_inc(x_53); -x_54 = lean_ctor_get(x_48, 4); -lean_inc(x_54); -x_55 = lean_ctor_get(x_48, 5); -lean_inc(x_55); -x_56 = lean_ctor_get(x_48, 6); +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; +x_55 = lean_ctor_get(x_23, 0); +x_56 = lean_ctor_get(x_23, 1); lean_inc(x_56); -x_57 = lean_ctor_get(x_48, 7); +lean_inc(x_55); +lean_dec(x_23); +x_57 = lean_ctor_get(x_55, 0); lean_inc(x_57); -if (lean_is_exclusive(x_48)) { - lean_ctor_release(x_48, 0); - lean_ctor_release(x_48, 1); - lean_ctor_release(x_48, 2); - lean_ctor_release(x_48, 3); - lean_ctor_release(x_48, 4); - lean_ctor_release(x_48, 5); - lean_ctor_release(x_48, 6); - lean_ctor_release(x_48, 7); - x_58 = x_48; -} else { - lean_dec_ref(x_48); - x_58 = lean_box(0); -} -x_59 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_59, 0, x_12); -lean_ctor_set(x_59, 1, x_14); -x_60 = l_Lean_Elab_Command_elabModuleDoc___closed__5; -x_61 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_60, x_50, x_59); -if (lean_is_scalar(x_58)) { - x_62 = lean_alloc_ctor(0, 8, 0); -} else { - x_62 = x_58; -} -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_51); -lean_ctor_set(x_62, 2, x_52); -lean_ctor_set(x_62, 3, x_53); -lean_ctor_set(x_62, 4, x_54); -lean_ctor_set(x_62, 5, x_55); -lean_ctor_set(x_62, 6, x_56); -lean_ctor_set(x_62, 7, x_57); -x_63 = lean_st_ref_set(x_3, x_62, x_49); -x_64 = lean_ctor_get(x_63, 1); +x_58 = lean_ctor_get(x_55, 1); +lean_inc(x_58); +x_59 = lean_ctor_get(x_55, 2); +lean_inc(x_59); +x_60 = lean_ctor_get(x_55, 3); +lean_inc(x_60); +x_61 = lean_ctor_get(x_55, 4); +lean_inc(x_61); +x_62 = lean_ctor_get(x_55, 5); +lean_inc(x_62); +x_63 = lean_ctor_get(x_55, 6); +lean_inc(x_63); +x_64 = lean_ctor_get(x_55, 7); 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; -} else { - lean_dec_ref(x_63); +if (lean_is_exclusive(x_55)) { + lean_ctor_release(x_55, 0); + lean_ctor_release(x_55, 1); + lean_ctor_release(x_55, 2); + lean_ctor_release(x_55, 3); + lean_ctor_release(x_55, 4); + lean_ctor_release(x_55, 5); + lean_ctor_release(x_55, 6); + lean_ctor_release(x_55, 7); + x_65 = x_55; +} else { + lean_dec_ref(x_55); x_65 = lean_box(0); } -x_66 = lean_box(0); +x_66 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_66, 0, x_12); +lean_ctor_set(x_66, 1, x_22); +x_67 = l_Lean_Elab_Command_elabModuleDoc___closed__5; +x_68 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_67, x_57, x_66); if (lean_is_scalar(x_65)) { - x_67 = lean_alloc_ctor(0, 2, 0); + x_69 = lean_alloc_ctor(0, 8, 0); } else { - x_67 = x_65; + x_69 = x_65; +} +lean_ctor_set(x_69, 0, x_68); +lean_ctor_set(x_69, 1, x_58); +lean_ctor_set(x_69, 2, x_59); +lean_ctor_set(x_69, 3, x_60); +lean_ctor_set(x_69, 4, x_61); +lean_ctor_set(x_69, 5, x_62); +lean_ctor_set(x_69, 6, x_63); +lean_ctor_set(x_69, 7, x_64); +x_70 = lean_st_ref_set(x_3, x_69, x_56); +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; +} else { + lean_dec_ref(x_70); + x_72 = lean_box(0); +} +x_73 = lean_box(0); +if (lean_is_scalar(x_72)) { + x_74 = lean_alloc_ctor(0, 2, 0); +} else { + x_74 = x_72; +} +lean_ctor_set(x_74, 0, x_73); +lean_ctor_set(x_74, 1, x_71); +return x_74; } -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, 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; -x_68 = l_Lean_MessageData_ofSyntax(x_6); -x_69 = l_Lean_indentD(x_68); -x_70 = l_Lean_Elab_Command_elabModuleDoc___closed__2; -x_71 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_71, 0, x_70); -lean_ctor_set(x_71, 1, x_69); -x_72 = l_Lean_Elab_Command_elabModuleDoc___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 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabModuleDoc___spec__1(x_1, x_73, x_2, x_3, x_4); -return 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_75 = l_Lean_MessageData_ofSyntax(x_6); +x_76 = l_Lean_indentD(x_75); +x_77 = l_Lean_Elab_Command_elabModuleDoc___closed__2; +x_78 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_78, 0, x_77); +lean_ctor_set(x_78, 1, x_76); +x_79 = l_Lean_Elab_Command_elabModuleDoc___closed__4; +x_80 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_80, 0, x_78); +lean_ctor_set(x_80, 1, x_79); +x_81 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabModuleDoc___spec__1(x_1, x_80, x_2, x_3, x_4); +return x_81; } } } @@ -1602,11 +1607,11 @@ lean_dec(x_1); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabModuleDoc___spec__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_getDeclarationRange_x3f___at_Lean_Elab_Command_elabModuleDoc___spec__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_getDeclarationRange___at_Lean_Elab_Command_elabModuleDoc___spec__2(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabModuleDoc___spec__2(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_1); return x_5; @@ -26179,42 +26184,97 @@ return x_69; LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___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; lean_object* x_10; uint8_t x_11; +lean_object* x_7; lean_object* x_8; lean_inc(x_4); -x_7 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabModuleDoc___spec__2(x_2, x_4, x_5, x_6); +x_7 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabModuleDoc___spec__2(x_2, 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); -lean_inc(x_4); -x_10 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabModuleDoc___spec__2(x_3, x_4, x_5, x_9); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) +if (lean_obj_tag(x_8) == 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_ctor_set(x_10, 1, x_12); -lean_ctor_set(x_10, 0, x_8); -x_14 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__6(x_1, x_10, x_4, x_5, x_13); +uint8_t x_9; lean_dec(x_4); +lean_dec(x_1); +x_9 = !lean_is_exclusive(x_7); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_7, 0); +lean_dec(x_10); +x_11 = lean_box(0); +lean_ctor_set(x_7, 0, x_11); +return x_7; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_7, 1); +lean_inc(x_12); +lean_dec(x_7); +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_12); 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_10, 0); -x_16 = lean_ctor_get(x_10, 1); -lean_inc(x_16); +x_15 = lean_ctor_get(x_7, 1); lean_inc(x_15); -lean_dec(x_10); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_8); -lean_ctor_set(x_17, 1, x_15); -x_18 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__6(x_1, x_17, x_4, x_5, x_16); +lean_dec(x_7); +x_16 = lean_ctor_get(x_8, 0); +lean_inc(x_16); +lean_dec(x_8); +lean_inc(x_4); +x_17 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabModuleDoc___spec__2(x_3, x_4, x_5, x_15); +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_4); -return x_18; +lean_dec(x_1); +x_19 = !lean_is_exclusive(x_17); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_17, 0); +lean_dec(x_20); +x_21 = lean_box(0); +lean_ctor_set(x_17, 0, x_21); +return x_17; +} +else +{ +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_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 +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_25 = lean_ctor_get(x_17, 1); +lean_inc(x_25); +lean_dec(x_17); +x_26 = lean_ctor_get(x_18, 0); +lean_inc(x_26); +lean_dec(x_18); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_16); +lean_ctor_set(x_27, 1, x_26); +x_28 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAddDeclDoc___spec__6(x_1, x_27, x_4, x_5, x_25); +lean_dec(x_4); +return x_28; +} } } } @@ -29235,300 +29295,1003 @@ x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOmit(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOmit(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; uint8_t x_6; +x_5 = l_Lean_Elab_Command_elabOmit___closed__2; +lean_inc(x_1); +x_6 = l_Lean_Syntax_isOfKind(x_1, x_5); +if (x_6 == 0) +{ +lean_object* x_7; +lean_dec(x_1); +x_7 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabNamespace___spec__1___rarg(x_4); +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; lean_object* x_14; lean_object* x_15; +x_8 = lean_unsigned_to_nat(1u); +x_9 = l_Lean_Syntax_getArg(x_1, x_8); +lean_dec(x_1); +x_10 = lean_box(0); +x_11 = l_Lean_Syntax_getArgs(x_9); +lean_dec(x_9); +x_12 = l_Lean_Elab_Command_elabSection___closed__4; +x_13 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__2; +x_14 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabOmit___lambda__1___boxed), 12, 4); +lean_closure_set(x_14, 0, x_11); +lean_closure_set(x_14, 1, x_12); +lean_closure_set(x_14, 2, x_13); +lean_closure_set(x_14, 3, x_10); +x_15 = l_Lean_Elab_Command_runTermElabM___rarg(x_14, x_2, x_3, x_4); +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_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_alloc_closure((void*)(l_Lean_Elab_Command_elabOmit___lambda__2), 3, 2); +lean_closure_set(x_18, 0, x_16); +lean_closure_set(x_18, 1, x_10); +x_19 = l_Lean_Elab_Command_modifyScope(x_18, x_2, x_3, x_17); +return x_19; +} +else +{ +uint8_t x_20; +x_20 = !lean_is_exclusive(x_15); +if (x_20 == 0) +{ +return x_15; +} +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_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabOmit___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) { +_start: +{ +lean_object* x_7; +x_7 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabOmit___spec__1(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_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___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: +{ +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_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___spec__3(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_3); +lean_dec(x_2); +lean_dec(x_1); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___spec__4___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_6 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___spec__4(x_4, x_5, x_3); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Elab_Command_elabOmit___spec__5___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_Elab_Command_elabOmit___spec__5(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_get_x3f___at_Lean_Elab_Command_elabOmit___spec__10___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_Elab_Command_elabOmit___spec__10(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11___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_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___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_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_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11(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_1); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___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_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__12___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_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___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_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; size_t x_17; lean_object* x_18; +x_15 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_16 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_17 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_18 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__12(x_15, x_2, x_3, x_4, x_16, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_9); +lean_dec(x_4); +lean_dec(x_2); +return x_18; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___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, 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_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__13(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_1); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Elab_Command_elabOmit___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_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_RBNode_forIn_visit___at_Lean_Elab_Command_elabOmit___spec__14(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); +return x_11; +} +} +LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Elab_Command_elabOmit___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_List_filterTR_loop___at_Lean_Elab_Command_elabOmit___spec__15(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOmit___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_Elab_Command_elabOmit___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_5); +lean_dec(x_3); +lean_dec(x_2); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOmit___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_Command_elabOmit(x_1, x_2, x_3, x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_5; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("elabOmit", 8, 8); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabOmit__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___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__1; +x_2 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__6; +x_3 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__3; +x_4 = l___regBuiltin_Lean_Elab_Command_elabOmit__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___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabOmit___boxed), 4, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabOmit__1(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___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__9; +x_3 = l_Lean_Elab_Command_elabOmit___closed__2; +x_4 = l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__2; +x_5 = l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__3; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean ", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_versionString; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__2; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__3; +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_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("\nTarget: ", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__4; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__6; +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_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = l_List_appendTR___rarg(x_1, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___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_Command_elabVersion___rarg___lambda__1___closed__8; +x_3 = l_List_appendTR___rarg(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabModuleDoc___closed__3; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__9; +x_3 = l_List_foldl___at_String_join___spec__1(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__10; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__12() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" Emscripten", 11, 11); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__12; +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_Command_elabVersion___rarg___lambda__1___closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__8; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__13; +x_3 = l_List_appendTR___rarg(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabModuleDoc___closed__3; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__14; +x_3 = l_List_foldl___at_String_join___spec__1(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__15; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__17() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" macOS", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___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_Command_elabVersion___rarg___lambda__1___closed__17; +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_Command_elabVersion___rarg___lambda__1___closed__19() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__18; +x_3 = l_List_appendTR___rarg(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__20() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__19; +x_3 = l_List_appendTR___rarg(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__21() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabModuleDoc___closed__3; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__20; +x_3 = l_List_foldl___at_String_join___spec__1(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__22() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__21; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__23() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__19; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__13; +x_3 = l_List_appendTR___rarg(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__24() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabModuleDoc___closed__3; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__23; +x_3 = l_List_foldl___at_String_join___spec__1(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__25() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__24; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__26() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" Windows", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__27() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__26; +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_Command_elabVersion___rarg___lambda__1___closed__28() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__27; +x_3 = l_List_appendTR___rarg(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__29() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__28; +x_3 = l_List_appendTR___rarg(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__30() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabModuleDoc___closed__3; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__29; +x_3 = l_List_foldl___at_String_join___spec__1(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__31() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__30; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__32() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__28; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__13; +x_3 = l_List_appendTR___rarg(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__33() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabModuleDoc___closed__3; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__32; +x_3 = l_List_foldl___at_String_join___spec__1(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__34() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__33; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__35() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__27; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__18; +x_3 = l_List_appendTR___rarg(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__36() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__35; +x_3 = l_List_appendTR___rarg(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__37() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabModuleDoc___closed__3; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__36; +x_3 = l_List_foldl___at_String_join___spec__1(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__38() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__37; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__39() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__35; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__13; +x_3 = l_List_appendTR___rarg(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__40() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_elabModuleDoc___closed__3; +x_2 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__39; +x_3 = l_List_foldl___at_String_join___spec__1(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__41() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__40; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion___rarg___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; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_6 = l_Lean_stringToMessageData(x_1); +x_7 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__7; +x_8 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_6); +x_9 = l_Lean_Elab_Command_elabModuleDoc___closed__4; +x_10 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_10, 0, x_8); +lean_ctor_set(x_10, 1, x_9); +x_11 = l_System_Platform_isWindows; +if (x_11 == 0) +{ +uint8_t x_12; +x_12 = l_System_Platform_isOSX; +if (x_12 == 0) +{ +uint8_t x_13; +x_13 = l_System_Platform_isEmscripten; +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; +x_14 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__11; +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_10); +lean_ctor_set(x_15, 1, x_14); +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 = 0; +x_18 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_16, x_17, x_3, x_4, x_5); +return x_18; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; +x_19 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__16; +x_20 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_20, 0, x_10); +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_9); +x_22 = 0; +x_23 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_21, x_22, x_3, x_4, x_5); +return x_23; +} +} +else +{ +uint8_t x_24; +x_24 = l_System_Platform_isEmscripten; +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; +x_25 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__22; +x_26 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_26, 0, x_10); +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_9); +x_28 = 0; +x_29 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_27, x_28, x_3, x_4, x_5); +return x_29; +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; +x_30 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__25; +x_31 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_31, 0, x_10); +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_9); +x_33 = 0; +x_34 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_32, x_33, x_3, x_4, x_5); +return x_34; +} +} +} +else { -lean_object* x_5; uint8_t x_6; -x_5 = l_Lean_Elab_Command_elabOmit___closed__2; -lean_inc(x_1); -x_6 = l_Lean_Syntax_isOfKind(x_1, x_5); -if (x_6 == 0) +uint8_t x_35; +x_35 = l_System_Platform_isOSX; +if (x_35 == 0) { -lean_object* x_7; -lean_dec(x_1); -x_7 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabNamespace___spec__1___rarg(x_4); -return x_7; +uint8_t x_36; +x_36 = l_System_Platform_isEmscripten; +if (x_36 == 0) +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; lean_object* x_41; +x_37 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__31; +x_38 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_38, 0, x_10); +lean_ctor_set(x_38, 1, x_37); +x_39 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_9); +x_40 = 0; +x_41 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_39, x_40, x_3, x_4, x_5); +return x_41; } 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; lean_object* x_14; lean_object* x_15; -x_8 = lean_unsigned_to_nat(1u); -x_9 = l_Lean_Syntax_getArg(x_1, x_8); -lean_dec(x_1); -x_10 = lean_box(0); -x_11 = l_Lean_Syntax_getArgs(x_9); -lean_dec(x_9); -x_12 = l_Lean_Elab_Command_elabSection___closed__4; -x_13 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__7___closed__2; -x_14 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabOmit___lambda__1___boxed), 12, 4); -lean_closure_set(x_14, 0, x_11); -lean_closure_set(x_14, 1, x_12); -lean_closure_set(x_14, 2, x_13); -lean_closure_set(x_14, 3, x_10); -x_15 = l_Lean_Elab_Command_runTermElabM___rarg(x_14, x_2, x_3, x_4); -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_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_alloc_closure((void*)(l_Lean_Elab_Command_elabOmit___lambda__2), 3, 2); -lean_closure_set(x_18, 0, x_16); -lean_closure_set(x_18, 1, x_10); -x_19 = l_Lean_Elab_Command_modifyScope(x_18, x_2, x_3, x_17); -return x_19; +lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; lean_object* x_46; +x_42 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__34; +x_43 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_43, 0, x_10); +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_9); +x_45 = 0; +x_46 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_44, x_45, x_3, x_4, x_5); +return x_46; +} } else { -uint8_t x_20; -x_20 = !lean_is_exclusive(x_15); -if (x_20 == 0) +uint8_t x_47; +x_47 = l_System_Platform_isEmscripten; +if (x_47 == 0) { -return x_15; +lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; +x_48 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__38; +x_49 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_49, 0, x_10); +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_9); +x_51 = 0; +x_52 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_50, x_51, x_3, x_4, x_5); +return x_52; } 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_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; +x_53 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__41; +x_54 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_54, 0, x_10); +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_9); +x_56 = 0; +x_57 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_55, x_56, x_3, x_4, x_5); +return x_57; } } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabOmit___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) { +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___closed__1() { _start: { -lean_object* x_7; -x_7 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabOmit___spec__1(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_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___boxed), 5, 0); +return x_1; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___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) { +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___closed__2() { _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_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___spec__3(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_3); -lean_dec(x_2); -lean_dec(x_1); -return x_16; +lean_object* x_1; lean_object* x_2; +x_1 = l_System_Platform_target; +x_2 = lean_string_utf8_byte_size(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static uint8_t _init_l_Lean_Elab_Command_elabVersion___rarg___closed__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_6 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabOmit___spec__4(x_4, x_5, x_3); -return x_6; +lean_object* x_1; lean_object* x_2; uint8_t x_3; +x_1 = l_Lean_Elab_Command_elabVersion___rarg___closed__2; +x_2 = lean_unsigned_to_nat(0u); +x_3 = lean_nat_dec_eq(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Elab_Command_elabOmit___spec__5___boxed(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_Elab_Command_elabVersion___rarg___closed__4() { _start: { -uint8_t x_3; lean_object* x_4; -x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Elab_Command_elabOmit___spec__5(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unknown", 7, 7); +return x_1; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Elab_Command_elabOmit___spec__10___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Elab_Command_elabOmit___spec__10(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -return x_3; -} +lean_object* x_4; uint8_t x_5; +x_4 = l_Lean_Elab_Command_elabVersion___rarg___closed__1; +x_5 = l_Lean_Elab_Command_elabVersion___rarg___closed__3; +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_6 = l_System_Platform_target; +x_7 = lean_box(0); +x_8 = lean_apply_5(x_4, x_6, x_7, x_1, x_2, x_3); +return x_8; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11___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_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11___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_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = l_Lean_Elab_Command_elabVersion___rarg___closed__4; +x_10 = lean_box(0); +x_11 = lean_apply_5(x_4, x_9, x_10, x_1, x_2, x_3); return x_11; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___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_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_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__11(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_1); -return x_16; -} } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___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_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion(lean_object* x_1) { _start: { -lean_object* x_10; -x_10 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__12___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_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabVersion___rarg), 3, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___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_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_Elab_Command_elabVersion___rarg___lambda__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_15; size_t x_16; size_t x_17; lean_object* x_18; -x_15 = lean_unbox_usize(x_1); -lean_dec(x_1); -x_16 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_17 = lean_unbox_usize(x_6); -lean_dec(x_6); -x_18 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__12(x_15, x_2, x_3, x_4, x_16, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -lean_dec(x_9); +lean_object* x_6; +x_6 = l_Lean_Elab_Command_elabVersion___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_2); -return x_18; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___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, 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_forInUnsafe_loop___at_Lean_Elab_Command_elabOmit___spec__13(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_1); -return x_14; -} -} -LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Elab_Command_elabOmit___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_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l_Lean_RBNode_forIn_visit___at_Lean_Elab_Command_elabOmit___spec__14(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); -return x_11; +return x_6; } } -LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Elab_Command_elabOmit___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabVersion___boxed(lean_object* x_1) { _start: { -lean_object* x_4; -x_4 = l_List_filterTR_loop___at_Lean_Elab_Command_elabOmit___spec__15(x_1, x_2, x_3); +lean_object* x_2; +x_2 = l_Lean_Elab_Command_elabVersion(x_1); lean_dec(x_1); -return x_4; +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOmit___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) { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__1() { _start: { -lean_object* x_13; -x_13 = l_Lean_Elab_Command_elabOmit___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_5); -lean_dec(x_3); -lean_dec(x_2); -return x_13; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("version", 7, 7); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabOmit___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__2() { _start: { -lean_object* x_5; -x_5 = l_Lean_Elab_Command_elabOmit(x_1, x_2, x_3, x_4); -lean_dec(x_3); -lean_dec(x_2); +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_Command_elabModuleDoc__1___closed__1; +x_2 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__2; +x_3 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__3; +x_4 = l___regBuiltin_Lean_Elab_Command_elabVersion__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___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("elabOmit", 8, 8); +x_1 = lean_mk_string_unchecked("elabVersion", 11, 11); return x_1; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___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_Command_elabModuleDoc__1___closed__1; x_2 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__6; x_3 = l___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__3; -x_4 = l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__1; +x_4 = l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__3; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__3() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabOmit___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabVersion___boxed), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabOmit__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabVersion__1(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___regBuiltin_Lean_Elab_Command_elabModuleDoc__1___closed__9; -x_3 = l_Lean_Elab_Command_elabOmit___closed__2; -x_4 = l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__2; -x_5 = l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__3; +x_3 = l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__2; +x_4 = l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__4; +x_5 = l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__5; x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } @@ -30226,6 +30989,7 @@ lean_object* initialize_Lean_Elab_Eval(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Elab_Command(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Elab_Open(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Elab_SetOption(uint8_t builtin, lean_object*); +lean_object* initialize_Init_System_Platform(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Elab_BuiltinCommand(uint8_t builtin, lean_object* w) { lean_object * res; @@ -30255,6 +31019,9 @@ lean_dec_ref(res); res = initialize_Lean_Elab_SetOption(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_System_Platform(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Elab_Command_elabModuleDoc___closed__1 = _init_l_Lean_Elab_Command_elabModuleDoc___closed__1(); lean_mark_persistent(l_Lean_Elab_Command_elabModuleDoc___closed__1); l_Lean_Elab_Command_elabModuleDoc___closed__2 = _init_l_Lean_Elab_Command_elabModuleDoc___closed__2(); @@ -31113,6 +31880,108 @@ lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_elabOmit__1___closed__3); if (builtin) {res = l___regBuiltin_Lean_Elab_Command_elabOmit__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +}l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__1 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__1); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__2 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__2); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__3 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__3); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__4 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__4); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__5 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__5); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__6 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__6); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__7 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__7); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__8 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__8); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__9 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__9); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__10 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__10); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__11 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__11(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__11); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__12 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__12(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__12); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__13 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__13(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__13); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__14 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__14(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__14); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__15 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__15(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__15); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__16 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__16(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__16); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__17 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__17(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__17); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__18 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__18(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__18); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__19 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__19(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__19); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__20 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__20(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__20); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__21 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__21(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__21); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__22 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__22(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__22); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__23 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__23(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__23); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__24 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__24(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__24); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__25 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__25(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__25); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__26 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__26(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__26); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__27 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__27(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__27); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__28 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__28(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__28); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__29 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__29(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__29); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__30 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__30(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__30); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__31 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__31(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__31); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__32 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__32(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__32); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__33 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__33(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__33); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__34 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__34(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__34); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__35 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__35(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__35); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__36 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__36(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__36); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__37 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__37(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__37); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__38 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__38(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__38); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__39 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__39(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__39); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__40 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__40(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__40); +l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__41 = _init_l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__41(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___lambda__1___closed__41); +l_Lean_Elab_Command_elabVersion___rarg___closed__1 = _init_l_Lean_Elab_Command_elabVersion___rarg___closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___closed__1); +l_Lean_Elab_Command_elabVersion___rarg___closed__2 = _init_l_Lean_Elab_Command_elabVersion___rarg___closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___closed__2); +l_Lean_Elab_Command_elabVersion___rarg___closed__3 = _init_l_Lean_Elab_Command_elabVersion___rarg___closed__3(); +l_Lean_Elab_Command_elabVersion___rarg___closed__4 = _init_l_Lean_Elab_Command_elabVersion___rarg___closed__4(); +lean_mark_persistent(l_Lean_Elab_Command_elabVersion___rarg___closed__4); +l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__1 = _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__1); +l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__2 = _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__2); +l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__3 = _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__3); +l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__4 = _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__4); +l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__5 = _init_l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__5(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_elabVersion__1___closed__5); +if (builtin) {res = l___regBuiltin_Lean_Elab_Command_elabVersion__1(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); }l_Lean_logWarning___at_Lean_Elab_Command_elabExit___spec__1___closed__1 = _init_l_Lean_logWarning___at_Lean_Elab_Command_elabExit___spec__1___closed__1(); lean_mark_persistent(l_Lean_logWarning___at_Lean_Elab_Command_elabExit___spec__1___closed__1); l_Lean_Elab_Command_elabExit___rarg___closed__1 = _init_l_Lean_Elab_Command_elabExit___rarg___closed__1(); diff --git a/stage0/stdlib/Lean/Elab/BuiltinEvalCommand.c b/stage0/stdlib/Lean/Elab/BuiltinEvalCommand.c index fc9cd3ce4e5d..e21468212948 100644 --- a/stage0/stdlib/Lean/Elab/BuiltinEvalCommand.c +++ b/stage0/stdlib/Lean/Elab/BuiltinEvalCommand.c @@ -2985,21 +2985,23 @@ return x_5; static lean_object* _init_l___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_addAndCompileExprForEval___closed__22() { _start: { -lean_object* x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; uint8_t x_6; lean_object* x_7; lean_object* x_8; x_1 = lean_box(0); -x_2 = 0; +x_2 = lean_box(0); x_3 = 0; -x_4 = 2; -x_5 = 1; -x_6 = l_Lean_collectAxioms___at___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_addAndCompileExprForEval___spec__1___closed__1; -x_7 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_7, 0, x_1); -lean_ctor_set(x_7, 1, x_6); -lean_ctor_set_uint8(x_7, sizeof(void*)*2, x_2); -lean_ctor_set_uint8(x_7, sizeof(void*)*2 + 1, x_3); -lean_ctor_set_uint8(x_7, sizeof(void*)*2 + 2, x_4); -lean_ctor_set_uint8(x_7, sizeof(void*)*2 + 3, x_5); -return x_7; +x_4 = 0; +x_5 = 2; +x_6 = 1; +x_7 = l_Lean_collectAxioms___at___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_addAndCompileExprForEval___spec__1___closed__1; +x_8 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_8, 0, x_2); +lean_ctor_set(x_8, 1, x_1); +lean_ctor_set(x_8, 2, x_7); +lean_ctor_set_uint8(x_8, sizeof(void*)*3, x_3); +lean_ctor_set_uint8(x_8, sizeof(void*)*3 + 1, x_4); +lean_ctor_set_uint8(x_8, sizeof(void*)*3 + 2, x_5); +lean_ctor_set_uint8(x_8, sizeof(void*)*3 + 3, x_6); +return x_8; } } static lean_object* _init_l___private_Lean_Elab_BuiltinEvalCommand_0__Lean_Elab_Command_addAndCompileExprForEval___closed__23() { diff --git a/stage0/stdlib/Lean/Elab/BuiltinNotation.c b/stage0/stdlib/Lean/Elab/BuiltinNotation.c index aaeb9122c31a..2854e2a845b5 100644 --- a/stage0/stdlib/Lean/Elab/BuiltinNotation.c +++ b/stage0/stdlib/Lean/Elab/BuiltinNotation.c @@ -422,6 +422,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Term_elabBorrowed_declRange__1___cl lean_object* l_Lean_Meta_withLetDecl___at_Lean_Elab_Term_elabLetDeclAux___spec__2___rarg(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_expr_eqv(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at_Lean_Elab_Term_elabAnonymousCtor___spec__4___rarg___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_elabSubst___lambda__6___closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabLeadingParserMacro___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_ResolveName_resolveNamespace(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_expandTuple_declRange__1___closed__5; @@ -503,6 +504,7 @@ static lean_object* l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__10; static lean_object* l___regBuiltin_Lean_Elab_Term_elabTrailingParserMacro_declRange__1___closed__3; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_expandCDot_x3f___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_expandCDot_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_elabSubst___lambda__6___closed__7; static lean_object* l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__2; static lean_object* l_Lean_Elab_Term_elabCDotFunctionAlias_x3f___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Term_elabShow__1___closed__1; @@ -652,6 +654,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Term_expandShow_declRange__1___clos static lean_object* l___regBuiltin_Lean_Elab_Term_elabHaveI_declRange__1___closed__1; static lean_object* l_Lean_Elab_Term_expandDbgTrace___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Term_elabRunElab_declRange__1___closed__5; +static lean_object* l_Lean_Elab_Term_elabSubst___lambda__6___closed__9; static lean_object* l_Lean_getConstInfoCtor___at_Lean_Elab_Term_elabAnonymousCtor___spec__1___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Term_expandUnreachable_declRange__1___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Term_elabSorry__1___closed__1; @@ -816,7 +819,6 @@ static lean_object* l_Lean_Elab_Term_expandAssert___closed__10; static lean_object* l_Lean_Elab_Term_elabStateRefT___lambda__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinNotation_0__Lean_Elab_Term_elabParserMacroAux(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_Lean_setImplementedBy___at_Lean_Elab_Term_elabUnsafe___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_Elab_Term_expandSuffices___closed__9; static lean_object* l___regBuiltin_Lean_Elab_Term_expandDbgTrace_declRange__1___closed__2; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_BuiltinNotation_0__Lean_Elab_Term_isSubstCandidate___spec__16(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabSubst___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*); @@ -918,7 +920,6 @@ static lean_object* l_Lean_Elab_Term_elabAnonymousCtor___closed__2; LEAN_EXPORT lean_object* l_Array_isEqvAux___at_Lean_Elab_Term_elabCDotFunctionAlias_x3f___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Term_elabCoeFunNotation_declRange__1___closed__5; -static lean_object* l_Lean_Elab_Term_expandSuffices___closed__8; 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_Elab_Term_expandAssert___closed__1; LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Elab_BuiltinNotation_0__Lean_Elab_Term_isSubstCandidate___spec__2___boxed(lean_object*, lean_object*, lean_object*); @@ -1091,6 +1092,7 @@ static lean_object* l_Lean_Elab_Term_elabStateRefT___lambda__1___closed__5; static lean_object* l_Lean_Elab_Term_expandHave___lambda__1___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_expandSuffices__1(lean_object*); extern lean_object* l_Lean_Compiler_implementedByAttr; +lean_object* l_Lean_Syntax_setKind(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_expandAssert___closed__6; static lean_object* l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; lean_object* lean_string_append(lean_object*, lean_object*); @@ -1153,7 +1155,6 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_expandShow__1(lean_object static lean_object* l___regBuiltin_Lean_Elab_Term_elabUnsafe_declRange__1___closed__6; static lean_object* l_Lean_Elab_Term_expandUnreachable___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_expandParen(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_expandSuffices___closed__7; static lean_object* l_Lean_Elab_Term_elabPanic___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_elabSubst__1(lean_object*); static lean_object* l_Lean_Elab_Term_elabLeadingParserMacro___lambda__1___closed__4; @@ -7878,34 +7879,6 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_expandSuffices___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Tactic", 6, 6); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Term_expandSuffices___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("tacticSeq", 9, 9); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Term_expandSuffices___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___regBuiltin_Lean_Elab_Term_elabCoe__1___closed__3; -x_2 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__8; -x_3 = l_Lean_Elab_Term_expandSuffices___closed__7; -x_4 = l_Lean_Elab_Term_expandSuffices___closed__8; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} LEAN_EXPORT lean_object* l_Lean_Elab_Term_expandSuffices(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -8003,577 +7976,481 @@ return x_31; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_32 = l_Lean_Syntax_getArg(x_25, x_8); -x_33 = l_Lean_Syntax_getArg(x_25, x_10); -lean_dec(x_25); -x_34 = l_Lean_Elab_Term_expandSuffices___closed__9; -lean_inc(x_33); -x_35 = l_Lean_Syntax_isOfKind(x_33, x_34); -if (x_35 == 0) -{ -lean_object* x_36; lean_object* x_37; -lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_23); -lean_dec(x_16); -lean_dec(x_9); -lean_dec(x_1); -x_36 = lean_box(1); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_3); -return x_37; -} -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t 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; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_38 = lean_unsigned_to_nat(3u); -x_39 = l_Lean_Syntax_getArg(x_1, x_38); +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; uint8_t 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; +x_32 = lean_unsigned_to_nat(3u); +x_33 = l_Lean_Syntax_getArg(x_1, x_32); lean_dec(x_1); -x_40 = lean_ctor_get(x_2, 5); -x_41 = 0; -x_42 = l_Lean_SourceInfo_fromRef(x_40, x_41); -x_43 = 1; -x_44 = l_Lean_SourceInfo_fromRef(x_9, x_43); +x_34 = l_Lean_Elab_Term_expandShow___closed__9; +x_35 = l_Lean_Syntax_setKind(x_25, x_34); +x_36 = lean_ctor_get(x_2, 5); +x_37 = 0; +x_38 = l_Lean_SourceInfo_fromRef(x_36, x_37); +x_39 = 1; +x_40 = l_Lean_SourceInfo_fromRef(x_9, x_39); lean_dec(x_9); -x_45 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; -x_46 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_46, 0, x_44); -lean_ctor_set(x_46, 1, x_45); -x_47 = l_Lean_Elab_Term_expandHave___closed__11; -lean_inc(x_42); -x_48 = l_Lean_Syntax_node1(x_42, x_47, x_16); -x_49 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; -x_50 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; -lean_inc(x_42); -x_51 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_51, 0, x_42); -lean_ctor_set(x_51, 1, x_49); -lean_ctor_set(x_51, 2, x_50); -x_52 = l_Lean_Elab_Term_elabShow___closed__11; -lean_inc(x_42); -x_53 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_53, 0, x_42); -lean_ctor_set(x_53, 1, x_52); -x_54 = l_Lean_Elab_Term_elabShow___closed__10; -lean_inc(x_42); -x_55 = l_Lean_Syntax_node2(x_42, x_54, x_53, x_23); -lean_inc(x_42); -x_56 = l_Lean_Syntax_node1(x_42, x_49, x_55); -x_57 = l_Lean_Elab_Term_elabShow___closed__12; -lean_inc(x_42); -x_58 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_58, 0, x_42); -lean_ctor_set(x_58, 1, x_57); -x_59 = l_Lean_Elab_Term_expandHave___closed__5; -lean_inc(x_42); -x_60 = l_Lean_Syntax_node5(x_42, x_59, x_48, x_51, x_56, x_58, x_39); -x_61 = l_Lean_Elab_Term_expandHave___closed__3; -lean_inc(x_42); -x_62 = l_Lean_Syntax_node1(x_42, x_61, x_60); -x_63 = l_Lean_Elab_Term_elabShow___closed__13; -lean_inc(x_42); -x_64 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_64, 0, x_42); -lean_ctor_set(x_64, 1, x_63); -x_65 = l_Lean_SourceInfo_fromRef(x_32, x_43); -lean_dec(x_32); -x_66 = l_Lean_Elab_Term_expandShow___closed__10; -x_67 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_67, 0, x_65); -lean_ctor_set(x_67, 1, x_66); -x_68 = l_Lean_Elab_Term_expandShow___closed__9; -lean_inc(x_42); -x_69 = l_Lean_Syntax_node2(x_42, x_68, x_67, x_33); -x_70 = l_Lean_Elab_Term_expandHave___closed__1; -x_71 = l_Lean_Syntax_node4(x_42, x_70, x_46, x_62, x_64, x_69); -x_72 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_72, 0, x_71); -lean_ctor_set(x_72, 1, x_3); -return x_72; -} +x_41 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; +x_42 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +x_43 = l_Lean_Elab_Term_expandHave___closed__11; +lean_inc(x_38); +x_44 = l_Lean_Syntax_node1(x_38, x_43, x_16); +x_45 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; +x_46 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; +lean_inc(x_38); +x_47 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_47, 0, x_38); +lean_ctor_set(x_47, 1, x_45); +lean_ctor_set(x_47, 2, x_46); +x_48 = l_Lean_Elab_Term_elabShow___closed__11; +lean_inc(x_38); +x_49 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_49, 0, x_38); +lean_ctor_set(x_49, 1, x_48); +x_50 = l_Lean_Elab_Term_elabShow___closed__10; +lean_inc(x_38); +x_51 = l_Lean_Syntax_node2(x_38, x_50, x_49, x_23); +lean_inc(x_38); +x_52 = l_Lean_Syntax_node1(x_38, x_45, x_51); +x_53 = l_Lean_Elab_Term_elabShow___closed__12; +lean_inc(x_38); +x_54 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_54, 0, x_38); +lean_ctor_set(x_54, 1, x_53); +x_55 = l_Lean_Elab_Term_expandHave___closed__5; +lean_inc(x_38); +x_56 = l_Lean_Syntax_node5(x_38, x_55, x_44, x_47, x_52, x_54, x_33); +x_57 = l_Lean_Elab_Term_expandHave___closed__3; +lean_inc(x_38); +x_58 = l_Lean_Syntax_node1(x_38, x_57, x_56); +x_59 = l_Lean_Elab_Term_elabShow___closed__13; +lean_inc(x_38); +x_60 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_60, 0, x_38); +lean_ctor_set(x_60, 1, x_59); +x_61 = l_Lean_Elab_Term_expandHave___closed__1; +x_62 = l_Lean_Syntax_node4(x_38, x_61, x_42, x_58, x_60, x_35); +x_63 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_63, 0, x_62); +lean_ctor_set(x_63, 1, x_3); +return x_63; } } else { -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; 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; -x_73 = l_Lean_Syntax_getArg(x_25, x_10); +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t 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; 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_64 = l_Lean_Syntax_getArg(x_25, x_10); lean_dec(x_25); -x_74 = lean_unsigned_to_nat(3u); -x_75 = l_Lean_Syntax_getArg(x_1, x_74); -lean_dec(x_1); -x_76 = lean_ctor_get(x_2, 5); -x_77 = 0; -x_78 = l_Lean_SourceInfo_fromRef(x_76, x_77); -x_79 = 1; -x_80 = l_Lean_SourceInfo_fromRef(x_9, x_79); +x_65 = lean_unsigned_to_nat(3u); +x_66 = l_Lean_Syntax_getArg(x_1, x_65); +lean_dec(x_1); +x_67 = lean_ctor_get(x_2, 5); +x_68 = 0; +x_69 = l_Lean_SourceInfo_fromRef(x_67, x_68); +x_70 = 1; +x_71 = l_Lean_SourceInfo_fromRef(x_9, x_70); lean_dec(x_9); -x_81 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; -x_82 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_82, 0, x_80); -lean_ctor_set(x_82, 1, x_81); -x_83 = l_Lean_Elab_Term_expandHave___closed__11; -lean_inc(x_78); -x_84 = l_Lean_Syntax_node1(x_78, x_83, x_16); -x_85 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; -x_86 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; -lean_inc(x_78); -x_87 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_87, 0, x_78); -lean_ctor_set(x_87, 1, x_85); -lean_ctor_set(x_87, 2, x_86); -x_88 = l_Lean_Elab_Term_elabShow___closed__11; -lean_inc(x_78); -x_89 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_89, 0, x_78); -lean_ctor_set(x_89, 1, x_88); -x_90 = l_Lean_Elab_Term_elabShow___closed__10; -lean_inc(x_78); -x_91 = l_Lean_Syntax_node2(x_78, x_90, x_89, x_23); -lean_inc(x_78); -x_92 = l_Lean_Syntax_node1(x_78, x_85, x_91); -x_93 = l_Lean_Elab_Term_elabShow___closed__12; -lean_inc(x_78); -x_94 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_94, 0, x_78); -lean_ctor_set(x_94, 1, x_93); -x_95 = l_Lean_Elab_Term_expandHave___closed__5; -lean_inc(x_78); -x_96 = l_Lean_Syntax_node5(x_78, x_95, x_84, x_87, x_92, x_94, x_75); -x_97 = l_Lean_Elab_Term_expandHave___closed__3; -lean_inc(x_78); -x_98 = l_Lean_Syntax_node1(x_78, x_97, x_96); -x_99 = l_Lean_Elab_Term_elabShow___closed__13; -lean_inc(x_78); -x_100 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_100, 0, x_78); -lean_ctor_set(x_100, 1, x_99); -x_101 = l_Lean_Elab_Term_expandHave___closed__1; -x_102 = l_Lean_Syntax_node4(x_78, x_101, x_82, x_98, x_100, x_73); -x_103 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_103, 0, x_102); -lean_ctor_set(x_103, 1, x_3); -return x_103; +x_72 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; +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 = l_Lean_Elab_Term_expandHave___closed__11; +lean_inc(x_69); +x_75 = l_Lean_Syntax_node1(x_69, x_74, x_16); +x_76 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; +x_77 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; +lean_inc(x_69); +x_78 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_78, 0, x_69); +lean_ctor_set(x_78, 1, x_76); +lean_ctor_set(x_78, 2, x_77); +x_79 = l_Lean_Elab_Term_elabShow___closed__11; +lean_inc(x_69); +x_80 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_80, 0, x_69); +lean_ctor_set(x_80, 1, x_79); +x_81 = l_Lean_Elab_Term_elabShow___closed__10; +lean_inc(x_69); +x_82 = l_Lean_Syntax_node2(x_69, x_81, x_80, x_23); +lean_inc(x_69); +x_83 = l_Lean_Syntax_node1(x_69, x_76, x_82); +x_84 = l_Lean_Elab_Term_elabShow___closed__12; +lean_inc(x_69); +x_85 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_85, 0, x_69); +lean_ctor_set(x_85, 1, x_84); +x_86 = l_Lean_Elab_Term_expandHave___closed__5; +lean_inc(x_69); +x_87 = l_Lean_Syntax_node5(x_69, x_86, x_75, x_78, x_83, x_85, x_66); +x_88 = l_Lean_Elab_Term_expandHave___closed__3; +lean_inc(x_69); +x_89 = l_Lean_Syntax_node1(x_69, x_88, x_87); +x_90 = l_Lean_Elab_Term_elabShow___closed__13; +lean_inc(x_69); +x_91 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_91, 0, x_69); +lean_ctor_set(x_91, 1, x_90); +x_92 = l_Lean_Elab_Term_expandHave___closed__1; +x_93 = l_Lean_Syntax_node4(x_69, x_92, x_73, x_89, x_91, x_64); +x_94 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_93); +lean_ctor_set(x_94, 1, x_3); +return x_94; } } } else { -lean_object* x_104; lean_object* x_105; uint8_t x_106; -x_104 = l_Lean_Syntax_getArg(x_16, x_8); +lean_object* x_95; lean_object* x_96; uint8_t x_97; +x_95 = l_Lean_Syntax_getArg(x_16, x_8); lean_dec(x_16); -x_105 = l_Lean_Elab_Term_expandHave___closed__15; -lean_inc(x_104); -x_106 = l_Lean_Syntax_isOfKind(x_104, x_105); -if (x_106 == 0) +x_96 = l_Lean_Elab_Term_expandHave___closed__15; +lean_inc(x_95); +x_97 = l_Lean_Syntax_isOfKind(x_95, x_96); +if (x_97 == 0) { -lean_object* x_107; uint8_t x_108; -x_107 = l_Lean_Elab_Term_expandHave___closed__17; -lean_inc(x_104); -x_108 = l_Lean_Syntax_isOfKind(x_104, x_107); -if (x_108 == 0) +lean_object* x_98; uint8_t x_99; +x_98 = l_Lean_Elab_Term_expandHave___closed__17; +lean_inc(x_95); +x_99 = l_Lean_Syntax_isOfKind(x_95, x_98); +if (x_99 == 0) { -lean_object* x_109; lean_object* x_110; -lean_dec(x_104); +lean_object* x_100; lean_object* x_101; +lean_dec(x_95); lean_dec(x_11); lean_dec(x_9); lean_dec(x_1); -x_109 = lean_box(1); -x_110 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_110, 0, x_109); -lean_ctor_set(x_110, 1, x_3); -return x_110; +x_100 = lean_box(1); +x_101 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_101, 0, x_100); +lean_ctor_set(x_101, 1, x_3); +return x_101; } else { -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_111 = l_Lean_Syntax_getArg(x_104, x_8); -lean_dec(x_104); -x_112 = l_Lean_Syntax_getArg(x_11, x_10); -x_113 = lean_unsigned_to_nat(2u); -x_114 = l_Lean_Syntax_getArg(x_11, x_113); +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_102 = l_Lean_Syntax_getArg(x_95, x_8); +lean_dec(x_95); +x_103 = l_Lean_Syntax_getArg(x_11, x_10); +x_104 = lean_unsigned_to_nat(2u); +x_105 = l_Lean_Syntax_getArg(x_11, x_104); lean_dec(x_11); -x_115 = l_Lean_Elab_Term_expandShow___closed__6; -lean_inc(x_114); -x_116 = l_Lean_Syntax_isOfKind(x_114, x_115); -if (x_116 == 0) +x_106 = l_Lean_Elab_Term_expandShow___closed__6; +lean_inc(x_105); +x_107 = l_Lean_Syntax_isOfKind(x_105, x_106); +if (x_107 == 0) { -lean_object* x_117; uint8_t x_118; -x_117 = l_Lean_Elab_Term_expandShow___closed__4; -lean_inc(x_114); -x_118 = l_Lean_Syntax_isOfKind(x_114, x_117); -if (x_118 == 0) +lean_object* x_108; uint8_t x_109; +x_108 = l_Lean_Elab_Term_expandShow___closed__4; +lean_inc(x_105); +x_109 = l_Lean_Syntax_isOfKind(x_105, x_108); +if (x_109 == 0) { -lean_object* x_119; lean_object* x_120; -lean_dec(x_114); -lean_dec(x_112); -lean_dec(x_111); +lean_object* x_110; lean_object* x_111; +lean_dec(x_105); +lean_dec(x_103); +lean_dec(x_102); lean_dec(x_9); lean_dec(x_1); -x_119 = lean_box(1); -x_120 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_120, 0, x_119); -lean_ctor_set(x_120, 1, x_3); -return x_120; +x_110 = lean_box(1); +x_111 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_111, 0, x_110); +lean_ctor_set(x_111, 1, x_3); +return x_111; } else { -lean_object* x_121; lean_object* x_122; lean_object* x_123; uint8_t x_124; -x_121 = l_Lean_Syntax_getArg(x_114, x_8); -x_122 = l_Lean_Syntax_getArg(x_114, x_10); -lean_dec(x_114); -x_123 = l_Lean_Elab_Term_expandSuffices___closed__9; -lean_inc(x_122); -x_124 = l_Lean_Syntax_isOfKind(x_122, x_123); -if (x_124 == 0) -{ -lean_object* x_125; lean_object* x_126; -lean_dec(x_122); -lean_dec(x_121); -lean_dec(x_112); -lean_dec(x_111); -lean_dec(x_9); +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; uint8_t x_117; lean_object* x_118; uint8_t 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; +x_112 = lean_unsigned_to_nat(3u); +x_113 = l_Lean_Syntax_getArg(x_1, x_112); lean_dec(x_1); -x_125 = lean_box(1); -x_126 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_126, 0, x_125); -lean_ctor_set(x_126, 1, x_3); -return x_126; +x_114 = l_Lean_Elab_Term_expandShow___closed__9; +x_115 = l_Lean_Syntax_setKind(x_105, x_114); +x_116 = lean_ctor_get(x_2, 5); +x_117 = 0; +x_118 = l_Lean_SourceInfo_fromRef(x_116, x_117); +x_119 = 1; +x_120 = l_Lean_SourceInfo_fromRef(x_9, x_119); +lean_dec(x_9); +x_121 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; +x_122 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_122, 0, x_120); +lean_ctor_set(x_122, 1, x_121); +x_123 = l_Lean_SourceInfo_fromRef(x_102, x_119); +lean_dec(x_102); +x_124 = l_Lean_Elab_Term_expandHave___lambda__2___closed__3; +x_125 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_125, 0, x_123); +lean_ctor_set(x_125, 1, x_124); +lean_inc(x_118); +x_126 = l_Lean_Syntax_node1(x_118, x_98, x_125); +x_127 = l_Lean_Elab_Term_expandHave___closed__11; +lean_inc(x_118); +x_128 = l_Lean_Syntax_node1(x_118, x_127, x_126); +x_129 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; +x_130 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; +lean_inc(x_118); +x_131 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_131, 0, x_118); +lean_ctor_set(x_131, 1, x_129); +lean_ctor_set(x_131, 2, x_130); +x_132 = l_Lean_Elab_Term_elabShow___closed__11; +lean_inc(x_118); +x_133 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_133, 0, x_118); +lean_ctor_set(x_133, 1, x_132); +x_134 = l_Lean_Elab_Term_elabShow___closed__10; +lean_inc(x_118); +x_135 = l_Lean_Syntax_node2(x_118, x_134, x_133, x_103); +lean_inc(x_118); +x_136 = l_Lean_Syntax_node1(x_118, x_129, x_135); +x_137 = l_Lean_Elab_Term_elabShow___closed__12; +lean_inc(x_118); +x_138 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_138, 0, x_118); +lean_ctor_set(x_138, 1, x_137); +x_139 = l_Lean_Elab_Term_expandHave___closed__5; +lean_inc(x_118); +x_140 = l_Lean_Syntax_node5(x_118, x_139, x_128, x_131, x_136, x_138, x_113); +x_141 = l_Lean_Elab_Term_expandHave___closed__3; +lean_inc(x_118); +x_142 = l_Lean_Syntax_node1(x_118, x_141, x_140); +x_143 = l_Lean_Elab_Term_elabShow___closed__13; +lean_inc(x_118); +x_144 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_144, 0, x_118); +lean_ctor_set(x_144, 1, x_143); +x_145 = l_Lean_Elab_Term_expandHave___closed__1; +x_146 = l_Lean_Syntax_node4(x_118, x_145, x_122, x_142, x_144, x_115); +x_147 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_147, 0, x_146); +lean_ctor_set(x_147, 1, x_3); +return x_147; +} } else { -lean_object* x_127; lean_object* x_128; lean_object* x_129; uint8_t x_130; lean_object* x_131; uint8_t 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; -x_127 = lean_unsigned_to_nat(3u); -x_128 = l_Lean_Syntax_getArg(x_1, x_127); -lean_dec(x_1); -x_129 = lean_ctor_get(x_2, 5); -x_130 = 0; -x_131 = l_Lean_SourceInfo_fromRef(x_129, x_130); -x_132 = 1; -x_133 = l_Lean_SourceInfo_fromRef(x_9, x_132); +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; uint8_t 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; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; +x_148 = l_Lean_Syntax_getArg(x_105, x_10); +lean_dec(x_105); +x_149 = lean_unsigned_to_nat(3u); +x_150 = l_Lean_Syntax_getArg(x_1, x_149); +lean_dec(x_1); +x_151 = lean_ctor_get(x_2, 5); +x_152 = 0; +x_153 = l_Lean_SourceInfo_fromRef(x_151, x_152); +x_154 = 1; +x_155 = l_Lean_SourceInfo_fromRef(x_9, x_154); lean_dec(x_9); -x_134 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; -x_135 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_135, 0, x_133); -lean_ctor_set(x_135, 1, x_134); -x_136 = l_Lean_SourceInfo_fromRef(x_111, x_132); -lean_dec(x_111); -x_137 = l_Lean_Elab_Term_expandHave___lambda__2___closed__3; -x_138 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_138, 0, x_136); -lean_ctor_set(x_138, 1, x_137); -lean_inc(x_131); -x_139 = l_Lean_Syntax_node1(x_131, x_107, x_138); -x_140 = l_Lean_Elab_Term_expandHave___closed__11; -lean_inc(x_131); -x_141 = l_Lean_Syntax_node1(x_131, x_140, x_139); -x_142 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; -x_143 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; -lean_inc(x_131); -x_144 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_144, 0, x_131); -lean_ctor_set(x_144, 1, x_142); -lean_ctor_set(x_144, 2, x_143); -x_145 = l_Lean_Elab_Term_elabShow___closed__11; -lean_inc(x_131); -x_146 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_146, 0, x_131); -lean_ctor_set(x_146, 1, x_145); -x_147 = l_Lean_Elab_Term_elabShow___closed__10; -lean_inc(x_131); -x_148 = l_Lean_Syntax_node2(x_131, x_147, x_146, x_112); -lean_inc(x_131); -x_149 = l_Lean_Syntax_node1(x_131, x_142, x_148); -x_150 = l_Lean_Elab_Term_elabShow___closed__12; -lean_inc(x_131); -x_151 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_151, 0, x_131); -lean_ctor_set(x_151, 1, x_150); -x_152 = l_Lean_Elab_Term_expandHave___closed__5; -lean_inc(x_131); -x_153 = l_Lean_Syntax_node5(x_131, x_152, x_141, x_144, x_149, x_151, x_128); -x_154 = l_Lean_Elab_Term_expandHave___closed__3; -lean_inc(x_131); -x_155 = l_Lean_Syntax_node1(x_131, x_154, x_153); -x_156 = l_Lean_Elab_Term_elabShow___closed__13; -lean_inc(x_131); +x_156 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; x_157 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_157, 0, x_131); +lean_ctor_set(x_157, 0, x_155); lean_ctor_set(x_157, 1, x_156); -x_158 = l_Lean_SourceInfo_fromRef(x_121, x_132); -lean_dec(x_121); -x_159 = l_Lean_Elab_Term_expandShow___closed__10; +x_158 = l_Lean_SourceInfo_fromRef(x_102, x_154); +lean_dec(x_102); +x_159 = l_Lean_Elab_Term_expandHave___lambda__2___closed__3; x_160 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_160, 0, x_158); lean_ctor_set(x_160, 1, x_159); -x_161 = l_Lean_Elab_Term_expandShow___closed__9; -lean_inc(x_131); -x_162 = l_Lean_Syntax_node2(x_131, x_161, x_160, x_122); -x_163 = l_Lean_Elab_Term_expandHave___closed__1; -x_164 = l_Lean_Syntax_node4(x_131, x_163, x_135, x_155, x_157, x_162); -x_165 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_165, 0, x_164); -lean_ctor_set(x_165, 1, x_3); -return x_165; -} -} -} -else -{ -lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; uint8_t x_170; lean_object* x_171; uint8_t 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; -x_166 = l_Lean_Syntax_getArg(x_114, x_10); -lean_dec(x_114); -x_167 = lean_unsigned_to_nat(3u); -x_168 = l_Lean_Syntax_getArg(x_1, x_167); -lean_dec(x_1); -x_169 = lean_ctor_get(x_2, 5); -x_170 = 0; -x_171 = l_Lean_SourceInfo_fromRef(x_169, x_170); -x_172 = 1; -x_173 = l_Lean_SourceInfo_fromRef(x_9, x_172); -lean_dec(x_9); -x_174 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; -x_175 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_175, 0, x_173); -lean_ctor_set(x_175, 1, x_174); -x_176 = l_Lean_SourceInfo_fromRef(x_111, x_172); -lean_dec(x_111); -x_177 = l_Lean_Elab_Term_expandHave___lambda__2___closed__3; -x_178 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_178, 0, x_176); -lean_ctor_set(x_178, 1, x_177); -lean_inc(x_171); -x_179 = l_Lean_Syntax_node1(x_171, x_107, x_178); -x_180 = l_Lean_Elab_Term_expandHave___closed__11; -lean_inc(x_171); -x_181 = l_Lean_Syntax_node1(x_171, x_180, x_179); -x_182 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; -x_183 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; -lean_inc(x_171); -x_184 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_184, 0, x_171); -lean_ctor_set(x_184, 1, x_182); -lean_ctor_set(x_184, 2, x_183); -x_185 = l_Lean_Elab_Term_elabShow___closed__11; -lean_inc(x_171); -x_186 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_186, 0, x_171); -lean_ctor_set(x_186, 1, x_185); -x_187 = l_Lean_Elab_Term_elabShow___closed__10; -lean_inc(x_171); -x_188 = l_Lean_Syntax_node2(x_171, x_187, x_186, x_112); -lean_inc(x_171); -x_189 = l_Lean_Syntax_node1(x_171, x_182, x_188); -x_190 = l_Lean_Elab_Term_elabShow___closed__12; -lean_inc(x_171); -x_191 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_191, 0, x_171); -lean_ctor_set(x_191, 1, x_190); -x_192 = l_Lean_Elab_Term_expandHave___closed__5; -lean_inc(x_171); -x_193 = l_Lean_Syntax_node5(x_171, x_192, x_181, x_184, x_189, x_191, x_168); -x_194 = l_Lean_Elab_Term_expandHave___closed__3; -lean_inc(x_171); -x_195 = l_Lean_Syntax_node1(x_171, x_194, x_193); -x_196 = l_Lean_Elab_Term_elabShow___closed__13; -lean_inc(x_171); -x_197 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_197, 0, x_171); -lean_ctor_set(x_197, 1, x_196); -x_198 = l_Lean_Elab_Term_expandHave___closed__1; -x_199 = l_Lean_Syntax_node4(x_171, x_198, x_175, x_195, x_197, x_166); -x_200 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_200, 0, x_199); -lean_ctor_set(x_200, 1, x_3); -return x_200; +lean_inc(x_153); +x_161 = l_Lean_Syntax_node1(x_153, x_98, x_160); +x_162 = l_Lean_Elab_Term_expandHave___closed__11; +lean_inc(x_153); +x_163 = l_Lean_Syntax_node1(x_153, x_162, x_161); +x_164 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; +x_165 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; +lean_inc(x_153); +x_166 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_166, 0, x_153); +lean_ctor_set(x_166, 1, x_164); +lean_ctor_set(x_166, 2, x_165); +x_167 = l_Lean_Elab_Term_elabShow___closed__11; +lean_inc(x_153); +x_168 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_168, 0, x_153); +lean_ctor_set(x_168, 1, x_167); +x_169 = l_Lean_Elab_Term_elabShow___closed__10; +lean_inc(x_153); +x_170 = l_Lean_Syntax_node2(x_153, x_169, x_168, x_103); +lean_inc(x_153); +x_171 = l_Lean_Syntax_node1(x_153, x_164, x_170); +x_172 = l_Lean_Elab_Term_elabShow___closed__12; +lean_inc(x_153); +x_173 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_173, 0, x_153); +lean_ctor_set(x_173, 1, x_172); +x_174 = l_Lean_Elab_Term_expandHave___closed__5; +lean_inc(x_153); +x_175 = l_Lean_Syntax_node5(x_153, x_174, x_163, x_166, x_171, x_173, x_150); +x_176 = l_Lean_Elab_Term_expandHave___closed__3; +lean_inc(x_153); +x_177 = l_Lean_Syntax_node1(x_153, x_176, x_175); +x_178 = l_Lean_Elab_Term_elabShow___closed__13; +lean_inc(x_153); +x_179 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_179, 0, x_153); +lean_ctor_set(x_179, 1, x_178); +x_180 = l_Lean_Elab_Term_expandHave___closed__1; +x_181 = l_Lean_Syntax_node4(x_153, x_180, x_157, x_177, x_179, x_148); +x_182 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_182, 0, x_181); +lean_ctor_set(x_182, 1, x_3); +return x_182; } } } else { -lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; uint8_t x_205; -x_201 = l_Lean_Syntax_getArg(x_11, x_10); -x_202 = lean_unsigned_to_nat(2u); -x_203 = l_Lean_Syntax_getArg(x_11, x_202); +lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; uint8_t x_187; +x_183 = l_Lean_Syntax_getArg(x_11, x_10); +x_184 = lean_unsigned_to_nat(2u); +x_185 = l_Lean_Syntax_getArg(x_11, x_184); lean_dec(x_11); -x_204 = l_Lean_Elab_Term_expandShow___closed__6; -lean_inc(x_203); -x_205 = l_Lean_Syntax_isOfKind(x_203, x_204); -if (x_205 == 0) -{ -lean_object* x_206; uint8_t x_207; -x_206 = l_Lean_Elab_Term_expandShow___closed__4; -lean_inc(x_203); -x_207 = l_Lean_Syntax_isOfKind(x_203, x_206); -if (x_207 == 0) -{ -lean_object* x_208; lean_object* x_209; -lean_dec(x_203); -lean_dec(x_201); -lean_dec(x_104); -lean_dec(x_9); -lean_dec(x_1); -x_208 = lean_box(1); -x_209 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_209, 0, x_208); -lean_ctor_set(x_209, 1, x_3); -return x_209; -} -else -{ -lean_object* x_210; lean_object* x_211; lean_object* x_212; uint8_t x_213; -x_210 = l_Lean_Syntax_getArg(x_203, x_8); -x_211 = l_Lean_Syntax_getArg(x_203, x_10); -lean_dec(x_203); -x_212 = l_Lean_Elab_Term_expandSuffices___closed__9; -lean_inc(x_211); -x_213 = l_Lean_Syntax_isOfKind(x_211, x_212); -if (x_213 == 0) +x_186 = l_Lean_Elab_Term_expandShow___closed__6; +lean_inc(x_185); +x_187 = l_Lean_Syntax_isOfKind(x_185, x_186); +if (x_187 == 0) +{ +lean_object* x_188; uint8_t x_189; +x_188 = l_Lean_Elab_Term_expandShow___closed__4; +lean_inc(x_185); +x_189 = l_Lean_Syntax_isOfKind(x_185, x_188); +if (x_189 == 0) { -lean_object* x_214; lean_object* x_215; -lean_dec(x_211); -lean_dec(x_210); -lean_dec(x_201); -lean_dec(x_104); +lean_object* x_190; lean_object* x_191; +lean_dec(x_185); +lean_dec(x_183); +lean_dec(x_95); lean_dec(x_9); lean_dec(x_1); -x_214 = lean_box(1); -x_215 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_215, 0, x_214); -lean_ctor_set(x_215, 1, x_3); -return x_215; +x_190 = lean_box(1); +x_191 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_191, 0, x_190); +lean_ctor_set(x_191, 1, x_3); +return x_191; } else { -lean_object* x_216; lean_object* x_217; lean_object* x_218; uint8_t x_219; lean_object* x_220; uint8_t 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; -x_216 = lean_unsigned_to_nat(3u); -x_217 = l_Lean_Syntax_getArg(x_1, x_216); +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; uint8_t 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_222; lean_object* x_223; +x_192 = lean_unsigned_to_nat(3u); +x_193 = l_Lean_Syntax_getArg(x_1, x_192); lean_dec(x_1); -x_218 = lean_ctor_get(x_2, 5); -x_219 = 0; -x_220 = l_Lean_SourceInfo_fromRef(x_218, x_219); -x_221 = 1; -x_222 = l_Lean_SourceInfo_fromRef(x_9, x_221); +x_194 = l_Lean_Elab_Term_expandShow___closed__9; +x_195 = l_Lean_Syntax_setKind(x_185, x_194); +x_196 = lean_ctor_get(x_2, 5); +x_197 = 0; +x_198 = l_Lean_SourceInfo_fromRef(x_196, x_197); +x_199 = 1; +x_200 = l_Lean_SourceInfo_fromRef(x_9, x_199); lean_dec(x_9); -x_223 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; -x_224 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_224, 0, x_222); -lean_ctor_set(x_224, 1, x_223); -x_225 = l_Lean_Elab_Term_expandHave___closed__11; -lean_inc(x_220); -x_226 = l_Lean_Syntax_node1(x_220, x_225, x_104); -x_227 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; -x_228 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; -lean_inc(x_220); -x_229 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_229, 0, x_220); -lean_ctor_set(x_229, 1, x_227); -lean_ctor_set(x_229, 2, x_228); -x_230 = l_Lean_Elab_Term_elabShow___closed__11; -lean_inc(x_220); -x_231 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_231, 0, x_220); -lean_ctor_set(x_231, 1, x_230); -x_232 = l_Lean_Elab_Term_elabShow___closed__10; -lean_inc(x_220); -x_233 = l_Lean_Syntax_node2(x_220, x_232, x_231, x_201); -lean_inc(x_220); -x_234 = l_Lean_Syntax_node1(x_220, x_227, x_233); -x_235 = l_Lean_Elab_Term_elabShow___closed__12; -lean_inc(x_220); -x_236 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_236, 0, x_220); -lean_ctor_set(x_236, 1, x_235); -x_237 = l_Lean_Elab_Term_expandHave___closed__5; -lean_inc(x_220); -x_238 = l_Lean_Syntax_node5(x_220, x_237, x_226, x_229, x_234, x_236, x_217); -x_239 = l_Lean_Elab_Term_expandHave___closed__3; -lean_inc(x_220); -x_240 = l_Lean_Syntax_node1(x_220, x_239, x_238); -x_241 = l_Lean_Elab_Term_elabShow___closed__13; -lean_inc(x_220); -x_242 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_242, 0, x_220); -lean_ctor_set(x_242, 1, x_241); -x_243 = l_Lean_SourceInfo_fromRef(x_210, x_221); -lean_dec(x_210); -x_244 = l_Lean_Elab_Term_expandShow___closed__10; +x_201 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; +x_202 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_202, 0, x_200); +lean_ctor_set(x_202, 1, x_201); +x_203 = l_Lean_Elab_Term_expandHave___closed__11; +lean_inc(x_198); +x_204 = l_Lean_Syntax_node1(x_198, x_203, x_95); +x_205 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; +x_206 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; +lean_inc(x_198); +x_207 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_207, 0, x_198); +lean_ctor_set(x_207, 1, x_205); +lean_ctor_set(x_207, 2, x_206); +x_208 = l_Lean_Elab_Term_elabShow___closed__11; +lean_inc(x_198); +x_209 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_209, 0, x_198); +lean_ctor_set(x_209, 1, x_208); +x_210 = l_Lean_Elab_Term_elabShow___closed__10; +lean_inc(x_198); +x_211 = l_Lean_Syntax_node2(x_198, x_210, x_209, x_183); +lean_inc(x_198); +x_212 = l_Lean_Syntax_node1(x_198, x_205, x_211); +x_213 = l_Lean_Elab_Term_elabShow___closed__12; +lean_inc(x_198); +x_214 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_214, 0, x_198); +lean_ctor_set(x_214, 1, x_213); +x_215 = l_Lean_Elab_Term_expandHave___closed__5; +lean_inc(x_198); +x_216 = l_Lean_Syntax_node5(x_198, x_215, x_204, x_207, x_212, x_214, x_193); +x_217 = l_Lean_Elab_Term_expandHave___closed__3; +lean_inc(x_198); +x_218 = l_Lean_Syntax_node1(x_198, x_217, x_216); +x_219 = l_Lean_Elab_Term_elabShow___closed__13; +lean_inc(x_198); +x_220 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_220, 0, x_198); +lean_ctor_set(x_220, 1, x_219); +x_221 = l_Lean_Elab_Term_expandHave___closed__1; +x_222 = l_Lean_Syntax_node4(x_198, x_221, x_202, x_218, x_220, x_195); +x_223 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_223, 0, x_222); +lean_ctor_set(x_223, 1, x_3); +return x_223; +} +} +else +{ +lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; uint8_t x_228; lean_object* x_229; uint8_t 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; +x_224 = l_Lean_Syntax_getArg(x_185, x_10); +lean_dec(x_185); +x_225 = lean_unsigned_to_nat(3u); +x_226 = l_Lean_Syntax_getArg(x_1, x_225); +lean_dec(x_1); +x_227 = lean_ctor_get(x_2, 5); +x_228 = 0; +x_229 = l_Lean_SourceInfo_fromRef(x_227, x_228); +x_230 = 1; +x_231 = l_Lean_SourceInfo_fromRef(x_9, x_230); +lean_dec(x_9); +x_232 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; +x_233 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_233, 0, x_231); +lean_ctor_set(x_233, 1, x_232); +x_234 = l_Lean_Elab_Term_expandHave___closed__11; +lean_inc(x_229); +x_235 = l_Lean_Syntax_node1(x_229, x_234, x_95); +x_236 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; +x_237 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; +lean_inc(x_229); +x_238 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_238, 0, x_229); +lean_ctor_set(x_238, 1, x_236); +lean_ctor_set(x_238, 2, x_237); +x_239 = l_Lean_Elab_Term_elabShow___closed__11; +lean_inc(x_229); +x_240 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_240, 0, x_229); +lean_ctor_set(x_240, 1, x_239); +x_241 = l_Lean_Elab_Term_elabShow___closed__10; +lean_inc(x_229); +x_242 = l_Lean_Syntax_node2(x_229, x_241, x_240, x_183); +lean_inc(x_229); +x_243 = l_Lean_Syntax_node1(x_229, x_236, x_242); +x_244 = l_Lean_Elab_Term_elabShow___closed__12; +lean_inc(x_229); x_245 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_245, 0, x_243); +lean_ctor_set(x_245, 0, x_229); lean_ctor_set(x_245, 1, x_244); -x_246 = l_Lean_Elab_Term_expandShow___closed__9; -lean_inc(x_220); -x_247 = l_Lean_Syntax_node2(x_220, x_246, x_245, x_211); -x_248 = l_Lean_Elab_Term_expandHave___closed__1; -x_249 = l_Lean_Syntax_node4(x_220, x_248, x_224, x_240, x_242, x_247); -x_250 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_250, 0, x_249); -lean_ctor_set(x_250, 1, x_3); -return x_250; -} -} -} -else -{ -lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; uint8_t x_255; lean_object* x_256; uint8_t 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; -x_251 = l_Lean_Syntax_getArg(x_203, x_10); -lean_dec(x_203); -x_252 = lean_unsigned_to_nat(3u); -x_253 = l_Lean_Syntax_getArg(x_1, x_252); -lean_dec(x_1); -x_254 = lean_ctor_get(x_2, 5); -x_255 = 0; -x_256 = l_Lean_SourceInfo_fromRef(x_254, x_255); -x_257 = 1; -x_258 = l_Lean_SourceInfo_fromRef(x_9, x_257); -lean_dec(x_9); -x_259 = l_Lean_Elab_Term_expandHave___lambda__4___closed__1; -x_260 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_260, 0, x_258); -lean_ctor_set(x_260, 1, x_259); -x_261 = l_Lean_Elab_Term_expandHave___closed__11; -lean_inc(x_256); -x_262 = l_Lean_Syntax_node1(x_256, x_261, x_104); -x_263 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; -x_264 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__4; -lean_inc(x_256); -x_265 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_265, 0, x_256); -lean_ctor_set(x_265, 1, x_263); -lean_ctor_set(x_265, 2, x_264); -x_266 = l_Lean_Elab_Term_elabShow___closed__11; -lean_inc(x_256); -x_267 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_267, 0, x_256); -lean_ctor_set(x_267, 1, x_266); -x_268 = l_Lean_Elab_Term_elabShow___closed__10; -lean_inc(x_256); -x_269 = l_Lean_Syntax_node2(x_256, x_268, x_267, x_201); -lean_inc(x_256); -x_270 = l_Lean_Syntax_node1(x_256, x_263, x_269); -x_271 = l_Lean_Elab_Term_elabShow___closed__12; -lean_inc(x_256); -x_272 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_272, 0, x_256); -lean_ctor_set(x_272, 1, x_271); -x_273 = l_Lean_Elab_Term_expandHave___closed__5; -lean_inc(x_256); -x_274 = l_Lean_Syntax_node5(x_256, x_273, x_262, x_265, x_270, x_272, x_253); -x_275 = l_Lean_Elab_Term_expandHave___closed__3; -lean_inc(x_256); -x_276 = l_Lean_Syntax_node1(x_256, x_275, x_274); -x_277 = l_Lean_Elab_Term_elabShow___closed__13; -lean_inc(x_256); -x_278 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_278, 0, x_256); -lean_ctor_set(x_278, 1, x_277); -x_279 = l_Lean_Elab_Term_expandHave___closed__1; -x_280 = l_Lean_Syntax_node4(x_256, x_279, x_260, x_276, x_278, x_251); -x_281 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_281, 0, x_280); -lean_ctor_set(x_281, 1, x_3); -return x_281; +x_246 = l_Lean_Elab_Term_expandHave___closed__5; +lean_inc(x_229); +x_247 = l_Lean_Syntax_node5(x_229, x_246, x_235, x_238, x_243, x_245, x_226); +x_248 = l_Lean_Elab_Term_expandHave___closed__3; +lean_inc(x_229); +x_249 = l_Lean_Syntax_node1(x_229, x_248, x_247); +x_250 = l_Lean_Elab_Term_elabShow___closed__13; +lean_inc(x_229); +x_251 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_251, 0, x_229); +lean_ctor_set(x_251, 1, x_250); +x_252 = l_Lean_Elab_Term_expandHave___closed__1; +x_253 = l_Lean_Syntax_node4(x_229, x_252, x_233, x_249, x_251, x_224); +x_254 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_254, 0, x_253); +lean_ctor_set(x_254, 1, x_3); +return x_254; } } } @@ -24958,23 +24835,51 @@ static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("tacticSeq1Indented", 18, 18); +x_1 = lean_mk_string_unchecked("Tactic", 6, 6); return x_1; } } static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__2() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("tacticSeq", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___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___regBuiltin_Lean_Elab_Term_elabCoe__1___closed__3; x_2 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__8; -x_3 = l_Lean_Elab_Term_expandSuffices___closed__7; -x_4 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__1; +x_3 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__1; +x_4 = l_Lean_Elab_Term_elabSubst___lambda__6___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_Elab_Term_elabSubst___lambda__6___closed__3() { +static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("tacticSeq1Indented", 18, 18); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___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___regBuiltin_Lean_Elab_Term_elabCoe__1___closed__3; +x_2 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__8; +x_3 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__1; +x_4 = l_Lean_Elab_Term_elabSubst___lambda__6___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_Elab_Term_elabSubst___lambda__6___closed__6() { _start: { lean_object* x_1; @@ -24982,19 +24887,19 @@ x_1 = lean_mk_string_unchecked("subst", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__4() { +static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___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___regBuiltin_Lean_Elab_Term_elabCoe__1___closed__3; x_2 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__8; -x_3 = l_Lean_Elab_Term_expandSuffices___closed__7; -x_4 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; +x_3 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__1; +x_4 = l_Lean_Elab_Term_elabSubst___lambda__6___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_Elab_Term_elabSubst___lambda__6___closed__5() { +static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__8() { _start: { lean_object* x_1; @@ -25002,14 +24907,14 @@ x_1 = lean_mk_string_unchecked("exact", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__6() { +static lean_object* _init_l_Lean_Elab_Term_elabSubst___lambda__6___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___regBuiltin_Lean_Elab_Term_elabCoe__1___closed__3; x_2 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__8; -x_3 = l_Lean_Elab_Term_expandSuffices___closed__7; -x_4 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; +x_3 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__1; +x_4 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__8; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -25036,7 +24941,7 @@ lean_inc(x_14); lean_ctor_set_tag(x_15, 2); lean_ctor_set(x_15, 1, x_19); lean_ctor_set(x_15, 0, x_14); -x_20 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; +x_20 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; lean_inc(x_14); x_21 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_21, 0, x_14); @@ -25044,7 +24949,7 @@ lean_ctor_set(x_21, 1, x_20); x_22 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; lean_inc(x_14); x_23 = l_Lean_Syntax_node1(x_14, x_22, x_1); -x_24 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__4; +x_24 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__7; lean_inc(x_14); x_25 = l_Lean_Syntax_node2(x_14, x_24, x_21, x_23); x_26 = l_Lean_Elab_Term_elabShow___closed__13; @@ -25052,20 +24957,20 @@ lean_inc(x_14); x_27 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_27, 0, x_14); lean_ctor_set(x_27, 1, x_26); -x_28 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; +x_28 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__8; lean_inc(x_14); x_29 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_29, 0, x_14); lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; +x_30 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__9; lean_inc(x_14); x_31 = l_Lean_Syntax_node2(x_14, x_30, x_29, x_4); lean_inc(x_14); x_32 = l_Lean_Syntax_node3(x_14, x_22, x_25, x_27, x_31); -x_33 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__2; +x_33 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; lean_inc(x_14); x_34 = l_Lean_Syntax_node1(x_14, x_33, x_32); -x_35 = l_Lean_Elab_Term_expandSuffices___closed__9; +x_35 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; lean_inc(x_14); x_36 = l_Lean_Syntax_node1(x_14, x_35, x_34); x_37 = l_Lean_Elab_Term_expandShow___closed__9; @@ -25095,7 +25000,7 @@ lean_inc(x_14); x_47 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_47, 0, x_14); lean_ctor_set(x_47, 1, x_46); -x_48 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; +x_48 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; lean_inc(x_14); x_49 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_49, 0, x_14); @@ -25103,7 +25008,7 @@ lean_ctor_set(x_49, 1, x_48); x_50 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; lean_inc(x_14); x_51 = l_Lean_Syntax_node1(x_14, x_50, x_1); -x_52 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__4; +x_52 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__7; lean_inc(x_14); x_53 = l_Lean_Syntax_node2(x_14, x_52, x_49, x_51); x_54 = l_Lean_Elab_Term_elabShow___closed__13; @@ -25111,20 +25016,20 @@ lean_inc(x_14); x_55 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_55, 0, x_14); lean_ctor_set(x_55, 1, x_54); -x_56 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; +x_56 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__8; lean_inc(x_14); x_57 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_57, 0, x_14); lean_ctor_set(x_57, 1, x_56); -x_58 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; +x_58 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__9; lean_inc(x_14); x_59 = l_Lean_Syntax_node2(x_14, x_58, x_57, x_4); lean_inc(x_14); x_60 = l_Lean_Syntax_node3(x_14, x_50, x_53, x_55, x_59); -x_61 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__2; +x_61 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; lean_inc(x_14); x_62 = l_Lean_Syntax_node1(x_14, x_61, x_60); -x_63 = l_Lean_Elab_Term_expandSuffices___closed__9; +x_63 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; lean_inc(x_14); x_64 = l_Lean_Syntax_node1(x_14, x_63, x_62); x_65 = l_Lean_Elab_Term_expandShow___closed__9; @@ -25190,7 +25095,7 @@ lean_inc(x_22); lean_ctor_set_tag(x_23, 2); lean_ctor_set(x_23, 1, x_27); lean_ctor_set(x_23, 0, x_22); -x_28 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; +x_28 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; lean_inc(x_22); lean_ctor_set_tag(x_13, 2); lean_ctor_set(x_13, 1, x_28); @@ -25198,7 +25103,7 @@ lean_ctor_set(x_13, 0, x_22); x_29 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; lean_inc(x_22); x_30 = l_Lean_Syntax_node1(x_22, x_29, x_5); -x_31 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__4; +x_31 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__7; lean_inc(x_22); x_32 = l_Lean_Syntax_node2(x_22, x_31, x_13, x_30); x_33 = l_Lean_Elab_Term_elabShow___closed__13; @@ -25206,20 +25111,20 @@ lean_inc(x_22); x_34 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_34, 0, x_22); lean_ctor_set(x_34, 1, x_33); -x_35 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; +x_35 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__8; lean_inc(x_22); x_36 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_36, 0, x_22); lean_ctor_set(x_36, 1, x_35); -x_37 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; +x_37 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__9; lean_inc(x_22); x_38 = l_Lean_Syntax_node2(x_22, x_37, x_36, x_4); lean_inc(x_22); x_39 = l_Lean_Syntax_node3(x_22, x_29, x_32, x_34, x_38); -x_40 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__2; +x_40 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; lean_inc(x_22); x_41 = l_Lean_Syntax_node1(x_22, x_40, x_39); -x_42 = l_Lean_Elab_Term_expandSuffices___closed__9; +x_42 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; lean_inc(x_22); x_43 = l_Lean_Syntax_node1(x_22, x_42, x_41); x_44 = l_Lean_Elab_Term_expandShow___closed__9; @@ -25249,7 +25154,7 @@ lean_inc(x_22); x_54 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_54, 0, x_22); lean_ctor_set(x_54, 1, x_53); -x_55 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; +x_55 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; lean_inc(x_22); lean_ctor_set_tag(x_13, 2); lean_ctor_set(x_13, 1, x_55); @@ -25257,7 +25162,7 @@ lean_ctor_set(x_13, 0, x_22); x_56 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; lean_inc(x_22); x_57 = l_Lean_Syntax_node1(x_22, x_56, x_5); -x_58 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__4; +x_58 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__7; lean_inc(x_22); x_59 = l_Lean_Syntax_node2(x_22, x_58, x_13, x_57); x_60 = l_Lean_Elab_Term_elabShow___closed__13; @@ -25265,20 +25170,20 @@ lean_inc(x_22); x_61 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_61, 0, x_22); lean_ctor_set(x_61, 1, x_60); -x_62 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; +x_62 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__8; lean_inc(x_22); x_63 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_63, 0, x_22); lean_ctor_set(x_63, 1, x_62); -x_64 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; +x_64 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__9; lean_inc(x_22); x_65 = l_Lean_Syntax_node2(x_22, x_64, x_63, x_4); lean_inc(x_22); x_66 = l_Lean_Syntax_node3(x_22, x_56, x_59, x_61, x_65); -x_67 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__2; +x_67 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; lean_inc(x_22); x_68 = l_Lean_Syntax_node1(x_22, x_67, x_66); -x_69 = l_Lean_Elab_Term_expandSuffices___closed__9; +x_69 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; lean_inc(x_22); x_70 = l_Lean_Syntax_node1(x_22, x_69, x_68); x_71 = l_Lean_Elab_Term_expandShow___closed__9; @@ -25348,7 +25253,7 @@ if (lean_is_scalar(x_89)) { } lean_ctor_set(x_91, 0, x_86); lean_ctor_set(x_91, 1, x_90); -x_92 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; +x_92 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; lean_inc(x_86); x_93 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_93, 0, x_86); @@ -25356,7 +25261,7 @@ lean_ctor_set(x_93, 1, x_92); x_94 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__3; lean_inc(x_86); x_95 = l_Lean_Syntax_node1(x_86, x_94, x_5); -x_96 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__4; +x_96 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__7; lean_inc(x_86); x_97 = l_Lean_Syntax_node2(x_86, x_96, x_93, x_95); x_98 = l_Lean_Elab_Term_elabShow___closed__13; @@ -25364,20 +25269,20 @@ lean_inc(x_86); x_99 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_99, 0, x_86); lean_ctor_set(x_99, 1, x_98); -x_100 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; +x_100 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__8; lean_inc(x_86); x_101 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_101, 0, x_86); lean_ctor_set(x_101, 1, x_100); -x_102 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; +x_102 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__9; lean_inc(x_86); x_103 = l_Lean_Syntax_node2(x_86, x_102, x_101, x_4); lean_inc(x_86); x_104 = l_Lean_Syntax_node3(x_86, x_94, x_97, x_99, x_103); -x_105 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__2; +x_105 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__5; lean_inc(x_86); x_106 = l_Lean_Syntax_node1(x_86, x_105, x_104); -x_107 = l_Lean_Elab_Term_expandSuffices___closed__9; +x_107 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; lean_inc(x_86); x_108 = l_Lean_Syntax_node1(x_86, x_107, x_106); x_109 = l_Lean_Elab_Term_expandShow___closed__9; @@ -27064,7 +26969,7 @@ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_obj x_1 = l___regBuiltin_Lean_Elab_Term_elabCoe__1___closed__3; x_2 = l_Lean_Elab_Term_elabAnonymousCtor___lambda__3___closed__8; x_3 = l___regBuiltin_Lean_Elab_Term_elabCoe__1___closed__5; -x_4 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__3; +x_4 = l_Lean_Elab_Term_elabSubst___lambda__6___closed__6; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -31442,7 +31347,7 @@ static lean_object* _init_l_Lean_Elab_Term_elabUnsafe___lambda__1___closed__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; x_1 = l_Lean_Elab_Term_elabUnsafe___lambda__1___closed__3; x_2 = l_Lean_Elab_Term_elabUnsafe___lambda__1___closed__4; -x_3 = lean_unsigned_to_nat(493u); +x_3 = lean_unsigned_to_nat(501u); x_4 = lean_unsigned_to_nat(54u); x_5 = l_Lean_Elab_Term_elabUnsafe___lambda__1___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -31455,7 +31360,7 @@ static lean_object* _init_l_Lean_Elab_Term_elabUnsafe___lambda__1___closed__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; x_1 = l_Lean_Elab_Term_elabUnsafe___lambda__1___closed__3; x_2 = l_Lean_Elab_Term_elabUnsafe___lambda__1___closed__4; -x_3 = lean_unsigned_to_nat(494u); +x_3 = lean_unsigned_to_nat(502u); x_4 = lean_unsigned_to_nat(55u); x_5 = l_Lean_Elab_Term_elabUnsafe___lambda__1___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -35202,12 +35107,6 @@ l_Lean_Elab_Term_expandSuffices___closed__5 = _init_l_Lean_Elab_Term_expandSuffi lean_mark_persistent(l_Lean_Elab_Term_expandSuffices___closed__5); l_Lean_Elab_Term_expandSuffices___closed__6 = _init_l_Lean_Elab_Term_expandSuffices___closed__6(); lean_mark_persistent(l_Lean_Elab_Term_expandSuffices___closed__6); -l_Lean_Elab_Term_expandSuffices___closed__7 = _init_l_Lean_Elab_Term_expandSuffices___closed__7(); -lean_mark_persistent(l_Lean_Elab_Term_expandSuffices___closed__7); -l_Lean_Elab_Term_expandSuffices___closed__8 = _init_l_Lean_Elab_Term_expandSuffices___closed__8(); -lean_mark_persistent(l_Lean_Elab_Term_expandSuffices___closed__8); -l_Lean_Elab_Term_expandSuffices___closed__9 = _init_l_Lean_Elab_Term_expandSuffices___closed__9(); -lean_mark_persistent(l_Lean_Elab_Term_expandSuffices___closed__9); l___regBuiltin_Lean_Elab_Term_expandSuffices__1___closed__1 = _init_l___regBuiltin_Lean_Elab_Term_expandSuffices__1___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_expandSuffices__1___closed__1); l___regBuiltin_Lean_Elab_Term_expandSuffices__1___closed__2 = _init_l___regBuiltin_Lean_Elab_Term_expandSuffices__1___closed__2(); @@ -35970,6 +35869,12 @@ l_Lean_Elab_Term_elabSubst___lambda__6___closed__5 = _init_l_Lean_Elab_Term_elab lean_mark_persistent(l_Lean_Elab_Term_elabSubst___lambda__6___closed__5); l_Lean_Elab_Term_elabSubst___lambda__6___closed__6 = _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__6(); lean_mark_persistent(l_Lean_Elab_Term_elabSubst___lambda__6___closed__6); +l_Lean_Elab_Term_elabSubst___lambda__6___closed__7 = _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__7(); +lean_mark_persistent(l_Lean_Elab_Term_elabSubst___lambda__6___closed__7); +l_Lean_Elab_Term_elabSubst___lambda__6___closed__8 = _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__8(); +lean_mark_persistent(l_Lean_Elab_Term_elabSubst___lambda__6___closed__8); +l_Lean_Elab_Term_elabSubst___lambda__6___closed__9 = _init_l_Lean_Elab_Term_elabSubst___lambda__6___closed__9(); +lean_mark_persistent(l_Lean_Elab_Term_elabSubst___lambda__6___closed__9); l_Lean_Elab_Term_elabSubst___closed__1 = _init_l_Lean_Elab_Term_elabSubst___closed__1(); lean_mark_persistent(l_Lean_Elab_Term_elabSubst___closed__1); l_Lean_Elab_Term_elabSubst___closed__2 = _init_l_Lean_Elab_Term_elabSubst___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Command.c b/stage0/stdlib/Lean/Elab/Command.c index dee76e855a04..574f83b172e7 100644 --- a/stage0/stdlib/Lean/Elab/Command.c +++ b/stage0/stdlib/Lean/Elab/Command.c @@ -549,6 +549,7 @@ static lean_object* l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instA static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommand___spec__20___at_Lean_Elab_Command_elabCommand___spec__21___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_getMainModule___rarg___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_mkState___closed__2; +lean_object* lean_thunk_get_own(lean_object*); lean_object* l_Lean_Elab_expandDeclIdCore(lean_object*); extern lean_object* l_Lean_Elab_builtinIncrementalElabs; static lean_object* l_Lean_Elab_Command_getBracketedBinderIds___closed__7; @@ -655,10 +656,12 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_liftTermE LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadLogCommandElabM___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadMacroAdapterCommandElabM___closed__3; +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabCommand___spec__19___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_addLinter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instInhabitedCommandElabM___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_4786____closed__2; LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__9___lambda__1___boxed(lean_object*, lean_object*); +lean_object* lean_mk_thunk(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__15___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Command_runTermElabM___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* l_Array_append___rarg(lean_object*, lean_object*); @@ -727,6 +730,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_getScopes(lean_object*); static lean_object* l___auto____x40_Lean_Elab_Command___hyg_456____closed__4; lean_object* l_Lean_Syntax_setArgs(lean_object*, lean_object*); extern lean_object* l_Lean_NameSet_empty; +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabCommand___spec__19___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadOptionsCommandElabM___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Command_runLinters___spec__6___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommand___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -18992,10 +18996,10 @@ return x_1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_instToSnapshotTreeMacroExpandedSnapshot___spec__1___lambda__1(lean_object* x_1) { _start: { -lean_object* x_2; +lean_object* x_2; lean_object* x_3; x_2 = lean_ctor_get(x_1, 1); -lean_inc(x_2); -return x_2; +x_3 = lean_thunk_get_own(x_2); +return x_3; } } static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Elab_Command_instToSnapshotTreeMacroExpandedSnapshot___spec__1___closed__1() { @@ -21755,29 +21759,39 @@ goto _start; } } } +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabCommand___spec__19___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; size_t x_5; size_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, 4); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_array_size(x_4); +x_6 = 0; +x_7 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_instToSnapshotTreeMacroExpandedSnapshot___spec__1(x_5, x_6, x_4); +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_3); +lean_ctor_set(x_8, 1, x_7); +return x_8; +} +} LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabCommand___spec__19(lean_object* x_1, lean_object* x_2) { _start: { -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_object* x_9; lean_object* x_10; +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_inc(x_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); -x_4 = lean_ctor_get(x_2, 0); -lean_inc(x_4); -x_5 = lean_ctor_get(x_2, 4); -lean_inc(x_5); -lean_dec(x_2); -x_6 = lean_array_size(x_5); -x_7 = 0; -x_8 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_instToSnapshotTreeMacroExpandedSnapshot___spec__1(x_6, x_7, x_5); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_4); -lean_ctor_set(x_9, 1, x_8); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_3); -lean_ctor_set(x_10, 1, x_9); -return x_10; +x_4 = lean_alloc_closure((void*)(l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabCommand___spec__19___lambda__1___boxed), 2, 1); +lean_closure_set(x_4, 0, x_2); +x_5 = lean_mk_thunk(x_4); +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_3); +lean_ctor_set(x_6, 1, x_5); +return x_6; } } static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommand___spec__20___closed__1() { @@ -26051,6 +26065,15 @@ lean_dec(x_1); return x_5; } } +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabCommand___spec__19___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabCommand___spec__19___lambda__1(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommand___spec__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: { @@ -27889,34 +27912,34 @@ x_23 = l_Lean_Syntax_hasMissing(x_1); x_24 = lean_st_ref_take(x_3, x_7); if (x_23 == 0) { -uint8_t x_293; +uint8_t x_339; lean_dec(x_11); -x_293 = 0; -x_25 = x_293; -goto block_292; +x_339 = 0; +x_25 = x_339; +goto block_338; } else { -lean_object* x_294; uint8_t x_295; -x_294 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__3___closed__2; -x_295 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_11, x_294); +lean_object* x_340; uint8_t x_341; +x_340 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__3___closed__2; +x_341 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_11, x_340); lean_dec(x_11); -if (x_295 == 0) +if (x_341 == 0) { -uint8_t x_296; -x_296 = 1; -x_25 = x_296; -goto block_292; +uint8_t x_342; +x_342 = 1; +x_25 = x_342; +goto block_338; } else { -uint8_t x_297; -x_297 = 0; -x_25 = x_297; -goto block_292; +uint8_t x_343; +x_343 = 0; +x_25 = x_343; +goto block_338; } } -block_292: +block_338: { lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; x_26 = lean_ctor_get(x_24, 0); @@ -27944,7 +27967,7 @@ lean_ctor_set_uint8(x_28, sizeof(void*)*10, x_25); x_29 = !lean_is_exclusive(x_26); 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_92; lean_object* x_93; lean_object* x_147; +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_104; lean_object* x_105; lean_object* x_171; x_30 = lean_ctor_get(x_26, 1); x_31 = l___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___rarg___closed__4; lean_ctor_set(x_26, 1, x_31); @@ -27961,74 +27984,74 @@ lean_dec(x_34); lean_inc(x_3); lean_inc(x_28); lean_inc(x_1); -x_147 = l_Lean_Elab_Command_elabCommand(x_1, x_28, x_3, x_36); -if (lean_obj_tag(x_147) == 0) +x_171 = l_Lean_Elab_Command_elabCommand(x_1, x_28, x_3, x_36); +if (lean_obj_tag(x_171) == 0) { -lean_object* x_148; lean_object* x_149; lean_object* x_150; -x_148 = lean_ctor_get(x_147, 1); -lean_inc(x_148); -lean_dec(x_147); -x_149 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__3___closed__1; +lean_object* x_172; lean_object* x_173; lean_object* x_174; +x_172 = lean_ctor_get(x_171, 1); +lean_inc(x_172); +lean_dec(x_171); +x_173 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__3___closed__1; lean_inc(x_1); -x_150 = l_Lean_Syntax_findAux(x_149, x_1); -if (lean_obj_tag(x_150) == 0) +x_174 = l_Lean_Syntax_findAux(x_173, x_1); +if (lean_obj_tag(x_174) == 0) { -lean_object* x_151; lean_object* x_152; -x_151 = lean_alloc_closure((void*)(l_Lean_Elab_Command_runLinters), 4, 1); -lean_closure_set(x_151, 0, x_1); +lean_object* x_175; lean_object* x_176; +x_175 = lean_alloc_closure((void*)(l_Lean_Elab_Command_runLinters), 4, 1); +lean_closure_set(x_175, 0, x_1); lean_inc(x_3); lean_inc(x_28); -x_152 = l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(x_151, x_28, x_3, x_148); -if (lean_obj_tag(x_152) == 0) +x_176 = l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(x_175, x_28, x_3, x_172); +if (lean_obj_tag(x_176) == 0) { -lean_object* x_153; lean_object* x_154; -x_153 = lean_ctor_get(x_152, 0); -lean_inc(x_153); -x_154 = lean_ctor_get(x_152, 1); -lean_inc(x_154); -lean_dec(x_152); -x_37 = x_153; -x_38 = x_154; -goto block_91; +lean_object* x_177; lean_object* x_178; +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_37 = x_177; +x_38 = x_178; +goto block_103; } else { -lean_object* x_155; lean_object* x_156; -x_155 = lean_ctor_get(x_152, 0); -lean_inc(x_155); -x_156 = lean_ctor_get(x_152, 1); -lean_inc(x_156); -lean_dec(x_152); -x_92 = x_155; -x_93 = x_156; -goto block_146; +lean_object* x_179; lean_object* x_180; +x_179 = lean_ctor_get(x_176, 0); +lean_inc(x_179); +x_180 = lean_ctor_get(x_176, 1); +lean_inc(x_180); +lean_dec(x_176); +x_104 = x_179; +x_105 = x_180; +goto block_170; } } else { -lean_object* x_157; -lean_dec(x_150); +lean_object* x_181; +lean_dec(x_174); lean_dec(x_1); -x_157 = lean_box(0); -x_37 = x_157; -x_38 = x_148; -goto block_91; +x_181 = lean_box(0); +x_37 = x_181; +x_38 = x_172; +goto block_103; } } else { -lean_object* x_158; lean_object* x_159; +lean_object* x_182; lean_object* x_183; lean_dec(x_1); -x_158 = lean_ctor_get(x_147, 0); -lean_inc(x_158); -x_159 = lean_ctor_get(x_147, 1); -lean_inc(x_159); -lean_dec(x_147); -x_92 = x_158; -x_93 = x_159; -goto block_146; +x_182 = lean_ctor_get(x_171, 0); +lean_inc(x_182); +x_183 = lean_ctor_get(x_171, 1); +lean_inc(x_183); +lean_dec(x_171); +x_104 = x_182; +x_105 = x_183; +goto block_170; } -block_91: +block_103: { 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_st_ref_get(x_3, x_38); @@ -28051,80 +28074,54 @@ x_47 = l_Lean_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel__ lean_dec(x_44); if (lean_obj_tag(x_47) == 0) { -if (lean_obj_tag(x_20) == 0) -{ -lean_object* x_48; lean_object* x_49; uint8_t x_50; +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; x_48 = lean_ctor_get(x_47, 1); lean_inc(x_48); lean_dec(x_47); -x_49 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_42, x_35, x_46, x_28, x_3, x_48); -lean_dec(x_3); -x_50 = !lean_is_exclusive(x_49); -if (x_50 == 0) -{ -lean_object* x_51; -x_51 = lean_ctor_get(x_49, 0); +x_49 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_4859____closed__5; +x_50 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Command_runLinters___spec__11(x_49, x_28, x_3, x_48); +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = lean_unbox(x_51); lean_dec(x_51); -lean_ctor_set(x_49, 0, x_37); -return x_49; -} -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_37); -lean_ctor_set(x_53, 1, x_52); -return x_53; -} -} -else +if (x_52 == 0) { -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_81; lean_object* x_82; -x_54 = lean_ctor_get(x_47, 1); -lean_inc(x_54); -lean_dec(x_47); -x_55 = lean_ctor_get(x_20, 0); -lean_inc(x_55); +lean_object* x_53; lean_object* x_54; uint8_t x_55; lean_dec(x_20); -x_56 = lean_ctor_get(x_55, 1); -lean_inc(x_56); -lean_dec(x_55); -x_57 = lean_io_promise_result(x_56); -x_81 = lean_io_get_task_state(x_57, x_54); -x_82 = lean_ctor_get(x_81, 0); -lean_inc(x_82); -if (lean_obj_tag(x_82) == 2) +x_53 = lean_ctor_get(x_50, 1); +lean_inc(x_53); +lean_dec(x_50); +x_54 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_42, x_35, x_46, x_28, x_3, x_53); +lean_dec(x_3); +x_55 = !lean_is_exclusive(x_54); +if (x_55 == 0) { -lean_object* x_83; uint8_t x_84; -x_83 = lean_ctor_get(x_81, 1); -lean_inc(x_83); -lean_dec(x_81); -x_84 = 1; -x_58 = x_84; -x_59 = x_83; -goto block_80; +lean_object* x_56; +x_56 = lean_ctor_get(x_54, 0); +lean_dec(x_56); +lean_ctor_set(x_54, 0, x_37); +return x_54; } else { -lean_object* x_85; uint8_t x_86; -lean_dec(x_82); -x_85 = lean_ctor_get(x_81, 1); -lean_inc(x_85); -lean_dec(x_81); -x_86 = 0; -x_58 = x_86; -x_59 = x_85; -goto block_80; +lean_object* x_57; lean_object* x_58; +x_57 = lean_ctor_get(x_54, 1); +lean_inc(x_57); +lean_dec(x_54); +x_58 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_58, 0, x_37); +lean_ctor_set(x_58, 1, x_57); +return x_58; } -block_80: +} +else { -if (x_58 == 0) +if (lean_obj_tag(x_20) == 0) { -lean_object* x_60; uint8_t x_61; -lean_dec(x_57); +lean_object* x_59; lean_object* x_60; uint8_t x_61; +x_59 = lean_ctor_get(x_50, 1); +lean_inc(x_59); +lean_dec(x_50); x_60 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_42, x_35, x_46, x_28, x_3, x_59); lean_dec(x_3); x_61 = !lean_is_exclusive(x_60); @@ -28150,25 +28147,51 @@ return x_64; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_65 = lean_task_get_own(x_57); -x_66 = lean_ctor_get(x_65, 1); +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; uint8_t x_69; lean_object* x_70; lean_object* x_93; lean_object* x_94; +x_65 = lean_ctor_get(x_50, 1); +lean_inc(x_65); +lean_dec(x_50); +x_66 = lean_ctor_get(x_20, 0); lean_inc(x_66); -lean_dec(x_65); -x_67 = lean_alloc_closure((void*)(l_Lean_Language_SnapshotTree_trace), 4, 1); -lean_closure_set(x_67, 0, x_66); -x_68 = l_Lean_Elab_Command_liftCoreM___rarg(x_67, x_28, x_3, x_59); -if (lean_obj_tag(x_68) == 0) +lean_dec(x_20); +x_67 = lean_ctor_get(x_66, 1); +lean_inc(x_67); +lean_dec(x_66); +x_68 = lean_io_promise_result(x_67); +x_93 = lean_io_get_task_state(x_68, x_65); +x_94 = lean_ctor_get(x_93, 0); +lean_inc(x_94); +if (lean_obj_tag(x_94) == 2) { -lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; -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_object* x_95; uint8_t x_96; +x_95 = lean_ctor_get(x_93, 1); +lean_inc(x_95); +lean_dec(x_93); +x_96 = 1; +x_69 = x_96; +x_70 = x_95; +goto block_92; +} +else +{ +lean_object* x_97; uint8_t x_98; +lean_dec(x_94); +x_97 = lean_ctor_get(x_93, 1); +lean_inc(x_97); +lean_dec(x_93); +x_98 = 0; +x_69 = x_98; +x_70 = x_97; +goto block_92; +} +block_92: +{ +if (x_69 == 0) +{ +lean_object* x_71; uint8_t x_72; lean_dec(x_68); -x_71 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_42, x_35, x_69, x_28, x_3, x_70); +x_71 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_42, x_35, x_46, x_28, x_3, x_70); lean_dec(x_3); -lean_dec(x_69); x_72 = !lean_is_exclusive(x_71); if (x_72 == 0) { @@ -28192,30 +28215,75 @@ return x_75; } else { -uint8_t x_76; +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_76 = lean_task_get_own(x_68); +x_77 = lean_ctor_get(x_76, 1); +lean_inc(x_77); +lean_dec(x_76); +x_78 = lean_thunk_get_own(x_77); +lean_dec(x_77); +x_79 = lean_alloc_closure((void*)(l_Lean_Language_SnapshotTree_trace), 4, 1); +lean_closure_set(x_79, 0, x_78); +x_80 = l_Lean_Elab_Command_liftCoreM___rarg(x_79, x_28, x_3, x_70); +if (lean_obj_tag(x_80) == 0) +{ +lean_object* x_81; lean_object* x_82; lean_object* x_83; uint8_t 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); +lean_dec(x_80); +x_83 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_42, x_35, x_81, x_28, x_3, x_82); +lean_dec(x_3); +lean_dec(x_81); +x_84 = !lean_is_exclusive(x_83); +if (x_84 == 0) +{ +lean_object* x_85; +x_85 = lean_ctor_get(x_83, 0); +lean_dec(x_85); +lean_ctor_set(x_83, 0, x_37); +return x_83; +} +else +{ +lean_object* x_86; lean_object* x_87; +x_86 = lean_ctor_get(x_83, 1); +lean_inc(x_86); +lean_dec(x_83); +x_87 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_87, 0, x_37); +lean_ctor_set(x_87, 1, x_86); +return x_87; +} +} +else +{ +uint8_t x_88; lean_dec(x_42); lean_dec(x_37); lean_dec(x_35); lean_dec(x_30); lean_dec(x_28); lean_dec(x_3); -x_76 = !lean_is_exclusive(x_68); -if (x_76 == 0) +x_88 = !lean_is_exclusive(x_80); +if (x_88 == 0) { -return x_68; +return x_80; } 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; +lean_object* x_89; lean_object* x_90; lean_object* x_91; +x_89 = lean_ctor_get(x_80, 0); +x_90 = lean_ctor_get(x_80, 1); +lean_inc(x_90); +lean_inc(x_89); +lean_dec(x_80); +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; +} } } } @@ -28224,7 +28292,7 @@ return x_79; } else { -uint8_t x_87; +uint8_t x_99; lean_dec(x_42); lean_dec(x_37); lean_dec(x_35); @@ -28232,217 +28300,263 @@ lean_dec(x_30); lean_dec(x_28); lean_dec(x_20); lean_dec(x_3); -x_87 = !lean_is_exclusive(x_47); -if (x_87 == 0) +x_99 = !lean_is_exclusive(x_47); +if (x_99 == 0) { return x_47; } else { -lean_object* x_88; lean_object* x_89; lean_object* x_90; -x_88 = lean_ctor_get(x_47, 0); -x_89 = lean_ctor_get(x_47, 1); -lean_inc(x_89); -lean_inc(x_88); +lean_object* x_100; lean_object* x_101; lean_object* x_102; +x_100 = lean_ctor_get(x_47, 0); +x_101 = lean_ctor_get(x_47, 1); +lean_inc(x_101); +lean_inc(x_100); lean_dec(x_47); -x_90 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_90, 0, x_88); -lean_ctor_set(x_90, 1, x_89); -return x_90; +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; } } } -block_146: +block_170: { -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; -x_94 = lean_st_ref_get(x_3, 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, 1); -lean_inc(x_97); -lean_dec(x_95); -x_98 = l_Lean_Elab_getInfoTrees___at_Lean_Elab_Command_elabCommandTopLevel___spec__1___rarg(x_3, x_96); -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 = lean_box(0); -x_102 = l_Lean_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel___spec__3(x_99, x_101, x_28, x_3, x_100); -lean_dec(x_99); -if (lean_obj_tag(x_102) == 0) +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; +x_106 = lean_st_ref_get(x_3, x_105); +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 = lean_ctor_get(x_107, 1); +lean_inc(x_109); +lean_dec(x_107); +x_110 = l_Lean_Elab_getInfoTrees___at_Lean_Elab_Command_elabCommandTopLevel___spec__1___rarg(x_3, x_108); +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_box(0); +x_114 = l_Lean_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel___spec__3(x_111, x_113, x_28, x_3, x_112); +lean_dec(x_111); +if (lean_obj_tag(x_114) == 0) +{ +lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; uint8_t x_119; +x_115 = lean_ctor_get(x_114, 1); +lean_inc(x_115); +lean_dec(x_114); +x_116 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_4859____closed__5; +x_117 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Command_runLinters___spec__11(x_116, x_28, x_3, x_115); +x_118 = lean_ctor_get(x_117, 0); +lean_inc(x_118); +x_119 = lean_unbox(x_118); +lean_dec(x_118); +if (x_119 == 0) +{ +lean_object* x_120; lean_object* x_121; uint8_t x_122; +lean_dec(x_20); +x_120 = lean_ctor_get(x_117, 1); +lean_inc(x_120); +lean_dec(x_117); +x_121 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_109, x_35, x_113, x_28, x_3, x_120); +lean_dec(x_3); +x_122 = !lean_is_exclusive(x_121); +if (x_122 == 0) +{ +lean_object* x_123; +x_123 = lean_ctor_get(x_121, 0); +lean_dec(x_123); +lean_ctor_set_tag(x_121, 1); +lean_ctor_set(x_121, 0, x_104); +return x_121; +} +else +{ +lean_object* x_124; lean_object* x_125; +x_124 = lean_ctor_get(x_121, 1); +lean_inc(x_124); +lean_dec(x_121); +x_125 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_125, 0, x_104); +lean_ctor_set(x_125, 1, x_124); +return x_125; +} +} +else { if (lean_obj_tag(x_20) == 0) { -lean_object* x_103; lean_object* x_104; uint8_t x_105; -x_103 = lean_ctor_get(x_102, 1); -lean_inc(x_103); -lean_dec(x_102); -x_104 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_97, x_35, x_101, x_28, x_3, x_103); +lean_object* x_126; lean_object* x_127; uint8_t x_128; +x_126 = lean_ctor_get(x_117, 1); +lean_inc(x_126); +lean_dec(x_117); +x_127 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_109, x_35, x_113, x_28, x_3, x_126); lean_dec(x_3); -x_105 = !lean_is_exclusive(x_104); -if (x_105 == 0) +x_128 = !lean_is_exclusive(x_127); +if (x_128 == 0) { -lean_object* x_106; -x_106 = lean_ctor_get(x_104, 0); -lean_dec(x_106); -lean_ctor_set_tag(x_104, 1); -lean_ctor_set(x_104, 0, x_92); -return x_104; +lean_object* x_129; +x_129 = lean_ctor_get(x_127, 0); +lean_dec(x_129); +lean_ctor_set_tag(x_127, 1); +lean_ctor_set(x_127, 0, x_104); +return x_127; } else { -lean_object* x_107; lean_object* x_108; -x_107 = lean_ctor_get(x_104, 1); -lean_inc(x_107); -lean_dec(x_104); -x_108 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_108, 0, x_92); -lean_ctor_set(x_108, 1, x_107); -return x_108; +lean_object* x_130; lean_object* x_131; +x_130 = lean_ctor_get(x_127, 1); +lean_inc(x_130); +lean_dec(x_127); +x_131 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_131, 0, x_104); +lean_ctor_set(x_131, 1, x_130); +return x_131; } } else { -lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; uint8_t x_113; lean_object* x_114; lean_object* x_136; lean_object* x_137; -x_109 = lean_ctor_get(x_102, 1); -lean_inc(x_109); -lean_dec(x_102); -x_110 = lean_ctor_get(x_20, 0); -lean_inc(x_110); +lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; uint8_t x_136; lean_object* x_137; lean_object* x_160; lean_object* x_161; +x_132 = lean_ctor_get(x_117, 1); +lean_inc(x_132); +lean_dec(x_117); +x_133 = lean_ctor_get(x_20, 0); +lean_inc(x_133); lean_dec(x_20); -x_111 = lean_ctor_get(x_110, 1); -lean_inc(x_111); -lean_dec(x_110); -x_112 = lean_io_promise_result(x_111); -x_136 = lean_io_get_task_state(x_112, x_109); -x_137 = lean_ctor_get(x_136, 0); -lean_inc(x_137); -if (lean_obj_tag(x_137) == 2) +x_134 = lean_ctor_get(x_133, 1); +lean_inc(x_134); +lean_dec(x_133); +x_135 = lean_io_promise_result(x_134); +x_160 = lean_io_get_task_state(x_135, x_132); +x_161 = lean_ctor_get(x_160, 0); +lean_inc(x_161); +if (lean_obj_tag(x_161) == 2) { -lean_object* x_138; uint8_t x_139; -x_138 = lean_ctor_get(x_136, 1); -lean_inc(x_138); -lean_dec(x_136); -x_139 = 1; -x_113 = x_139; -x_114 = x_138; -goto block_135; +lean_object* x_162; uint8_t x_163; +x_162 = lean_ctor_get(x_160, 1); +lean_inc(x_162); +lean_dec(x_160); +x_163 = 1; +x_136 = x_163; +x_137 = x_162; +goto block_159; } else { -lean_object* x_140; uint8_t x_141; -lean_dec(x_137); -x_140 = lean_ctor_get(x_136, 1); -lean_inc(x_140); -lean_dec(x_136); -x_141 = 0; -x_113 = x_141; -x_114 = x_140; -goto block_135; +lean_object* x_164; uint8_t x_165; +lean_dec(x_161); +x_164 = lean_ctor_get(x_160, 1); +lean_inc(x_164); +lean_dec(x_160); +x_165 = 0; +x_136 = x_165; +x_137 = x_164; +goto block_159; } -block_135: +block_159: { -if (x_113 == 0) +if (x_136 == 0) { -lean_object* x_115; uint8_t x_116; -lean_dec(x_112); -x_115 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_97, x_35, x_101, x_28, x_3, x_114); +lean_object* x_138; uint8_t x_139; +lean_dec(x_135); +x_138 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_109, x_35, x_113, x_28, x_3, x_137); lean_dec(x_3); -x_116 = !lean_is_exclusive(x_115); -if (x_116 == 0) +x_139 = !lean_is_exclusive(x_138); +if (x_139 == 0) { -lean_object* x_117; -x_117 = lean_ctor_get(x_115, 0); -lean_dec(x_117); -lean_ctor_set_tag(x_115, 1); -lean_ctor_set(x_115, 0, x_92); -return x_115; +lean_object* x_140; +x_140 = lean_ctor_get(x_138, 0); +lean_dec(x_140); +lean_ctor_set_tag(x_138, 1); +lean_ctor_set(x_138, 0, x_104); +return x_138; } else { -lean_object* x_118; lean_object* x_119; -x_118 = lean_ctor_get(x_115, 1); -lean_inc(x_118); -lean_dec(x_115); -x_119 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_119, 0, x_92); -lean_ctor_set(x_119, 1, x_118); -return x_119; +lean_object* x_141; lean_object* x_142; +x_141 = lean_ctor_get(x_138, 1); +lean_inc(x_141); +lean_dec(x_138); +x_142 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_142, 0, x_104); +lean_ctor_set(x_142, 1, x_141); +return x_142; } } else { -lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; -x_120 = lean_task_get_own(x_112); -x_121 = lean_ctor_get(x_120, 1); -lean_inc(x_121); -lean_dec(x_120); -x_122 = lean_alloc_closure((void*)(l_Lean_Language_SnapshotTree_trace), 4, 1); -lean_closure_set(x_122, 0, x_121); -x_123 = l_Lean_Elab_Command_liftCoreM___rarg(x_122, x_28, x_3, x_114); -if (lean_obj_tag(x_123) == 0) +lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_143 = lean_task_get_own(x_135); +x_144 = lean_ctor_get(x_143, 1); +lean_inc(x_144); +lean_dec(x_143); +x_145 = lean_thunk_get_own(x_144); +lean_dec(x_144); +x_146 = lean_alloc_closure((void*)(l_Lean_Language_SnapshotTree_trace), 4, 1); +lean_closure_set(x_146, 0, x_145); +x_147 = l_Lean_Elab_Command_liftCoreM___rarg(x_146, x_28, x_3, x_137); +if (lean_obj_tag(x_147) == 0) { -lean_object* x_124; lean_object* x_125; lean_object* x_126; uint8_t x_127; -x_124 = lean_ctor_get(x_123, 0); -lean_inc(x_124); -x_125 = lean_ctor_get(x_123, 1); -lean_inc(x_125); -lean_dec(x_123); -x_126 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_97, x_35, x_124, x_28, x_3, x_125); +lean_object* x_148; lean_object* x_149; lean_object* x_150; uint8_t x_151; +x_148 = lean_ctor_get(x_147, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_147, 1); +lean_inc(x_149); +lean_dec(x_147); +x_150 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_30, x_109, x_35, x_148, x_28, x_3, x_149); lean_dec(x_3); -lean_dec(x_124); -x_127 = !lean_is_exclusive(x_126); -if (x_127 == 0) +lean_dec(x_148); +x_151 = !lean_is_exclusive(x_150); +if (x_151 == 0) { -lean_object* x_128; -x_128 = lean_ctor_get(x_126, 0); -lean_dec(x_128); -lean_ctor_set_tag(x_126, 1); -lean_ctor_set(x_126, 0, x_92); -return x_126; +lean_object* x_152; +x_152 = lean_ctor_get(x_150, 0); +lean_dec(x_152); +lean_ctor_set_tag(x_150, 1); +lean_ctor_set(x_150, 0, x_104); +return x_150; } else { -lean_object* x_129; lean_object* x_130; -x_129 = lean_ctor_get(x_126, 1); -lean_inc(x_129); -lean_dec(x_126); -x_130 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_130, 0, x_92); -lean_ctor_set(x_130, 1, x_129); -return x_130; +lean_object* x_153; lean_object* x_154; +x_153 = lean_ctor_get(x_150, 1); +lean_inc(x_153); +lean_dec(x_150); +x_154 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_154, 0, x_104); +lean_ctor_set(x_154, 1, x_153); +return x_154; } } else { -uint8_t x_131; -lean_dec(x_97); -lean_dec(x_92); +uint8_t x_155; +lean_dec(x_109); +lean_dec(x_104); lean_dec(x_35); lean_dec(x_30); lean_dec(x_28); lean_dec(x_3); -x_131 = !lean_is_exclusive(x_123); -if (x_131 == 0) +x_155 = !lean_is_exclusive(x_147); +if (x_155 == 0) { -return x_123; +return x_147; } else { -lean_object* x_132; lean_object* x_133; lean_object* x_134; -x_132 = lean_ctor_get(x_123, 0); -x_133 = lean_ctor_get(x_123, 1); -lean_inc(x_133); -lean_inc(x_132); -lean_dec(x_123); -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; +lean_object* x_156; lean_object* x_157; lean_object* x_158; +x_156 = lean_ctor_get(x_147, 0); +x_157 = lean_ctor_get(x_147, 1); +lean_inc(x_157); +lean_inc(x_156); +lean_dec(x_147); +x_158 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_158, 0, x_156); +lean_ctor_set(x_158, 1, x_157); +return x_158; +} } } } @@ -28451,330 +28565,373 @@ return x_134; } else { -uint8_t x_142; -lean_dec(x_97); -lean_dec(x_92); +uint8_t x_166; +lean_dec(x_109); +lean_dec(x_104); lean_dec(x_35); lean_dec(x_30); lean_dec(x_28); lean_dec(x_20); lean_dec(x_3); -x_142 = !lean_is_exclusive(x_102); -if (x_142 == 0) +x_166 = !lean_is_exclusive(x_114); +if (x_166 == 0) { -return x_102; +return x_114; } else { -lean_object* x_143; lean_object* x_144; lean_object* x_145; -x_143 = lean_ctor_get(x_102, 0); -x_144 = lean_ctor_get(x_102, 1); -lean_inc(x_144); -lean_inc(x_143); -lean_dec(x_102); -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_object* x_167; lean_object* x_168; lean_object* x_169; +x_167 = lean_ctor_get(x_114, 0); +x_168 = lean_ctor_get(x_114, 1); +lean_inc(x_168); +lean_inc(x_167); +lean_dec(x_114); +x_169 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_169, 0, x_167); +lean_ctor_set(x_169, 1, x_168); +return x_169; } } } } 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; 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_227; lean_object* x_228; lean_object* x_279; -x_160 = lean_ctor_get(x_26, 0); -x_161 = lean_ctor_get(x_26, 1); -x_162 = lean_ctor_get(x_26, 2); -x_163 = lean_ctor_get(x_26, 3); -x_164 = lean_ctor_get(x_26, 4); -x_165 = lean_ctor_get(x_26, 5); -x_166 = lean_ctor_get(x_26, 6); -x_167 = lean_ctor_get(x_26, 7); -lean_inc(x_167); -lean_inc(x_166); -lean_inc(x_165); -lean_inc(x_164); -lean_inc(x_163); -lean_inc(x_162); -lean_inc(x_161); -lean_inc(x_160); +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_262; lean_object* x_263; lean_object* x_325; +x_184 = lean_ctor_get(x_26, 0); +x_185 = lean_ctor_get(x_26, 1); +x_186 = lean_ctor_get(x_26, 2); +x_187 = lean_ctor_get(x_26, 3); +x_188 = lean_ctor_get(x_26, 4); +x_189 = lean_ctor_get(x_26, 5); +x_190 = lean_ctor_get(x_26, 6); +x_191 = lean_ctor_get(x_26, 7); +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_inc(x_184); lean_dec(x_26); -x_168 = l___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___rarg___closed__4; -x_169 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_169, 0, x_160); -lean_ctor_set(x_169, 1, x_168); -lean_ctor_set(x_169, 2, x_162); -lean_ctor_set(x_169, 3, x_163); -lean_ctor_set(x_169, 4, x_164); -lean_ctor_set(x_169, 5, x_165); -lean_ctor_set(x_169, 6, x_166); -lean_ctor_set(x_169, 7, x_167); -x_170 = lean_st_ref_set(x_3, x_169, x_27); -x_171 = lean_ctor_get(x_170, 1); -lean_inc(x_171); -lean_dec(x_170); -x_172 = l_Lean_Elab_getResetInfoTrees___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__3___rarg(x_3, x_171); -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_192 = l___private_Lean_Elab_Command_0__Lean_Elab_Command_runCore___rarg___closed__4; +x_193 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_193, 0, x_184); +lean_ctor_set(x_193, 1, x_192); +lean_ctor_set(x_193, 2, x_186); +lean_ctor_set(x_193, 3, x_187); +lean_ctor_set(x_193, 4, x_188); +lean_ctor_set(x_193, 5, x_189); +lean_ctor_set(x_193, 6, x_190); +lean_ctor_set(x_193, 7, x_191); +x_194 = lean_st_ref_set(x_3, x_193, x_27); +x_195 = lean_ctor_get(x_194, 1); +lean_inc(x_195); +lean_dec(x_194); +x_196 = l_Lean_Elab_getResetInfoTrees___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__3___rarg(x_3, x_195); +x_197 = lean_ctor_get(x_196, 0); +lean_inc(x_197); +x_198 = lean_ctor_get(x_196, 1); +lean_inc(x_198); +lean_dec(x_196); lean_inc(x_3); lean_inc(x_28); lean_inc(x_1); -x_279 = l_Lean_Elab_Command_elabCommand(x_1, x_28, x_3, x_174); -if (lean_obj_tag(x_279) == 0) -{ -lean_object* x_280; lean_object* x_281; lean_object* x_282; -x_280 = lean_ctor_get(x_279, 1); -lean_inc(x_280); -lean_dec(x_279); -x_281 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__3___closed__1; +x_325 = l_Lean_Elab_Command_elabCommand(x_1, x_28, x_3, x_198); +if (lean_obj_tag(x_325) == 0) +{ +lean_object* x_326; lean_object* x_327; lean_object* x_328; +x_326 = lean_ctor_get(x_325, 1); +lean_inc(x_326); +lean_dec(x_325); +x_327 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__3___closed__1; lean_inc(x_1); -x_282 = l_Lean_Syntax_findAux(x_281, x_1); -if (lean_obj_tag(x_282) == 0) +x_328 = l_Lean_Syntax_findAux(x_327, x_1); +if (lean_obj_tag(x_328) == 0) { -lean_object* x_283; lean_object* x_284; -x_283 = lean_alloc_closure((void*)(l_Lean_Elab_Command_runLinters), 4, 1); -lean_closure_set(x_283, 0, x_1); +lean_object* x_329; lean_object* x_330; +x_329 = lean_alloc_closure((void*)(l_Lean_Elab_Command_runLinters), 4, 1); +lean_closure_set(x_329, 0, x_1); lean_inc(x_3); lean_inc(x_28); -x_284 = l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(x_283, x_28, x_3, x_280); -if (lean_obj_tag(x_284) == 0) +x_330 = l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(x_329, x_28, x_3, x_326); +if (lean_obj_tag(x_330) == 0) { -lean_object* x_285; lean_object* x_286; -x_285 = lean_ctor_get(x_284, 0); -lean_inc(x_285); -x_286 = lean_ctor_get(x_284, 1); -lean_inc(x_286); -lean_dec(x_284); -x_175 = x_285; -x_176 = x_286; -goto block_226; +lean_object* x_331; lean_object* x_332; +x_331 = lean_ctor_get(x_330, 0); +lean_inc(x_331); +x_332 = lean_ctor_get(x_330, 1); +lean_inc(x_332); +lean_dec(x_330); +x_199 = x_331; +x_200 = x_332; +goto block_261; } else { -lean_object* x_287; lean_object* x_288; -x_287 = lean_ctor_get(x_284, 0); -lean_inc(x_287); -x_288 = lean_ctor_get(x_284, 1); -lean_inc(x_288); -lean_dec(x_284); -x_227 = x_287; -x_228 = x_288; -goto block_278; +lean_object* x_333; lean_object* x_334; +x_333 = lean_ctor_get(x_330, 0); +lean_inc(x_333); +x_334 = lean_ctor_get(x_330, 1); +lean_inc(x_334); +lean_dec(x_330); +x_262 = x_333; +x_263 = x_334; +goto block_324; } } else { -lean_object* x_289; -lean_dec(x_282); +lean_object* x_335; +lean_dec(x_328); lean_dec(x_1); -x_289 = lean_box(0); -x_175 = x_289; -x_176 = x_280; -goto block_226; +x_335 = lean_box(0); +x_199 = x_335; +x_200 = x_326; +goto block_261; } } else { -lean_object* x_290; lean_object* x_291; +lean_object* x_336; lean_object* x_337; lean_dec(x_1); -x_290 = lean_ctor_get(x_279, 0); -lean_inc(x_290); -x_291 = lean_ctor_get(x_279, 1); -lean_inc(x_291); -lean_dec(x_279); -x_227 = x_290; -x_228 = x_291; -goto block_278; -} -block_226: -{ -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; -x_177 = lean_st_ref_get(x_3, x_176); -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_180 = lean_ctor_get(x_178, 1); -lean_inc(x_180); -lean_dec(x_178); -x_181 = l_Lean_Elab_getInfoTrees___at_Lean_Elab_Command_elabCommandTopLevel___spec__1___rarg(x_3, x_179); -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_box(0); -x_185 = l_Lean_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel___spec__3(x_182, x_184, x_28, x_3, x_183); -lean_dec(x_182); -if (lean_obj_tag(x_185) == 0) +x_336 = lean_ctor_get(x_325, 0); +lean_inc(x_336); +x_337 = lean_ctor_get(x_325, 1); +lean_inc(x_337); +lean_dec(x_325); +x_262 = x_336; +x_263 = x_337; +goto block_324; +} +block_261: +{ +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; +x_201 = lean_st_ref_get(x_3, x_200); +x_202 = lean_ctor_get(x_201, 0); +lean_inc(x_202); +x_203 = lean_ctor_get(x_201, 1); +lean_inc(x_203); +lean_dec(x_201); +x_204 = lean_ctor_get(x_202, 1); +lean_inc(x_204); +lean_dec(x_202); +x_205 = l_Lean_Elab_getInfoTrees___at_Lean_Elab_Command_elabCommandTopLevel___spec__1___rarg(x_3, x_203); +x_206 = lean_ctor_get(x_205, 0); +lean_inc(x_206); +x_207 = lean_ctor_get(x_205, 1); +lean_inc(x_207); +lean_dec(x_205); +x_208 = lean_box(0); +x_209 = l_Lean_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel___spec__3(x_206, x_208, x_28, x_3, x_207); +lean_dec(x_206); +if (lean_obj_tag(x_209) == 0) +{ +lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; uint8_t x_214; +x_210 = lean_ctor_get(x_209, 1); +lean_inc(x_210); +lean_dec(x_209); +x_211 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_4859____closed__5; +x_212 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Command_runLinters___spec__11(x_211, x_28, x_3, x_210); +x_213 = lean_ctor_get(x_212, 0); +lean_inc(x_213); +x_214 = lean_unbox(x_213); +lean_dec(x_213); +if (x_214 == 0) +{ +lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; +lean_dec(x_20); +x_215 = lean_ctor_get(x_212, 1); +lean_inc(x_215); +lean_dec(x_212); +x_216 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_185, x_204, x_197, x_208, x_28, x_3, x_215); +lean_dec(x_3); +x_217 = lean_ctor_get(x_216, 1); +lean_inc(x_217); +if (lean_is_exclusive(x_216)) { + lean_ctor_release(x_216, 0); + lean_ctor_release(x_216, 1); + x_218 = x_216; +} else { + lean_dec_ref(x_216); + x_218 = lean_box(0); +} +if (lean_is_scalar(x_218)) { + x_219 = lean_alloc_ctor(0, 2, 0); +} else { + x_219 = x_218; +} +lean_ctor_set(x_219, 0, x_199); +lean_ctor_set(x_219, 1, x_217); +return x_219; +} +else { if (lean_obj_tag(x_20) == 0) { -lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; -x_186 = lean_ctor_get(x_185, 1); -lean_inc(x_186); -lean_dec(x_185); -x_187 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_161, x_180, x_173, x_184, x_28, x_3, x_186); +lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; +x_220 = lean_ctor_get(x_212, 1); +lean_inc(x_220); +lean_dec(x_212); +x_221 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_185, x_204, x_197, x_208, x_28, x_3, x_220); lean_dec(x_3); -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; +x_222 = lean_ctor_get(x_221, 1); +lean_inc(x_222); +if (lean_is_exclusive(x_221)) { + lean_ctor_release(x_221, 0); + lean_ctor_release(x_221, 1); + x_223 = x_221; } else { - lean_dec_ref(x_187); - x_189 = lean_box(0); + lean_dec_ref(x_221); + x_223 = lean_box(0); } -if (lean_is_scalar(x_189)) { - x_190 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_223)) { + x_224 = lean_alloc_ctor(0, 2, 0); } else { - x_190 = x_189; + x_224 = x_223; } -lean_ctor_set(x_190, 0, x_175); -lean_ctor_set(x_190, 1, x_188); -return x_190; +lean_ctor_set(x_224, 0, x_199); +lean_ctor_set(x_224, 1, x_222); +return x_224; } else { -lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; uint8_t x_195; lean_object* x_196; lean_object* x_216; lean_object* x_217; -x_191 = lean_ctor_get(x_185, 1); -lean_inc(x_191); -lean_dec(x_185); -x_192 = lean_ctor_get(x_20, 0); -lean_inc(x_192); +lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; uint8_t x_229; lean_object* x_230; lean_object* x_251; lean_object* x_252; +x_225 = lean_ctor_get(x_212, 1); +lean_inc(x_225); +lean_dec(x_212); +x_226 = lean_ctor_get(x_20, 0); +lean_inc(x_226); lean_dec(x_20); -x_193 = lean_ctor_get(x_192, 1); -lean_inc(x_193); -lean_dec(x_192); -x_194 = lean_io_promise_result(x_193); -x_216 = lean_io_get_task_state(x_194, x_191); -x_217 = lean_ctor_get(x_216, 0); -lean_inc(x_217); -if (lean_obj_tag(x_217) == 2) +x_227 = lean_ctor_get(x_226, 1); +lean_inc(x_227); +lean_dec(x_226); +x_228 = lean_io_promise_result(x_227); +x_251 = lean_io_get_task_state(x_228, x_225); +x_252 = lean_ctor_get(x_251, 0); +lean_inc(x_252); +if (lean_obj_tag(x_252) == 2) { -lean_object* x_218; uint8_t x_219; -x_218 = lean_ctor_get(x_216, 1); -lean_inc(x_218); -lean_dec(x_216); -x_219 = 1; -x_195 = x_219; -x_196 = x_218; -goto block_215; +lean_object* x_253; uint8_t x_254; +x_253 = lean_ctor_get(x_251, 1); +lean_inc(x_253); +lean_dec(x_251); +x_254 = 1; +x_229 = x_254; +x_230 = x_253; +goto block_250; } else { -lean_object* x_220; uint8_t x_221; -lean_dec(x_217); -x_220 = lean_ctor_get(x_216, 1); -lean_inc(x_220); -lean_dec(x_216); -x_221 = 0; -x_195 = x_221; -x_196 = x_220; -goto block_215; +lean_object* x_255; uint8_t x_256; +lean_dec(x_252); +x_255 = lean_ctor_get(x_251, 1); +lean_inc(x_255); +lean_dec(x_251); +x_256 = 0; +x_229 = x_256; +x_230 = x_255; +goto block_250; } -block_215: +block_250: { -if (x_195 == 0) +if (x_229 == 0) { -lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; -lean_dec(x_194); -x_197 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_161, x_180, x_173, x_184, x_28, x_3, x_196); +lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; +lean_dec(x_228); +x_231 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_185, x_204, x_197, x_208, x_28, x_3, x_230); lean_dec(x_3); -x_198 = lean_ctor_get(x_197, 1); -lean_inc(x_198); -if (lean_is_exclusive(x_197)) { - lean_ctor_release(x_197, 0); - lean_ctor_release(x_197, 1); - x_199 = x_197; +x_232 = lean_ctor_get(x_231, 1); +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_197); - x_199 = lean_box(0); + lean_dec_ref(x_231); + x_233 = lean_box(0); } -if (lean_is_scalar(x_199)) { - x_200 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_233)) { + x_234 = lean_alloc_ctor(0, 2, 0); } else { - x_200 = x_199; + x_234 = x_233; } -lean_ctor_set(x_200, 0, x_175); -lean_ctor_set(x_200, 1, x_198); -return x_200; +lean_ctor_set(x_234, 0, x_199); +lean_ctor_set(x_234, 1, x_232); +return x_234; } else { -lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; -x_201 = lean_task_get_own(x_194); -x_202 = lean_ctor_get(x_201, 1); -lean_inc(x_202); -lean_dec(x_201); -x_203 = lean_alloc_closure((void*)(l_Lean_Language_SnapshotTree_trace), 4, 1); -lean_closure_set(x_203, 0, x_202); -x_204 = l_Lean_Elab_Command_liftCoreM___rarg(x_203, x_28, x_3, x_196); -if (lean_obj_tag(x_204) == 0) -{ -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_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_Elab_Command_elabCommandTopLevel___lambda__1(x_161, x_180, x_173, x_205, x_28, x_3, x_206); +lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; +x_235 = lean_task_get_own(x_228); +x_236 = lean_ctor_get(x_235, 1); +lean_inc(x_236); +lean_dec(x_235); +x_237 = lean_thunk_get_own(x_236); +lean_dec(x_236); +x_238 = lean_alloc_closure((void*)(l_Lean_Language_SnapshotTree_trace), 4, 1); +lean_closure_set(x_238, 0, x_237); +x_239 = l_Lean_Elab_Command_liftCoreM___rarg(x_238, x_28, x_3, x_230); +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; +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_Elab_Command_elabCommandTopLevel___lambda__1(x_185, x_204, x_197, x_240, x_28, x_3, x_241); lean_dec(x_3); -lean_dec(x_205); -x_208 = lean_ctor_get(x_207, 1); -lean_inc(x_208); -if (lean_is_exclusive(x_207)) { - lean_ctor_release(x_207, 0); - lean_ctor_release(x_207, 1); - x_209 = x_207; +lean_dec(x_240); +x_243 = lean_ctor_get(x_242, 1); +lean_inc(x_243); +if (lean_is_exclusive(x_242)) { + lean_ctor_release(x_242, 0); + lean_ctor_release(x_242, 1); + x_244 = x_242; } else { - lean_dec_ref(x_207); - x_209 = lean_box(0); + lean_dec_ref(x_242); + x_244 = lean_box(0); } -if (lean_is_scalar(x_209)) { - x_210 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_244)) { + x_245 = lean_alloc_ctor(0, 2, 0); } else { - x_210 = x_209; + x_245 = x_244; } -lean_ctor_set(x_210, 0, x_175); -lean_ctor_set(x_210, 1, x_208); -return x_210; +lean_ctor_set(x_245, 0, x_199); +lean_ctor_set(x_245, 1, x_243); +return x_245; } else { -lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; -lean_dec(x_180); -lean_dec(x_175); -lean_dec(x_173); -lean_dec(x_161); +lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; +lean_dec(x_204); +lean_dec(x_199); +lean_dec(x_197); +lean_dec(x_185); lean_dec(x_28); lean_dec(x_3); -x_211 = lean_ctor_get(x_204, 0); -lean_inc(x_211); -x_212 = lean_ctor_get(x_204, 1); -lean_inc(x_212); -if (lean_is_exclusive(x_204)) { - lean_ctor_release(x_204, 0); - lean_ctor_release(x_204, 1); - x_213 = x_204; +x_246 = lean_ctor_get(x_239, 0); +lean_inc(x_246); +x_247 = lean_ctor_get(x_239, 1); +lean_inc(x_247); +if (lean_is_exclusive(x_239)) { + lean_ctor_release(x_239, 0); + lean_ctor_release(x_239, 1); + x_248 = x_239; } else { - lean_dec_ref(x_204); - x_213 = lean_box(0); + lean_dec_ref(x_239); + x_248 = lean_box(0); } -if (lean_is_scalar(x_213)) { - x_214 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_248)) { + x_249 = lean_alloc_ctor(1, 2, 0); } else { - x_214 = x_213; + x_249 = x_248; +} +lean_ctor_set(x_249, 0, x_246); +lean_ctor_set(x_249, 1, x_247); +return x_249; } -lean_ctor_set(x_214, 0, x_211); -lean_ctor_set(x_214, 1, x_212); -return x_214; } } } @@ -28782,224 +28939,268 @@ return x_214; } else { -lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; -lean_dec(x_180); -lean_dec(x_175); -lean_dec(x_173); -lean_dec(x_161); +lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; +lean_dec(x_204); +lean_dec(x_199); +lean_dec(x_197); +lean_dec(x_185); lean_dec(x_28); lean_dec(x_20); lean_dec(x_3); -x_222 = lean_ctor_get(x_185, 0); -lean_inc(x_222); -x_223 = lean_ctor_get(x_185, 1); -lean_inc(x_223); -if (lean_is_exclusive(x_185)) { - lean_ctor_release(x_185, 0); - lean_ctor_release(x_185, 1); - x_224 = x_185; +x_257 = lean_ctor_get(x_209, 0); +lean_inc(x_257); +x_258 = lean_ctor_get(x_209, 1); +lean_inc(x_258); +if (lean_is_exclusive(x_209)) { + lean_ctor_release(x_209, 0); + lean_ctor_release(x_209, 1); + x_259 = x_209; } else { - lean_dec_ref(x_185); - x_224 = lean_box(0); + lean_dec_ref(x_209); + x_259 = lean_box(0); } -if (lean_is_scalar(x_224)) { - x_225 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_259)) { + x_260 = lean_alloc_ctor(1, 2, 0); } else { - x_225 = x_224; + x_260 = x_259; } -lean_ctor_set(x_225, 0, x_222); -lean_ctor_set(x_225, 1, x_223); -return x_225; +lean_ctor_set(x_260, 0, x_257); +lean_ctor_set(x_260, 1, x_258); +return x_260; } } -block_278: +block_324: { -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_229 = lean_st_ref_get(x_3, x_228); -x_230 = lean_ctor_get(x_229, 0); -lean_inc(x_230); -x_231 = lean_ctor_get(x_229, 1); -lean_inc(x_231); -lean_dec(x_229); -x_232 = lean_ctor_get(x_230, 1); -lean_inc(x_232); -lean_dec(x_230); -x_233 = l_Lean_Elab_getInfoTrees___at_Lean_Elab_Command_elabCommandTopLevel___spec__1___rarg(x_3, 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); -lean_dec(x_233); -x_236 = lean_box(0); -x_237 = l_Lean_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel___spec__3(x_234, x_236, x_28, x_3, x_235); -lean_dec(x_234); -if (lean_obj_tag(x_237) == 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; lean_object* x_270; lean_object* x_271; lean_object* x_272; +x_264 = lean_st_ref_get(x_3, x_263); +x_265 = lean_ctor_get(x_264, 0); +lean_inc(x_265); +x_266 = lean_ctor_get(x_264, 1); +lean_inc(x_266); +lean_dec(x_264); +x_267 = lean_ctor_get(x_265, 1); +lean_inc(x_267); +lean_dec(x_265); +x_268 = l_Lean_Elab_getInfoTrees___at_Lean_Elab_Command_elabCommandTopLevel___spec__1___rarg(x_3, x_266); +x_269 = lean_ctor_get(x_268, 0); +lean_inc(x_269); +x_270 = lean_ctor_get(x_268, 1); +lean_inc(x_270); +lean_dec(x_268); +x_271 = lean_box(0); +x_272 = l_Lean_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel___spec__3(x_269, x_271, x_28, x_3, x_270); +lean_dec(x_269); +if (lean_obj_tag(x_272) == 0) +{ +lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; uint8_t x_277; +x_273 = lean_ctor_get(x_272, 1); +lean_inc(x_273); +lean_dec(x_272); +x_274 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_4859____closed__5; +x_275 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Command_runLinters___spec__11(x_274, x_28, x_3, x_273); +x_276 = lean_ctor_get(x_275, 0); +lean_inc(x_276); +x_277 = lean_unbox(x_276); +lean_dec(x_276); +if (x_277 == 0) +{ +lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; +lean_dec(x_20); +x_278 = lean_ctor_get(x_275, 1); +lean_inc(x_278); +lean_dec(x_275); +x_279 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_185, x_267, x_197, x_271, x_28, x_3, x_278); +lean_dec(x_3); +x_280 = lean_ctor_get(x_279, 1); +lean_inc(x_280); +if (lean_is_exclusive(x_279)) { + lean_ctor_release(x_279, 0); + lean_ctor_release(x_279, 1); + x_281 = x_279; +} else { + lean_dec_ref(x_279); + x_281 = lean_box(0); +} +if (lean_is_scalar(x_281)) { + x_282 = lean_alloc_ctor(1, 2, 0); +} else { + x_282 = x_281; + lean_ctor_set_tag(x_282, 1); +} +lean_ctor_set(x_282, 0, x_262); +lean_ctor_set(x_282, 1, x_280); +return x_282; +} +else { if (lean_obj_tag(x_20) == 0) { -lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; -x_238 = lean_ctor_get(x_237, 1); -lean_inc(x_238); -lean_dec(x_237); -x_239 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_161, x_232, x_173, x_236, x_28, x_3, x_238); +lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; +x_283 = lean_ctor_get(x_275, 1); +lean_inc(x_283); +lean_dec(x_275); +x_284 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_185, x_267, x_197, x_271, x_28, x_3, x_283); lean_dec(x_3); -x_240 = lean_ctor_get(x_239, 1); -lean_inc(x_240); -if (lean_is_exclusive(x_239)) { - lean_ctor_release(x_239, 0); - lean_ctor_release(x_239, 1); - x_241 = x_239; +x_285 = lean_ctor_get(x_284, 1); +lean_inc(x_285); +if (lean_is_exclusive(x_284)) { + lean_ctor_release(x_284, 0); + lean_ctor_release(x_284, 1); + x_286 = x_284; } else { - lean_dec_ref(x_239); - x_241 = lean_box(0); + lean_dec_ref(x_284); + x_286 = lean_box(0); } -if (lean_is_scalar(x_241)) { - x_242 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_286)) { + x_287 = lean_alloc_ctor(1, 2, 0); } else { - x_242 = x_241; - lean_ctor_set_tag(x_242, 1); + x_287 = x_286; + lean_ctor_set_tag(x_287, 1); } -lean_ctor_set(x_242, 0, x_227); -lean_ctor_set(x_242, 1, x_240); -return x_242; +lean_ctor_set(x_287, 0, x_262); +lean_ctor_set(x_287, 1, x_285); +return x_287; } else { -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_268; lean_object* x_269; -x_243 = lean_ctor_get(x_237, 1); -lean_inc(x_243); -lean_dec(x_237); -x_244 = lean_ctor_get(x_20, 0); -lean_inc(x_244); +lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; uint8_t x_292; lean_object* x_293; lean_object* x_314; lean_object* x_315; +x_288 = lean_ctor_get(x_275, 1); +lean_inc(x_288); +lean_dec(x_275); +x_289 = lean_ctor_get(x_20, 0); +lean_inc(x_289); lean_dec(x_20); -x_245 = lean_ctor_get(x_244, 1); -lean_inc(x_245); -lean_dec(x_244); -x_246 = lean_io_promise_result(x_245); -x_268 = lean_io_get_task_state(x_246, x_243); -x_269 = lean_ctor_get(x_268, 0); -lean_inc(x_269); -if (lean_obj_tag(x_269) == 2) -{ -lean_object* x_270; uint8_t x_271; -x_270 = lean_ctor_get(x_268, 1); -lean_inc(x_270); -lean_dec(x_268); -x_271 = 1; -x_247 = x_271; -x_248 = x_270; -goto block_267; +x_290 = lean_ctor_get(x_289, 1); +lean_inc(x_290); +lean_dec(x_289); +x_291 = lean_io_promise_result(x_290); +x_314 = lean_io_get_task_state(x_291, x_288); +x_315 = lean_ctor_get(x_314, 0); +lean_inc(x_315); +if (lean_obj_tag(x_315) == 2) +{ +lean_object* x_316; uint8_t x_317; +x_316 = lean_ctor_get(x_314, 1); +lean_inc(x_316); +lean_dec(x_314); +x_317 = 1; +x_292 = x_317; +x_293 = x_316; +goto block_313; } else { -lean_object* x_272; uint8_t x_273; -lean_dec(x_269); -x_272 = lean_ctor_get(x_268, 1); -lean_inc(x_272); -lean_dec(x_268); -x_273 = 0; -x_247 = x_273; -x_248 = x_272; -goto block_267; +lean_object* x_318; uint8_t x_319; +lean_dec(x_315); +x_318 = lean_ctor_get(x_314, 1); +lean_inc(x_318); +lean_dec(x_314); +x_319 = 0; +x_292 = x_319; +x_293 = x_318; +goto block_313; } -block_267: +block_313: { -if (x_247 == 0) +if (x_292 == 0) { -lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; -lean_dec(x_246); -x_249 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_161, x_232, x_173, x_236, x_28, x_3, x_248); +lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; +lean_dec(x_291); +x_294 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_185, x_267, x_197, x_271, x_28, x_3, x_293); lean_dec(x_3); -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; +x_295 = lean_ctor_get(x_294, 1); +lean_inc(x_295); +if (lean_is_exclusive(x_294)) { + lean_ctor_release(x_294, 0); + lean_ctor_release(x_294, 1); + x_296 = x_294; } else { - lean_dec_ref(x_249); - x_251 = lean_box(0); + lean_dec_ref(x_294); + x_296 = lean_box(0); } -if (lean_is_scalar(x_251)) { - x_252 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_296)) { + x_297 = lean_alloc_ctor(1, 2, 0); } else { - x_252 = x_251; - lean_ctor_set_tag(x_252, 1); + x_297 = x_296; + lean_ctor_set_tag(x_297, 1); } -lean_ctor_set(x_252, 0, x_227); -lean_ctor_set(x_252, 1, x_250); -return x_252; +lean_ctor_set(x_297, 0, x_262); +lean_ctor_set(x_297, 1, x_295); +return x_297; } else { -lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; -x_253 = lean_task_get_own(x_246); -x_254 = lean_ctor_get(x_253, 1); -lean_inc(x_254); -lean_dec(x_253); -x_255 = lean_alloc_closure((void*)(l_Lean_Language_SnapshotTree_trace), 4, 1); -lean_closure_set(x_255, 0, x_254); -x_256 = l_Lean_Elab_Command_liftCoreM___rarg(x_255, x_28, x_3, x_248); -if (lean_obj_tag(x_256) == 0) -{ -lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; -x_257 = lean_ctor_get(x_256, 0); -lean_inc(x_257); -x_258 = lean_ctor_get(x_256, 1); -lean_inc(x_258); -lean_dec(x_256); -x_259 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_161, x_232, x_173, x_257, x_28, x_3, x_258); +lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; +x_298 = lean_task_get_own(x_291); +x_299 = lean_ctor_get(x_298, 1); +lean_inc(x_299); +lean_dec(x_298); +x_300 = lean_thunk_get_own(x_299); +lean_dec(x_299); +x_301 = lean_alloc_closure((void*)(l_Lean_Language_SnapshotTree_trace), 4, 1); +lean_closure_set(x_301, 0, x_300); +x_302 = l_Lean_Elab_Command_liftCoreM___rarg(x_301, x_28, x_3, x_293); +if (lean_obj_tag(x_302) == 0) +{ +lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; +x_303 = lean_ctor_get(x_302, 0); +lean_inc(x_303); +x_304 = lean_ctor_get(x_302, 1); +lean_inc(x_304); +lean_dec(x_302); +x_305 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__1(x_185, x_267, x_197, x_303, x_28, x_3, x_304); lean_dec(x_3); -lean_dec(x_257); -x_260 = lean_ctor_get(x_259, 1); -lean_inc(x_260); -if (lean_is_exclusive(x_259)) { - lean_ctor_release(x_259, 0); - lean_ctor_release(x_259, 1); - x_261 = x_259; +lean_dec(x_303); +x_306 = lean_ctor_get(x_305, 1); +lean_inc(x_306); +if (lean_is_exclusive(x_305)) { + lean_ctor_release(x_305, 0); + lean_ctor_release(x_305, 1); + x_307 = x_305; } else { - lean_dec_ref(x_259); - x_261 = lean_box(0); + lean_dec_ref(x_305); + x_307 = lean_box(0); } -if (lean_is_scalar(x_261)) { - x_262 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_307)) { + x_308 = lean_alloc_ctor(1, 2, 0); } else { - x_262 = x_261; - lean_ctor_set_tag(x_262, 1); + x_308 = x_307; + lean_ctor_set_tag(x_308, 1); } -lean_ctor_set(x_262, 0, x_227); -lean_ctor_set(x_262, 1, x_260); -return x_262; +lean_ctor_set(x_308, 0, x_262); +lean_ctor_set(x_308, 1, x_306); +return x_308; } else { -lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; -lean_dec(x_232); -lean_dec(x_227); -lean_dec(x_173); -lean_dec(x_161); +lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; +lean_dec(x_267); +lean_dec(x_262); +lean_dec(x_197); +lean_dec(x_185); lean_dec(x_28); lean_dec(x_3); -x_263 = lean_ctor_get(x_256, 0); -lean_inc(x_263); -x_264 = lean_ctor_get(x_256, 1); -lean_inc(x_264); -if (lean_is_exclusive(x_256)) { - lean_ctor_release(x_256, 0); - lean_ctor_release(x_256, 1); - x_265 = x_256; +x_309 = lean_ctor_get(x_302, 0); +lean_inc(x_309); +x_310 = lean_ctor_get(x_302, 1); +lean_inc(x_310); +if (lean_is_exclusive(x_302)) { + lean_ctor_release(x_302, 0); + lean_ctor_release(x_302, 1); + x_311 = x_302; } else { - lean_dec_ref(x_256); - x_265 = lean_box(0); + lean_dec_ref(x_302); + x_311 = lean_box(0); } -if (lean_is_scalar(x_265)) { - x_266 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_311)) { + x_312 = lean_alloc_ctor(1, 2, 0); } else { - x_266 = x_265; + x_312 = x_311; +} +lean_ctor_set(x_312, 0, x_309); +lean_ctor_set(x_312, 1, x_310); +return x_312; } -lean_ctor_set(x_266, 0, x_263); -lean_ctor_set(x_266, 1, x_264); -return x_266; } } } @@ -29007,34 +29208,34 @@ return x_266; } else { -lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; -lean_dec(x_232); -lean_dec(x_227); -lean_dec(x_173); -lean_dec(x_161); +lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; +lean_dec(x_267); +lean_dec(x_262); +lean_dec(x_197); +lean_dec(x_185); lean_dec(x_28); lean_dec(x_20); lean_dec(x_3); -x_274 = lean_ctor_get(x_237, 0); -lean_inc(x_274); -x_275 = lean_ctor_get(x_237, 1); -lean_inc(x_275); -if (lean_is_exclusive(x_237)) { - lean_ctor_release(x_237, 0); - lean_ctor_release(x_237, 1); - x_276 = x_237; +x_320 = lean_ctor_get(x_272, 0); +lean_inc(x_320); +x_321 = lean_ctor_get(x_272, 1); +lean_inc(x_321); +if (lean_is_exclusive(x_272)) { + lean_ctor_release(x_272, 0); + lean_ctor_release(x_272, 1); + x_322 = x_272; } else { - lean_dec_ref(x_237); - x_276 = lean_box(0); + lean_dec_ref(x_272); + x_322 = lean_box(0); } -if (lean_is_scalar(x_276)) { - x_277 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_322)) { + x_323 = lean_alloc_ctor(1, 2, 0); } else { - x_277 = x_276; + x_323 = x_322; } -lean_ctor_set(x_277, 0, x_274); -lean_ctor_set(x_277, 1, x_275); -return x_277; +lean_ctor_set(x_323, 0, x_320); +lean_ctor_set(x_323, 1, x_321); +return x_323; } } } @@ -33648,7 +33849,7 @@ static lean_object* _init_l_Lean_Elab_Command_modifyScope___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_Elab_Command_modifyScope___closed__1; x_2 = l_Lean_Elab_Command_modifyScope___closed__2; -x_3 = lean_unsigned_to_nat(689u); +x_3 = lean_unsigned_to_nat(690u); x_4 = lean_unsigned_to_nat(16u); x_5 = l_Lean_Elab_Command_modifyScope___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -37710,7 +37911,7 @@ lean_object* x_10; uint8_t x_11; lean_object* x_12; x_10 = lean_ctor_get(x_9, 1); lean_inc(x_10); lean_dec(x_9); -x_11 = lean_ctor_get_uint8(x_2, sizeof(void*)*2); +x_11 = lean_ctor_get_uint8(x_2, sizeof(void*)*3); lean_inc(x_6); x_12 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Command_expandDeclId___spec__6(x_11, x_1, x_6, x_7, x_10); if (lean_obj_tag(x_12) == 0) @@ -38647,7 +38848,7 @@ lean_inc(x_27); x_28 = lean_ctor_get(x_25, 1); lean_inc(x_28); lean_dec(x_25); -x_29 = lean_ctor_get(x_3, 0); +x_29 = lean_ctor_get(x_3, 1); lean_inc(x_29); lean_dec(x_3); lean_inc(x_27); diff --git a/stage0/stdlib/Lean/Elab/ComputedFields.c b/stage0/stdlib/Lean/Elab/ComputedFields.c index bddfa98091f0..15bf8086e5e1 100644 --- a/stage0/stdlib/Lean/Elab/ComputedFields.c +++ b/stage0/stdlib/Lean/Elab/ComputedFields.c @@ -126,7 +126,6 @@ lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLetDeclImp___rarg(lean static lean_object* l_Lean_Elab_ComputedFields_initFn____x40_Lean_Elab_ComputedFields___hyg_5____closed__2; 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_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_overrideComputedFields___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*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___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_EXPORT lean_object* l_Lean_Meta_whnfEasyCases___at_Lean_Elab_ComputedFields_getComputedFieldValue___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_ComputedFields_overrideComputedFields___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*); @@ -202,7 +201,7 @@ uint8_t l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_ComputedFields_setComputedFields___spec__2___lambda__2___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescope___at_Lean_Elab_ComputedFields_mkImplType___spec__1___rarg___boxed(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_Lean_Meta_withLocalDecls___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +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*); lean_object* l_Lean_Expr_instantiateLevelParams(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Elab_ComputedFields_overrideCasesOn___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* l_Lean_compileDecls(lean_object*, lean_object*, lean_object*, lean_object*); @@ -215,7 +214,6 @@ LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Elab_ComputedFields_setComputedFie static lean_object* l_Lean_Elab_ComputedFields_initFn____x40_Lean_Elab_ComputedFields___hyg_5____closed__9; 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_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___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_Meta_getConfig(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); 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*); uint8_t l_Lean_LocalDecl_isImplementationDetail(lean_object*); @@ -268,7 +266,6 @@ LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_ComputedFields_setComp lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_setEnv___at_Lean_Elab_ComputedFields_overrideCasesOn___spec__10___boxed(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_Lean_Meta_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_ComputedFields_getComputedFieldValue___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_ComputedFields_overrideCasesOn___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*); static lean_object* l_Lean_Elab_ComputedFields_initFn____x40_Lean_Elab_ComputedFields___hyg_5____lambda__1___closed__3; @@ -290,7 +287,6 @@ uint8_t l_Lean_Expr_occurs(lean_object*, lean_object*); static lean_object* l_Lean_setImplementedBy___at_Lean_Elab_ComputedFields_overrideCasesOn___spec__8___closed__1; static lean_object* l_Lean_logAt___at_Lean_Elab_ComputedFields_setComputedFields___spec__2___closed__1; size_t lean_usize_add(size_t, size_t); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__3(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_ComputedFields_overrideCasesOn___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_forallTelescope___at_Lean_Elab_ComputedFields_mkImplType___spec__1___rarg___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); @@ -304,7 +300,6 @@ lean_object* l_Lean_Meta_setInlineAttribute(lean_object*, uint8_t, lean_object*, lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_ComputedFields_getComputedFieldValue___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Compiler_implementedByAttr; -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_setImplementedBy___at_Lean_Elab_ComputedFields_overrideConstructors___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_setEnv___at_Lean_Elab_ComputedFields_overrideCasesOn___spec__10___closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_ComputedFields_validateComputedFields___spec__3(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -316,19 +311,16 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_ComputedFields_ lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_overrideConstructors___spec__4___boxed(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_Meta_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, 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_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_overrideComputedFields___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_nat_add(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_ComputedFields_setComputedFields___spec__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_ComputedFields_mkComputedFieldOverrides___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_ComputedFields_overrideCasesOn(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__4(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_ComputedFields_overrideComputedFields(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Attribute_Builtin_ensureNoArgs___spec__2(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_withLocalDeclsD___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__2(lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Message_0__Lean_beqMessageSeverity____x40_Lean_Message___hyg_106_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_ComputedFields_overrideComputedFields___spec__3(lean_object*, lean_object*, lean_object*, 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_object*, lean_object*, lean_object*, lean_object*); @@ -9507,208 +9499,6 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___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; size_t x_8; size_t x_9; uint8_t x_10; -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 = 1; -x_9 = lean_usize_add(x_2, x_8); -x_10 = !lean_is_exclusive(x_5); -if (x_10 == 0) -{ -lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = lean_ctor_get(x_5, 0); -x_12 = 0; -x_13 = lean_box(x_12); -lean_ctor_set(x_5, 0, x_13); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_11); -lean_ctor_set(x_14, 1, x_5); -x_15 = lean_array_uset(x_7, x_2, x_14); -x_2 = x_9; -x_3 = x_15; -goto _start; -} -else -{ -lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_17 = lean_ctor_get(x_5, 0); -x_18 = lean_ctor_get(x_5, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_5); -x_19 = 0; -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_18); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_17); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_array_uset(x_7, x_2, x_22); -x_2 = x_9; -x_3 = x_23; -goto _start; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5___rarg___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_array_push(x_1, x_5); -x_12 = l_Lean_Meta_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5___rarg(x_2, x_3, x_4, x_11, x_6, x_7, x_8, x_9, x_10); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5___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; uint8_t x_12; -x_10 = lean_array_get_size(x_4); -x_11 = lean_array_get_size(x_1); -x_12 = lean_nat_dec_lt(x_10, x_11); -lean_dec(x_11); -if (x_12 == 0) -{ -lean_object* x_13; -lean_dec(x_10); -lean_dec(x_3); -lean_dec(x_1); -x_13 = lean_apply_6(x_2, x_4, x_5, x_6, x_7, x_8, x_9); -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; -x_14 = lean_array_fget(x_1, x_10); -lean_dec(x_10); -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 0); -lean_inc(x_16); -lean_dec(x_14); -x_17 = lean_ctor_get(x_15, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_dec(x_15); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_19 = lean_apply_6(x_18, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; uint8_t 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 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5___rarg___lambda__1), 10, 4); -lean_closure_set(x_22, 0, x_4); -lean_closure_set(x_22, 1, x_1); -lean_closure_set(x_22, 2, x_2); -lean_closure_set(x_22, 3, x_3); -x_23 = 0; -x_24 = lean_unbox(x_17); -lean_dec(x_17); -x_25 = l_Lean_Meta_withLocalDecl___at_Lean_Meta_GeneralizeTelescope_generalizeTelescopeAux___spec__1___rarg(x_16, x_24, x_20, x_22, x_23, x_5, x_6, x_7, x_8, x_21); -return x_25; -} -else -{ -uint8_t x_26; -lean_dec(x_17); -lean_dec(x_16); -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_19); -if (x_26 == 0) -{ -return x_19; -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_19, 0); -x_28 = lean_ctor_get(x_19, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_19); -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_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5___rarg), 9, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___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) { -_start: -{ -lean_object* x_9; lean_object* x_10; -x_9 = l_List_mapM_loop___at_Lean_Elab_ComputedFields_mkImplType___spec__2___lambda__1___closed__3; -x_10 = l_Lean_Meta_withLocalDecls_loop___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__5___rarg(x_2, x_3, x_1, x_9, x_4, x_5, x_6, x_7, x_8); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__4(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__4___rarg), 8, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___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: -{ -size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_array_size(x_2); -x_10 = 0; -x_11 = l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__3(x_9, x_10, x_2); -x_12 = l_Lean_Meta_withLocalDecls___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__4___rarg(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__2(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDeclsD___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__2___rarg), 8, 0); -return x_2; -} -} LEAN_EXPORT lean_object* l_Lean_Elab_ComputedFields_mkComputedFieldOverrides___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: { @@ -9915,7 +9705,7 @@ lean_closure_set(x_21, 3, x_3); lean_closure_set(x_21, 4, x_17); lean_closure_set(x_21, 5, x_5); x_22 = l_instInhabitedPUnit; -x_23 = l_Lean_Meta_withLocalDeclsD___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__2___rarg(x_22, x_20, x_21, x_6, x_7, x_8, x_9, x_10); +x_23 = l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(x_22, x_20, x_21, x_6, x_7, x_8, x_9, x_10); return x_23; } } @@ -10090,18 +9880,6 @@ x_9 = l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_mkComputedFieldOverri return x_9; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___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_6 = l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_mkComputedFieldOverrides___spec__3(x_4, x_5, x_3); -return x_6; -} -} LEAN_EXPORT lean_object* l_Lean_Elab_ComputedFields_mkComputedFieldOverrides___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: { diff --git a/stage0/stdlib/Lean/Elab/DeclModifiers.c b/stage0/stdlib/Lean/Elab/DeclModifiers.c index 89c360f5591b..c4de9ab6a254 100644 --- a/stage0/stdlib/Lean/Elab/DeclModifiers.c +++ b/stage0/stdlib/Lean/Elab/DeclModifiers.c @@ -33,7 +33,7 @@ static lean_object* l_Lean_Elab_expandOptDocComment_x3f___rarg___closed__1; lean_object* lean_private_to_user_name(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_checkIfShadowingStructureField___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___rarg___lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*); static lean_object* l_Lean_Elab_Modifiers_filterAttrs___closed__1; static lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__7; static lean_object* l_Lean_Elab_instToStringVisibility___closed__2; @@ -42,7 +42,7 @@ lean_object* l_Lean_Syntax_formatStxAux(lean_object*, uint8_t, lean_object*, lea LEAN_EXPORT lean_object* l_Lean_Elab_expandDeclId___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_expandDeclIdCore___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_checkIfShadowingStructureField___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_Lean_Elab_elabModifiers___rarg___lambda__2(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*, uint8_t); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2(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*, uint8_t); static lean_object* l_Lean_Elab_instToFormatModifiers___closed__3; static lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__6; lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); @@ -58,7 +58,6 @@ static lean_object* l_Lean_Elab_applyVisibility___rarg___lambda__2___closed__1; uint8_t lean_usize_dec_eq(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_instToStringModifiers___lambda__1(lean_object*); lean_object* l_Lean_Syntax_getArgs(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___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*); static lean_object* l_Lean_Elab_instToFormatModifiers___closed__9; static lean_object* l_Lean_Elab_mkDeclName___rarg___closed__3; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_expandDeclId___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -97,7 +96,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_checkIfShadowingStructureField___rarg___lam static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___rarg___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_RecKind_noConfusion(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Visibility_toCtorIdx___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___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_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3(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*); uint8_t l_Lean_isReservedName(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Elab_RecKind_toCtorIdx___boxed(lean_object*); @@ -274,7 +273,7 @@ uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Modifiers_filterAttrs___spec__1___boxed(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_Elab_instToFormatModifiers___closed__29; -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___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_forInUnsafe_loop___at_Lean_Elab_checkIfShadowingStructureField___spec__1___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_Lean_Elab_instToFormatModifiers___closed__24; static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___rarg___lambda__1___closed__1; @@ -1175,20 +1174,22 @@ return x_2; static lean_object* _init_l_Lean_Elab_instInhabitedModifiers___closed__2() { _start: { -lean_object* x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; x_1 = lean_box(0); -x_2 = 0; +x_2 = lean_box(0); x_3 = 0; x_4 = 0; -x_5 = l_Lean_Elab_instInhabitedModifiers___closed__1; -x_6 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -lean_ctor_set_uint8(x_6, sizeof(void*)*2, x_2); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 1, x_3); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 2, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 3, x_3); -return x_6; +x_5 = 0; +x_6 = l_Lean_Elab_instInhabitedModifiers___closed__1; +x_7 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_7, 0, x_2); +lean_ctor_set(x_7, 1, x_1); +lean_ctor_set(x_7, 2, x_6); +lean_ctor_set_uint8(x_7, sizeof(void*)*3, x_3); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 1, x_4); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 2, x_5); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 3, x_4); +return x_7; } } static lean_object* _init_l_Lean_Elab_instInhabitedModifiers() { @@ -1203,7 +1204,7 @@ LEAN_EXPORT uint8_t l_Lean_Elab_Modifiers_isPrivate(lean_object* x_1) { _start: { uint8_t x_2; lean_object* x_3; -x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); +x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); x_3 = lean_box(x_2); if (lean_obj_tag(x_3) == 2) { @@ -1234,7 +1235,7 @@ LEAN_EXPORT uint8_t l_Lean_Elab_Modifiers_isProtected(lean_object* x_1) { _start: { uint8_t x_2; lean_object* x_3; -x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); +x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); x_3 = lean_box(x_2); if (lean_obj_tag(x_3) == 1) { @@ -1265,7 +1266,7 @@ LEAN_EXPORT uint8_t l_Lean_Elab_Modifiers_isPartial(lean_object* x_1) { _start: { uint8_t x_2; lean_object* x_3; -x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 2); +x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 2); x_3 = lean_box(x_2); if (lean_obj_tag(x_3) == 0) { @@ -1296,7 +1297,7 @@ LEAN_EXPORT uint8_t l_Lean_Elab_Modifiers_isNonrec(lean_object* x_1) { _start: { uint8_t x_2; lean_object* x_3; -x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 2); +x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 2); x_3 = lean_box(x_2); if (lean_obj_tag(x_3) == 1) { @@ -1331,32 +1332,35 @@ x_3 = !lean_is_exclusive(x_1); if (x_3 == 0) { lean_object* x_4; lean_object* x_5; -x_4 = lean_ctor_get(x_1, 1); +x_4 = lean_ctor_get(x_1, 2); x_5 = lean_array_push(x_4, x_2); -lean_ctor_set(x_1, 1, x_5); +lean_ctor_set(x_1, 2, x_5); return x_1; } else { -lean_object* x_6; uint8_t 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_6; lean_object* x_7; uint8_t x_8; uint8_t x_9; uint8_t x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_6 = lean_ctor_get(x_1, 0); -x_7 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); -x_8 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); -x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 2); -x_10 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); -x_11 = lean_ctor_get(x_1, 1); -lean_inc(x_11); +x_7 = lean_ctor_get(x_1, 1); +x_8 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); +x_10 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 2); +x_11 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); +x_12 = lean_ctor_get(x_1, 2); +lean_inc(x_12); +lean_inc(x_7); lean_inc(x_6); lean_dec(x_1); -x_12 = lean_array_push(x_11, x_2); -x_13 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_13, 0, x_6); -lean_ctor_set(x_13, 1, x_12); -lean_ctor_set_uint8(x_13, sizeof(void*)*2, x_7); -lean_ctor_set_uint8(x_13, sizeof(void*)*2 + 1, x_8); -lean_ctor_set_uint8(x_13, sizeof(void*)*2 + 2, x_9); -lean_ctor_set_uint8(x_13, sizeof(void*)*2 + 3, x_10); -return x_13; +x_13 = lean_array_push(x_12, x_2); +x_14 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_14, 0, x_6); +lean_ctor_set(x_14, 1, x_7); +lean_ctor_set(x_14, 2, x_13); +lean_ctor_set_uint8(x_14, sizeof(void*)*3, x_8); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 1, x_9); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 2, x_10); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 3, x_11); +return x_14; } } } @@ -1415,7 +1419,7 @@ x_3 = !lean_is_exclusive(x_1); if (x_3 == 0) { lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; -x_4 = lean_ctor_get(x_1, 1); +x_4 = lean_ctor_get(x_1, 2); x_5 = lean_array_get_size(x_4); x_6 = lean_unsigned_to_nat(0u); x_7 = lean_nat_dec_lt(x_6, x_5); @@ -1426,7 +1430,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); x_8 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; -lean_ctor_set(x_1, 1, x_8); +lean_ctor_set(x_1, 2, x_8); return x_1; } else @@ -1440,7 +1444,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); x_10 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; -lean_ctor_set(x_1, 1, x_10); +lean_ctor_set(x_1, 2, x_10); return x_1; } else @@ -1452,79 +1456,84 @@ lean_dec(x_5); x_13 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; x_14 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Modifiers_filterAttrs___spec__1(x_2, x_4, x_11, x_12, x_13); lean_dec(x_4); -lean_ctor_set(x_1, 1, x_14); +lean_ctor_set(x_1, 2, x_14); return x_1; } } } else { -lean_object* x_15; uint8_t 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; uint8_t x_23; +lean_object* x_15; lean_object* x_16; uint8_t x_17; uint8_t x_18; uint8_t x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; x_15 = lean_ctor_get(x_1, 0); -x_16 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); -x_17 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); -x_18 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 2); -x_19 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); -x_20 = lean_ctor_get(x_1, 1); -lean_inc(x_20); +x_16 = lean_ctor_get(x_1, 1); +x_17 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); +x_18 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); +x_19 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 2); +x_20 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); +x_21 = lean_ctor_get(x_1, 2); +lean_inc(x_21); +lean_inc(x_16); lean_inc(x_15); lean_dec(x_1); -x_21 = lean_array_get_size(x_20); -x_22 = lean_unsigned_to_nat(0u); -x_23 = lean_nat_dec_lt(x_22, x_21); -if (x_23 == 0) +x_22 = lean_array_get_size(x_21); +x_23 = lean_unsigned_to_nat(0u); +x_24 = lean_nat_dec_lt(x_23, x_22); +if (x_24 == 0) { -lean_object* x_24; lean_object* x_25; +lean_object* x_25; lean_object* x_26; +lean_dec(x_22); lean_dec(x_21); -lean_dec(x_20); lean_dec(x_2); -x_24 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; -x_25 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_25, 0, x_15); -lean_ctor_set(x_25, 1, x_24); -lean_ctor_set_uint8(x_25, sizeof(void*)*2, x_16); -lean_ctor_set_uint8(x_25, sizeof(void*)*2 + 1, x_17); -lean_ctor_set_uint8(x_25, sizeof(void*)*2 + 2, x_18); -lean_ctor_set_uint8(x_25, sizeof(void*)*2 + 3, x_19); -return x_25; +x_25 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; +x_26 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_26, 0, x_15); +lean_ctor_set(x_26, 1, x_16); +lean_ctor_set(x_26, 2, x_25); +lean_ctor_set_uint8(x_26, sizeof(void*)*3, x_17); +lean_ctor_set_uint8(x_26, sizeof(void*)*3 + 1, x_18); +lean_ctor_set_uint8(x_26, sizeof(void*)*3 + 2, x_19); +lean_ctor_set_uint8(x_26, sizeof(void*)*3 + 3, x_20); +return x_26; } else { -uint8_t x_26; -x_26 = lean_nat_dec_le(x_21, x_21); -if (x_26 == 0) +uint8_t x_27; +x_27 = lean_nat_dec_le(x_22, x_22); +if (x_27 == 0) { -lean_object* x_27; lean_object* x_28; +lean_object* x_28; lean_object* x_29; +lean_dec(x_22); lean_dec(x_21); -lean_dec(x_20); lean_dec(x_2); -x_27 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; -x_28 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_28, 0, x_15); -lean_ctor_set(x_28, 1, x_27); -lean_ctor_set_uint8(x_28, sizeof(void*)*2, x_16); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 1, x_17); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 2, x_18); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 3, x_19); -return x_28; +x_28 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; +x_29 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_29, 0, x_15); +lean_ctor_set(x_29, 1, x_16); +lean_ctor_set(x_29, 2, x_28); +lean_ctor_set_uint8(x_29, sizeof(void*)*3, x_17); +lean_ctor_set_uint8(x_29, sizeof(void*)*3 + 1, x_18); +lean_ctor_set_uint8(x_29, sizeof(void*)*3 + 2, x_19); +lean_ctor_set_uint8(x_29, sizeof(void*)*3 + 3, x_20); +return x_29; } else { -size_t x_29; size_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_29 = 0; -x_30 = lean_usize_of_nat(x_21); +size_t x_30; size_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_30 = 0; +x_31 = lean_usize_of_nat(x_22); +lean_dec(x_22); +x_32 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; +x_33 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Modifiers_filterAttrs___spec__1(x_2, x_21, x_30, x_31, x_32); lean_dec(x_21); -x_31 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; -x_32 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Modifiers_filterAttrs___spec__1(x_2, x_20, x_29, x_30, x_31); -lean_dec(x_20); -x_33 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_33, 0, x_15); -lean_ctor_set(x_33, 1, x_32); -lean_ctor_set_uint8(x_33, sizeof(void*)*2, x_16); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 1, x_17); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 2, x_18); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 3, x_19); -return x_33; +x_34 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_34, 0, x_15); +lean_ctor_set(x_34, 1, x_16); +lean_ctor_set(x_34, 2, x_33); +lean_ctor_set_uint8(x_34, sizeof(void*)*3, x_17); +lean_ctor_set_uint8(x_34, sizeof(void*)*3 + 1, x_18); +lean_ctor_set_uint8(x_34, sizeof(void*)*3 + 2, x_19); +lean_ctor_set_uint8(x_34, sizeof(void*)*3 + 3, x_20); +return x_34; } } } @@ -2055,13 +2064,13 @@ LEAN_EXPORT lean_object* l_Lean_Elab_instToFormatModifiers(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; uint8_t 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; -x_2 = lean_ctor_get(x_1, 0); +x_2 = lean_ctor_get(x_1, 1); lean_inc(x_2); -x_3 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); -x_4 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); -x_5 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 2); -x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); -x_7 = lean_ctor_get(x_1, 1); +x_3 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); +x_4 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); +x_5 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 2); +x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); +x_7 = lean_ctor_get(x_1, 2); lean_inc(x_7); lean_dec(x_1); x_8 = lean_array_to_list(x_7); @@ -2267,13 +2276,13 @@ LEAN_EXPORT lean_object* l_Lean_Elab_instToStringModifiers___lambda__2(lean_obje _start: { lean_object* x_2; uint8_t x_3; uint8_t 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; -x_2 = lean_ctor_get(x_1, 0); +x_2 = lean_ctor_get(x_1, 1); lean_inc(x_2); -x_3 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); -x_4 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); -x_5 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 2); -x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); -x_7 = lean_ctor_get(x_1, 1); +x_3 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); +x_4 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); +x_5 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 2); +x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); +x_7 = lean_ctor_get(x_1, 2); lean_inc(x_7); lean_dec(x_1); x_8 = lean_array_to_list(x_7); @@ -2662,102 +2671,108 @@ lean_dec(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__1(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_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___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, uint8_t x_7, lean_object* x_8) { _start: { -lean_object* x_8; lean_object* x_9; uint8_t x_10; uint8_t x_11; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); -lean_dec(x_1); -x_9 = lean_ctor_get(x_8, 1); +lean_object* x_9; lean_object* x_10; uint8_t x_11; uint8_t x_12; +x_9 = lean_ctor_get(x_1, 0); lean_inc(x_9); -lean_dec(x_8); -x_10 = l_Lean_Syntax_isNone(x_2); -x_11 = l_Lean_Syntax_isNone(x_3); -if (x_10 == 0) -{ +lean_dec(x_1); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = l_Lean_Syntax_isNone(x_2); +x_12 = l_Lean_Syntax_isNone(x_3); if (x_11 == 0) { -uint8_t x_12; lean_object* x_13; lean_object* x_14; -x_12 = 1; -x_13 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_13, 0, x_4); -lean_ctor_set(x_13, 1, x_7); -lean_ctor_set_uint8(x_13, sizeof(void*)*2, x_5); -lean_ctor_set_uint8(x_13, sizeof(void*)*2 + 1, x_12); -lean_ctor_set_uint8(x_13, sizeof(void*)*2 + 2, x_6); -lean_ctor_set_uint8(x_13, sizeof(void*)*2 + 3, x_12); -x_14 = lean_apply_2(x_9, lean_box(0), x_13); -return x_14; +if (x_12 == 0) +{ +uint8_t x_13; lean_object* x_14; lean_object* x_15; +x_13 = 1; +x_14 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_14, 0, x_4); +lean_ctor_set(x_14, 1, x_5); +lean_ctor_set(x_14, 2, x_8); +lean_ctor_set_uint8(x_14, sizeof(void*)*3, x_6); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 1, x_13); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 2, x_7); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 3, x_13); +x_15 = lean_apply_2(x_10, lean_box(0), x_14); +return x_15; } else { -uint8_t x_15; uint8_t x_16; lean_object* x_17; lean_object* x_18; -x_15 = 1; -x_16 = 0; -x_17 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_17, 0, x_4); -lean_ctor_set(x_17, 1, x_7); -lean_ctor_set_uint8(x_17, sizeof(void*)*2, x_5); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 1, x_15); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 2, x_6); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 3, x_16); -x_18 = lean_apply_2(x_9, lean_box(0), x_17); -return x_18; +uint8_t x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; +x_16 = 1; +x_17 = 0; +x_18 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_18, 0, x_4); +lean_ctor_set(x_18, 1, x_5); +lean_ctor_set(x_18, 2, x_8); +lean_ctor_set_uint8(x_18, sizeof(void*)*3, x_6); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 1, x_16); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 2, x_7); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 3, x_17); +x_19 = lean_apply_2(x_10, lean_box(0), x_18); +return x_19; } } else { -if (x_11 == 0) +if (x_12 == 0) { -uint8_t x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; -x_19 = 0; -x_20 = 1; -x_21 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_21, 0, x_4); -lean_ctor_set(x_21, 1, x_7); -lean_ctor_set_uint8(x_21, sizeof(void*)*2, x_5); -lean_ctor_set_uint8(x_21, sizeof(void*)*2 + 1, x_19); -lean_ctor_set_uint8(x_21, sizeof(void*)*2 + 2, x_6); -lean_ctor_set_uint8(x_21, sizeof(void*)*2 + 3, x_20); -x_22 = lean_apply_2(x_9, lean_box(0), x_21); -return x_22; +uint8_t x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; +x_20 = 0; +x_21 = 1; +x_22 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_22, 0, x_4); +lean_ctor_set(x_22, 1, x_5); +lean_ctor_set(x_22, 2, x_8); +lean_ctor_set_uint8(x_22, sizeof(void*)*3, x_6); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 1, x_20); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 2, x_7); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 3, x_21); +x_23 = lean_apply_2(x_10, lean_box(0), x_22); +return x_23; } else { -uint8_t x_23; lean_object* x_24; lean_object* x_25; -x_23 = 0; -x_24 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_24, 0, x_4); -lean_ctor_set(x_24, 1, x_7); -lean_ctor_set_uint8(x_24, sizeof(void*)*2, x_5); -lean_ctor_set_uint8(x_24, sizeof(void*)*2 + 1, x_23); -lean_ctor_set_uint8(x_24, sizeof(void*)*2 + 2, x_6); -lean_ctor_set_uint8(x_24, sizeof(void*)*2 + 3, x_23); -x_25 = lean_apply_2(x_9, lean_box(0), x_24); -return x_25; +uint8_t x_24; lean_object* x_25; lean_object* x_26; +x_24 = 0; +x_25 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_25, 0, x_4); +lean_ctor_set(x_25, 1, x_5); +lean_ctor_set(x_25, 2, x_8); +lean_ctor_set_uint8(x_25, sizeof(void*)*3, x_6); +lean_ctor_set_uint8(x_25, sizeof(void*)*3 + 1, x_24); +lean_ctor_set_uint8(x_25, sizeof(void*)*3 + 2, x_7); +lean_ctor_set_uint8(x_25, sizeof(void*)*3 + 3, x_24); +x_26 = lean_apply_2(x_10, lean_box(0), x_25); +return x_26; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2(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, 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) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2(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, uint8_t x_18) { _start: { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_18 = lean_box(x_17); -x_19 = lean_box(x_5); +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_19 = lean_box(x_18); +x_20 = lean_box(x_6); lean_inc(x_1); -x_20 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___lambda__1___boxed), 7, 6); -lean_closure_set(x_20, 0, x_1); -lean_closure_set(x_20, 1, x_2); -lean_closure_set(x_20, 2, x_3); -lean_closure_set(x_20, 3, x_4); -lean_closure_set(x_20, 4, x_18); -lean_closure_set(x_20, 5, x_19); -x_21 = l_Lean_Syntax_getOptional_x3f(x_6); -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; +x_21 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___lambda__1___boxed), 8, 7); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, x_2); +lean_closure_set(x_21, 2, x_3); +lean_closure_set(x_21, 3, x_4); +lean_closure_set(x_21, 4, x_5); +lean_closure_set(x_21, 5, x_19); +lean_closure_set(x_21, 6, x_20); +x_22 = l_Lean_Syntax_getOptional_x3f(x_7); +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_dec(x_17); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); @@ -2767,32 +2782,31 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); -x_22 = lean_ctor_get(x_1, 1); -lean_inc(x_22); -x_23 = lean_ctor_get(x_1, 0); +x_23 = lean_ctor_get(x_1, 1); lean_inc(x_23); -lean_dec(x_1); -x_24 = lean_ctor_get(x_23, 1); +x_24 = lean_ctor_get(x_1, 0); lean_inc(x_24); -lean_dec(x_23); -x_25 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; -x_26 = lean_apply_2(x_24, lean_box(0), x_25); -x_27 = lean_apply_4(x_22, lean_box(0), lean_box(0), x_26, x_20); -return x_27; +lean_dec(x_1); +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = l_Lean_Elab_Modifiers_filterAttrs___closed__1; +x_27 = lean_apply_2(x_25, lean_box(0), x_26); +x_28 = lean_apply_4(x_23, lean_box(0), lean_box(0), x_27, x_21); +return x_28; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_28 = lean_ctor_get(x_21, 0); -lean_inc(x_28); -lean_dec(x_21); -x_29 = lean_ctor_get(x_1, 1); +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_29 = lean_ctor_get(x_22, 0); lean_inc(x_29); -x_30 = l_Lean_Elab_elabDeclAttrs___rarg(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_28); -lean_dec(x_28); -x_31 = lean_apply_4(x_29, lean_box(0), lean_box(0), x_30, x_20); -return x_31; +lean_dec(x_22); +x_30 = lean_ctor_get(x_1, 1); +lean_inc(x_30); +x_31 = l_Lean_Elab_elabDeclAttrs___rarg(x_1, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_29); +lean_dec(x_29); +x_32 = lean_apply_4(x_30, lean_box(0), lean_box(0), x_31, x_21); +return x_32; } } } @@ -2861,114 +2875,115 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___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, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___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, 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_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_box(x_4); -lean_inc(x_8); +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_box(x_5); +lean_inc(x_9); lean_inc(x_1); -x_19 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___lambda__2___boxed), 17, 16); -lean_closure_set(x_19, 0, x_1); -lean_closure_set(x_19, 1, x_2); -lean_closure_set(x_19, 2, x_3); -lean_closure_set(x_19, 3, x_17); -lean_closure_set(x_19, 4, x_18); -lean_closure_set(x_19, 5, x_5); -lean_closure_set(x_19, 6, x_6); -lean_closure_set(x_19, 7, x_7); -lean_closure_set(x_19, 8, x_8); -lean_closure_set(x_19, 9, x_9); -lean_closure_set(x_19, 10, x_10); -lean_closure_set(x_19, 11, x_11); -lean_closure_set(x_19, 12, x_12); -lean_closure_set(x_19, 13, x_13); -lean_closure_set(x_19, 14, x_14); -lean_closure_set(x_19, 15, x_15); -x_20 = l_Lean_Syntax_getOptional_x3f(x_16); -if (lean_obj_tag(x_20) == 0) -{ -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_dec(x_8); -x_21 = lean_ctor_get(x_1, 1); -lean_inc(x_21); -x_22 = lean_ctor_get(x_1, 0); +x_20 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___lambda__2___boxed), 18, 17); +lean_closure_set(x_20, 0, x_1); +lean_closure_set(x_20, 1, x_2); +lean_closure_set(x_20, 2, x_3); +lean_closure_set(x_20, 3, x_4); +lean_closure_set(x_20, 4, x_18); +lean_closure_set(x_20, 5, x_19); +lean_closure_set(x_20, 6, x_6); +lean_closure_set(x_20, 7, x_7); +lean_closure_set(x_20, 8, x_8); +lean_closure_set(x_20, 9, x_9); +lean_closure_set(x_20, 10, x_10); +lean_closure_set(x_20, 11, x_11); +lean_closure_set(x_20, 12, x_12); +lean_closure_set(x_20, 13, x_13); +lean_closure_set(x_20, 14, x_14); +lean_closure_set(x_20, 15, x_15); +lean_closure_set(x_20, 16, x_16); +x_21 = l_Lean_Syntax_getOptional_x3f(x_17); +if (lean_obj_tag(x_21) == 0) +{ +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_dec(x_9); +x_22 = lean_ctor_get(x_1, 1); lean_inc(x_22); -lean_dec(x_1); -x_23 = lean_ctor_get(x_22, 1); +x_23 = lean_ctor_get(x_1, 0); lean_inc(x_23); -lean_dec(x_22); -x_24 = 0; -x_25 = lean_box(x_24); -x_26 = lean_apply_2(x_23, lean_box(0), x_25); -x_27 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_26, x_19); -return x_27; +lean_dec(x_1); +x_24 = lean_ctor_get(x_23, 1); +lean_inc(x_24); +lean_dec(x_23); +x_25 = 0; +x_26 = lean_box(x_25); +x_27 = lean_apply_2(x_24, lean_box(0), x_26); +x_28 = lean_apply_4(x_22, lean_box(0), lean_box(0), x_27, x_20); +return x_28; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; -x_28 = lean_ctor_get(x_20, 0); -lean_inc(x_28); -lean_dec(x_20); -lean_inc(x_28); -x_29 = l_Lean_Syntax_getKind(x_28); -x_30 = l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__4; -x_31 = lean_name_eq(x_29, x_30); -if (x_31 == 0) -{ -lean_object* x_32; uint8_t x_33; -x_32 = l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__5; -x_33 = lean_name_eq(x_29, x_32); -lean_dec(x_29); -if (x_33 == 0) -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_34 = lean_ctor_get(x_1, 1); -lean_inc(x_34); -x_35 = l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__7; -x_36 = l_Lean_throwErrorAt___rarg(x_1, x_8, x_28, x_35); -x_37 = lean_apply_4(x_34, lean_box(0), lean_box(0), x_36, x_19); -return x_37; +lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_29 = lean_ctor_get(x_21, 0); +lean_inc(x_29); +lean_dec(x_21); +lean_inc(x_29); +x_30 = l_Lean_Syntax_getKind(x_29); +x_31 = l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__4; +x_32 = lean_name_eq(x_30, x_31); +if (x_32 == 0) +{ +lean_object* x_33; uint8_t x_34; +x_33 = l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__5; +x_34 = lean_name_eq(x_30, x_33); +lean_dec(x_30); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_35 = lean_ctor_get(x_1, 1); +lean_inc(x_35); +x_36 = l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__7; +x_37 = l_Lean_throwErrorAt___rarg(x_1, x_9, x_29, x_36); +x_38 = lean_apply_4(x_35, lean_box(0), lean_box(0), x_37, x_20); +return x_38; } else { -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_dec(x_28); -lean_dec(x_8); -x_38 = lean_ctor_get(x_1, 1); -lean_inc(x_38); -x_39 = lean_ctor_get(x_1, 0); +lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +lean_dec(x_29); +lean_dec(x_9); +x_39 = lean_ctor_get(x_1, 1); lean_inc(x_39); -lean_dec(x_1); -x_40 = lean_ctor_get(x_39, 1); +x_40 = lean_ctor_get(x_1, 0); lean_inc(x_40); -lean_dec(x_39); -x_41 = 1; -x_42 = lean_box(x_41); -x_43 = lean_apply_2(x_40, lean_box(0), x_42); -x_44 = lean_apply_4(x_38, lean_box(0), lean_box(0), x_43, x_19); -return x_44; +lean_dec(x_1); +x_41 = lean_ctor_get(x_40, 1); +lean_inc(x_41); +lean_dec(x_40); +x_42 = 1; +x_43 = lean_box(x_42); +x_44 = lean_apply_2(x_41, lean_box(0), x_43); +x_45 = lean_apply_4(x_39, lean_box(0), lean_box(0), x_44, x_20); +return x_45; } } else { -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_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_dec(x_30); lean_dec(x_29); -lean_dec(x_28); -lean_dec(x_8); -x_45 = lean_ctor_get(x_1, 1); -lean_inc(x_45); -x_46 = lean_ctor_get(x_1, 0); +lean_dec(x_9); +x_46 = lean_ctor_get(x_1, 1); lean_inc(x_46); -lean_dec(x_1); -x_47 = lean_ctor_get(x_46, 1); +x_47 = lean_ctor_get(x_1, 0); lean_inc(x_47); -lean_dec(x_46); -x_48 = 2; -x_49 = lean_box(x_48); -x_50 = lean_apply_2(x_47, lean_box(0), x_49); -x_51 = lean_apply_4(x_45, lean_box(0), lean_box(0), x_50, x_19); -return x_51; +lean_dec(x_1); +x_48 = lean_ctor_get(x_47, 1); +lean_inc(x_48); +lean_dec(x_47); +x_49 = 2; +x_50 = lean_box(x_49); +x_51 = lean_apply_2(x_48, lean_box(0), x_50); +x_52 = lean_apply_4(x_46, lean_box(0), lean_box(0), x_51, x_20); +return x_52; } } } @@ -3059,23 +3074,24 @@ lean_object* x_28; lean_object* x_29; x_28 = lean_box(x_27); lean_inc(x_4); lean_inc(x_1); -x_29 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___lambda__3___boxed), 17, 16); +x_29 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___lambda__3___boxed), 18, 17); lean_closure_set(x_29, 0, x_1); lean_closure_set(x_29, 1, x_20); lean_closure_set(x_29, 2, x_22); -lean_closure_set(x_29, 3, x_28); -lean_closure_set(x_29, 4, x_16); -lean_closure_set(x_29, 5, x_2); -lean_closure_set(x_29, 6, x_3); -lean_closure_set(x_29, 7, x_4); -lean_closure_set(x_29, 8, x_5); -lean_closure_set(x_29, 9, x_6); -lean_closure_set(x_29, 10, x_7); -lean_closure_set(x_29, 11, x_8); -lean_closure_set(x_29, 12, x_9); -lean_closure_set(x_29, 13, x_10); -lean_closure_set(x_29, 14, x_11); -lean_closure_set(x_29, 15, x_18); +lean_closure_set(x_29, 3, x_12); +lean_closure_set(x_29, 4, x_28); +lean_closure_set(x_29, 5, x_16); +lean_closure_set(x_29, 6, x_2); +lean_closure_set(x_29, 7, x_3); +lean_closure_set(x_29, 8, x_4); +lean_closure_set(x_29, 9, x_5); +lean_closure_set(x_29, 10, x_6); +lean_closure_set(x_29, 11, x_7); +lean_closure_set(x_29, 12, x_8); +lean_closure_set(x_29, 13, x_9); +lean_closure_set(x_29, 14, x_10); +lean_closure_set(x_29, 15, x_11); +lean_closure_set(x_29, 16, x_18); if (lean_obj_tag(x_26) == 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; @@ -3118,22 +3134,22 @@ LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___boxed), 12, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg), 12, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___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_EXPORT lean_object* l_Lean_Elab_elabModifiers___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: { -uint8_t x_8; uint8_t x_9; lean_object* x_10; -x_8 = lean_unbox(x_5); -lean_dec(x_5); +uint8_t x_9; uint8_t x_10; lean_object* x_11; x_9 = lean_unbox(x_6); lean_dec(x_6); -x_10 = l_Lean_Elab_elabModifiers___rarg___lambda__1(x_1, x_2, x_3, x_4, x_8, x_9, x_7); +x_10 = lean_unbox(x_7); +lean_dec(x_7); +x_11 = l_Lean_Elab_elabModifiers___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_9, x_10, x_8); lean_dec(x_3); lean_dec(x_2); -return x_10; +return x_11; } } LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2___boxed(lean_object** _args) { @@ -3154,16 +3170,17 @@ 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_18; uint8_t x_19; lean_object* x_20; -x_18 = lean_unbox(x_5); -lean_dec(x_5); -x_19 = lean_unbox(x_17); -lean_dec(x_17); -x_20 = l_Lean_Elab_elabModifiers___rarg___lambda__2(x_1, x_2, x_3, x_4, x_18, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_19); +uint8_t x_19; uint8_t x_20; lean_object* x_21; +x_19 = lean_unbox(x_6); lean_dec(x_6); -return x_20; +x_20 = lean_unbox(x_18); +lean_dec(x_18); +x_21 = l_Lean_Elab_elabModifiers___rarg___lambda__2(x_1, x_2, x_3, x_4, x_5, x_19, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_20); +lean_dec(x_7); +return x_21; } } LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3___boxed(lean_object** _args) { @@ -3184,23 +3201,15 @@ 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_18; lean_object* x_19; -x_18 = lean_unbox(x_4); -lean_dec(x_4); -x_19 = l_Lean_Elab_elabModifiers___rarg___lambda__3(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_13, x_14, x_15, x_16, x_17); -lean_dec(x_16); -return x_19; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___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) { -_start: -{ -lean_object* x_13; -x_13 = l_Lean_Elab_elabModifiers___rarg(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_12); -return x_13; +uint8_t x_19; lean_object* x_20; +x_19 = lean_unbox(x_5); +lean_dec(x_5); +x_20 = l_Lean_Elab_elabModifiers___rarg___lambda__3(x_1, x_2, x_3, x_4, x_19, 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); +return x_20; } } LEAN_EXPORT lean_object* l_Lean_Elab_applyVisibility___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { @@ -3919,7 +3928,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___rarg___lambda__3(lean_object* _start: { uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); +x_11 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); lean_inc(x_4); lean_inc(x_2); x_12 = l_Lean_Elab_applyVisibility___rarg(x_2, x_3, x_4, x_5, x_11, x_6); @@ -4478,7 +4487,7 @@ lean_inc(x_8); x_9 = lean_ctor_get(x_7, 1); lean_inc(x_9); lean_dec(x_7); -x_10 = lean_ctor_get(x_1, 0); +x_10 = lean_ctor_get(x_1, 1); lean_inc(x_10); lean_dec(x_1); lean_inc(x_8); diff --git a/stage0/stdlib/Lean/Elab/Declaration.c b/stage0/stdlib/Lean/Elab/Declaration.c index d821ce959d6e..a157385d0ba5 100644 --- a/stage0/stdlib/Lean/Elab/Declaration.c +++ b/stage0/stdlib/Lean/Elab/Declaration.c @@ -26,7 +26,6 @@ static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__37; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___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_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDefName___closed__3; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__8; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAttr(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement__1___closed__2; @@ -45,7 +44,6 @@ static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration_declRange__1___closed__2; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___closed__3; lean_object* l_Lean_addDocString_x27___at_Lean_Elab_Command_expandDeclId___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___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___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1(lean_object*); @@ -66,6 +64,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration__1(lea static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__7; static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___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___regBuiltin_Lean_Elab_Command_expandMutualNamespace__1___closed__2; @@ -74,6 +73,7 @@ lean_object* l_Lean_Elab_Command_getLevelNames___rarg(lean_object*, lean_object* LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandMutualPreamble(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getHeadInfo(lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__11; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___closed__5; uint8_t l_Lean_Exception_isInterrupt(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabInitialize__1___closed__1; @@ -92,8 +92,8 @@ LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Command_expandMutualNamespace___ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandMutualElement___spec__1___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___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*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__13; lean_object* l_Lean_Syntax_getId(lean_object*); static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -107,6 +107,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__3; 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_Elab_Command_elabInitialize___lambda__1___closed__48; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6(lean_object*, size_t, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive___boxed(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__2; @@ -129,21 +130,17 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__4___closed__11; 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*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__4; -lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); lean_object* l_Lean_Elab_Command_elabCommand(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration_declRange__1___closed__7; static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__6; -lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__4; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Macro_throwError___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabDeclaration___closed__1; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__17; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_declRange__1___closed__1; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__9; LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_elabMutualInductive(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___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_Elab_Command_elabClassInductive___closed__3; @@ -152,6 +149,7 @@ lean_object* l_Lean_logAt___at_Lean_Elab_Command_runLinters___spec__2(lean_objec lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkIdentFrom(lean_object*, lean_object*, uint8_t); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__13; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__8; lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement_declRange__1(lean_object*); @@ -171,6 +169,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___clo lean_object* l_EStateM_instMonad(lean_object*, lean_object*); uint8_t l_Lean_MapDeclarationExtension_contains___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__12; lean_object* l_List_head_x21___rarg(lean_object*, lean_object*); lean_object* l_Lean_Elab_applyVisibility___at_Lean_Elab_Command_expandDeclId___spec__6(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); @@ -208,7 +207,6 @@ lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialIn static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange__1___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement__1___closed__1; lean_object* l_Lean_Elab_Modifiers_addAttr(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -218,7 +216,6 @@ static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_induc LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; LEAN_EXPORT uint8_t l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___lambda__2(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__3; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5___closed__1; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__6; @@ -227,10 +224,9 @@ lean_object* l_Lean_Elab_Term_ensureNoUnassignedMVars(lean_object*, lean_object* static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace__1___closed__1; lean_object* lean_st_ref_take(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__30; -static lean_object* l_Lean_Elab_Command_expandNamespacedDeclaration___closed__6; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__1; extern lean_object* l_Lean_Elab_Command_commandElabAttribute; -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble__1(lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__3___closed__6; @@ -241,11 +237,13 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declara static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual_declRange__1___closed__1; lean_object* l_Lean_mkPrivateName(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__13; +static lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__7; static lean_object* l_Lean_Elab_Command_elabAttr___closed__1; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___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*); +static lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; uint8_t l_Lean_Elab_Modifiers_isProtected(lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive(lean_object*); lean_object* l_Lean_Syntax_node6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -284,20 +282,19 @@ lean_object* l_Lean_Elab_elabAttrs___at_Lean_Elab_Command_elabMutualDef___spec__ lean_object* l_Lean_Elab_Command_liftTermElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_replacePrefix(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabDeclaration___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabAxiom___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__38; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__2; lean_object* l_Lean_Elab_addBuiltinIncrementalElab(lean_object*, lean_object*); uint8_t l_Lean_Elab_Command_isDefLike(lean_object*); lean_object* l_Lean_Syntax_getOptional_x3f(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__5; lean_object* lean_array_to_list(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement_declRange__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Command_findCommonPrefix_findCommon___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___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*); static lean_object* l_Lean_Elab_Command_elabInitialize___closed__3; -static lean_object* l_Lean_Elab_Command_expandNamespacedDeclaration___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_declRange__1___closed__4; lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); lean_object* l_Lean_Syntax_node3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -305,11 +302,10 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___lambda__2___boxed( LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___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_Command_elabMutual_declRange__1___closed__6; lean_object* l_Lean_Name_append(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__5; static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual_declRange__1___closed__3; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__12; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_declRange__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabAxiom___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__6___closed__2; lean_object* l_Lean_Elab_expandDeclSig(lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__9; @@ -317,7 +313,6 @@ static lean_object* l_Lean_Elab_Command_elabInitialize___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDeclIdName___closed__3; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive___spec__1___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__4; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___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_Elab_Command_getCurrMacroScope(lean_object*, lean_object*, lean_object*); @@ -350,9 +345,11 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandNamespacedDeclaration___boxed static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration_declRange__1___closed__5; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDefName___closed__1; static lean_object* l_panic___at_Lean_Elab_Command_elabAttr___spec__3___closed__1; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__7; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__12; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__19; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__4; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_expandMutualNamespace___spec__3___closed__1; uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); @@ -372,7 +369,6 @@ lean_object* l_Lean_TSyntax_getDocString(lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration_declRange__1___closed__4; static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__2; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__10; extern lean_object* l_Std_Format_defWidth; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_declRange__1___closed__5; lean_object* l_Lean_MacroScopesView_review(lean_object*); @@ -397,7 +393,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_splitMutualPreamble(lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__10; lean_object* l_panic___at_Lean_Parser_SyntaxStack_back___spec__1(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__2; lean_object* l_Lean_Syntax_node4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDeclIdName___closed__4; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_elabMutualInductive___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -421,6 +416,7 @@ static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__6___closed__3; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__32; LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___boxed(lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__9; lean_object* l_Lean_Elab_getOptDerivingClasses(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_expandMutualPreamble___closed__3; static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__6___closed__3; @@ -442,7 +438,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration(lean_object*, lean_ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration__2(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualDef___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabInitialize__1(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__11; static lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandMutualNamespace(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -455,10 +450,11 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declara LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandMutualElement___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_expandNamespacedDeclaration___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace__1___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__31; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___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*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_elabBinders___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -493,7 +489,6 @@ lean_object* l_Lean_throwError___at___private_Lean_Elab_Command_0__Lean_Elab_Com LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ensureNonAmbiguous___at_Lean_Elab_Command_elabAttr___spec__2___closed__4; LEAN_EXPORT lean_object* l_Lean_Linter_logLintIf___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange__1___closed__1; lean_object* l_Lean_Syntax_setInfo(lean_object*, lean_object*); @@ -504,6 +499,8 @@ static lean_object* l_Lean_Elab_Command_expandNamespacedDeclaration___closed__1; lean_object* l_Array_mkArray1___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___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* l_Lean_Elab_Command_liftCoreM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_findCommonPrefix(lean_object*); @@ -515,6 +512,7 @@ lean_object* l_Array_ofSubarray___rarg(lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__3___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___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*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__3; extern lean_object* l_Lean_instInhabitedDeclarationRanges; lean_object* lean_erase_macro_scopes(lean_object*); lean_object* l_List_toString___at_Lean_ensureNoOverload___spec__2(lean_object*); @@ -528,7 +526,6 @@ lean_object* lean_array_mk(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration__1___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__6___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_Lean_Elab_Command_elabInitialize___lambda__1___closed__6; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr__1___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr_declRange__1___closed__6; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__1; @@ -554,7 +551,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration_declRange__1(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration__1___closed__4; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024_(lean_object*); lean_object* l_instInhabitedOfMonad___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___boxed(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedSyntax; @@ -583,6 +579,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_d static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange__1___closed__7; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive___spec__1(lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration_declRange__1(lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__10; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabMutual___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; lean_object* lean_array_get_size(lean_object*); @@ -603,6 +600,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_ static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration_declRange__1___closed__1; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009_(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration_declRange__1___closed__5; static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__3___closed__1; lean_object* lean_nat_add(lean_object*, lean_object*); @@ -633,7 +631,6 @@ uint8_t l_Lean_Elab_Modifiers_isPartial(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInitialize___lambda__1___closed__1; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabInitialize__1___closed__3; lean_object* l_Lean_addDecl(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__10; @@ -642,6 +639,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual__1___closed__1; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__17; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__10; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__6; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__13; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__14; LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_elabAttr___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__3___closed__1; @@ -1659,237 +1657,146 @@ lean_dec(x_2); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabAxiom___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_5; uint8_t x_6; lean_object* x_7; lean_object* x_8; -x_5 = lean_ctor_get(x_2, 1); -lean_inc(x_5); -lean_dec(x_2); -x_6 = 0; -x_7 = l_Lean_Syntax_getPos_x3f(x_1, x_6); -x_8 = l_Lean_Syntax_getTailPos_x3f(x_1, x_6); -if (lean_obj_tag(x_7) == 0) +uint8_t x_5; lean_object* x_6; +x_5 = 0; +x_6 = l_Lean_Syntax_getRange_x3f(x_1, x_5); +if (lean_obj_tag(x_6) == 0) { -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = lean_unsigned_to_nat(0u); -lean_inc(x_5); -x_10 = l_Lean_FileMap_toPosition(x_5, x_9); -lean_inc(x_10); -x_11 = l_Lean_FileMap_leanPosToLspPos(x_5, x_10); -if (lean_obj_tag(x_8) == 0) +lean_object* x_7; lean_object* x_8; +lean_dec(x_2); +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_4); +return x_8; +} +else { -uint8_t x_12; -lean_dec(x_5); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +uint8_t x_9; +x_9 = !lean_is_exclusive(x_6); +if (x_9 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_11, 1); -x_14 = lean_ctor_get(x_11, 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; uint8_t x_17; +x_10 = lean_ctor_get(x_6, 0); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +lean_dec(x_2); +x_12 = lean_ctor_get(x_10, 0); +lean_inc(x_12); +lean_inc(x_11); +x_13 = l_Lean_FileMap_toPosition(x_11, x_12); +lean_dec(x_12); +x_14 = lean_ctor_get(x_10, 1); +lean_inc(x_14); +lean_dec(x_10); +lean_inc(x_11); +x_15 = l_Lean_FileMap_toPosition(x_11, x_14); lean_dec(x_14); lean_inc(x_13); -lean_inc(x_10); -x_15 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_15, 0, x_10); -lean_ctor_set(x_15, 1, x_13); -lean_ctor_set(x_15, 2, x_10); -lean_ctor_set(x_15, 3, x_13); -lean_ctor_set(x_11, 1, x_4); -lean_ctor_set(x_11, 0, x_15); -return x_11; -} -else +x_16 = l_Lean_FileMap_leanPosToLspPos(x_11, x_13); +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) { -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_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_18 = lean_ctor_get(x_16, 1); +x_19 = lean_ctor_get(x_16, 0); +lean_dec(x_19); +lean_inc(x_15); +x_20 = l_Lean_FileMap_leanPosToLspPos(x_11, x_15); lean_dec(x_11); -lean_inc(x_16); -lean_inc(x_10); -x_17 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_17, 0, x_10); -lean_ctor_set(x_17, 1, x_16); -lean_ctor_set(x_17, 2, x_10); -lean_ctor_set(x_17, 3, 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_4); -return x_18; -} +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_22, 0, x_13); +lean_ctor_set(x_22, 1, x_18); +lean_ctor_set(x_22, 2, x_15); +lean_ctor_set(x_22, 3, x_21); +lean_ctor_set(x_6, 0, x_22); +lean_ctor_set(x_16, 1, x_4); +lean_ctor_set(x_16, 0, x_6); +return x_16; } else { -uint8_t x_19; -x_19 = !lean_is_exclusive(x_11); -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; -x_20 = lean_ctor_get(x_11, 1); -x_21 = lean_ctor_get(x_11, 0); -lean_dec(x_21); -x_22 = lean_ctor_get(x_8, 0); -lean_inc(x_22); -lean_dec(x_8); -lean_inc(x_5); -x_23 = l_Lean_FileMap_toPosition(x_5, x_22); -lean_dec(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_16, 1); lean_inc(x_23); -x_24 = l_Lean_FileMap_leanPosToLspPos(x_5, x_23); -lean_dec(x_5); +lean_dec(x_16); +lean_inc(x_15); +x_24 = l_Lean_FileMap_leanPosToLspPos(x_11, x_15); +lean_dec(x_11); x_25 = lean_ctor_get(x_24, 1); lean_inc(x_25); lean_dec(x_24); x_26 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_26, 0, x_10); -lean_ctor_set(x_26, 1, x_20); -lean_ctor_set(x_26, 2, x_23); +lean_ctor_set(x_26, 0, x_13); +lean_ctor_set(x_26, 1, x_23); +lean_ctor_set(x_26, 2, x_15); lean_ctor_set(x_26, 3, x_25); -lean_ctor_set(x_11, 1, x_4); -lean_ctor_set(x_11, 0, x_26); -return x_11; +lean_ctor_set(x_6, 0, x_26); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_6); +lean_ctor_set(x_27, 1, x_4); +return x_27; +} } 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_ctor_get(x_11, 1); -lean_inc(x_27); -lean_dec(x_11); -x_28 = lean_ctor_get(x_8, 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; +x_28 = lean_ctor_get(x_6, 0); lean_inc(x_28); -lean_dec(x_8); -lean_inc(x_5); -x_29 = l_Lean_FileMap_toPosition(x_5, x_28); +lean_dec(x_6); +x_29 = lean_ctor_get(x_2, 1); +lean_inc(x_29); +lean_dec(x_2); +x_30 = lean_ctor_get(x_28, 0); +lean_inc(x_30); +lean_inc(x_29); +x_31 = l_Lean_FileMap_toPosition(x_29, x_30); +lean_dec(x_30); +x_32 = lean_ctor_get(x_28, 1); +lean_inc(x_32); lean_dec(x_28); lean_inc(x_29); -x_30 = l_Lean_FileMap_leanPosToLspPos(x_5, x_29); -lean_dec(x_5); -x_31 = lean_ctor_get(x_30, 1); +x_33 = l_Lean_FileMap_toPosition(x_29, x_32); +lean_dec(x_32); lean_inc(x_31); -lean_dec(x_30); -x_32 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_32, 0, x_10); -lean_ctor_set(x_32, 1, x_27); -lean_ctor_set(x_32, 2, x_29); -lean_ctor_set(x_32, 3, 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_4); -return x_33; -} -} -} -else -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_7, 0); -lean_inc(x_34); -lean_dec(x_7); -lean_inc(x_5); -x_35 = l_Lean_FileMap_toPosition(x_5, x_34); -lean_dec(x_34); -lean_inc(x_35); -x_36 = l_Lean_FileMap_leanPosToLspPos(x_5, x_35); -if (lean_obj_tag(x_8) == 0) -{ -uint8_t x_37; -lean_dec(x_5); -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, 1); -x_39 = lean_ctor_get(x_36, 0); -lean_dec(x_39); -lean_inc(x_38); -lean_inc(x_35); -x_40 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_40, 0, x_35); -lean_ctor_set(x_40, 1, x_38); -lean_ctor_set(x_40, 2, x_35); -lean_ctor_set(x_40, 3, x_38); -lean_ctor_set(x_36, 1, x_4); -lean_ctor_set(x_36, 0, x_40); -return x_36; -} -else -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_36, 1); -lean_inc(x_41); -lean_dec(x_36); -lean_inc(x_41); +x_34 = l_Lean_FileMap_leanPosToLspPos(x_29, x_31); +x_35 = lean_ctor_get(x_34, 1); lean_inc(x_35); -x_42 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_42, 0, x_35); -lean_ctor_set(x_42, 1, x_41); -lean_ctor_set(x_42, 2, x_35); -lean_ctor_set(x_42, 3, 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_4); -return x_43; -} -} -else -{ -uint8_t x_44; -x_44 = !lean_is_exclusive(x_36); -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 = lean_ctor_get(x_36, 1); -x_46 = lean_ctor_get(x_36, 0); -lean_dec(x_46); -x_47 = lean_ctor_get(x_8, 0); -lean_inc(x_47); -lean_dec(x_8); -lean_inc(x_5); -x_48 = l_Lean_FileMap_toPosition(x_5, x_47); -lean_dec(x_47); -lean_inc(x_48); -x_49 = l_Lean_FileMap_leanPosToLspPos(x_5, x_48); -lean_dec(x_5); -x_50 = lean_ctor_get(x_49, 1); -lean_inc(x_50); -lean_dec(x_49); -x_51 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_51, 0, x_35); -lean_ctor_set(x_51, 1, x_45); -lean_ctor_set(x_51, 2, x_48); -lean_ctor_set(x_51, 3, x_50); -lean_ctor_set(x_36, 1, x_4); -lean_ctor_set(x_36, 0, x_51); -return x_36; +if (lean_is_exclusive(x_34)) { + lean_ctor_release(x_34, 0); + lean_ctor_release(x_34, 1); + x_36 = x_34; +} else { + lean_dec_ref(x_34); + x_36 = lean_box(0); } -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; -x_52 = lean_ctor_get(x_36, 1); -lean_inc(x_52); -lean_dec(x_36); -x_53 = lean_ctor_get(x_8, 0); -lean_inc(x_53); -lean_dec(x_8); -lean_inc(x_5); -x_54 = l_Lean_FileMap_toPosition(x_5, x_53); -lean_dec(x_53); -lean_inc(x_54); -x_55 = l_Lean_FileMap_leanPosToLspPos(x_5, x_54); -lean_dec(x_5); -x_56 = lean_ctor_get(x_55, 1); -lean_inc(x_56); -lean_dec(x_55); -x_57 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_57, 0, x_35); -lean_ctor_set(x_57, 1, x_52); -lean_ctor_set(x_57, 2, x_54); -lean_ctor_set(x_57, 3, x_56); -x_58 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_58, 0, x_57); -lean_ctor_set(x_58, 1, x_4); -return x_58; +lean_inc(x_33); +x_37 = l_Lean_FileMap_leanPosToLspPos(x_29, x_33); +lean_dec(x_29); +x_38 = lean_ctor_get(x_37, 1); +lean_inc(x_38); +lean_dec(x_37); +x_39 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_39, 0, x_31); +lean_ctor_set(x_39, 1, x_35); +lean_ctor_set(x_39, 2, x_33); +lean_ctor_set(x_39, 3, x_38); +x_40 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_40, 0, x_39); +if (lean_is_scalar(x_36)) { + x_41 = lean_alloc_ctor(0, 2, 0); +} else { + x_41 = x_36; } +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_4); +return x_41; } } } @@ -2128,98 +2035,198 @@ return x_69; } } } -static lean_object* _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__1() { +static lean_object* _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("example", 7, 7); +x_1 = lean_mk_string_unchecked("null", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__2() { +static lean_object* _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___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_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__1; -x_2 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__2; -x_3 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__3; -x_4 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__1; -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; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__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_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___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) { _start: { -lean_object* x_6; lean_object* x_7; uint8_t x_8; -lean_inc(x_2); -x_6 = l_Lean_Syntax_getKind(x_2); -x_7 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__2; -x_8 = lean_name_eq(x_6, x_7); -lean_dec(x_6); -if (x_8 == 0) -{ -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_inc(x_3); -x_9 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2(x_2, x_3, x_4, x_5); -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_getDeclarationSelectionRef(x_2); -lean_inc(x_3); -x_13 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2(x_12, x_3, x_4, x_11); -lean_dec(x_12); -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 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; +x_8 = lean_box(0); +lean_inc(x_1); +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_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_2); +lean_ctor_set(x_10, 1, x_9); +x_11 = lean_array_mk(x_10); +x_12 = lean_box(2); +x_13 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; +x_14 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +lean_ctor_set(x_14, 2, x_11); +lean_inc(x_5); +x_15 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabAxiom___spec__2(x_14, x_5, x_6, x_7); +lean_dec(x_14); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +if (lean_obj_tag(x_16) == 0) { -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_ctor_set(x_13, 1, x_15); -lean_ctor_set(x_13, 0, x_10); -x_17 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3(x_1, x_13, x_3, x_4, x_16); +uint8_t x_17; +lean_dec(x_5); lean_dec(x_3); -return x_17; +lean_dec(x_1); +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 = lean_box(0); +lean_ctor_set(x_15, 0, x_19); +return x_15; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -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(0, 2, 0); -lean_ctor_set(x_20, 0, x_10); -lean_ctor_set(x_20, 1, x_18); -x_21 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3(x_1, x_20, x_3, x_4, x_19); -lean_dec(x_3); -return x_21; +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_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_22; lean_object* x_23; +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_15, 1); +lean_inc(x_23); +lean_dec(x_15); +x_24 = lean_ctor_get(x_16, 0); +lean_inc(x_24); +lean_dec(x_16); +x_25 = l_Lean_Elab_getDeclarationSelectionRef(x_1); +lean_inc(x_5); +x_26 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabAxiom___spec__2(x_25, x_5, x_6, x_23); +lean_dec(x_25); +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +if (lean_obj_tag(x_27) == 0) +{ +uint8_t x_28; +lean_dec(x_24); +lean_dec(x_5); lean_dec(x_3); -lean_dec(x_2); -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_5); -return x_23; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___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: +x_28 = !lean_is_exclusive(x_26); +if (x_28 == 0) { -lean_object* x_10; -lean_inc(x_3); -x_10 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__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_29; lean_object* x_30; +x_29 = lean_ctor_get(x_26, 0); +lean_dec(x_29); +x_30 = lean_box(0); +lean_ctor_set(x_26, 0, x_30); +return x_26; +} +else +{ +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_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 +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +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_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_24); +lean_ctor_set(x_36, 1, x_35); +x_37 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3(x_3, x_36, x_5, x_6, x_34); +lean_dec(x_5); +return x_37; +} +} +} +} +static lean_object* _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("example", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__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_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__1; +x_2 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__2; +x_3 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__3; +x_4 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___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) { +_start: +{ +lean_object* x_7; lean_object* x_8; uint8_t x_9; +lean_inc(x_3); +x_7 = l_Lean_Syntax_getKind(x_3); +x_8 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__2; +x_9 = lean_name_eq(x_7, x_8); +lean_dec(x_7); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_box(0); +x_11 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1(x_3, x_2, x_1, x_10, x_4, x_5, x_6); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +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_6); +return x_13; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___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_inc(x_3); +x_10 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__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; lean_object* x_14; uint8_t x_15; lean_object* x_16; x_11 = lean_ctor_get(x_10, 0); @@ -2652,7 +2659,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__4(lean_object* _start: { lean_object* x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_1, 1); +x_17 = lean_ctor_get(x_1, 2); lean_inc(x_17); x_18 = 2; lean_inc(x_15); @@ -2803,7 +2810,7 @@ x_62 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_62, 0, x_2); lean_ctor_set(x_62, 1, x_57); lean_ctor_set(x_62, 2, x_60); -x_63 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); +x_63 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); lean_dec(x_1); x_64 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_64, 0, x_62); @@ -2916,7 +2923,7 @@ x_95 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_95, 0, x_2); lean_ctor_set(x_95, 1, x_57); lean_ctor_set(x_95, 2, x_93); -x_96 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); +x_96 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); lean_dec(x_1); x_97 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_97, 0, x_95); @@ -3014,7 +3021,7 @@ x_122 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_122, 0, x_2); lean_ctor_set(x_122, 1, x_117); lean_ctor_set(x_122, 2, x_119); -x_123 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); +x_123 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); lean_dec(x_1); x_124 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_124, 0, x_122); @@ -3173,7 +3180,7 @@ x_162 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_162, 0, x_2); lean_ctor_set(x_162, 1, x_156); lean_ctor_set(x_162, 2, x_159); -x_163 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); +x_163 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); lean_dec(x_1); x_164 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_164, 0, x_162); @@ -3443,7 +3450,7 @@ x_224 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_224, 0, x_2); lean_ctor_set(x_224, 1, x_218); lean_ctor_set(x_224, 2, x_221); -x_225 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); +x_225 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); lean_dec(x_1); x_226 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_226, 0, x_224); @@ -3773,7 +3780,7 @@ lean_inc(x_1); x_16 = l_Lean_Elab_Command_expandDeclId(x_7, x_1, x_3, x_4, 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; lean_object* x_23; lean_object* x_24; +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; x_17 = lean_ctor_get(x_16, 0); lean_inc(x_17); x_18 = lean_ctor_get(x_16, 1); @@ -3784,29 +3791,31 @@ lean_inc(x_19); x_20 = lean_ctor_get(x_17, 2); lean_inc(x_20); lean_dec(x_17); +x_21 = lean_ctor_get(x_1, 0); +lean_inc(x_21); lean_inc(x_3); lean_inc(x_2); lean_inc(x_19); -x_21 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1(x_19, x_2, x_3, x_4, x_18); -x_22 = lean_ctor_get(x_21, 1); -lean_inc(x_22); -lean_dec(x_21); -x_23 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabAxiom___lambda__5___boxed), 16, 8); -lean_closure_set(x_23, 0, x_11); -lean_closure_set(x_23, 1, x_1); -lean_closure_set(x_23, 2, x_19); -lean_closure_set(x_23, 3, x_12); -lean_closure_set(x_23, 4, x_14); -lean_closure_set(x_23, 5, x_20); -lean_closure_set(x_23, 6, x_2); -lean_closure_set(x_23, 7, x_7); -x_24 = l_Lean_Elab_Command_runTermElabM___rarg(x_23, x_3, x_4, x_22); +x_22 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1(x_19, x_21, x_2, x_3, x_4, x_18); +x_23 = lean_ctor_get(x_22, 1); +lean_inc(x_23); +lean_dec(x_22); +x_24 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabAxiom___lambda__5___boxed), 16, 8); +lean_closure_set(x_24, 0, x_11); +lean_closure_set(x_24, 1, x_1); +lean_closure_set(x_24, 2, x_19); +lean_closure_set(x_24, 3, x_12); +lean_closure_set(x_24, 4, x_14); +lean_closure_set(x_24, 5, x_20); +lean_closure_set(x_24, 6, x_2); +lean_closure_set(x_24, 7, x_7); +x_25 = l_Lean_Elab_Command_runTermElabM___rarg(x_24, x_3, x_4, x_23); lean_dec(x_3); -return x_24; +return x_25; } else { -uint8_t x_25; +uint8_t x_26; lean_dec(x_14); lean_dec(x_12); lean_dec(x_11); @@ -3814,32 +3823,32 @@ lean_dec(x_7); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_25 = !lean_is_exclusive(x_16); -if (x_25 == 0) +x_26 = !lean_is_exclusive(x_16); +if (x_26 == 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_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_16, 0); +x_28 = lean_ctor_get(x_16, 1); +lean_inc(x_28); 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; +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_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__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_getDeclarationRange_x3f___at_Lean_Elab_Command_elabAxiom___spec__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_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabAxiom___spec__2(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_1); return x_5; @@ -3855,13 +3864,23 @@ lean_dec(x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__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_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___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) { _start: { -lean_object* x_6; -x_6 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1(x_1, x_2, x_3, x_4, x_5); +lean_object* x_8; +x_8 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_6); lean_dec(x_4); -return x_6; +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___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) { +_start: +{ +lean_object* x_7; +x_7 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_5); +return x_7; } } LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___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) { @@ -3930,7 +3949,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___priva _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_6 = lean_ctor_get(x_1, 1); +x_6 = lean_ctor_get(x_1, 2); x_7 = lean_array_get_size(x_6); x_8 = lean_unsigned_to_nat(0u); x_9 = lean_nat_dec_eq(x_7, x_8); @@ -3975,7 +3994,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___priva _start: { uint8_t x_6; -x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); +x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); if (x_6 == 0) { lean_object* x_7; lean_object* x_8; @@ -4085,7 +4104,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___priva _start: { uint8_t x_5; -x_5 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); +x_5 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); if (x_5 == 0) { lean_object* x_6; lean_object* x_7; @@ -4122,42 +4141,97 @@ return x_13; LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___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_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +lean_object* x_7; lean_object* x_8; lean_inc(x_4); -x_7 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2(x_2, x_4, x_5, x_6); +x_7 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabAxiom___spec__2(x_2, 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); -lean_inc(x_4); -x_10 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2(x_3, x_4, x_5, x_9); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) +if (lean_obj_tag(x_8) == 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_ctor_set(x_10, 1, x_12); -lean_ctor_set(x_10, 0, x_8); -x_14 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3(x_1, x_10, x_4, x_5, x_13); +uint8_t x_9; lean_dec(x_4); +lean_dec(x_1); +x_9 = !lean_is_exclusive(x_7); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_7, 0); +lean_dec(x_10); +x_11 = lean_box(0); +lean_ctor_set(x_7, 0, x_11); +return x_7; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_7, 1); +lean_inc(x_12); +lean_dec(x_7); +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_12); 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_10, 0); -x_16 = lean_ctor_get(x_10, 1); -lean_inc(x_16); +x_15 = lean_ctor_get(x_7, 1); lean_inc(x_15); -lean_dec(x_10); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_8); -lean_ctor_set(x_17, 1, x_15); -x_18 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3(x_1, x_17, x_4, x_5, x_16); +lean_dec(x_7); +x_16 = lean_ctor_get(x_8, 0); +lean_inc(x_16); +lean_dec(x_8); +lean_inc(x_4); +x_17 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Command_elabAxiom___spec__2(x_3, x_4, x_5, x_15); +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_4); -return x_18; +lean_dec(x_1); +x_19 = !lean_is_exclusive(x_17); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_17, 0); +lean_dec(x_20); +x_21 = lean_box(0); +lean_ctor_set(x_17, 0, x_21); +return x_17; +} +else +{ +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_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 +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_25 = lean_ctor_get(x_17, 1); +lean_inc(x_25); +lean_dec(x_17); +x_26 = lean_ctor_get(x_18, 0); +lean_inc(x_26); +lean_dec(x_18); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_16); +lean_ctor_set(x_27, 1, x_26); +x_28 = l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3(x_1, x_27, x_4, x_5, x_25); +lean_dec(x_4); +return x_28; +} } } } @@ -4177,7 +4251,7 @@ x_10 = lean_unsigned_to_nat(3u); x_11 = l_Lean_Syntax_getIdAt(x_2, x_10); x_12 = l_Lean_Name_append(x_3, x_11); x_13 = l_Lean_Syntax_getArg(x_2, x_10); -x_14 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); +x_14 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); x_15 = l_Lean_Elab_Command_getRef(x_5, x_6, x_9); x_16 = lean_ctor_get(x_15, 0); lean_inc(x_16); @@ -4235,7 +4309,7 @@ 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_1, 0); +x_38 = lean_ctor_get(x_1, 1); lean_inc(x_38); lean_inc(x_5); lean_inc(x_31); @@ -4510,41 +4584,47 @@ return x_20; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___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) { _start: { -lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_8 = l_Lean_TSyntax_getDocString(x_1); -x_9 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_9, 0, x_8); -x_10 = !lean_is_exclusive(x_3); -if (x_10 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_3); +if (x_8 == 0) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_3, 0); -lean_dec(x_11); -lean_ctor_set(x_3, 0, x_9); +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = lean_ctor_get(x_3, 1); +lean_dec(x_9); +x_10 = l_Lean_TSyntax_getDocString(x_1); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_ctor_set(x_3, 1, x_11); x_12 = lean_box(0); x_13 = lean_apply_5(x_2, x_3, x_12, x_5, x_6, x_7); return x_13; } else { -uint8_t x_14; uint8_t x_15; uint8_t x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_14 = lean_ctor_get_uint8(x_3, sizeof(void*)*2); -x_15 = lean_ctor_get_uint8(x_3, sizeof(void*)*2 + 1); -x_16 = lean_ctor_get_uint8(x_3, sizeof(void*)*2 + 2); -x_17 = lean_ctor_get_uint8(x_3, sizeof(void*)*2 + 3); -x_18 = lean_ctor_get(x_3, 1); -lean_inc(x_18); +lean_object* x_14; uint8_t x_15; uint8_t x_16; uint8_t 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; +x_14 = lean_ctor_get(x_3, 0); +x_15 = lean_ctor_get_uint8(x_3, sizeof(void*)*3); +x_16 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 1); +x_17 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 2); +x_18 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 3); +x_19 = lean_ctor_get(x_3, 2); +lean_inc(x_19); +lean_inc(x_14); lean_dec(x_3); -x_19 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_19, 0, x_9); -lean_ctor_set(x_19, 1, x_18); -lean_ctor_set_uint8(x_19, sizeof(void*)*2, x_14); -lean_ctor_set_uint8(x_19, sizeof(void*)*2 + 1, x_15); -lean_ctor_set_uint8(x_19, sizeof(void*)*2 + 2, x_16); -lean_ctor_set_uint8(x_19, sizeof(void*)*2 + 3, x_17); -x_20 = lean_box(0); -x_21 = lean_apply_5(x_2, x_19, x_20, x_5, x_6, x_7); -return x_21; +x_20 = l_Lean_TSyntax_getDocString(x_1); +x_21 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_21, 0, x_20); +x_22 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_22, 0, x_14); +lean_ctor_set(x_22, 1, x_21); +lean_ctor_set(x_22, 2, x_19); +lean_ctor_set_uint8(x_22, sizeof(void*)*3, x_15); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 1, x_16); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 2, x_17); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 3, x_18); +x_23 = lean_box(0); +x_24 = lean_apply_5(x_2, x_22, x_23, x_5, x_6, x_7); +return x_24; } } } @@ -4640,7 +4720,6 @@ lean_ctor_set(x_30, 9, x_28); lean_ctor_set_uint8(x_30, sizeof(void*)*10, x_29); lean_inc(x_30); x_31 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_15, x_30, x_7, x_18); -lean_dec(x_15); 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; @@ -4713,7 +4792,7 @@ else { lean_object* x_49; lean_dec(x_11); -x_49 = lean_ctor_get(x_32, 0); +x_49 = lean_ctor_get(x_32, 1); lean_inc(x_49); if (lean_obj_tag(x_49) == 0) { @@ -5219,7 +5298,7 @@ lean_inc(x_1); x_15 = l_Lean_Elab_Command_expandDeclId(x_14, x_1, x_3, x_4, x_7); 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; lean_object* x_23; lean_object* x_24; lean_object* x_25; size_t x_26; size_t x_27; lean_object* x_28; +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; size_t x_27; size_t x_28; lean_object* x_29; x_16 = lean_ctor_get(x_15, 0); lean_inc(x_16); x_17 = lean_ctor_get(x_15, 1); @@ -5232,160 +5311,162 @@ lean_inc(x_19); x_20 = lean_ctor_get(x_16, 2); lean_inc(x_20); lean_dec(x_16); +x_21 = lean_ctor_get(x_1, 0); +lean_inc(x_21); lean_inc(x_3); lean_inc(x_2); lean_inc(x_19); -x_21 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1(x_19, x_2, x_3, x_4, x_17); -x_22 = lean_ctor_get(x_21, 1); -lean_inc(x_22); -lean_dec(x_21); -x_23 = lean_unsigned_to_nat(4u); -x_24 = l_Lean_Syntax_getArg(x_2, x_23); -x_25 = l_Lean_Syntax_getArgs(x_24); -lean_dec(x_24); -x_26 = lean_array_size(x_25); -x_27 = 0; +x_22 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1(x_19, x_21, x_2, x_3, x_4, x_17); +x_23 = lean_ctor_get(x_22, 1); +lean_inc(x_23); +lean_dec(x_22); +x_24 = lean_unsigned_to_nat(4u); +x_25 = l_Lean_Syntax_getArg(x_2, x_24); +x_26 = l_Lean_Syntax_getArgs(x_25); +lean_dec(x_25); +x_27 = lean_array_size(x_26); +x_28 = 0; lean_inc(x_4); lean_inc(x_19); lean_inc(x_1); -x_28 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3(x_1, x_19, x_26, x_27, x_25, x_3, x_4, x_22); -if (lean_obj_tag(x_28) == 0) +x_29 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3(x_1, x_19, x_27, x_28, x_26, x_3, x_4, x_23); +if (lean_obj_tag(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; -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; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_30 = lean_ctor_get(x_29, 0); lean_inc(x_30); -lean_dec(x_28); -x_31 = lean_unsigned_to_nat(5u); -x_32 = l_Lean_Syntax_getArg(x_2, x_31); -x_33 = l_Lean_Syntax_getOptional_x3f(x_32); -lean_dec(x_32); -if (lean_obj_tag(x_33) == 0) +x_31 = lean_ctor_get(x_29, 1); +lean_inc(x_31); +lean_dec(x_29); +x_32 = lean_unsigned_to_nat(5u); +x_33 = l_Lean_Syntax_getArg(x_2, x_32); +x_34 = l_Lean_Syntax_getOptional_x3f(x_33); +lean_dec(x_33); +if (lean_obj_tag(x_34) == 0) { -lean_object* x_80; -x_80 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__4; -x_34 = x_80; -goto block_79; +lean_object* x_81; +x_81 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__4; +x_35 = x_81; +goto block_80; } else { -lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_81 = lean_ctor_get(x_33, 0); -lean_inc(x_81); -lean_dec(x_33); -x_82 = l_Lean_Syntax_getArg(x_81, x_13); -lean_dec(x_81); -x_83 = l_Lean_Syntax_getArgs(x_82); +lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_82 = lean_ctor_get(x_34, 0); +lean_inc(x_82); +lean_dec(x_34); +x_83 = l_Lean_Syntax_getArg(x_82, x_13); lean_dec(x_82); -x_34 = x_83; -goto block_79; +x_84 = l_Lean_Syntax_getArgs(x_83); +lean_dec(x_83); +x_35 = x_84; +goto block_80; } -block_79: +block_80: { -size_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; -x_35 = lean_array_size(x_34); -x_36 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__4(x_35, x_27, x_34, x_3, x_4, x_30); -x_37 = lean_ctor_get(x_36, 0); -lean_inc(x_37); -x_38 = lean_ctor_get(x_36, 1); +size_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; +x_36 = lean_array_size(x_35); +x_37 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__4(x_36, x_28, x_35, x_3, x_4, x_31); +x_38 = lean_ctor_get(x_37, 0); lean_inc(x_38); -lean_dec(x_36); -x_39 = lean_unsigned_to_nat(6u); -x_40 = l_Lean_Syntax_getArg(x_2, x_39); -x_41 = lean_alloc_closure((void*)(l_Lean_Elab_getOptDerivingClasses), 4, 1); -lean_closure_set(x_41, 0, x_40); -x_42 = l_Lean_Elab_Command_liftCoreM___rarg(x_41, x_3, x_4, x_38); -if (lean_obj_tag(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; uint8_t x_50; -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_unsigned_to_nat(3u); -x_46 = l_Lean_Syntax_getArg(x_2, x_45); -x_47 = lean_unsigned_to_nat(0u); -x_48 = l_Lean_Syntax_getArg(x_46, x_47); -x_49 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; -x_50 = l_Lean_Syntax_isToken(x_49, x_48); -lean_dec(x_48); -if (x_50 == 0) -{ -lean_object* x_51; lean_object* x_52; -lean_dec(x_46); -x_51 = lean_box(0); -x_52 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___lambda__1(x_2, x_14, x_1, x_18, x_19, x_20, x_11, x_12, x_29, x_43, x_37, x_51, x_3, x_4, x_44); +x_39 = lean_ctor_get(x_37, 1); +lean_inc(x_39); +lean_dec(x_37); +x_40 = lean_unsigned_to_nat(6u); +x_41 = l_Lean_Syntax_getArg(x_2, x_40); +x_42 = lean_alloc_closure((void*)(l_Lean_Elab_getOptDerivingClasses), 4, 1); +lean_closure_set(x_42, 0, x_41); +x_43 = l_Lean_Elab_Command_liftCoreM___rarg(x_42, x_3, x_4, x_39); +if (lean_obj_tag(x_43) == 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; uint8_t x_51; +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_unsigned_to_nat(3u); +x_47 = l_Lean_Syntax_getArg(x_2, x_46); +x_48 = lean_unsigned_to_nat(0u); +x_49 = l_Lean_Syntax_getArg(x_47, x_48); +x_50 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; +x_51 = l_Lean_Syntax_isToken(x_50, x_49); +lean_dec(x_49); +if (x_51 == 0) +{ +lean_object* x_52; lean_object* x_53; +lean_dec(x_47); +x_52 = lean_box(0); +x_53 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___lambda__1(x_2, x_14, x_1, x_18, x_19, x_20, x_11, x_12, x_30, x_44, x_38, x_52, x_3, x_4, x_45); lean_dec(x_4); lean_dec(x_3); -return x_52; +return x_53; } 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; uint8_t 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_53 = l_Lean_Syntax_getArg(x_2, x_47); -x_54 = l_Lean_Elab_Command_getRef(x_3, x_4, x_44); -x_55 = lean_ctor_get(x_54, 0); -lean_inc(x_55); -x_56 = lean_ctor_get(x_54, 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; 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; +x_54 = l_Lean_Syntax_getArg(x_2, x_48); +x_55 = l_Lean_Elab_Command_getRef(x_3, x_4, x_45); +x_56 = lean_ctor_get(x_55, 0); lean_inc(x_56); -lean_dec(x_54); -x_57 = l_Lean_replaceRef(x_53, x_55); +x_57 = lean_ctor_get(x_55, 1); +lean_inc(x_57); lean_dec(x_55); -lean_dec(x_53); -x_58 = lean_ctor_get(x_3, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_3, 1); +x_58 = l_Lean_replaceRef(x_54, x_56); +lean_dec(x_56); +lean_dec(x_54); +x_59 = lean_ctor_get(x_3, 0); lean_inc(x_59); -x_60 = lean_ctor_get(x_3, 2); +x_60 = lean_ctor_get(x_3, 1); lean_inc(x_60); -x_61 = lean_ctor_get(x_3, 3); +x_61 = lean_ctor_get(x_3, 2); lean_inc(x_61); -x_62 = lean_ctor_get(x_3, 4); +x_62 = lean_ctor_get(x_3, 3); lean_inc(x_62); -x_63 = lean_ctor_get(x_3, 5); +x_63 = lean_ctor_get(x_3, 4); lean_inc(x_63); -x_64 = lean_ctor_get(x_3, 7); +x_64 = lean_ctor_get(x_3, 5); lean_inc(x_64); -x_65 = lean_ctor_get(x_3, 8); +x_65 = lean_ctor_get(x_3, 7); lean_inc(x_65); -x_66 = lean_ctor_get(x_3, 9); +x_66 = lean_ctor_get(x_3, 8); lean_inc(x_66); -x_67 = lean_ctor_get_uint8(x_3, sizeof(void*)*10); -x_68 = lean_alloc_ctor(0, 10, 1); -lean_ctor_set(x_68, 0, x_58); -lean_ctor_set(x_68, 1, x_59); -lean_ctor_set(x_68, 2, x_60); -lean_ctor_set(x_68, 3, x_61); -lean_ctor_set(x_68, 4, x_62); -lean_ctor_set(x_68, 5, x_63); -lean_ctor_set(x_68, 6, x_57); -lean_ctor_set(x_68, 7, x_64); -lean_ctor_set(x_68, 8, x_65); -lean_ctor_set(x_68, 9, x_66); -lean_ctor_set_uint8(x_68, sizeof(void*)*10, x_67); -x_69 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__5; -x_70 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__4; -x_71 = l_Lean_Linter_logLintIf___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5(x_69, x_46, x_70, x_68, x_4, x_56); -lean_dec(x_46); -x_72 = lean_ctor_get(x_71, 0); -lean_inc(x_72); -x_73 = lean_ctor_get(x_71, 1); +x_67 = lean_ctor_get(x_3, 9); +lean_inc(x_67); +x_68 = lean_ctor_get_uint8(x_3, sizeof(void*)*10); +x_69 = lean_alloc_ctor(0, 10, 1); +lean_ctor_set(x_69, 0, x_59); +lean_ctor_set(x_69, 1, x_60); +lean_ctor_set(x_69, 2, x_61); +lean_ctor_set(x_69, 3, x_62); +lean_ctor_set(x_69, 4, x_63); +lean_ctor_set(x_69, 5, x_64); +lean_ctor_set(x_69, 6, x_58); +lean_ctor_set(x_69, 7, x_65); +lean_ctor_set(x_69, 8, x_66); +lean_ctor_set(x_69, 9, x_67); +lean_ctor_set_uint8(x_69, sizeof(void*)*10, x_68); +x_70 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__5; +x_71 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__4; +x_72 = l_Lean_Linter_logLintIf___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__5(x_70, x_47, x_71, x_69, x_4, x_57); +lean_dec(x_47); +x_73 = lean_ctor_get(x_72, 0); lean_inc(x_73); -lean_dec(x_71); -x_74 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___lambda__1(x_2, x_14, x_1, x_18, x_19, x_20, x_11, x_12, x_29, x_43, x_37, x_72, x_3, x_4, x_73); +x_74 = lean_ctor_get(x_72, 1); +lean_inc(x_74); +lean_dec(x_72); +x_75 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___lambda__1(x_2, x_14, x_1, x_18, x_19, x_20, x_11, x_12, x_30, x_44, x_38, x_73, x_3, x_4, x_74); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_72); -return x_74; +lean_dec(x_73); +return x_75; } } else { -uint8_t x_75; -lean_dec(x_37); -lean_dec(x_29); +uint8_t x_76; +lean_dec(x_38); +lean_dec(x_30); lean_dec(x_20); lean_dec(x_19); lean_dec(x_18); @@ -5396,30 +5477,30 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_75 = !lean_is_exclusive(x_42); -if (x_75 == 0) +x_76 = !lean_is_exclusive(x_43); +if (x_76 == 0) { -return x_42; +return x_43; } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_42, 0); -x_77 = lean_ctor_get(x_42, 1); +lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_77 = lean_ctor_get(x_43, 0); +x_78 = lean_ctor_get(x_43, 1); +lean_inc(x_78); lean_inc(x_77); -lean_inc(x_76); -lean_dec(x_42); -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_dec(x_43); +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 { -uint8_t x_84; +uint8_t x_85; lean_dec(x_20); lean_dec(x_19); lean_dec(x_18); @@ -5430,29 +5511,29 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_84 = !lean_is_exclusive(x_28); -if (x_84 == 0) +x_85 = !lean_is_exclusive(x_29); +if (x_85 == 0) { -return x_28; +return x_29; } else { -lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_85 = lean_ctor_get(x_28, 0); -x_86 = lean_ctor_get(x_28, 1); +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_inc(x_85); -lean_dec(x_28); -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_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_88; +uint8_t x_89; lean_dec(x_14); lean_dec(x_12); lean_dec(x_11); @@ -5460,50 +5541,50 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_88 = !lean_is_exclusive(x_15); -if (x_88 == 0) +x_89 = !lean_is_exclusive(x_15); +if (x_89 == 0) { return x_15; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_89 = lean_ctor_get(x_15, 0); -x_90 = lean_ctor_get(x_15, 1); +lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_90 = lean_ctor_get(x_15, 0); +x_91 = lean_ctor_get(x_15, 1); +lean_inc(x_91); lean_inc(x_90); -lean_inc(x_89); lean_dec(x_15); -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; +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_92; +uint8_t x_93; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_92 = !lean_is_exclusive(x_6); -if (x_92 == 0) +x_93 = !lean_is_exclusive(x_6); +if (x_93 == 0) { return x_6; } else { -lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_93 = lean_ctor_get(x_6, 0); -x_94 = lean_ctor_get(x_6, 1); +lean_object* x_94; lean_object* x_95; lean_object* x_96; +x_94 = lean_ctor_get(x_6, 0); +x_95 = lean_ctor_get(x_6, 1); +lean_inc(x_95); lean_inc(x_94); -lean_inc(x_93); lean_dec(x_6); -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; +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; } } } @@ -5806,41 +5887,23 @@ static lean_object* _init_l_Lean_Elab_Command_expandNamespacedDeclaration___clos _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("null", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_expandNamespacedDeclaration___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_Command_expandNamespacedDeclaration___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3() { -_start: -{ -lean_object* x_1; x_1 = lean_mk_string_unchecked("namespace", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandNamespacedDeclaration___closed__4() { +static lean_object* _init_l_Lean_Elab_Command_expandNamespacedDeclaration___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_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__1; x_2 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__2; x_3 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__3; -x_4 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3; +x_4 = l_Lean_Elab_Command_expandNamespacedDeclaration___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_Elab_Command_expandNamespacedDeclaration___closed__5() { +static lean_object* _init_l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3() { _start: { lean_object* x_1; @@ -5848,14 +5911,14 @@ x_1 = lean_mk_string_unchecked("end", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandNamespacedDeclaration___closed__6() { +static lean_object* _init_l_Lean_Elab_Command_expandNamespacedDeclaration___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___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__1; x_2 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__2; x_3 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__3; -x_4 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__5; +x_4 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -5930,24 +5993,24 @@ x_25 = l_Lean_replaceRef(x_21, x_24); lean_dec(x_21); x_26 = l_Lean_SourceInfo_fromRef(x_25, x_22); lean_dec(x_25); -x_27 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3; +x_27 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__1; lean_inc(x_26); lean_ctor_set_tag(x_12, 2); lean_ctor_set(x_12, 1, x_27); lean_ctor_set(x_12, 0, x_26); -x_28 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__4; +x_28 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; lean_inc(x_23); lean_inc(x_26); x_29 = l_Lean_Syntax_node2(x_26, x_28, x_12, x_23); -x_30 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__5; +x_30 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3; lean_inc(x_26); x_31 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_31, 0, x_26); lean_ctor_set(x_31, 1, x_30); -x_32 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_32 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; lean_inc(x_26); x_33 = l_Lean_Syntax_node1(x_26, x_32, x_23); -x_34 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__6; +x_34 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__4; lean_inc(x_26); x_35 = l_Lean_Syntax_node2(x_26, x_34, x_31, x_33); x_36 = l_Lean_Syntax_node3(x_26, x_32, x_29, x_17, x_35); @@ -5975,24 +6038,24 @@ x_46 = l_Lean_replaceRef(x_42, x_45); lean_dec(x_42); x_47 = l_Lean_SourceInfo_fromRef(x_46, x_43); lean_dec(x_46); -x_48 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3; +x_48 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__1; lean_inc(x_47); x_49 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_49, 0, x_47); lean_ctor_set(x_49, 1, x_48); -x_50 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__4; +x_50 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; lean_inc(x_44); lean_inc(x_47); x_51 = l_Lean_Syntax_node2(x_47, x_50, x_49, x_44); -x_52 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__5; +x_52 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3; lean_inc(x_47); x_53 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_53, 0, x_47); lean_ctor_set(x_53, 1, x_52); -x_54 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_54 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; lean_inc(x_47); x_55 = l_Lean_Syntax_node1(x_47, x_54, x_44); -x_56 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__6; +x_56 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__4; lean_inc(x_47); x_57 = l_Lean_Syntax_node2(x_47, x_56, x_53, x_55); x_58 = l_Lean_Syntax_node3(x_47, x_54, x_51, x_38, x_57); @@ -6031,7 +6094,7 @@ x_70 = l_Lean_replaceRef(x_66, x_69); lean_dec(x_66); x_71 = l_Lean_SourceInfo_fromRef(x_70, x_67); lean_dec(x_70); -x_72 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3; +x_72 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__1; lean_inc(x_71); if (lean_is_scalar(x_62)) { x_73 = lean_alloc_ctor(2, 2, 0); @@ -6041,19 +6104,19 @@ if (lean_is_scalar(x_62)) { } lean_ctor_set(x_73, 0, x_71); lean_ctor_set(x_73, 1, x_72); -x_74 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__4; +x_74 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; lean_inc(x_68); lean_inc(x_71); x_75 = l_Lean_Syntax_node2(x_71, x_74, x_73, x_68); -x_76 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__5; +x_76 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3; lean_inc(x_71); x_77 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_77, 0, x_71); lean_ctor_set(x_77, 1, x_76); -x_78 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_78 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; lean_inc(x_71); x_79 = l_Lean_Syntax_node1(x_71, x_78, x_68); -x_80 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__6; +x_80 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__4; lean_inc(x_71); x_81 = l_Lean_Syntax_node2(x_71, x_80, x_77, x_79); x_82 = l_Lean_Syntax_node3(x_71, x_78, x_75, x_61, x_81); @@ -6480,43 +6543,43 @@ lean_inc(x_6); x_8 = l_Lean_Elab_Command_isDefLike(x_6); if (x_8 == 0) { -lean_object* x_9; uint8_t x_10; -x_9 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__15; -x_10 = lean_name_eq(x_7, x_9); -if (x_10 == 0) -{ -lean_object* x_11; uint8_t x_12; -x_11 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__17; +lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_9 = lean_unsigned_to_nat(0u); +x_10 = l_Lean_Syntax_getArg(x_1, x_9); +lean_dec(x_1); +x_11 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__15; x_12 = lean_name_eq(x_7, x_11); if (x_12 == 0) { lean_object* x_13; uint8_t x_14; -x_13 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__19; +x_13 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__17; x_14 = lean_name_eq(x_7, x_13); if (x_14 == 0) { lean_object* x_15; uint8_t x_16; -x_15 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__21; +x_15 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__19; x_16 = lean_name_eq(x_7, x_15); -lean_dec(x_7); if (x_16 == 0) { -uint8_t x_17; lean_object* x_18; lean_object* x_19; +lean_object* x_17; uint8_t x_18; +x_17 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__21; +x_18 = lean_name_eq(x_7, x_17); +lean_dec(x_7); +if (x_18 == 0) +{ +uint8_t x_19; lean_object* x_20; lean_object* x_21; +lean_dec(x_10); lean_dec(x_6); -lean_dec(x_1); -x_17 = 1; -x_18 = l_Lean_Elab_Command_elabDeclaration___closed__3; -x_19 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_17, x_18, x_2, x_3, x_4); -return x_19; +x_19 = 1; +x_20 = l_Lean_Elab_Command_elabDeclaration___closed__3; +x_21 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_19, x_20, x_2, x_3, x_4); +return x_21; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; -x_20 = lean_unsigned_to_nat(0u); -x_21 = l_Lean_Syntax_getArg(x_1, x_20); -lean_dec(x_1); -x_22 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabDeclaration___lambda__1___boxed), 5, 2); -lean_closure_set(x_22, 0, x_21); +lean_object* x_22; uint8_t x_23; lean_object* x_24; +x_22 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabDeclaration___lambda__1), 5, 2); +lean_closure_set(x_22, 0, x_10); lean_closure_set(x_22, 1, x_6); x_23 = 1; x_24 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_23, x_22, x_2, x_3, x_4); @@ -6525,89 +6588,53 @@ return x_24; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; +lean_object* x_25; uint8_t x_26; lean_object* x_27; lean_dec(x_7); -x_25 = lean_unsigned_to_nat(0u); -x_26 = l_Lean_Syntax_getArg(x_1, x_25); -lean_dec(x_1); -x_27 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabDeclaration___lambda__2___boxed), 5, 2); -lean_closure_set(x_27, 0, x_26); -lean_closure_set(x_27, 1, x_6); -x_28 = 1; -x_29 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_28, x_27, x_2, x_3, x_4); -return x_29; +x_25 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabDeclaration___lambda__2), 5, 2); +lean_closure_set(x_25, 0, x_10); +lean_closure_set(x_25, 1, x_6); +x_26 = 1; +x_27 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_26, x_25, x_2, x_3, x_4); +return x_27; } } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; +lean_object* x_28; uint8_t x_29; lean_object* x_30; lean_dec(x_7); -x_30 = lean_unsigned_to_nat(0u); -x_31 = l_Lean_Syntax_getArg(x_1, x_30); -lean_dec(x_1); -x_32 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabDeclaration___lambda__3___boxed), 5, 2); -lean_closure_set(x_32, 0, x_31); -lean_closure_set(x_32, 1, x_6); -x_33 = 1; -x_34 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_33, x_32, x_2, x_3, x_4); -return x_34; +x_28 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabDeclaration___lambda__3), 5, 2); +lean_closure_set(x_28, 0, x_10); +lean_closure_set(x_28, 1, x_6); +x_29 = 1; +x_30 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_29, x_28, x_2, x_3, x_4); +return x_30; } } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; lean_object* x_39; +lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_dec(x_7); -x_35 = lean_unsigned_to_nat(0u); -x_36 = l_Lean_Syntax_getArg(x_1, x_35); -lean_dec(x_1); -x_37 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabDeclaration___lambda__4___boxed), 5, 2); -lean_closure_set(x_37, 0, x_36); -lean_closure_set(x_37, 1, x_6); -x_38 = 1; -x_39 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_38, x_37, x_2, x_3, x_4); -return x_39; +x_31 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabDeclaration___lambda__4___boxed), 5, 2); +lean_closure_set(x_31, 0, x_10); +lean_closure_set(x_31, 1, x_6); +x_32 = 1; +x_33 = l_Lean_Elab_Command_withoutCommandIncrementality___rarg(x_32, x_31, x_2, x_3, x_4); +return x_33; } } else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_dec(x_7); lean_dec(x_6); -x_40 = lean_box(0); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_1); -lean_ctor_set(x_41, 1, x_40); -x_42 = lean_array_mk(x_41); -x_43 = l_Lean_Elab_Command_elabMutualDef(x_42, x_2, x_3, x_4); -return x_43; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___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_Lean_Elab_Command_elabDeclaration___lambda__1(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_1); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__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_Lean_Elab_Command_elabDeclaration___lambda__2(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_1); -return 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); +x_36 = lean_array_mk(x_35); +x_37 = l_Lean_Elab_Command_elabMutualDef(x_36, x_2, x_3, x_4); +return x_37; } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__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_Elab_Command_elabDeclaration___lambda__3(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_1); -return x_6; } } LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { @@ -6616,7 +6643,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration___lambda__4___boxed lean_object* x_6; x_6 = l_Lean_Elab_Command_elabDeclaration___lambda__4(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); -lean_dec(x_1); return x_6; } } @@ -6908,7 +6934,6 @@ x_11 = lean_array_uset(x_3, x_2, x_10); x_12 = l_Lean_Syntax_getArg(x_9, x_10); lean_inc(x_4); x_13 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_12, x_4, x_5, x_6); -lean_dec(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; lean_object* x_18; @@ -7673,7 +7698,7 @@ static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Elab_Command_expandMu 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_Elab_Declaration_0__Lean_Elab_Command_setDeclIdName___closed__5; x_2 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_expandMutualNamespace___spec__3___closed__1; -x_3 = lean_unsigned_to_nat(308u); +x_3 = lean_unsigned_to_nat(309u); x_4 = lean_unsigned_to_nat(40u); x_5 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_expandMutualNamespace___spec__3___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -7824,7 +7849,7 @@ x_11 = lean_ctor_get(x_9, 0); x_12 = 0; x_13 = l_Lean_mkIdentFrom(x_4, x_2, x_12); x_14 = lean_box(2); -x_15 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_15 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; x_16 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); @@ -7836,23 +7861,23 @@ lean_inc(x_19); lean_dec(x_6); x_20 = l_Lean_SourceInfo_fromRef(x_19, x_12); lean_dec(x_19); -x_21 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3; +x_21 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__1; lean_inc(x_20); x_22 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_22, 0, x_20); lean_ctor_set(x_22, 1, x_21); -x_23 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__4; +x_23 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; lean_inc(x_13); lean_inc(x_20); x_24 = l_Lean_Syntax_node2(x_20, x_23, x_22, x_13); -x_25 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__5; +x_25 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3; lean_inc(x_20); x_26 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_26, 0, x_20); lean_ctor_set(x_26, 1, x_25); lean_inc(x_20); x_27 = l_Lean_Syntax_node1(x_20, x_15, x_13); -x_28 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__6; +x_28 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__4; lean_inc(x_20); x_29 = l_Lean_Syntax_node2(x_20, x_28, x_26, x_27); x_30 = l_Lean_Syntax_node3(x_20, x_15, x_24, x_18, x_29); @@ -7870,7 +7895,7 @@ lean_dec(x_9); x_33 = 0; x_34 = l_Lean_mkIdentFrom(x_4, x_2, x_33); x_35 = lean_box(2); -x_36 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_36 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; x_37 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_37, 0, x_35); lean_ctor_set(x_37, 1, x_36); @@ -7882,23 +7907,23 @@ lean_inc(x_40); lean_dec(x_6); x_41 = l_Lean_SourceInfo_fromRef(x_40, x_33); lean_dec(x_40); -x_42 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3; +x_42 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__1; lean_inc(x_41); x_43 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_43, 0, x_41); lean_ctor_set(x_43, 1, x_42); -x_44 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__4; +x_44 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; lean_inc(x_34); lean_inc(x_41); x_45 = l_Lean_Syntax_node2(x_41, x_44, x_43, x_34); -x_46 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__5; +x_46 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3; lean_inc(x_41); x_47 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_47, 0, x_41); lean_ctor_set(x_47, 1, x_46); lean_inc(x_41); x_48 = l_Lean_Syntax_node1(x_41, x_36, x_34); -x_49 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__6; +x_49 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__4; lean_inc(x_41); x_50 = l_Lean_Syntax_node2(x_41, x_49, x_47, x_48); x_51 = l_Lean_Syntax_node3(x_41, x_36, x_45, x_39, x_50); @@ -8701,7 +8726,7 @@ x_22 = lean_ctor_get(x_11, 0); lean_inc(x_22); lean_dec(x_11); x_23 = lean_box(2); -x_24 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_24 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; x_25 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_25, 0, x_23); lean_ctor_set(x_25, 1, x_24); @@ -8720,7 +8745,7 @@ x_28 = lean_ctor_get(x_11, 0); lean_inc(x_28); lean_dec(x_11); x_29 = lean_box(2); -x_30 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_30 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; x_31 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_31, 0, x_29); lean_ctor_set(x_31, 1, x_30); @@ -8993,7 +9018,7 @@ lean_inc(x_17); lean_ctor_set_tag(x_11, 2); lean_ctor_set(x_11, 1, x_18); lean_ctor_set(x_11, 0, x_17); -x_19 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_19 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; x_20 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; lean_inc(x_17); x_21 = lean_alloc_ctor(1, 3, 0); @@ -9010,12 +9035,12 @@ lean_ctor_set(x_25, 0, x_24); lean_ctor_set(x_25, 1, x_19); lean_ctor_set(x_25, 2, x_14); x_26 = l_Lean_Syntax_setArg(x_1, x_4, x_25); -x_27 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__5; +x_27 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3; lean_inc(x_17); x_28 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_28, 0, x_17); lean_ctor_set(x_28, 1, x_27); -x_29 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__6; +x_29 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__4; x_30 = l_Lean_Syntax_node2(x_17, x_29, x_28, x_21); x_31 = lean_box(0); x_32 = lean_alloc_ctor(1, 2, 0); @@ -9061,7 +9086,7 @@ lean_inc(x_47); x_49 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_49, 0, x_47); lean_ctor_set(x_49, 1, x_48); -x_50 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_50 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; x_51 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; lean_inc(x_47); x_52 = lean_alloc_ctor(1, 3, 0); @@ -9078,12 +9103,12 @@ lean_ctor_set(x_56, 0, x_55); lean_ctor_set(x_56, 1, x_50); lean_ctor_set(x_56, 2, x_44); x_57 = l_Lean_Syntax_setArg(x_1, x_4, x_56); -x_58 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__5; +x_58 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3; lean_inc(x_47); x_59 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_59, 0, x_47); lean_ctor_set(x_59, 1, x_58); -x_60 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__6; +x_60 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__4; x_61 = l_Lean_Syntax_node2(x_47, x_60, x_59, x_52); x_62 = lean_box(0); x_63 = lean_alloc_ctor(1, 2, 0); @@ -11577,7 +11602,7 @@ lean_inc(x_41); lean_ctor_set_tag(x_46, 2); lean_ctor_set(x_46, 1, x_50); lean_ctor_set(x_46, 0, x_41); -x_51 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_51 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; x_52 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; lean_inc(x_41); x_53 = lean_alloc_ctor(1, 3, 0); @@ -11747,7 +11772,7 @@ lean_inc(x_41); x_122 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_122, 0, x_41); lean_ctor_set(x_122, 1, x_121); -x_123 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_123 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; x_124 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; lean_inc(x_41); x_125 = lean_alloc_ctor(1, 3, 0); @@ -11936,7 +11961,7 @@ if (lean_is_scalar(x_196)) { } lean_ctor_set(x_198, 0, x_41); lean_ctor_set(x_198, 1, x_197); -x_199 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_199 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; x_200 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; lean_inc(x_41); x_201 = lean_alloc_ctor(1, 3, 0); @@ -12141,7 +12166,7 @@ if (lean_is_scalar(x_279)) { } lean_ctor_set(x_281, 0, x_271); lean_ctor_set(x_281, 1, x_280); -x_282 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_282 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; x_283 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; lean_inc(x_271); x_284 = lean_alloc_ctor(1, 3, 0); @@ -12361,532 +12386,522 @@ return x_5; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInitialize___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; uint8_t x_12; +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_unsigned_to_nat(0u); +x_12 = l_Lean_Syntax_getArg(x_1, x_11); +x_13 = lean_unsigned_to_nat(1u); +x_14 = l_Lean_Syntax_getArg(x_1, x_13); lean_inc(x_8); -lean_inc(x_1); lean_inc(x_6); -x_11 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1(x_6, x_1, 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, 1); -x_14 = lean_ctor_get(x_11, 0); -lean_dec(x_14); -x_15 = l_Lean_Elab_Command_getRef(x_8, x_9, x_13); +x_15 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1(x_6, x_12, x_14, x_8, x_9, x_10); x_16 = !lean_is_exclusive(x_15); if (x_16 == 0) { -lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_17 = lean_ctor_get(x_15, 0); -x_18 = lean_ctor_get(x_15, 1); -x_19 = 0; -x_20 = l_Lean_SourceInfo_fromRef(x_17, x_19); -lean_dec(x_17); -x_21 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_18); -x_22 = !lean_is_exclusive(x_21); -if (x_22 == 0) +lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_17 = lean_ctor_get(x_15, 1); +x_18 = lean_ctor_get(x_15, 0); +lean_dec(x_18); +x_19 = l_Lean_Elab_Command_getRef(x_8, x_9, x_17); +x_20 = !lean_is_exclusive(x_19); +if (x_20 == 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_Elab_Command_getMainModule___rarg(x_9, x_24); +lean_object* x_21; lean_object* x_22; uint8_t 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 = 0; +x_24 = l_Lean_SourceInfo_fromRef(x_21, x_23); +lean_dec(x_21); +x_25 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_22); 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; 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_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; x_27 = lean_ctor_get(x_25, 0); x_28 = lean_ctor_get(x_25, 1); -x_29 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; -x_30 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -lean_inc(x_20); -x_31 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_31, 0, x_20); -lean_ctor_set(x_31, 1, x_29); -lean_ctor_set(x_31, 2, x_30); -x_32 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; -lean_inc(x_20); -lean_ctor_set_tag(x_25, 2); -lean_ctor_set(x_25, 1, x_32); -lean_ctor_set(x_25, 0, x_20); -x_33 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; -lean_inc(x_23); +x_29 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_28); +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; 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; +x_31 = lean_ctor_get(x_29, 0); +x_32 = lean_ctor_get(x_29, 1); +x_33 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; +x_34 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +lean_inc(x_24); +x_35 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_35, 0, x_24); +lean_ctor_set(x_35, 1, x_33); +lean_ctor_set(x_35, 2, x_34); +x_36 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; +lean_inc(x_24); +lean_ctor_set_tag(x_29, 2); +lean_ctor_set(x_29, 1, x_36); +lean_ctor_set(x_29, 0, x_24); +x_37 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; lean_inc(x_27); -x_34 = l_Lean_addMacroScope(x_27, x_33, x_23); -x_35 = lean_box(0); -x_36 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; -lean_inc(x_20); -x_37 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_37, 0, x_20); -lean_ctor_set(x_37, 1, x_36); -lean_ctor_set(x_37, 2, x_34); -lean_ctor_set(x_37, 3, x_35); -x_38 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; -lean_inc(x_31); -lean_inc(x_20); -x_39 = l_Lean_Syntax_node2(x_20, x_38, x_37, x_31); -x_40 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; -lean_inc(x_20); -lean_ctor_set_tag(x_21, 2); -lean_ctor_set(x_21, 1, x_40); -lean_ctor_set(x_21, 0, x_20); -x_41 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; -x_42 = l_Lean_addMacroScope(x_27, x_41, x_23); -x_43 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; -x_44 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; -lean_inc(x_20); -x_45 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_45, 0, x_20); -lean_ctor_set(x_45, 1, x_43); -lean_ctor_set(x_45, 2, x_42); -lean_ctor_set(x_45, 3, x_44); -lean_inc(x_20); -x_46 = l_Lean_Syntax_node1(x_20, x_29, x_2); -x_47 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; -lean_inc(x_20); -x_48 = l_Lean_Syntax_node2(x_20, x_47, x_45, x_46); -x_49 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; -lean_inc(x_20); -x_50 = l_Lean_Syntax_node2(x_20, x_49, x_21, x_48); -lean_inc(x_20); -x_51 = l_Lean_Syntax_node1(x_20, x_29, x_50); -x_52 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; lean_inc(x_31); -lean_inc(x_20); -x_53 = l_Lean_Syntax_node2(x_20, x_52, x_31, x_51); -x_54 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; -lean_inc(x_20); +x_38 = l_Lean_addMacroScope(x_31, x_37, x_27); +x_39 = lean_box(0); +x_40 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; +lean_inc(x_24); +x_41 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_41, 0, x_24); +lean_ctor_set(x_41, 1, x_40); +lean_ctor_set(x_41, 2, x_38); +lean_ctor_set(x_41, 3, x_39); +x_42 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; +lean_inc(x_35); +lean_inc(x_24); +x_43 = l_Lean_Syntax_node2(x_24, x_42, x_41, x_35); +x_44 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; +lean_inc(x_24); +lean_ctor_set_tag(x_25, 2); +lean_ctor_set(x_25, 1, x_44); +lean_ctor_set(x_25, 0, x_24); +x_45 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; +x_46 = l_Lean_addMacroScope(x_31, x_45, x_27); +x_47 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; +x_48 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; +lean_inc(x_24); +x_49 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_49, 0, x_24); +lean_ctor_set(x_49, 1, x_47); +lean_ctor_set(x_49, 2, x_46); +lean_ctor_set(x_49, 3, x_48); +lean_inc(x_24); +x_50 = l_Lean_Syntax_node1(x_24, x_33, x_2); +x_51 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; +lean_inc(x_24); +x_52 = l_Lean_Syntax_node2(x_24, x_51, x_49, x_50); +x_53 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; +lean_inc(x_24); +x_54 = l_Lean_Syntax_node2(x_24, x_53, x_25, x_52); +lean_inc(x_24); +x_55 = l_Lean_Syntax_node1(x_24, x_33, x_54); +x_56 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; +lean_inc(x_35); +lean_inc(x_24); +x_57 = l_Lean_Syntax_node2(x_24, x_56, x_35, x_55); +x_58 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; +lean_inc(x_24); +lean_ctor_set_tag(x_19, 2); +lean_ctor_set(x_19, 1, x_58); +lean_ctor_set(x_19, 0, x_24); +x_59 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; +lean_inc(x_24); lean_ctor_set_tag(x_15, 2); -lean_ctor_set(x_15, 1, x_54); -lean_ctor_set(x_15, 0, x_20); -x_55 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; -lean_inc(x_20); -lean_ctor_set_tag(x_11, 2); -lean_ctor_set(x_11, 1, x_55); -lean_ctor_set(x_11, 0, x_20); -x_56 = lean_mk_syntax_ident(x_6); -x_57 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; -lean_inc(x_20); -x_58 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_58, 0, x_20); -lean_ctor_set(x_58, 1, x_57); -x_59 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; -lean_inc(x_20); -x_60 = l_Lean_Syntax_node2(x_20, x_59, x_58, x_3); -x_61 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; -lean_inc(x_31); -lean_inc(x_20); -x_62 = l_Lean_Syntax_node4(x_20, x_61, x_11, x_31, x_56, x_60); -x_63 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; -lean_inc_n(x_31, 2); -lean_inc(x_20); -x_64 = l_Lean_Syntax_node2(x_20, x_63, x_31, x_31); -x_65 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; -lean_inc(x_31); -lean_inc(x_20); -x_66 = l_Lean_Syntax_node4(x_20, x_65, x_15, x_62, x_64, x_31); -x_67 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; -lean_inc(x_31); -lean_inc(x_20); -x_68 = l_Lean_Syntax_node5(x_20, x_67, x_25, x_39, x_53, x_66, x_31); +lean_ctor_set(x_15, 1, x_59); +lean_ctor_set(x_15, 0, x_24); +x_60 = lean_mk_syntax_ident(x_6); +x_61 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; +lean_inc(x_24); +x_62 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_62, 0, x_24); +lean_ctor_set(x_62, 1, x_61); +x_63 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; +lean_inc(x_24); +x_64 = l_Lean_Syntax_node2(x_24, x_63, x_62, x_3); +x_65 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; +lean_inc(x_35); +lean_inc(x_24); +x_66 = l_Lean_Syntax_node4(x_24, x_65, x_15, x_35, x_60, x_64); +x_67 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; +lean_inc_n(x_35, 2); +lean_inc(x_24); +x_68 = l_Lean_Syntax_node2(x_24, x_67, x_35, x_35); +x_69 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; +lean_inc(x_35); +lean_inc(x_24); +x_70 = l_Lean_Syntax_node4(x_24, x_69, x_19, x_66, x_68, x_35); +x_71 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; +lean_inc(x_35); +lean_inc(x_24); +x_72 = l_Lean_Syntax_node5(x_24, x_71, x_29, x_43, x_57, x_70, x_35); if (lean_obj_tag(x_4) == 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; -x_69 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; -lean_inc(x_20); -x_70 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_70, 0, x_20); -lean_ctor_set(x_70, 1, x_29); -lean_ctor_set(x_70, 2, x_69); -lean_inc_n(x_31, 4); -lean_inc(x_20); -x_71 = l_Lean_Syntax_node6(x_20, x_5, x_31, x_31, x_31, x_31, x_70, x_31); -x_72 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_20); -x_73 = l_Lean_Syntax_node2(x_20, x_72, x_71, x_68); -x_74 = l_Lean_Syntax_node2(x_20, x_29, x_73, x_1); -x_75 = l_Lean_Elab_Command_elabCommand(x_74, x_8, x_9, x_28); -return x_75; +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 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; +lean_inc(x_24); +x_74 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_74, 0, x_24); +lean_ctor_set(x_74, 1, x_33); +lean_ctor_set(x_74, 2, x_73); +lean_inc_n(x_35, 4); +lean_inc(x_24); +x_75 = l_Lean_Syntax_node6(x_24, x_5, x_35, x_35, x_35, x_35, x_74, x_35); +x_76 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_24); +x_77 = l_Lean_Syntax_node2(x_24, x_76, x_75, x_72); +x_78 = l_Lean_Syntax_node2(x_24, x_33, x_77, x_1); +x_79 = l_Lean_Elab_Command_elabCommand(x_78, x_8, x_9, x_32); +return x_79; } else { -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; -x_76 = lean_ctor_get(x_4, 0); -x_77 = 1; -x_78 = l_Lean_SourceInfo_fromRef(x_76, x_77); -x_79 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; -x_80 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_80, 0, x_78); -lean_ctor_set(x_80, 1, x_79); -x_81 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; -lean_inc(x_20); -x_82 = l_Lean_Syntax_node1(x_20, x_81, x_80); -x_83 = l_Array_mkArray1___rarg(x_82); -x_84 = l_Array_append___rarg(x_30, x_83); -lean_dec(x_83); -lean_inc(x_20); -x_85 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_85, 0, x_20); -lean_ctor_set(x_85, 1, x_29); -lean_ctor_set(x_85, 2, x_84); -lean_inc_n(x_31, 4); -lean_inc(x_20); -x_86 = l_Lean_Syntax_node6(x_20, x_5, x_31, x_31, x_31, x_31, x_85, x_31); -x_87 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_20); -x_88 = l_Lean_Syntax_node2(x_20, x_87, x_86, x_68); -x_89 = l_Lean_Syntax_node2(x_20, x_29, x_88, x_1); -x_90 = l_Lean_Elab_Command_elabCommand(x_89, x_8, x_9, x_28); -return x_90; +lean_object* x_80; uint8_t 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_4, 0); +x_81 = 1; +x_82 = l_Lean_SourceInfo_fromRef(x_80, x_81); +x_83 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; +x_84 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_83); +x_85 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; +lean_inc(x_24); +x_86 = l_Lean_Syntax_node1(x_24, x_85, x_84); +x_87 = l_Array_mkArray1___rarg(x_86); +x_88 = l_Array_append___rarg(x_34, x_87); +lean_dec(x_87); +lean_inc(x_24); +x_89 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_89, 0, x_24); +lean_ctor_set(x_89, 1, x_33); +lean_ctor_set(x_89, 2, x_88); +lean_inc_n(x_35, 4); +lean_inc(x_24); +x_90 = l_Lean_Syntax_node6(x_24, x_5, x_35, x_35, x_35, x_35, x_89, x_35); +x_91 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_24); +x_92 = l_Lean_Syntax_node2(x_24, x_91, x_90, x_72); +x_93 = l_Lean_Syntax_node2(x_24, x_33, x_92, x_1); +x_94 = l_Lean_Elab_Command_elabCommand(x_93, x_8, x_9, x_32); +return x_94; } } 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; 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; -x_91 = lean_ctor_get(x_25, 0); -x_92 = lean_ctor_get(x_25, 1); -lean_inc(x_92); -lean_inc(x_91); -lean_dec(x_25); -x_93 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; -x_94 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -lean_inc(x_20); -x_95 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_95, 0, x_20); -lean_ctor_set(x_95, 1, x_93); -lean_ctor_set(x_95, 2, x_94); -x_96 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; -lean_inc(x_20); -x_97 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_97, 0, x_20); -lean_ctor_set(x_97, 1, x_96); -x_98 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; -lean_inc(x_23); -lean_inc(x_91); -x_99 = l_Lean_addMacroScope(x_91, x_98, x_23); -x_100 = lean_box(0); -x_101 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; -lean_inc(x_20); -x_102 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_102, 0, x_20); -lean_ctor_set(x_102, 1, x_101); -lean_ctor_set(x_102, 2, x_99); -lean_ctor_set(x_102, 3, x_100); -x_103 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; +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; +x_95 = lean_ctor_get(x_29, 0); +x_96 = lean_ctor_get(x_29, 1); +lean_inc(x_96); lean_inc(x_95); -lean_inc(x_20); -x_104 = l_Lean_Syntax_node2(x_20, x_103, x_102, x_95); -x_105 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; -lean_inc(x_20); -lean_ctor_set_tag(x_21, 2); -lean_ctor_set(x_21, 1, x_105); -lean_ctor_set(x_21, 0, x_20); -x_106 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; -x_107 = l_Lean_addMacroScope(x_91, x_106, x_23); -x_108 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; -x_109 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; -lean_inc(x_20); -x_110 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_110, 0, x_20); -lean_ctor_set(x_110, 1, x_108); -lean_ctor_set(x_110, 2, x_107); -lean_ctor_set(x_110, 3, x_109); -lean_inc(x_20); -x_111 = l_Lean_Syntax_node1(x_20, x_93, x_2); -x_112 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; -lean_inc(x_20); -x_113 = l_Lean_Syntax_node2(x_20, x_112, x_110, x_111); -x_114 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; -lean_inc(x_20); -x_115 = l_Lean_Syntax_node2(x_20, x_114, x_21, x_113); -lean_inc(x_20); -x_116 = l_Lean_Syntax_node1(x_20, x_93, x_115); -x_117 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; +lean_dec(x_29); +x_97 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; +x_98 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +lean_inc(x_24); +x_99 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_99, 0, x_24); +lean_ctor_set(x_99, 1, x_97); +lean_ctor_set(x_99, 2, x_98); +x_100 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; +lean_inc(x_24); +x_101 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_101, 0, x_24); +lean_ctor_set(x_101, 1, x_100); +x_102 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; +lean_inc(x_27); lean_inc(x_95); -lean_inc(x_20); -x_118 = l_Lean_Syntax_node2(x_20, x_117, x_95, x_116); -x_119 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; -lean_inc(x_20); +x_103 = l_Lean_addMacroScope(x_95, x_102, x_27); +x_104 = lean_box(0); +x_105 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; +lean_inc(x_24); +x_106 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_106, 0, x_24); +lean_ctor_set(x_106, 1, x_105); +lean_ctor_set(x_106, 2, x_103); +lean_ctor_set(x_106, 3, x_104); +x_107 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; +lean_inc(x_99); +lean_inc(x_24); +x_108 = l_Lean_Syntax_node2(x_24, x_107, x_106, x_99); +x_109 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; +lean_inc(x_24); +lean_ctor_set_tag(x_25, 2); +lean_ctor_set(x_25, 1, x_109); +lean_ctor_set(x_25, 0, x_24); +x_110 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; +x_111 = l_Lean_addMacroScope(x_95, x_110, x_27); +x_112 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; +x_113 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; +lean_inc(x_24); +x_114 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_114, 0, x_24); +lean_ctor_set(x_114, 1, x_112); +lean_ctor_set(x_114, 2, x_111); +lean_ctor_set(x_114, 3, x_113); +lean_inc(x_24); +x_115 = l_Lean_Syntax_node1(x_24, x_97, x_2); +x_116 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; +lean_inc(x_24); +x_117 = l_Lean_Syntax_node2(x_24, x_116, x_114, x_115); +x_118 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; +lean_inc(x_24); +x_119 = l_Lean_Syntax_node2(x_24, x_118, x_25, x_117); +lean_inc(x_24); +x_120 = l_Lean_Syntax_node1(x_24, x_97, x_119); +x_121 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; +lean_inc(x_99); +lean_inc(x_24); +x_122 = l_Lean_Syntax_node2(x_24, x_121, x_99, x_120); +x_123 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; +lean_inc(x_24); +lean_ctor_set_tag(x_19, 2); +lean_ctor_set(x_19, 1, x_123); +lean_ctor_set(x_19, 0, x_24); +x_124 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; +lean_inc(x_24); lean_ctor_set_tag(x_15, 2); -lean_ctor_set(x_15, 1, x_119); -lean_ctor_set(x_15, 0, x_20); -x_120 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; -lean_inc(x_20); -lean_ctor_set_tag(x_11, 2); -lean_ctor_set(x_11, 1, x_120); -lean_ctor_set(x_11, 0, x_20); -x_121 = lean_mk_syntax_ident(x_6); -x_122 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; -lean_inc(x_20); -x_123 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_123, 0, x_20); -lean_ctor_set(x_123, 1, x_122); -x_124 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; -lean_inc(x_20); -x_125 = l_Lean_Syntax_node2(x_20, x_124, x_123, x_3); -x_126 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; -lean_inc(x_95); -lean_inc(x_20); -x_127 = l_Lean_Syntax_node4(x_20, x_126, x_11, x_95, x_121, x_125); -x_128 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; -lean_inc_n(x_95, 2); -lean_inc(x_20); -x_129 = l_Lean_Syntax_node2(x_20, x_128, x_95, x_95); -x_130 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; -lean_inc(x_95); -lean_inc(x_20); -x_131 = l_Lean_Syntax_node4(x_20, x_130, x_15, x_127, x_129, x_95); -x_132 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; -lean_inc(x_95); -lean_inc(x_20); -x_133 = l_Lean_Syntax_node5(x_20, x_132, x_97, x_104, x_118, x_131, x_95); +lean_ctor_set(x_15, 1, x_124); +lean_ctor_set(x_15, 0, x_24); +x_125 = lean_mk_syntax_ident(x_6); +x_126 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; +lean_inc(x_24); +x_127 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_127, 0, x_24); +lean_ctor_set(x_127, 1, x_126); +x_128 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; +lean_inc(x_24); +x_129 = l_Lean_Syntax_node2(x_24, x_128, x_127, x_3); +x_130 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; +lean_inc(x_99); +lean_inc(x_24); +x_131 = l_Lean_Syntax_node4(x_24, x_130, x_15, x_99, x_125, x_129); +x_132 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; +lean_inc_n(x_99, 2); +lean_inc(x_24); +x_133 = l_Lean_Syntax_node2(x_24, x_132, x_99, x_99); +x_134 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; +lean_inc(x_99); +lean_inc(x_24); +x_135 = l_Lean_Syntax_node4(x_24, x_134, x_19, x_131, x_133, x_99); +x_136 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; +lean_inc(x_99); +lean_inc(x_24); +x_137 = l_Lean_Syntax_node5(x_24, x_136, x_101, x_108, x_122, x_135, x_99); if (lean_obj_tag(x_4) == 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; -x_134 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; -lean_inc(x_20); -x_135 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_135, 0, x_20); -lean_ctor_set(x_135, 1, x_93); -lean_ctor_set(x_135, 2, x_134); -lean_inc_n(x_95, 4); -lean_inc(x_20); -x_136 = l_Lean_Syntax_node6(x_20, x_5, x_95, x_95, x_95, x_95, x_135, x_95); -x_137 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_20); -x_138 = l_Lean_Syntax_node2(x_20, x_137, x_136, x_133); -x_139 = l_Lean_Syntax_node2(x_20, x_93, x_138, x_1); -x_140 = l_Lean_Elab_Command_elabCommand(x_139, x_8, x_9, x_92); -return x_140; +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_138 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; +lean_inc(x_24); +x_139 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_139, 0, x_24); +lean_ctor_set(x_139, 1, x_97); +lean_ctor_set(x_139, 2, x_138); +lean_inc_n(x_99, 4); +lean_inc(x_24); +x_140 = l_Lean_Syntax_node6(x_24, x_5, x_99, x_99, x_99, x_99, x_139, x_99); +x_141 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_24); +x_142 = l_Lean_Syntax_node2(x_24, x_141, x_140, x_137); +x_143 = l_Lean_Syntax_node2(x_24, x_97, x_142, x_1); +x_144 = l_Lean_Elab_Command_elabCommand(x_143, x_8, x_9, x_96); +return x_144; } else { -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; -x_141 = lean_ctor_get(x_4, 0); -x_142 = 1; -x_143 = l_Lean_SourceInfo_fromRef(x_141, x_142); -x_144 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; -x_145 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_145, 0, x_143); -lean_ctor_set(x_145, 1, x_144); -x_146 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; -lean_inc(x_20); -x_147 = l_Lean_Syntax_node1(x_20, x_146, x_145); -x_148 = l_Array_mkArray1___rarg(x_147); -x_149 = l_Array_append___rarg(x_94, x_148); -lean_dec(x_148); -lean_inc(x_20); -x_150 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_150, 0, x_20); -lean_ctor_set(x_150, 1, x_93); -lean_ctor_set(x_150, 2, x_149); -lean_inc_n(x_95, 4); -lean_inc(x_20); -x_151 = l_Lean_Syntax_node6(x_20, x_5, x_95, x_95, x_95, x_95, x_150, x_95); -x_152 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_20); -x_153 = l_Lean_Syntax_node2(x_20, x_152, x_151, x_133); -x_154 = l_Lean_Syntax_node2(x_20, x_93, x_153, x_1); -x_155 = l_Lean_Elab_Command_elabCommand(x_154, x_8, x_9, x_92); -return x_155; +lean_object* x_145; uint8_t 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; +x_145 = lean_ctor_get(x_4, 0); +x_146 = 1; +x_147 = l_Lean_SourceInfo_fromRef(x_145, x_146); +x_148 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; +x_149 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_149, 0, x_147); +lean_ctor_set(x_149, 1, x_148); +x_150 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; +lean_inc(x_24); +x_151 = l_Lean_Syntax_node1(x_24, x_150, x_149); +x_152 = l_Array_mkArray1___rarg(x_151); +x_153 = l_Array_append___rarg(x_98, x_152); +lean_dec(x_152); +lean_inc(x_24); +x_154 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_154, 0, x_24); +lean_ctor_set(x_154, 1, x_97); +lean_ctor_set(x_154, 2, x_153); +lean_inc_n(x_99, 4); +lean_inc(x_24); +x_155 = l_Lean_Syntax_node6(x_24, x_5, x_99, x_99, x_99, x_99, x_154, x_99); +x_156 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_24); +x_157 = l_Lean_Syntax_node2(x_24, x_156, x_155, x_137); +x_158 = l_Lean_Syntax_node2(x_24, x_97, x_157, x_1); +x_159 = l_Lean_Elab_Command_elabCommand(x_158, x_8, x_9, x_96); +return x_159; } } } else { -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; -x_156 = lean_ctor_get(x_21, 0); -x_157 = lean_ctor_get(x_21, 1); -lean_inc(x_157); -lean_inc(x_156); -lean_dec(x_21); -x_158 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_157); -x_159 = lean_ctor_get(x_158, 0); -lean_inc(x_159); -x_160 = lean_ctor_get(x_158, 1); +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; +x_160 = lean_ctor_get(x_25, 0); +x_161 = lean_ctor_get(x_25, 1); +lean_inc(x_161); lean_inc(x_160); -if (lean_is_exclusive(x_158)) { - lean_ctor_release(x_158, 0); - lean_ctor_release(x_158, 1); - x_161 = x_158; +lean_dec(x_25); +x_162 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_161); +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_158); - x_161 = lean_box(0); + lean_dec_ref(x_162); + x_165 = lean_box(0); } -x_162 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; -x_163 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -lean_inc(x_20); -x_164 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_164, 0, x_20); -lean_ctor_set(x_164, 1, x_162); -lean_ctor_set(x_164, 2, x_163); -x_165 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; -lean_inc(x_20); -if (lean_is_scalar(x_161)) { - x_166 = lean_alloc_ctor(2, 2, 0); +x_166 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; +x_167 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +lean_inc(x_24); +x_168 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_168, 0, x_24); +lean_ctor_set(x_168, 1, x_166); +lean_ctor_set(x_168, 2, x_167); +x_169 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; +lean_inc(x_24); +if (lean_is_scalar(x_165)) { + x_170 = lean_alloc_ctor(2, 2, 0); } else { - x_166 = x_161; - lean_ctor_set_tag(x_166, 2); + x_170 = x_165; + lean_ctor_set_tag(x_170, 2); } -lean_ctor_set(x_166, 0, x_20); -lean_ctor_set(x_166, 1, x_165); -x_167 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; -lean_inc(x_156); -lean_inc(x_159); -x_168 = l_Lean_addMacroScope(x_159, x_167, x_156); -x_169 = lean_box(0); -x_170 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; -lean_inc(x_20); -x_171 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_171, 0, x_20); -lean_ctor_set(x_171, 1, x_170); -lean_ctor_set(x_171, 2, x_168); -lean_ctor_set(x_171, 3, x_169); -x_172 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; -lean_inc(x_164); -lean_inc(x_20); -x_173 = l_Lean_Syntax_node2(x_20, x_172, x_171, x_164); -x_174 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; -lean_inc(x_20); -x_175 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_175, 0, x_20); +lean_ctor_set(x_170, 0, x_24); +lean_ctor_set(x_170, 1, x_169); +x_171 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; +lean_inc(x_160); +lean_inc(x_163); +x_172 = l_Lean_addMacroScope(x_163, x_171, x_160); +x_173 = lean_box(0); +x_174 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; +lean_inc(x_24); +x_175 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_175, 0, x_24); lean_ctor_set(x_175, 1, x_174); -x_176 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; -x_177 = l_Lean_addMacroScope(x_159, x_176, x_156); -x_178 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; -x_179 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; -lean_inc(x_20); -x_180 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_180, 0, x_20); -lean_ctor_set(x_180, 1, x_178); -lean_ctor_set(x_180, 2, x_177); -lean_ctor_set(x_180, 3, x_179); -lean_inc(x_20); -x_181 = l_Lean_Syntax_node1(x_20, x_162, x_2); -x_182 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; -lean_inc(x_20); -x_183 = l_Lean_Syntax_node2(x_20, x_182, x_180, x_181); -x_184 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; -lean_inc(x_20); -x_185 = l_Lean_Syntax_node2(x_20, x_184, x_175, x_183); -lean_inc(x_20); -x_186 = l_Lean_Syntax_node1(x_20, x_162, x_185); -x_187 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; -lean_inc(x_164); -lean_inc(x_20); -x_188 = l_Lean_Syntax_node2(x_20, x_187, x_164, x_186); -x_189 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; -lean_inc(x_20); +lean_ctor_set(x_175, 2, x_172); +lean_ctor_set(x_175, 3, x_173); +x_176 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; +lean_inc(x_168); +lean_inc(x_24); +x_177 = l_Lean_Syntax_node2(x_24, x_176, x_175, x_168); +x_178 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; +lean_inc(x_24); +x_179 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_179, 0, x_24); +lean_ctor_set(x_179, 1, x_178); +x_180 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; +x_181 = l_Lean_addMacroScope(x_163, x_180, x_160); +x_182 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; +x_183 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; +lean_inc(x_24); +x_184 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_184, 0, x_24); +lean_ctor_set(x_184, 1, x_182); +lean_ctor_set(x_184, 2, x_181); +lean_ctor_set(x_184, 3, x_183); +lean_inc(x_24); +x_185 = l_Lean_Syntax_node1(x_24, x_166, x_2); +x_186 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; +lean_inc(x_24); +x_187 = l_Lean_Syntax_node2(x_24, x_186, x_184, x_185); +x_188 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; +lean_inc(x_24); +x_189 = l_Lean_Syntax_node2(x_24, x_188, x_179, x_187); +lean_inc(x_24); +x_190 = l_Lean_Syntax_node1(x_24, x_166, x_189); +x_191 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; +lean_inc(x_168); +lean_inc(x_24); +x_192 = l_Lean_Syntax_node2(x_24, x_191, x_168, x_190); +x_193 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; +lean_inc(x_24); +lean_ctor_set_tag(x_19, 2); +lean_ctor_set(x_19, 1, x_193); +lean_ctor_set(x_19, 0, x_24); +x_194 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; +lean_inc(x_24); lean_ctor_set_tag(x_15, 2); -lean_ctor_set(x_15, 1, x_189); -lean_ctor_set(x_15, 0, x_20); -x_190 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; -lean_inc(x_20); -lean_ctor_set_tag(x_11, 2); -lean_ctor_set(x_11, 1, x_190); -lean_ctor_set(x_11, 0, x_20); -x_191 = lean_mk_syntax_ident(x_6); -x_192 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; -lean_inc(x_20); -x_193 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_193, 0, x_20); -lean_ctor_set(x_193, 1, x_192); -x_194 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; -lean_inc(x_20); -x_195 = l_Lean_Syntax_node2(x_20, x_194, x_193, x_3); -x_196 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; -lean_inc(x_164); -lean_inc(x_20); -x_197 = l_Lean_Syntax_node4(x_20, x_196, x_11, x_164, x_191, x_195); -x_198 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; -lean_inc_n(x_164, 2); -lean_inc(x_20); -x_199 = l_Lean_Syntax_node2(x_20, x_198, x_164, x_164); -x_200 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; -lean_inc(x_164); -lean_inc(x_20); -x_201 = l_Lean_Syntax_node4(x_20, x_200, x_15, x_197, x_199, x_164); -x_202 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; -lean_inc(x_164); -lean_inc(x_20); -x_203 = l_Lean_Syntax_node5(x_20, x_202, x_166, x_173, x_188, x_201, x_164); +lean_ctor_set(x_15, 1, x_194); +lean_ctor_set(x_15, 0, x_24); +x_195 = lean_mk_syntax_ident(x_6); +x_196 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; +lean_inc(x_24); +x_197 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_197, 0, x_24); +lean_ctor_set(x_197, 1, x_196); +x_198 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; +lean_inc(x_24); +x_199 = l_Lean_Syntax_node2(x_24, x_198, x_197, x_3); +x_200 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; +lean_inc(x_168); +lean_inc(x_24); +x_201 = l_Lean_Syntax_node4(x_24, x_200, x_15, x_168, x_195, x_199); +x_202 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; +lean_inc_n(x_168, 2); +lean_inc(x_24); +x_203 = l_Lean_Syntax_node2(x_24, x_202, x_168, x_168); +x_204 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; +lean_inc(x_168); +lean_inc(x_24); +x_205 = l_Lean_Syntax_node4(x_24, x_204, x_19, x_201, x_203, x_168); +x_206 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; +lean_inc(x_168); +lean_inc(x_24); +x_207 = l_Lean_Syntax_node5(x_24, x_206, x_170, x_177, x_192, x_205, x_168); if (lean_obj_tag(x_4) == 0) { -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_204 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; -lean_inc(x_20); -x_205 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_205, 0, x_20); -lean_ctor_set(x_205, 1, x_162); -lean_ctor_set(x_205, 2, x_204); -lean_inc_n(x_164, 4); -lean_inc(x_20); -x_206 = l_Lean_Syntax_node6(x_20, x_5, x_164, x_164, x_164, x_164, x_205, x_164); -x_207 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_20); -x_208 = l_Lean_Syntax_node2(x_20, x_207, x_206, x_203); -x_209 = l_Lean_Syntax_node2(x_20, x_162, x_208, x_1); -x_210 = l_Lean_Elab_Command_elabCommand(x_209, x_8, x_9, x_160); -return x_210; +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_208 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; +lean_inc(x_24); +x_209 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_209, 0, x_24); +lean_ctor_set(x_209, 1, x_166); +lean_ctor_set(x_209, 2, x_208); +lean_inc_n(x_168, 4); +lean_inc(x_24); +x_210 = l_Lean_Syntax_node6(x_24, x_5, x_168, x_168, x_168, x_168, x_209, x_168); +x_211 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_24); +x_212 = l_Lean_Syntax_node2(x_24, x_211, x_210, x_207); +x_213 = l_Lean_Syntax_node2(x_24, x_166, x_212, x_1); +x_214 = l_Lean_Elab_Command_elabCommand(x_213, x_8, x_9, x_164); +return x_214; } else { -lean_object* x_211; uint8_t 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; -x_211 = lean_ctor_get(x_4, 0); -x_212 = 1; -x_213 = l_Lean_SourceInfo_fromRef(x_211, x_212); -x_214 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; -x_215 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_215, 0, x_213); -lean_ctor_set(x_215, 1, x_214); -x_216 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; -lean_inc(x_20); -x_217 = l_Lean_Syntax_node1(x_20, x_216, x_215); -x_218 = l_Array_mkArray1___rarg(x_217); -x_219 = l_Array_append___rarg(x_163, x_218); -lean_dec(x_218); -lean_inc(x_20); -x_220 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_220, 0, x_20); -lean_ctor_set(x_220, 1, x_162); -lean_ctor_set(x_220, 2, x_219); -lean_inc_n(x_164, 4); -lean_inc(x_20); -x_221 = l_Lean_Syntax_node6(x_20, x_5, x_164, x_164, x_164, x_164, x_220, x_164); -x_222 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_20); -x_223 = l_Lean_Syntax_node2(x_20, x_222, x_221, x_203); -x_224 = l_Lean_Syntax_node2(x_20, x_162, x_223, x_1); -x_225 = l_Lean_Elab_Command_elabCommand(x_224, x_8, x_9, x_160); -return x_225; +lean_object* x_215; uint8_t 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; +x_215 = lean_ctor_get(x_4, 0); +x_216 = 1; +x_217 = l_Lean_SourceInfo_fromRef(x_215, x_216); +x_218 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; +x_219 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_219, 0, x_217); +lean_ctor_set(x_219, 1, x_218); +x_220 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; +lean_inc(x_24); +x_221 = l_Lean_Syntax_node1(x_24, x_220, x_219); +x_222 = l_Array_mkArray1___rarg(x_221); +x_223 = l_Array_append___rarg(x_167, x_222); +lean_dec(x_222); +lean_inc(x_24); +x_224 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_224, 0, x_24); +lean_ctor_set(x_224, 1, x_166); +lean_ctor_set(x_224, 2, x_223); +lean_inc_n(x_168, 4); +lean_inc(x_24); +x_225 = l_Lean_Syntax_node6(x_24, x_5, x_168, x_168, x_168, x_168, x_224, x_168); +x_226 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_24); +x_227 = l_Lean_Syntax_node2(x_24, x_226, x_225, x_207); +x_228 = l_Lean_Syntax_node2(x_24, x_166, x_227, x_1); +x_229 = l_Lean_Elab_Command_elabCommand(x_228, x_8, x_9, x_164); +return x_229; } } } else { -lean_object* x_226; lean_object* x_227; uint8_t 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; -x_226 = lean_ctor_get(x_15, 0); -x_227 = lean_ctor_get(x_15, 1); -lean_inc(x_227); -lean_inc(x_226); -lean_dec(x_15); -x_228 = 0; -x_229 = l_Lean_SourceInfo_fromRef(x_226, x_228); -lean_dec(x_226); -x_230 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_227); -x_231 = lean_ctor_get(x_230, 0); +lean_object* x_230; lean_object* x_231; uint8_t 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; +x_230 = lean_ctor_get(x_19, 0); +x_231 = lean_ctor_get(x_19, 1); lean_inc(x_231); -x_232 = lean_ctor_get(x_230, 1); -lean_inc(x_232); -if (lean_is_exclusive(x_230)) { - lean_ctor_release(x_230, 0); - lean_ctor_release(x_230, 1); - x_233 = x_230; -} else { - lean_dec_ref(x_230); - x_233 = lean_box(0); -} -x_234 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_232); +lean_inc(x_230); +lean_dec(x_19); +x_232 = 0; +x_233 = l_Lean_SourceInfo_fromRef(x_230, x_232); +lean_dec(x_230); +x_234 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_231); x_235 = lean_ctor_get(x_234, 0); lean_inc(x_235); x_236 = lean_ctor_get(x_234, 1); @@ -12899,196 +12914,196 @@ if (lean_is_exclusive(x_234)) { lean_dec_ref(x_234); x_237 = lean_box(0); } -x_238 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; -x_239 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -lean_inc(x_229); -x_240 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_240, 0, x_229); -lean_ctor_set(x_240, 1, x_238); -lean_ctor_set(x_240, 2, x_239); -x_241 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; -lean_inc(x_229); -if (lean_is_scalar(x_237)) { - x_242 = lean_alloc_ctor(2, 2, 0); -} else { - x_242 = x_237; - lean_ctor_set_tag(x_242, 2); -} -lean_ctor_set(x_242, 0, x_229); -lean_ctor_set(x_242, 1, x_241); -x_243 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; -lean_inc(x_231); -lean_inc(x_235); -x_244 = l_Lean_addMacroScope(x_235, x_243, x_231); -x_245 = lean_box(0); -x_246 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; -lean_inc(x_229); -x_247 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_247, 0, x_229); -lean_ctor_set(x_247, 1, x_246); -lean_ctor_set(x_247, 2, x_244); -lean_ctor_set(x_247, 3, x_245); -x_248 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; +x_238 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_236); +x_239 = lean_ctor_get(x_238, 0); +lean_inc(x_239); +x_240 = lean_ctor_get(x_238, 1); lean_inc(x_240); -lean_inc(x_229); -x_249 = l_Lean_Syntax_node2(x_229, x_248, x_247, x_240); -x_250 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; -lean_inc(x_229); -if (lean_is_scalar(x_233)) { - x_251 = lean_alloc_ctor(2, 2, 0); +if (lean_is_exclusive(x_238)) { + lean_ctor_release(x_238, 0); + lean_ctor_release(x_238, 1); + x_241 = x_238; } else { - x_251 = x_233; - lean_ctor_set_tag(x_251, 2); + lean_dec_ref(x_238); + x_241 = lean_box(0); +} +x_242 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; +x_243 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +lean_inc(x_233); +x_244 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_244, 0, x_233); +lean_ctor_set(x_244, 1, x_242); +lean_ctor_set(x_244, 2, x_243); +x_245 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; +lean_inc(x_233); +if (lean_is_scalar(x_241)) { + x_246 = lean_alloc_ctor(2, 2, 0); +} else { + x_246 = x_241; + lean_ctor_set_tag(x_246, 2); } -lean_ctor_set(x_251, 0, x_229); +lean_ctor_set(x_246, 0, x_233); +lean_ctor_set(x_246, 1, x_245); +x_247 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; +lean_inc(x_235); +lean_inc(x_239); +x_248 = l_Lean_addMacroScope(x_239, x_247, x_235); +x_249 = lean_box(0); +x_250 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; +lean_inc(x_233); +x_251 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_251, 0, x_233); lean_ctor_set(x_251, 1, x_250); -x_252 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; -x_253 = l_Lean_addMacroScope(x_235, x_252, x_231); -x_254 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; -x_255 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; -lean_inc(x_229); -x_256 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_256, 0, x_229); -lean_ctor_set(x_256, 1, x_254); -lean_ctor_set(x_256, 2, x_253); -lean_ctor_set(x_256, 3, x_255); -lean_inc(x_229); -x_257 = l_Lean_Syntax_node1(x_229, x_238, x_2); -x_258 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; -lean_inc(x_229); -x_259 = l_Lean_Syntax_node2(x_229, x_258, x_256, x_257); -x_260 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; -lean_inc(x_229); -x_261 = l_Lean_Syntax_node2(x_229, x_260, x_251, x_259); -lean_inc(x_229); -x_262 = l_Lean_Syntax_node1(x_229, x_238, x_261); -x_263 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; -lean_inc(x_240); -lean_inc(x_229); -x_264 = l_Lean_Syntax_node2(x_229, x_263, x_240, x_262); -x_265 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; -lean_inc(x_229); -x_266 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_266, 0, x_229); -lean_ctor_set(x_266, 1, x_265); -x_267 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; -lean_inc(x_229); -lean_ctor_set_tag(x_11, 2); -lean_ctor_set(x_11, 1, x_267); -lean_ctor_set(x_11, 0, x_229); -x_268 = lean_mk_syntax_ident(x_6); -x_269 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; -lean_inc(x_229); +lean_ctor_set(x_251, 2, x_248); +lean_ctor_set(x_251, 3, x_249); +x_252 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; +lean_inc(x_244); +lean_inc(x_233); +x_253 = l_Lean_Syntax_node2(x_233, x_252, x_251, x_244); +x_254 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; +lean_inc(x_233); +if (lean_is_scalar(x_237)) { + x_255 = lean_alloc_ctor(2, 2, 0); +} else { + x_255 = x_237; + lean_ctor_set_tag(x_255, 2); +} +lean_ctor_set(x_255, 0, x_233); +lean_ctor_set(x_255, 1, x_254); +x_256 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; +x_257 = l_Lean_addMacroScope(x_239, x_256, x_235); +x_258 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; +x_259 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; +lean_inc(x_233); +x_260 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_260, 0, x_233); +lean_ctor_set(x_260, 1, x_258); +lean_ctor_set(x_260, 2, x_257); +lean_ctor_set(x_260, 3, x_259); +lean_inc(x_233); +x_261 = l_Lean_Syntax_node1(x_233, x_242, x_2); +x_262 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; +lean_inc(x_233); +x_263 = l_Lean_Syntax_node2(x_233, x_262, x_260, x_261); +x_264 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; +lean_inc(x_233); +x_265 = l_Lean_Syntax_node2(x_233, x_264, x_255, x_263); +lean_inc(x_233); +x_266 = l_Lean_Syntax_node1(x_233, x_242, x_265); +x_267 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; +lean_inc(x_244); +lean_inc(x_233); +x_268 = l_Lean_Syntax_node2(x_233, x_267, x_244, x_266); +x_269 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; +lean_inc(x_233); x_270 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_270, 0, x_229); +lean_ctor_set(x_270, 0, x_233); lean_ctor_set(x_270, 1, x_269); -x_271 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; -lean_inc(x_229); -x_272 = l_Lean_Syntax_node2(x_229, x_271, x_270, x_3); -x_273 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; -lean_inc(x_240); -lean_inc(x_229); -x_274 = l_Lean_Syntax_node4(x_229, x_273, x_11, x_240, x_268, x_272); -x_275 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; -lean_inc_n(x_240, 2); -lean_inc(x_229); -x_276 = l_Lean_Syntax_node2(x_229, x_275, x_240, x_240); -x_277 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; -lean_inc(x_240); -lean_inc(x_229); -x_278 = l_Lean_Syntax_node4(x_229, x_277, x_266, x_274, x_276, x_240); -x_279 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; -lean_inc(x_240); -lean_inc(x_229); -x_280 = l_Lean_Syntax_node5(x_229, x_279, x_242, x_249, x_264, x_278, x_240); +x_271 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; +lean_inc(x_233); +lean_ctor_set_tag(x_15, 2); +lean_ctor_set(x_15, 1, x_271); +lean_ctor_set(x_15, 0, x_233); +x_272 = lean_mk_syntax_ident(x_6); +x_273 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; +lean_inc(x_233); +x_274 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_274, 0, x_233); +lean_ctor_set(x_274, 1, x_273); +x_275 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; +lean_inc(x_233); +x_276 = l_Lean_Syntax_node2(x_233, x_275, x_274, x_3); +x_277 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; +lean_inc(x_244); +lean_inc(x_233); +x_278 = l_Lean_Syntax_node4(x_233, x_277, x_15, x_244, x_272, x_276); +x_279 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; +lean_inc_n(x_244, 2); +lean_inc(x_233); +x_280 = l_Lean_Syntax_node2(x_233, x_279, x_244, x_244); +x_281 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; +lean_inc(x_244); +lean_inc(x_233); +x_282 = l_Lean_Syntax_node4(x_233, x_281, x_270, x_278, x_280, x_244); +x_283 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; +lean_inc(x_244); +lean_inc(x_233); +x_284 = l_Lean_Syntax_node5(x_233, x_283, x_246, x_253, x_268, x_282, x_244); if (lean_obj_tag(x_4) == 0) { -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; -x_281 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; -lean_inc(x_229); -x_282 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_282, 0, x_229); -lean_ctor_set(x_282, 1, x_238); -lean_ctor_set(x_282, 2, x_281); -lean_inc_n(x_240, 4); -lean_inc(x_229); -x_283 = l_Lean_Syntax_node6(x_229, x_5, x_240, x_240, x_240, x_240, x_282, x_240); -x_284 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_229); -x_285 = l_Lean_Syntax_node2(x_229, x_284, x_283, x_280); -x_286 = l_Lean_Syntax_node2(x_229, x_238, x_285, x_1); -x_287 = l_Lean_Elab_Command_elabCommand(x_286, x_8, x_9, x_236); -return x_287; -} -else -{ -lean_object* x_288; uint8_t 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; -x_288 = lean_ctor_get(x_4, 0); -x_289 = 1; -x_290 = l_Lean_SourceInfo_fromRef(x_288, x_289); -x_291 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; -x_292 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_292, 0, x_290); -lean_ctor_set(x_292, 1, x_291); -x_293 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; -lean_inc(x_229); -x_294 = l_Lean_Syntax_node1(x_229, x_293, x_292); -x_295 = l_Array_mkArray1___rarg(x_294); -x_296 = l_Array_append___rarg(x_239, x_295); -lean_dec(x_295); -lean_inc(x_229); -x_297 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_297, 0, x_229); -lean_ctor_set(x_297, 1, x_238); -lean_ctor_set(x_297, 2, x_296); -lean_inc_n(x_240, 4); -lean_inc(x_229); -x_298 = l_Lean_Syntax_node6(x_229, x_5, x_240, x_240, x_240, x_240, x_297, x_240); -x_299 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_229); -x_300 = l_Lean_Syntax_node2(x_229, x_299, x_298, x_280); -x_301 = l_Lean_Syntax_node2(x_229, x_238, x_300, x_1); -x_302 = l_Lean_Elab_Command_elabCommand(x_301, x_8, x_9, x_236); -return x_302; -} -} -} -else -{ -lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; uint8_t 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; -x_303 = lean_ctor_get(x_11, 1); -lean_inc(x_303); -lean_dec(x_11); -x_304 = l_Lean_Elab_Command_getRef(x_8, x_9, x_303); -x_305 = lean_ctor_get(x_304, 0); -lean_inc(x_305); -x_306 = lean_ctor_get(x_304, 1); -lean_inc(x_306); -if (lean_is_exclusive(x_304)) { - lean_ctor_release(x_304, 0); - lean_ctor_release(x_304, 1); - x_307 = x_304; -} else { - lean_dec_ref(x_304); - x_307 = lean_box(0); -} -x_308 = 0; -x_309 = l_Lean_SourceInfo_fromRef(x_305, x_308); -lean_dec(x_305); -x_310 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_306); -x_311 = lean_ctor_get(x_310, 0); -lean_inc(x_311); -x_312 = lean_ctor_get(x_310, 1); -lean_inc(x_312); -if (lean_is_exclusive(x_310)) { - lean_ctor_release(x_310, 0); - lean_ctor_release(x_310, 1); - x_313 = x_310; +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; +x_285 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; +lean_inc(x_233); +x_286 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_286, 0, x_233); +lean_ctor_set(x_286, 1, x_242); +lean_ctor_set(x_286, 2, x_285); +lean_inc_n(x_244, 4); +lean_inc(x_233); +x_287 = l_Lean_Syntax_node6(x_233, x_5, x_244, x_244, x_244, x_244, x_286, x_244); +x_288 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_233); +x_289 = l_Lean_Syntax_node2(x_233, x_288, x_287, x_284); +x_290 = l_Lean_Syntax_node2(x_233, x_242, x_289, x_1); +x_291 = l_Lean_Elab_Command_elabCommand(x_290, x_8, x_9, x_240); +return x_291; +} +else +{ +lean_object* x_292; uint8_t 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; +x_292 = lean_ctor_get(x_4, 0); +x_293 = 1; +x_294 = l_Lean_SourceInfo_fromRef(x_292, x_293); +x_295 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; +x_296 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_296, 0, x_294); +lean_ctor_set(x_296, 1, x_295); +x_297 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; +lean_inc(x_233); +x_298 = l_Lean_Syntax_node1(x_233, x_297, x_296); +x_299 = l_Array_mkArray1___rarg(x_298); +x_300 = l_Array_append___rarg(x_243, x_299); +lean_dec(x_299); +lean_inc(x_233); +x_301 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_301, 0, x_233); +lean_ctor_set(x_301, 1, x_242); +lean_ctor_set(x_301, 2, x_300); +lean_inc_n(x_244, 4); +lean_inc(x_233); +x_302 = l_Lean_Syntax_node6(x_233, x_5, x_244, x_244, x_244, x_244, x_301, x_244); +x_303 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_233); +x_304 = l_Lean_Syntax_node2(x_233, x_303, x_302, x_284); +x_305 = l_Lean_Syntax_node2(x_233, x_242, x_304, x_1); +x_306 = l_Lean_Elab_Command_elabCommand(x_305, x_8, x_9, x_240); +return x_306; +} +} +} +else +{ +lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; uint8_t 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; +x_307 = lean_ctor_get(x_15, 1); +lean_inc(x_307); +lean_dec(x_15); +x_308 = l_Lean_Elab_Command_getRef(x_8, x_9, x_307); +x_309 = lean_ctor_get(x_308, 0); +lean_inc(x_309); +x_310 = lean_ctor_get(x_308, 1); +lean_inc(x_310); +if (lean_is_exclusive(x_308)) { + lean_ctor_release(x_308, 0); + lean_ctor_release(x_308, 1); + x_311 = x_308; } else { - lean_dec_ref(x_310); - x_313 = lean_box(0); + lean_dec_ref(x_308); + x_311 = lean_box(0); } -x_314 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_312); +x_312 = 0; +x_313 = l_Lean_SourceInfo_fromRef(x_309, x_312); +lean_dec(x_309); +x_314 = l_Lean_Elab_Command_getCurrMacroScope(x_8, x_9, x_310); x_315 = lean_ctor_get(x_314, 0); lean_inc(x_315); x_316 = lean_ctor_get(x_314, 1); @@ -13101,162 +13116,175 @@ if (lean_is_exclusive(x_314)) { lean_dec_ref(x_314); x_317 = lean_box(0); } -x_318 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; -x_319 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -lean_inc(x_309); -x_320 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_320, 0, x_309); -lean_ctor_set(x_320, 1, x_318); -lean_ctor_set(x_320, 2, x_319); -x_321 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; -lean_inc(x_309); -if (lean_is_scalar(x_317)) { - x_322 = lean_alloc_ctor(2, 2, 0); -} else { - x_322 = x_317; - lean_ctor_set_tag(x_322, 2); -} -lean_ctor_set(x_322, 0, x_309); -lean_ctor_set(x_322, 1, x_321); -x_323 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; -lean_inc(x_311); -lean_inc(x_315); -x_324 = l_Lean_addMacroScope(x_315, x_323, x_311); -x_325 = lean_box(0); -x_326 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; -lean_inc(x_309); -x_327 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_327, 0, x_309); -lean_ctor_set(x_327, 1, x_326); -lean_ctor_set(x_327, 2, x_324); -lean_ctor_set(x_327, 3, x_325); -x_328 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; +x_318 = l_Lean_Elab_Command_getMainModule___rarg(x_9, x_316); +x_319 = lean_ctor_get(x_318, 0); +lean_inc(x_319); +x_320 = lean_ctor_get(x_318, 1); lean_inc(x_320); -lean_inc(x_309); -x_329 = l_Lean_Syntax_node2(x_309, x_328, x_327, x_320); -x_330 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; -lean_inc(x_309); -if (lean_is_scalar(x_313)) { - x_331 = lean_alloc_ctor(2, 2, 0); +if (lean_is_exclusive(x_318)) { + lean_ctor_release(x_318, 0); + lean_ctor_release(x_318, 1); + x_321 = x_318; +} else { + lean_dec_ref(x_318); + x_321 = lean_box(0); +} +x_322 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; +x_323 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +lean_inc(x_313); +x_324 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_324, 0, x_313); +lean_ctor_set(x_324, 1, x_322); +lean_ctor_set(x_324, 2, x_323); +x_325 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__14; +lean_inc(x_313); +if (lean_is_scalar(x_321)) { + x_326 = lean_alloc_ctor(2, 2, 0); } else { - x_331 = x_313; - lean_ctor_set_tag(x_331, 2); + x_326 = x_321; + lean_ctor_set_tag(x_326, 2); } -lean_ctor_set(x_331, 0, x_309); +lean_ctor_set(x_326, 0, x_313); +lean_ctor_set(x_326, 1, x_325); +x_327 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__19; +lean_inc(x_315); +lean_inc(x_319); +x_328 = l_Lean_addMacroScope(x_319, x_327, x_315); +x_329 = lean_box(0); +x_330 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__18; +lean_inc(x_313); +x_331 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_331, 0, x_313); lean_ctor_set(x_331, 1, x_330); -x_332 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; -x_333 = l_Lean_addMacroScope(x_315, x_332, x_311); -x_334 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; -x_335 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; -lean_inc(x_309); -x_336 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_336, 0, x_309); -lean_ctor_set(x_336, 1, x_334); -lean_ctor_set(x_336, 2, x_333); -lean_ctor_set(x_336, 3, x_335); -lean_inc(x_309); -x_337 = l_Lean_Syntax_node1(x_309, x_318, x_2); -x_338 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; -lean_inc(x_309); -x_339 = l_Lean_Syntax_node2(x_309, x_338, x_336, x_337); -x_340 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; -lean_inc(x_309); -x_341 = l_Lean_Syntax_node2(x_309, x_340, x_331, x_339); -lean_inc(x_309); -x_342 = l_Lean_Syntax_node1(x_309, x_318, x_341); -x_343 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; -lean_inc(x_320); -lean_inc(x_309); -x_344 = l_Lean_Syntax_node2(x_309, x_343, x_320, x_342); -x_345 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; -lean_inc(x_309); -if (lean_is_scalar(x_307)) { - x_346 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_331, 2, x_328); +lean_ctor_set(x_331, 3, x_329); +x_332 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__16; +lean_inc(x_324); +lean_inc(x_313); +x_333 = l_Lean_Syntax_node2(x_313, x_332, x_331, x_324); +x_334 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__24; +lean_inc(x_313); +if (lean_is_scalar(x_317)) { + x_335 = lean_alloc_ctor(2, 2, 0); } else { - x_346 = x_307; - lean_ctor_set_tag(x_346, 2); -} -lean_ctor_set(x_346, 0, x_309); -lean_ctor_set(x_346, 1, x_345); -x_347 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; -lean_inc(x_309); -x_348 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_348, 0, x_309); -lean_ctor_set(x_348, 1, x_347); -x_349 = lean_mk_syntax_ident(x_6); -x_350 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; -lean_inc(x_309); -x_351 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_351, 0, x_309); -lean_ctor_set(x_351, 1, x_350); -x_352 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; -lean_inc(x_309); -x_353 = l_Lean_Syntax_node2(x_309, x_352, x_351, x_3); -x_354 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; -lean_inc(x_320); -lean_inc(x_309); -x_355 = l_Lean_Syntax_node4(x_309, x_354, x_348, x_320, x_349, x_353); -x_356 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; -lean_inc_n(x_320, 2); -lean_inc(x_309); -x_357 = l_Lean_Syntax_node2(x_309, x_356, x_320, x_320); -x_358 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; -lean_inc(x_320); -lean_inc(x_309); -x_359 = l_Lean_Syntax_node4(x_309, x_358, x_346, x_355, x_357, x_320); -x_360 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; -lean_inc(x_320); -lean_inc(x_309); -x_361 = l_Lean_Syntax_node5(x_309, x_360, x_322, x_329, x_344, x_359, x_320); + x_335 = x_317; + lean_ctor_set_tag(x_335, 2); +} +lean_ctor_set(x_335, 0, x_313); +lean_ctor_set(x_335, 1, x_334); +x_336 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__29; +x_337 = l_Lean_addMacroScope(x_319, x_336, x_315); +x_338 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__28; +x_339 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__33; +lean_inc(x_313); +x_340 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_340, 0, x_313); +lean_ctor_set(x_340, 1, x_338); +lean_ctor_set(x_340, 2, x_337); +lean_ctor_set(x_340, 3, x_339); +lean_inc(x_313); +x_341 = l_Lean_Syntax_node1(x_313, x_322, x_2); +x_342 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__26; +lean_inc(x_313); +x_343 = l_Lean_Syntax_node2(x_313, x_342, x_340, x_341); +x_344 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__23; +lean_inc(x_313); +x_345 = l_Lean_Syntax_node2(x_313, x_344, x_335, x_343); +lean_inc(x_313); +x_346 = l_Lean_Syntax_node1(x_313, x_322, x_345); +x_347 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__21; +lean_inc(x_324); +lean_inc(x_313); +x_348 = l_Lean_Syntax_node2(x_313, x_347, x_324, x_346); +x_349 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; +lean_inc(x_313); +if (lean_is_scalar(x_311)) { + x_350 = lean_alloc_ctor(2, 2, 0); +} else { + x_350 = x_311; + lean_ctor_set_tag(x_350, 2); +} +lean_ctor_set(x_350, 0, x_313); +lean_ctor_set(x_350, 1, x_349); +x_351 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__3; +lean_inc(x_313); +x_352 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_352, 0, x_313); +lean_ctor_set(x_352, 1, x_351); +x_353 = lean_mk_syntax_ident(x_6); +x_354 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__43; +lean_inc(x_313); +x_355 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_355, 0, x_313); +lean_ctor_set(x_355, 1, x_354); +x_356 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__44; +lean_inc(x_313); +x_357 = l_Lean_Syntax_node2(x_313, x_356, x_355, x_3); +x_358 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__2; +lean_inc(x_324); +lean_inc(x_313); +x_359 = l_Lean_Syntax_node4(x_313, x_358, x_352, x_324, x_353, x_357); +x_360 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__47; +lean_inc_n(x_324, 2); +lean_inc(x_313); +x_361 = l_Lean_Syntax_node2(x_313, x_360, x_324, x_324); +x_362 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__42; +lean_inc(x_324); +lean_inc(x_313); +x_363 = l_Lean_Syntax_node4(x_313, x_362, x_350, x_359, x_361, x_324); +x_364 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__9; +lean_inc(x_324); +lean_inc(x_313); +x_365 = l_Lean_Syntax_node5(x_313, x_364, x_326, x_333, x_348, x_363, x_324); if (lean_obj_tag(x_4) == 0) { -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; -x_362 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; -lean_inc(x_309); -x_363 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_363, 0, x_309); -lean_ctor_set(x_363, 1, x_318); -lean_ctor_set(x_363, 2, x_362); -lean_inc_n(x_320, 4); -lean_inc(x_309); -x_364 = l_Lean_Syntax_node6(x_309, x_5, x_320, x_320, x_320, x_320, x_363, x_320); -x_365 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_309); -x_366 = l_Lean_Syntax_node2(x_309, x_365, x_364, x_361); -x_367 = l_Lean_Syntax_node2(x_309, x_318, x_366, x_1); -x_368 = l_Lean_Elab_Command_elabCommand(x_367, x_8, x_9, x_316); -return x_368; -} -else -{ -lean_object* x_369; uint8_t 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; -x_369 = lean_ctor_get(x_4, 0); -x_370 = 1; -x_371 = l_Lean_SourceInfo_fromRef(x_369, x_370); -x_372 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; -x_373 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_373, 0, x_371); -lean_ctor_set(x_373, 1, x_372); -x_374 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; -lean_inc(x_309); -x_375 = l_Lean_Syntax_node1(x_309, x_374, x_373); -x_376 = l_Array_mkArray1___rarg(x_375); -x_377 = l_Array_append___rarg(x_319, x_376); -lean_dec(x_376); -lean_inc(x_309); -x_378 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_378, 0, x_309); -lean_ctor_set(x_378, 1, x_318); -lean_ctor_set(x_378, 2, x_377); -lean_inc_n(x_320, 4); -lean_inc(x_309); -x_379 = l_Lean_Syntax_node6(x_309, x_5, x_320, x_320, x_320, x_320, x_378, x_320); -x_380 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; -lean_inc(x_309); -x_381 = l_Lean_Syntax_node2(x_309, x_380, x_379, x_361); -x_382 = l_Lean_Syntax_node2(x_309, x_318, x_381, x_1); -x_383 = l_Lean_Elab_Command_elabCommand(x_382, x_8, x_9, x_316); -return x_383; +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; +x_366 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__48; +lean_inc(x_313); +x_367 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_367, 0, x_313); +lean_ctor_set(x_367, 1, x_322); +lean_ctor_set(x_367, 2, x_366); +lean_inc_n(x_324, 4); +lean_inc(x_313); +x_368 = l_Lean_Syntax_node6(x_313, x_5, x_324, x_324, x_324, x_324, x_367, x_324); +x_369 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_313); +x_370 = l_Lean_Syntax_node2(x_313, x_369, x_368, x_365); +x_371 = l_Lean_Syntax_node2(x_313, x_322, x_370, x_1); +x_372 = l_Lean_Elab_Command_elabCommand(x_371, x_8, x_9, x_320); +return x_372; +} +else +{ +lean_object* x_373; uint8_t 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; +x_373 = lean_ctor_get(x_4, 0); +x_374 = 1; +x_375 = l_Lean_SourceInfo_fromRef(x_373, x_374); +x_376 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__4; +x_377 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_377, 0, x_375); +lean_ctor_set(x_377, 1, x_376); +x_378 = l_Lean_Elab_Command_elabInitialize___lambda__2___closed__5; +lean_inc(x_313); +x_379 = l_Lean_Syntax_node1(x_313, x_378, x_377); +x_380 = l_Array_mkArray1___rarg(x_379); +x_381 = l_Array_append___rarg(x_323, x_380); +lean_dec(x_380); +lean_inc(x_313); +x_382 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_382, 0, x_313); +lean_ctor_set(x_382, 1, x_322); +lean_ctor_set(x_382, 2, x_381); +lean_inc_n(x_324, 4); +lean_inc(x_313); +x_383 = l_Lean_Syntax_node6(x_313, x_5, x_324, x_324, x_324, x_324, x_382, x_324); +x_384 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__5; +lean_inc(x_313); +x_385 = l_Lean_Syntax_node2(x_313, x_384, x_383, x_365); +x_386 = l_Lean_Syntax_node2(x_313, x_322, x_385, x_1); +x_387 = l_Lean_Elab_Command_elabCommand(x_386, x_8, x_9, x_320); +return x_387; } } } @@ -13294,7 +13322,7 @@ static lean_object* _init_l_Lean_Elab_Command_elabInitialize___lambda__3___close { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(2); -x_2 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_2 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; x_3 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__4; x_4 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_4, 0, x_1); @@ -13423,7 +13451,7 @@ lean_inc(x_44); lean_ctor_set_tag(x_49, 2); lean_ctor_set(x_49, 1, x_53); lean_ctor_set(x_49, 0, x_44); -x_54 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_54 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; x_55 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; lean_inc(x_44); x_56 = lean_alloc_ctor(1, 3, 0); @@ -13609,7 +13637,7 @@ lean_inc(x_44); x_117 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_117, 0, x_44); lean_ctor_set(x_117, 1, x_116); -x_118 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_118 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; x_119 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; lean_inc(x_44); x_120 = lean_alloc_ctor(1, 3, 0); @@ -13814,7 +13842,7 @@ if (lean_is_scalar(x_183)) { } lean_ctor_set(x_185, 0, x_44); lean_ctor_set(x_185, 1, x_184); -x_186 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_186 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; x_187 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; lean_inc(x_44); x_188 = lean_alloc_ctor(1, 3, 0); @@ -14035,7 +14063,7 @@ if (lean_is_scalar(x_258)) { } lean_ctor_set(x_260, 0, x_250); lean_ctor_set(x_260, 1, x_259); -x_261 = l_Lean_Elab_Command_expandNamespacedDeclaration___closed__2; +x_261 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2; x_262 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; lean_inc(x_250); x_263 = lean_alloc_ctor(1, 3, 0); @@ -15205,7 +15233,7 @@ x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__1() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -15215,37 +15243,37 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__2() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__1; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__1; x_2 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__3() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__2; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__2; x_2 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__4() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__3; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__3; x_2 = l_Lean_Elab_Command_elabInitialize___lambda__1___closed__17; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__5() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__5() { _start: { lean_object* x_1; @@ -15253,37 +15281,37 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__6() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__4; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__4; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__7() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__6; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__6; x_2 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isNamedDef___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__8() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__7; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__7; x_2 = l_Lean_Elab_Command_elabAxiom___lambda__4___closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__9() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__9() { _start: { lean_object* x_1; @@ -15291,17 +15319,17 @@ x_1 = lean_mk_string_unchecked("Declaration", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__10() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__8; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__9; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__8; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__9; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__11() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__11() { _start: { lean_object* x_1; @@ -15309,33 +15337,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__12() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__10; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__11; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__10; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__11; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__13() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__12; -x_2 = lean_unsigned_to_nat(9024u); +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__12; +x_2 = lean_unsigned_to_nat(9009u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009_(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_Command_elabAxiom___lambda__4___closed__7; x_3 = 0; -x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__13; +x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__13; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -15453,6 +15481,10 @@ l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDefName___closed__4 = lean_mark_persistent(l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_setDefName___closed__4); l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3___closed__1 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3___closed__1(); lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3___closed__1); +l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__1 = _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__1); +l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2 = _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___lambda__1___closed__2); l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__1 = _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__1(); lean_mark_persistent(l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__1); l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__2 = _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__2(); @@ -15547,10 +15579,6 @@ l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3 = _init_l_Lean_Elab_ lean_mark_persistent(l_Lean_Elab_Command_expandNamespacedDeclaration___closed__3); l_Lean_Elab_Command_expandNamespacedDeclaration___closed__4 = _init_l_Lean_Elab_Command_expandNamespacedDeclaration___closed__4(); lean_mark_persistent(l_Lean_Elab_Command_expandNamespacedDeclaration___closed__4); -l_Lean_Elab_Command_expandNamespacedDeclaration___closed__5 = _init_l_Lean_Elab_Command_expandNamespacedDeclaration___closed__5(); -lean_mark_persistent(l_Lean_Elab_Command_expandNamespacedDeclaration___closed__5); -l_Lean_Elab_Command_expandNamespacedDeclaration___closed__6 = _init_l_Lean_Elab_Command_expandNamespacedDeclaration___closed__6(); -lean_mark_persistent(l_Lean_Elab_Command_expandNamespacedDeclaration___closed__6); l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration__1___closed__1 = _init_l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration__1___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration__1___closed__1); l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration__1___closed__2 = _init_l___regBuiltin_Lean_Elab_Command_expandNamespacedDeclaration__1___closed__2(); @@ -15995,33 +16023,33 @@ lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_elabInitialize__1___closed if (builtin) {res = l___regBuiltin_Lean_Elab_Command_elabInitialize__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__1); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__2); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__3(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__3); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__4(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__4); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__5(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__5); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__6(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__6); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__7 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__7(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__7); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__8 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__8(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__8); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__9 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__9(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__9); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__10 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__10(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__10); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__11 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__11(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__11); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__12 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__12(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__12); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__13 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__13(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024____closed__13); -if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9024_(lean_io_mk_world()); +}l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__1); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__2); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__3); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__4(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__4); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__5(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__5); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__6(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__6); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__7 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__7(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__7); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__8 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__8(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__8); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__9 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__9(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__9); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__10 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__10(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__10); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__11 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__11(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__11); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__12 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__12(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__12); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__13 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__13(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009____closed__13); +if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_9009_(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/DeclarationRange.c b/stage0/stdlib/Lean/Elab/DeclarationRange.c index 675fa967f956..e8ac762aca59 100644 --- a/stage0/stdlib/Lean/Elab/DeclarationRange.c +++ b/stage0/stdlib/Lean/Elab/DeclarationRange.c @@ -13,192 +13,143 @@ #ifdef __cplusplus extern "C" { #endif +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addDeclarationRanges___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges(lean_object*); -lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); -lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange(lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationSelectionRef(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_addDeclarationRanges___rarg___closed__2; lean_object* l_Lean_Syntax_getKind(lean_object*); +static lean_object* l_Lean_Elab_addDeclarationRanges___rarg___lambda__3___closed__1; uint8_t lean_name_eq(lean_object*, lean_object*); +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_Elab_addDeclarationRanges___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isIdent(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FileMap_leanPosToLspPos(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_getDeclarationSelectionRef___closed__2; uint8_t l_Lean_Syntax_isNone(lean_object*); static lean_object* l_Lean_Elab_getDeclarationSelectionRef___closed__1; +lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges(lean_object*); +lean_object* lean_array_mk(lean_object*); +static lean_object* l_Lean_Elab_addDeclarationRanges___rarg___lambda__3___closed__2; static lean_object* l_Lean_Elab_addDeclarationRanges___rarg___closed__1; lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_getDeclarationSelectionRef___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_getDeclarationSelectionRef___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_getDeclarationSelectionRef___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_4 = 0; -x_5 = l_Lean_Syntax_getPos_x3f(x_1, x_4); -x_6 = l_Lean_Syntax_getTailPos_x3f(x_1, x_4); -if (lean_obj_tag(x_5) == 0) -{ -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_2, 0); -lean_inc(x_7); -lean_dec(x_2); -x_8 = lean_ctor_get(x_7, 1); -lean_inc(x_8); -lean_dec(x_7); -x_9 = lean_unsigned_to_nat(0u); +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; 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_4 = lean_ctor_get(x_1, 0); lean_inc(x_3); -x_10 = l_Lean_FileMap_toPosition(x_3, x_9); -lean_inc(x_10); -x_11 = l_Lean_FileMap_leanPosToLspPos(x_3, x_10); -if (lean_obj_tag(x_6) == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; -lean_dec(x_3); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -lean_inc(x_12); -lean_inc(x_10); -x_13 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_13, 0, x_10); -lean_ctor_set(x_13, 1, x_12); -lean_ctor_set(x_13, 2, x_10); -lean_ctor_set(x_13, 3, x_12); -x_14 = lean_apply_2(x_8, lean_box(0), 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; lean_object* x_21; -x_15 = lean_ctor_get(x_11, 1); -lean_inc(x_15); -lean_dec(x_11); -x_16 = lean_ctor_get(x_6, 0); -lean_inc(x_16); -lean_dec(x_6); +x_5 = l_Lean_FileMap_toPosition(x_3, x_4); +x_6 = lean_ctor_get(x_1, 1); lean_inc(x_3); -x_17 = l_Lean_FileMap_toPosition(x_3, x_16); -lean_dec(x_16); -lean_inc(x_17); -x_18 = l_Lean_FileMap_leanPosToLspPos(x_3, x_17); +x_7 = l_Lean_FileMap_toPosition(x_3, x_6); +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); +lean_dec(x_2); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +lean_inc(x_5); +x_10 = l_Lean_FileMap_leanPosToLspPos(x_3, x_5); +x_11 = lean_ctor_get(x_10, 1); +lean_inc(x_11); +lean_dec(x_10); +lean_inc(x_7); +x_12 = l_Lean_FileMap_leanPosToLspPos(x_3, x_7); lean_dec(x_3); -x_19 = lean_ctor_get(x_18, 1); -lean_inc(x_19); -lean_dec(x_18); -x_20 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_20, 0, x_10); -lean_ctor_set(x_20, 1, x_15); -lean_ctor_set(x_20, 2, x_17); -lean_ctor_set(x_20, 3, x_19); -x_21 = lean_apply_2(x_8, lean_box(0), x_20); -return x_21; +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_14, 0, x_5); +lean_ctor_set(x_14, 1, x_11); +lean_ctor_set(x_14, 2, x_7); +lean_ctor_set(x_14, 3, x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_14); +x_16 = lean_apply_2(x_9, lean_box(0), x_15); +return x_16; } } -else +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: { -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_2, 0); -lean_inc(x_22); -lean_dec(x_2); -x_23 = lean_ctor_get(x_22, 1); -lean_inc(x_23); -lean_dec(x_22); -x_24 = lean_ctor_get(x_5, 0); -lean_inc(x_24); -lean_dec(x_5); -lean_inc(x_3); -x_25 = l_Lean_FileMap_toPosition(x_3, x_24); -lean_dec(x_24); -lean_inc(x_25); -x_26 = l_Lean_FileMap_leanPosToLspPos(x_3, x_25); -if (lean_obj_tag(x_6) == 0) +uint8_t x_4; lean_object* x_5; +x_4 = 0; +x_5 = l_Lean_Syntax_getRange_x3f(x_3, x_4); +if (lean_obj_tag(x_5) == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -lean_dec(x_3); -x_27 = lean_ctor_get(x_26, 1); -lean_inc(x_27); -lean_dec(x_26); -lean_inc(x_27); -lean_inc(x_25); -x_28 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_28, 0, x_25); -lean_ctor_set(x_28, 1, x_27); -lean_ctor_set(x_28, 2, x_25); -lean_ctor_set(x_28, 3, x_27); -x_29 = lean_apply_2(x_23, lean_box(0), x_28); -return x_29; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_dec(x_2); +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_box(0); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; } 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 = lean_ctor_get(x_26, 1); -lean_inc(x_30); -lean_dec(x_26); -x_31 = lean_ctor_get(x_6, 0); -lean_inc(x_31); -lean_dec(x_6); -lean_inc(x_3); -x_32 = l_Lean_FileMap_toPosition(x_3, x_31); -lean_dec(x_31); -lean_inc(x_32); -x_33 = l_Lean_FileMap_leanPosToLspPos(x_3, x_32); -lean_dec(x_3); -x_34 = lean_ctor_get(x_33, 1); -lean_inc(x_34); -lean_dec(x_33); -x_35 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_35, 0, x_25); -lean_ctor_set(x_35, 1, x_30); -lean_ctor_set(x_35, 2, x_32); -lean_ctor_set(x_35, 3, x_34); -x_36 = lean_apply_2(x_23, lean_box(0), x_35); -return x_36; -} +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_Lean_Elab_getDeclarationRange_x3f___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_12, 0, x_10); +lean_closure_set(x_12, 1, x_1); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_2, x_12); +return x_13; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f(lean_object* x_1) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_4 = lean_ctor_get(x_1, 1); -lean_inc(x_4); -x_5 = lean_alloc_closure((void*)(l_Lean_Elab_getDeclarationRange___rarg___lambda__1___boxed), 3, 2); -lean_closure_set(x_5, 0, x_3); -lean_closure_set(x_5, 1, x_1); -x_6 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_2, x_5); -return x_6; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_getDeclarationRange_x3f___rarg___boxed), 3, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_getDeclarationRange___rarg), 3, 0); -return x_2; +lean_object* x_4; +x_4 = l_Lean_Elab_getDeclarationRange_x3f___rarg___lambda__1(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Lean_Elab_getDeclarationRange___rarg___lambda__1(x_1, x_2, x_3); -lean_dec(x_1); +x_4 = l_Lean_Elab_getDeclarationRange_x3f___rarg(x_1, x_2, x_3); +lean_dec(x_3); return x_4; } } @@ -317,29 +268,130 @@ return x_17; LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___rarg___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; lean_object* x_7; -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -x_7 = l_Lean_addDeclarationRanges___rarg(x_2, x_3, x_4, x_6); -return x_7; +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_box(0); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_2); +lean_ctor_set(x_11, 1, x_10); +x_12 = l_Lean_addDeclarationRanges___rarg(x_1, x_3, x_4, x_11); +return x_12; +} } } LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___rarg___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: { +if (lean_obj_tag(x_7) == 0) +{ lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_8 = l_Lean_Elab_getDeclarationSelectionRef(x_1); -lean_inc(x_2); -x_9 = l_Lean_Elab_getDeclarationRange___rarg(x_2, x_3, x_8); -x_10 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRanges___rarg___lambda__1), 5, 4); -lean_closure_set(x_10, 0, x_7); -lean_closure_set(x_10, 1, x_2); -lean_closure_set(x_10, 2, x_4); -lean_closure_set(x_10, 3, x_5); -x_11 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_9, x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +lean_dec(x_1); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_box(0); +x_11 = lean_apply_2(x_9, lean_box(0), x_10); return x_11; } +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_12 = lean_ctor_get(x_7, 0); +lean_inc(x_12); +lean_dec(x_7); +x_13 = l_Lean_Elab_getDeclarationSelectionRef(x_2); +lean_inc(x_1); +x_14 = l_Lean_Elab_getDeclarationRange_x3f___rarg(x_1, x_3, x_13); +lean_dec(x_13); +x_15 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRanges___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_15, 0, x_1); +lean_closure_set(x_15, 1, x_12); +lean_closure_set(x_15, 2, x_4); +lean_closure_set(x_15, 3, x_5); +x_16 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_14, x_15); +return x_16; +} +} +} +static lean_object* _init_l_Lean_Elab_addDeclarationRanges___rarg___lambda__3___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("null", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_addDeclarationRanges___rarg___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_Lean_Elab_addDeclarationRanges___rarg___lambda__3___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___rarg___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) { +_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; lean_object* x_18; +x_8 = lean_box(0); +lean_inc(x_1); +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_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_2); +lean_ctor_set(x_10, 1, x_9); +x_11 = lean_array_mk(x_10); +x_12 = lean_box(2); +x_13 = l_Lean_Elab_addDeclarationRanges___rarg___lambda__3___closed__2; +x_14 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +lean_ctor_set(x_14, 2, x_11); +x_15 = lean_ctor_get(x_3, 1); +lean_inc(x_15); +lean_inc(x_4); +lean_inc(x_3); +x_16 = l_Lean_Elab_getDeclarationRange_x3f___rarg(x_3, x_4, x_14); +lean_dec(x_14); +lean_inc(x_15); +x_17 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRanges___rarg___lambda__2), 7, 6); +lean_closure_set(x_17, 0, x_3); +lean_closure_set(x_17, 1, x_1); +lean_closure_set(x_17, 2, x_4); +lean_closure_set(x_17, 3, x_5); +lean_closure_set(x_17, 4, x_6); +lean_closure_set(x_17, 5, x_15); +x_18 = lean_apply_4(x_15, lean_box(0), lean_box(0), x_16, x_17); +return x_18; +} } static lean_object* _init_l_Lean_Elab_addDeclarationRanges___rarg___closed__1() { _start: @@ -361,51 +413,52 @@ x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___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_Lean_Elab_addDeclarationRanges___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_6; lean_object* x_7; uint8_t x_8; -lean_inc(x_5); -x_6 = l_Lean_Syntax_getKind(x_5); -x_7 = l_Lean_Elab_addDeclarationRanges___rarg___closed__2; -x_8 = lean_name_eq(x_6, x_7); -lean_dec(x_6); -if (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_1, 1); -lean_inc(x_9); -lean_inc(x_5); -lean_inc(x_3); +lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; lean_inc(x_1); -x_10 = l_Lean_Elab_getDeclarationRange___rarg(x_1, x_3, x_5); -lean_inc(x_9); -x_11 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRanges___rarg___lambda__2), 7, 6); -lean_closure_set(x_11, 0, x_5); -lean_closure_set(x_11, 1, x_1); -lean_closure_set(x_11, 2, x_3); -lean_closure_set(x_11, 3, x_2); -lean_closure_set(x_11, 4, x_4); -lean_closure_set(x_11, 5, x_9); -x_12 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_10, x_11); -return x_12; +lean_inc(x_6); +x_7 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRanges___rarg___lambda__3___boxed), 7, 6); +lean_closure_set(x_7, 0, x_6); +lean_closure_set(x_7, 1, x_5); +lean_closure_set(x_7, 2, x_1); +lean_closure_set(x_7, 3, x_3); +lean_closure_set(x_7, 4, x_2); +lean_closure_set(x_7, 5, x_4); +x_8 = l_Lean_Syntax_getKind(x_6); +x_9 = l_Lean_Elab_addDeclarationRanges___rarg___closed__2; +x_10 = lean_name_eq(x_8, x_9); +lean_dec(x_8); +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; +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +lean_dec(x_1); +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_box(0); +x_15 = lean_apply_2(x_13, lean_box(0), x_14); +x_16 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_15, x_7); +return x_16; } else { -lean_object* x_13; lean_object* x_14; 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_13 = lean_ctor_get(x_1, 0); -lean_inc(x_13); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_dec(x_7); +x_17 = lean_ctor_get(x_1, 0); +lean_inc(x_17); lean_dec(x_1); -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -lean_dec(x_13); -x_15 = lean_box(0); -x_16 = lean_apply_2(x_14, lean_box(0), x_15); -return x_16; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_19 = lean_box(0); +x_20 = lean_apply_2(x_18, lean_box(0), x_19); +return x_20; } } } @@ -413,23 +466,64 @@ LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRanges___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRanges___rarg), 6, 0); return x_2; } } +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___rarg___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_Lean_Elab_addDeclarationRanges___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___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) { +_start: +{ +lean_object* x_8; +x_8 = l_Lean_Elab_addDeclarationRanges___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_7); +return x_8; +} +} LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___rarg___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; lean_object* x_10; +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +lean_dec(x_1); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_box(0); +x_11 = lean_apply_2(x_9, lean_box(0), x_10); +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_7, 0); +lean_inc(x_12); +lean_dec(x_7); lean_inc(x_1); -x_8 = l_Lean_Elab_getDeclarationRange___rarg(x_1, x_2, x_3); -x_9 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRanges___rarg___lambda__1), 5, 4); -lean_closure_set(x_9, 0, x_7); -lean_closure_set(x_9, 1, x_1); -lean_closure_set(x_9, 2, x_4); -lean_closure_set(x_9, 3, x_5); -x_10 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_8, x_9); -return x_10; +x_13 = l_Lean_Elab_getDeclarationRange_x3f___rarg(x_1, x_2, x_3); +x_14 = lean_alloc_closure((void*)(l_Lean_Elab_addDeclarationRanges___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_14, 0, x_1); +lean_closure_set(x_14, 1, x_12); +lean_closure_set(x_14, 2, x_4); +lean_closure_set(x_14, 3, x_5); +x_15 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_13, x_14); +return x_15; +} } } LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___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) { @@ -440,9 +534,9 @@ x_7 = lean_ctor_get(x_1, 1); lean_inc(x_7); lean_inc(x_3); lean_inc(x_1); -x_8 = l_Lean_Elab_getDeclarationRange___rarg(x_1, x_3, x_5); +x_8 = l_Lean_Elab_getDeclarationRange_x3f___rarg(x_1, x_3, x_5); lean_inc(x_7); -x_9 = lean_alloc_closure((void*)(l_Lean_Elab_addAuxDeclarationRanges___rarg___lambda__1), 7, 6); +x_9 = lean_alloc_closure((void*)(l_Lean_Elab_addAuxDeclarationRanges___rarg___lambda__1___boxed), 7, 6); lean_closure_set(x_9, 0, x_1); lean_closure_set(x_9, 1, x_3); lean_closure_set(x_9, 2, x_6); @@ -457,10 +551,28 @@ LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_addAuxDeclarationRanges___rarg), 6, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_addAuxDeclarationRanges___rarg___boxed), 6, 0); return x_2; } } +LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___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) { +_start: +{ +lean_object* x_8; +x_8 = l_Lean_Elab_addAuxDeclarationRanges___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_3); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___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_Elab_addAuxDeclarationRanges___rarg(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_5); +return x_7; +} +} lean_object* initialize_Lean_Log(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Parser_Command(uint8_t builtin, lean_object*); lean_object* initialize_Lean_DeclarationRange(uint8_t builtin, lean_object*); @@ -492,6 +604,10 @@ l_Lean_Elab_getDeclarationSelectionRef___closed__4 = _init_l_Lean_Elab_getDeclar lean_mark_persistent(l_Lean_Elab_getDeclarationSelectionRef___closed__4); l_Lean_Elab_getDeclarationSelectionRef___closed__5 = _init_l_Lean_Elab_getDeclarationSelectionRef___closed__5(); lean_mark_persistent(l_Lean_Elab_getDeclarationSelectionRef___closed__5); +l_Lean_Elab_addDeclarationRanges___rarg___lambda__3___closed__1 = _init_l_Lean_Elab_addDeclarationRanges___rarg___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Elab_addDeclarationRanges___rarg___lambda__3___closed__1); +l_Lean_Elab_addDeclarationRanges___rarg___lambda__3___closed__2 = _init_l_Lean_Elab_addDeclarationRanges___rarg___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Elab_addDeclarationRanges___rarg___lambda__3___closed__2); l_Lean_Elab_addDeclarationRanges___rarg___closed__1 = _init_l_Lean_Elab_addDeclarationRanges___rarg___closed__1(); lean_mark_persistent(l_Lean_Elab_addDeclarationRanges___rarg___closed__1); l_Lean_Elab_addDeclarationRanges___rarg___closed__2 = _init_l_Lean_Elab_addDeclarationRanges___rarg___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/DefView.c b/stage0/stdlib/Lean/Elab/DefView.c index fdefcf32ea6c..2d58b955f865 100644 --- a/stage0/stdlib/Lean/Elab/DefView.c +++ b/stage0/stdlib/Lean/Elab/DefView.c @@ -1005,20 +1005,22 @@ return x_6; static lean_object* _init_l_Lean_Elab_instInhabitedDefView___closed__1() { _start: { -lean_object* x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; x_1 = lean_box(0); -x_2 = 0; +x_2 = lean_box(0); x_3 = 0; x_4 = 0; -x_5 = l_Lean_Elab_instInhabitedDefViewElabHeaderData___closed__1; -x_6 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -lean_ctor_set_uint8(x_6, sizeof(void*)*2, x_2); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 1, x_3); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 2, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 3, x_3); -return x_6; +x_5 = 0; +x_6 = l_Lean_Elab_instInhabitedDefViewElabHeaderData___closed__1; +x_7 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_7, 0, x_2); +lean_ctor_set(x_7, 1, x_1); +lean_ctor_set(x_7, 2, x_6); +lean_ctor_set_uint8(x_7, sizeof(void*)*3, x_3); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 1, x_4); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 2, x_5); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 3, x_4); +return x_7; } } static lean_object* _init_l_Lean_Elab_instInhabitedDefView___closed__2() { @@ -1112,7 +1114,7 @@ LEAN_EXPORT uint8_t l_Lean_Elab_DefView_isInstance(lean_object* x_1) { { 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, 2); -x_3 = lean_ctor_get(x_2, 1); +x_3 = lean_ctor_get(x_2, 2); x_4 = lean_array_get_size(x_3); x_5 = lean_unsigned_to_nat(0u); x_6 = lean_nat_dec_lt(x_5, x_4); @@ -4899,7 +4901,7 @@ uint8_t x_15; lean_dec(x_10); lean_dec(x_9); lean_dec(x_2); -x_15 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); +x_15 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); lean_dec(x_1); if (x_15 == 0) { diff --git a/stage0/stdlib/Lean/Elab/Deriving/FromToJson.c b/stage0/stdlib/Lean/Elab/Deriving/FromToJson.c index cbe35a926aaf..62fff02aac01 100644 --- a/stage0/stdlib/Lean/Elab/Deriving/FromToJson.c +++ b/stage0/stdlib/Lean/Elab/Deriving/FromToJson.c @@ -42,6 +42,7 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__1 static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__14; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__5; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__16; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6656____closed__16; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -66,6 +67,7 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deri lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Array_qpartition___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__5; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__3___closed__3; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__13; @@ -78,6 +80,7 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___lamb lean_object* l_Lean_Elab_Deriving_mkInstanceCmds(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_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; lean_object* l_Lean_Elab_Deriving_mkDiscrs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__12; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonAuxFunction___lambda__1___closed__7; @@ -87,7 +90,6 @@ lean_object* l_Lean_Elab_Command_elabCommand(lean_object*, lean_object*, lean_ob lean_object* lean_array_fget(lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__3___closed__3; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___spec__1___closed__2; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___lambda__1___closed__12; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__5; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__6; @@ -103,6 +105,7 @@ static lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Elab_Deriving_FromToJson LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkJsonField___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___spec__1___closed__25; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__13; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isInductive___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__40; @@ -113,12 +116,12 @@ uint8_t l_Lean_Expr_isAppOf(lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__6; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__4___lambda__1___closed__2; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__11; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___lambda__1___closed__5; lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Deriving_mkContext___spec__1(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*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___closed__4; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__24; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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* l_Lean_stringToMessageData(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___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_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__12; @@ -141,7 +144,6 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__8(lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__12; LEAN_EXPORT lean_object* l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___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*); static lean_object* l___private_Lean_Elab_Deriving_FromToJson_0__Lean_Elab_Deriving_FromToJson_mkToJsonInstance___closed__1; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___closed__2; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__2; @@ -162,7 +164,6 @@ lean_object* l_Array_mapMUnsafe_map___at___aux__Init__NotationExtra______macroRu static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___spec__1___closed__20; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__3___closed__8; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__9; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonAuxFunction___lambda__1___closed__12; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__3___closed__4; @@ -179,20 +180,26 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonMutualBlock___closed static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__8; lean_object* l_Lean_Elab_registerDerivingHandler(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Substring_takeRightWhileAux___at_Lean_Elab_Deriving_FromToJson_mkJsonField___spec__2___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__2___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_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct___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_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__11; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__31; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___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*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___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_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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_Elab_Deriving_mkLet(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__3___closed__13; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; lean_object* l_Array_zip___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct___closed__4; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___closed__4; lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__2___closed__6; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___lambda__1___closed__6; lean_object* l_Lean_MessageData_ofSyntax(lean_object*); @@ -213,8 +220,6 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__1 static lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6656____closed__13; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___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___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___lambda__1___closed__7; static lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6656____closed__14; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__9; @@ -253,8 +258,8 @@ static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mk static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__5___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__5(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; lean_object* lean_array_to_list(lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonAuxFunction___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_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__2___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); @@ -290,6 +295,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct(l static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___spec__1___closed__16; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__2___closed__7; lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; LEAN_EXPORT lean_object* l_Substring_takeRightWhileAux___at_Lean_Elab_Deriving_FromToJson_mkJsonField___spec__2(lean_object*, lean_object*, lean_object*); lean_object* lean_string_utf8_prev(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___closed__10; @@ -300,7 +306,6 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Elab_Deriving_FromT static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__20; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__5___lambda__1___closed__7; static lean_object* l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__1___closed__2; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___spec__1___closed__9; static lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6656____closed__8; lean_object* lean_mk_syntax_ident(lean_object*); @@ -317,7 +322,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJs LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); static lean_object* l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__1___closed__3; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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* l_Lean_MessageData_ofExpr(lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__5___lambda__1___closed__1; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonMutualBlock___closed__2; @@ -329,9 +333,9 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJs LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___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_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__4; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___spec__1___closed__5; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; static lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6656____closed__10; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___spec__1___closed__13; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___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_Elab_Deriving_FromToJson_mkFromJsonMutualBlock(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__25; lean_object* l_Lean_LocalDecl_userName(lean_object*); @@ -340,14 +344,15 @@ lean_object* l_Lean_Syntax_node4(lean_object*, lean_object*, lean_object*, lean_ LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___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_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__14; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__34; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__1; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct___closed__2; static lean_object* l___private_Lean_Elab_Deriving_FromToJson_0__Lean_Elab_Deriving_FromToJson_mkToJsonInstance___closed__2; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__13; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___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_Deriving_FromToJson_mkToJsonBodyForInduct___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonAuxFunction(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; static lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6656____closed__17; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__20; uint8_t l_Lean_Name_hasMacroScopes(lean_object*); @@ -363,7 +368,6 @@ static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mk static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__8; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___lambda__1___closed__3; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__21; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9; lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(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*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__3___closed__5; @@ -374,7 +378,6 @@ uint8_t lean_nat_dec_lt(lean_object*, lean_object*); lean_object* lean_environment_main_module(lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__10; LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Deriving_FromToJson_0__Lean_Elab_Deriving_FromToJson_mkFromJsonInstance___spec__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__9; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___closed__18; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct___closed__3; @@ -405,7 +408,6 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct___cl lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___closed__17; lean_object* l_Lean_mkSepArray(lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__3___closed__10; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__2___closed__8; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___closed__12; @@ -425,14 +427,13 @@ uint8_t l_Lean_isStructure(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__25; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonAuxFunction___lambda__1___closed__8; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__19; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___closed__1; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___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*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct___closed__8; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__29; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3; lean_object* l_Lean_Name_getString_x21(lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonMutualBlock(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___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*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__4; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__19; lean_object* lean_erase_macro_scopes(lean_object*); @@ -460,7 +461,6 @@ LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJs static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__1; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__2; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__5___lambda__1___closed__8; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___closed__1; size_t lean_usize_add(size_t, size_t); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__3; @@ -476,6 +476,7 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___lamb size_t lean_array_size(lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonAuxFunction___lambda__1___closed__3; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__18; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__26; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__11; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__3___closed__1; @@ -486,7 +487,6 @@ LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mk static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__2___closed__3; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___spec__5___lambda__1___closed__9; lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__5; LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Deriving_FromToJson_0__Lean_Elab_Deriving_FromToJson_mkToJsonInstance___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__3___closed__6; @@ -508,6 +508,7 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct___cl static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__10; uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBody(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6; uint8_t lean_usize_dec_lt(size_t, size_t); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonAuxFunction___lambda__1___closed__16; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__1___closed__21; @@ -541,7 +542,6 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___clos LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct_mkAlts___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*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___spec__3___closed__4; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__7; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1; lean_object* l_Lean_Syntax_mkNumLit(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__12; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForStruct___closed__15; @@ -4590,7 +4590,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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) { _start: { lean_object* x_17; uint8_t x_18; @@ -4870,7 +4870,7 @@ return x_134; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -5696,7 +5696,7 @@ lean_object* x_191; lean_object* x_192; lean_object* x_193; uint8_t x_194; x_191 = lean_ctor_get(x_5, 0); x_192 = lean_mk_empty_array_with_capacity(x_17); lean_inc(x_10); -x_193 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__2(x_1, x_2, x_4, x_191, x_4, x_17, x_18, lean_box(0), x_192, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_193 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__2(x_1, x_2, x_4, x_191, x_4, x_17, x_18, lean_box(0), x_192, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_4); x_194 = !lean_is_exclusive(x_193); if (x_194 == 0) @@ -6300,7 +6300,7 @@ x_453 = lean_array_mk(x_452); x_454 = lean_array_get_size(x_453); x_455 = lean_mk_empty_array_with_capacity(x_454); lean_inc(x_10); -x_456 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__3(x_1, x_2, x_450, x_453, x_453, x_454, x_18, lean_box(0), x_455, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_456 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___spec__3(x_1, x_2, x_450, x_453, x_453, x_454, x_18, lean_box(0), x_455, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_453); x_457 = !lean_is_exclusive(x_456); if (x_457 == 0) @@ -7133,11 +7133,11 @@ lean_dec(x_1); return x_15; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; -x_17 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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); lean_dec(x_15); lean_dec(x_13); lean_dec(x_12); @@ -7150,11 +7150,11 @@ lean_dec(x_1); return x_17; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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, lean_object* x_16) { _start: { lean_object* x_17; -x_17 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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, x_16); +x_17 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonBodyForInduct___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, x_16); lean_dec(x_15); lean_dec(x_13); lean_dec(x_12); @@ -9664,7 +9664,7 @@ goto _start; } } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1() { _start: { lean_object* x_1; @@ -9672,61 +9672,61 @@ x_1 = lean_mk_string_unchecked("fromJson\?", 9, 9); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1; +x_1 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1; +x_2 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Elab_Deriving_FromToJson_mkToJsonHeader___closed__1; x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__1; -x_3 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1; +x_3 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4; +x_2 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___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_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5; +x_2 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5; 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_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7() { _start: { lean_object* x_1; @@ -9734,17 +9734,17 @@ x_1 = lean_mk_string_unchecked("term__[_]_!", 11, 11); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7; +x_2 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9() { _start: { lean_object* x_1; @@ -9752,26 +9752,26 @@ x_1 = lean_mk_string_unchecked("jsons", 5, 5); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9; +x_1 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___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_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9; +x_2 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12() { _start: { lean_object* x_1; @@ -9779,17 +9779,17 @@ x_1 = lean_mk_string_unchecked("group", 5, 5); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12; +x_2 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14() { _start: { lean_object* x_1; @@ -9797,7 +9797,7 @@ x_1 = lean_mk_string_unchecked("!", 1, 1); return x_1; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___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) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___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; @@ -9842,29 +9842,29 @@ x_35 = lean_ctor_get(x_33, 0); lean_inc(x_35); lean_dec(x_33); x_36 = lean_environment_main_module(x_35); -x_37 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3; +x_37 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3; lean_inc(x_30); lean_inc(x_36); x_38 = l_Lean_addMacroScope(x_36, x_37, x_30); x_39 = lean_box(0); -x_40 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2; -x_41 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6; +x_40 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2; +x_41 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6; lean_inc(x_29); x_42 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_42, 0, x_29); lean_ctor_set(x_42, 1, x_40); lean_ctor_set(x_42, 2, x_38); lean_ctor_set(x_42, 3, x_41); -x_43 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; +x_43 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; x_44 = l_Lean_addMacroScope(x_36, x_43, x_30); -x_45 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; +x_45 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; lean_inc(x_29); x_46 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_46, 0, x_29); lean_ctor_set(x_46, 1, x_45); lean_ctor_set(x_46, 2, x_44); lean_ctor_set(x_46, 3, x_39); -x_47 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; +x_47 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; x_48 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__25; lean_inc(x_29); x_49 = lean_alloc_ctor(1, 3, 0); @@ -9885,12 +9885,12 @@ lean_inc(x_29); lean_ctor_set_tag(x_20, 2); lean_ctor_set(x_20, 1, x_54); lean_ctor_set(x_20, 0, x_29); -x_55 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; +x_55 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; lean_inc(x_29); x_56 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_56, 0, x_29); lean_ctor_set(x_56, 1, x_55); -x_57 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; +x_57 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; lean_inc(x_49); lean_inc(x_29); x_58 = l_Lean_Syntax_node7(x_29, x_57, x_46, x_49, x_31, x_53, x_20, x_49, x_56); @@ -9924,29 +9924,29 @@ x_70 = lean_ctor_get(x_68, 0); lean_inc(x_70); lean_dec(x_68); x_71 = lean_environment_main_module(x_70); -x_72 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3; +x_72 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3; lean_inc(x_30); lean_inc(x_71); x_73 = l_Lean_addMacroScope(x_71, x_72, x_30); x_74 = lean_box(0); -x_75 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2; -x_76 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6; +x_75 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2; +x_76 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6; lean_inc(x_29); x_77 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_77, 0, x_29); lean_ctor_set(x_77, 1, x_75); lean_ctor_set(x_77, 2, x_73); lean_ctor_set(x_77, 3, x_76); -x_78 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; +x_78 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; x_79 = l_Lean_addMacroScope(x_71, x_78, x_30); -x_80 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; +x_80 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; lean_inc(x_29); x_81 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_81, 0, x_29); lean_ctor_set(x_81, 1, x_80); lean_ctor_set(x_81, 2, x_79); lean_ctor_set(x_81, 3, x_74); -x_82 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; +x_82 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; x_83 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__25; lean_inc(x_29); x_84 = lean_alloc_ctor(1, 3, 0); @@ -9967,12 +9967,12 @@ lean_inc(x_29); lean_ctor_set_tag(x_20, 2); lean_ctor_set(x_20, 1, x_90); lean_ctor_set(x_20, 0, x_29); -x_91 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; +x_91 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; lean_inc(x_29); x_92 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_92, 0, x_29); lean_ctor_set(x_92, 1, x_91); -x_93 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; +x_93 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; lean_inc(x_84); lean_inc(x_29); x_94 = l_Lean_Syntax_node7(x_29, x_93, x_81, x_84, x_86, x_89, x_20, x_84, x_92); @@ -10016,17 +10016,17 @@ x_112 = lean_ctor_get(x_110, 0); lean_inc(x_112); lean_dec(x_110); x_113 = lean_environment_main_module(x_112); -x_114 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; +x_114 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; x_115 = l_Lean_addMacroScope(x_113, x_114, x_107); x_116 = lean_box(0); -x_117 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; +x_117 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; lean_inc(x_106); x_118 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_118, 0, x_106); lean_ctor_set(x_118, 1, x_117); lean_ctor_set(x_118, 2, x_115); lean_ctor_set(x_118, 3, x_116); -x_119 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; +x_119 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; x_120 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__25; lean_inc(x_106); x_121 = lean_alloc_ctor(1, 3, 0); @@ -10047,12 +10047,12 @@ lean_inc(x_106); lean_ctor_set_tag(x_20, 2); lean_ctor_set(x_20, 1, x_126); lean_ctor_set(x_20, 0, x_106); -x_127 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; +x_127 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; lean_inc(x_106); x_128 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_128, 0, x_106); lean_ctor_set(x_128, 1, x_127); -x_129 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; +x_129 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; lean_inc(x_121); lean_inc(x_106); x_130 = l_Lean_Syntax_node7(x_106, x_129, x_118, x_121, x_108, x_125, x_20, x_121, x_128); @@ -10087,17 +10087,17 @@ x_142 = lean_ctor_get(x_140, 0); lean_inc(x_142); lean_dec(x_140); x_143 = lean_environment_main_module(x_142); -x_144 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; +x_144 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; x_145 = l_Lean_addMacroScope(x_143, x_144, x_107); x_146 = lean_box(0); -x_147 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; +x_147 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; lean_inc(x_106); x_148 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_148, 0, x_106); lean_ctor_set(x_148, 1, x_147); lean_ctor_set(x_148, 2, x_145); lean_ctor_set(x_148, 3, x_146); -x_149 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; +x_149 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; x_150 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__25; lean_inc(x_106); x_151 = lean_alloc_ctor(1, 3, 0); @@ -10118,12 +10118,12 @@ lean_inc(x_106); lean_ctor_set_tag(x_20, 2); lean_ctor_set(x_20, 1, x_157); lean_ctor_set(x_20, 0, x_106); -x_158 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; +x_158 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; lean_inc(x_106); x_159 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_159, 0, x_106); lean_ctor_set(x_159, 1, x_158); -x_160 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; +x_160 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; lean_inc(x_151); lean_inc(x_106); x_161 = l_Lean_Syntax_node7(x_106, x_160, x_148, x_151, x_153, x_156, x_20, x_151, x_159); @@ -10185,29 +10185,29 @@ x_183 = lean_ctor_get(x_180, 0); lean_inc(x_183); lean_dec(x_180); x_184 = lean_environment_main_module(x_183); -x_185 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3; +x_185 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3; lean_inc(x_178); lean_inc(x_184); x_186 = l_Lean_addMacroScope(x_184, x_185, x_178); x_187 = lean_box(0); -x_188 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2; -x_189 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6; +x_188 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2; +x_189 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6; lean_inc(x_177); x_190 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_190, 0, x_177); lean_ctor_set(x_190, 1, x_188); lean_ctor_set(x_190, 2, x_186); lean_ctor_set(x_190, 3, x_189); -x_191 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; +x_191 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; x_192 = l_Lean_addMacroScope(x_184, x_191, x_178); -x_193 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; +x_193 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; lean_inc(x_177); x_194 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_194, 0, x_177); lean_ctor_set(x_194, 1, x_193); lean_ctor_set(x_194, 2, x_192); lean_ctor_set(x_194, 3, x_187); -x_195 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; +x_195 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; x_196 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__25; lean_inc(x_177); x_197 = lean_alloc_ctor(1, 3, 0); @@ -10233,12 +10233,12 @@ lean_inc(x_177); x_204 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_204, 0, x_177); lean_ctor_set(x_204, 1, x_203); -x_205 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; +x_205 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; lean_inc(x_177); x_206 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_206, 0, x_177); lean_ctor_set(x_206, 1, x_205); -x_207 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; +x_207 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; lean_inc(x_197); lean_inc(x_177); x_208 = l_Lean_Syntax_node7(x_177, x_207, x_194, x_197, x_199, x_202, x_204, x_197, x_206); @@ -10287,17 +10287,17 @@ x_226 = lean_ctor_get(x_223, 0); lean_inc(x_226); lean_dec(x_223); x_227 = lean_environment_main_module(x_226); -x_228 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; +x_228 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; x_229 = l_Lean_addMacroScope(x_227, x_228, x_221); x_230 = lean_box(0); -x_231 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; +x_231 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; lean_inc(x_220); x_232 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_232, 0, x_220); lean_ctor_set(x_232, 1, x_231); lean_ctor_set(x_232, 2, x_229); lean_ctor_set(x_232, 3, x_230); -x_233 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; +x_233 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13; x_234 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonHeader___closed__25; lean_inc(x_220); x_235 = lean_alloc_ctor(1, 3, 0); @@ -10323,12 +10323,12 @@ lean_inc(x_220); x_242 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_242, 0, x_220); lean_ctor_set(x_242, 1, x_241); -x_243 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; +x_243 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14; lean_inc(x_220); x_244 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_244, 0, x_220); lean_ctor_set(x_244, 1, x_243); -x_245 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; +x_245 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8; lean_inc(x_235); lean_inc(x_220); x_246 = l_Lean_Syntax_node7(x_220, x_245, x_232, x_235, x_237, x_240, x_242, x_235, x_244); @@ -10806,9 +10806,9 @@ lean_inc(x_17); x_69 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_69, 0, x_17); lean_ctor_set(x_69, 1, x_68); -x_70 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; +x_70 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; x_71 = l_Lean_addMacroScope(x_23, x_70, x_18); -x_72 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; +x_72 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; lean_inc(x_17); x_73 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_73, 0, x_17); @@ -11017,9 +11017,9 @@ lean_inc(x_17); x_161 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_161, 0, x_17); lean_ctor_set(x_161, 1, x_160); -x_162 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; +x_162 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11; x_163 = l_Lean_addMacroScope(x_115, x_162, x_18); -x_164 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; +x_164 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10; lean_inc(x_17); x_165 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_165, 0, x_17); @@ -11322,7 +11322,7 @@ lean_object* x_33; lean_object* x_34; uint8_t x_35; x_33 = lean_mk_syntax_ident(x_32); lean_inc(x_11); lean_inc(x_30); -x_34 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3(x_2, x_22, x_33, x_22, x_30, x_16, lean_box(0), x_31, x_7, x_8, x_9, x_10, x_11, x_12, x_21); +x_34 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3(x_2, x_22, x_33, x_22, x_30, x_16, lean_box(0), x_31, x_7, x_8, x_9, x_10, x_11, x_12, x_21); lean_dec(x_22); x_35 = !lean_is_exclusive(x_34); if (x_35 == 0) @@ -12113,11 +12113,11 @@ x_6 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyFo return x_6; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___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) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___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_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___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); +x_16 = l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___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_12); lean_dec(x_11); @@ -18624,34 +18624,34 @@ l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__12 = _init_l_L lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__12); l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__13 = _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__13(); lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForStruct___closed__13); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13); -l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__1); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__2); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__3); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__4); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__5); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__6); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__7); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__8); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__9); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__10); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__11); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__12); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__13); +l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__3___closed__14); l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__1 = _init_l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__1(); lean_mark_persistent(l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__1); l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__2 = _init_l_List_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonBodyForInduct_mkAlts___spec__7___lambda__2___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Frontend.c b/stage0/stdlib/Lean/Elab/Frontend.c index 72ec511f4ad8..f2c5977b0a92 100644 --- a/stage0/stdlib/Lean/Elab/Frontend.c +++ b/stage0/stdlib/Lean/Elab/Frontend.c @@ -72,19 +72,20 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_runFrontend___ static lean_object* l_Array_filterMapM___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__3___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__2(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_runCommandElabM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__6(lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_process___closed__2; LEAN_EXPORT lean_object* l_Array_filterMapM___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__3___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_setParserState___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_mkInputContext(lean_object*, lean_object*, uint8_t); lean_object* lean_st_mk_ref(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(lean_object*, size_t, size_t, lean_object*); lean_object* l_Array_toPArray_x27___rarg(lean_object*); static lean_object* l_Lean_Elab_runFrontend___closed__4; lean_object* lean_io_mono_nanos_now(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_elabCommandAtFrontend___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Option_set___at_Lean_Elab_Term_withoutMacroStackAtErr___spec__1(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_processCommand___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(size_t, size_t, lean_object*); extern lean_object* l_Lean_Language_Lean_internal_cmdlineSnapshots; lean_object* lean_task_get_own(lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); @@ -113,6 +114,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_runFrontend___lambda__1(lean_object*, lean_ static lean_object* l_Lean_Elab_runFrontend___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_processCommand(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__4(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_runFrontend___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_firstFrontendMacroScope; extern lean_object* l_Lean_Elab_Command_instInhabitedScope; @@ -121,6 +123,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_setCommandState(lean_object*, lean LEAN_EXPORT lean_object* l_Lean_Elab_process(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_updateCmdPos___rarg(lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Language_SnapshotTask_map___rarg(lean_object*, lean_object*, lean_object*, uint8_t); lean_object* l_Lean_MessageLog_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_runFrontend___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, double, lean_object*, lean_object*); @@ -136,7 +139,6 @@ extern lean_object* l_Lean_trace_profiler_output; lean_object* lean_array_get_size(lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_setParserState(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); lean_object* lean_mk_empty_environment(uint32_t, lean_object*); static lean_object* l_Lean_Elab_Frontend_processCommand___closed__1; @@ -2063,18 +2065,25 @@ 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; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; size_t x_12; size_t x_13; lean_object* x_14; 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, 2); +x_8 = lean_ctor_get(x_5, 4); 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; +x_9 = l_Lean_Language_SnapshotTask_get___rarg(x_8); +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +lean_dec(x_9); +x_11 = lean_ctor_get(x_10, 2); +lean_inc(x_11); +lean_dec(x_10); +x_12 = 1; +x_13 = lean_usize_add(x_2, x_12); +x_14 = lean_array_uset(x_7, x_2, x_11); +x_2 = x_13; +x_3 = x_14; goto _start; } } @@ -2157,7 +2166,34 @@ return x_12; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(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_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(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_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 lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__6(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -2187,28 +2223,28 @@ x_6 = lean_task_get_own(x_3); x_7 = !lean_is_exclusive(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_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); -x_10 = lean_ctor_get(x_8, 1); -lean_inc(x_10); -x_11 = lean_array_push(x_4, x_10); +lean_inc(x_8); +x_10 = lean_array_push(x_4, x_8); if (lean_obj_tag(x_9) == 0) { -lean_object* x_12; lean_object* x_13; size_t x_14; size_t 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; 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_11; lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_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; lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_inc(x_2); -x_12 = l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go(x_2); -x_13 = l_Lean_Language_SnapshotTree_getAll(x_12); -x_14 = lean_array_size(x_13); -x_15 = 0; -lean_inc(x_13); -x_16 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__1(x_14, x_15, x_13); -x_17 = lean_array_get_size(x_16); -x_18 = lean_unsigned_to_nat(0u); -x_19 = lean_nat_dec_lt(x_18, x_17); -x_20 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__2(x_14, x_15, x_13); +x_11 = l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go(x_2); +x_12 = l_Lean_Language_SnapshotTree_getAll(x_11); +x_13 = lean_array_size(x_12); +x_14 = 0; +x_15 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__1(x_13, x_14, x_12); +x_16 = lean_array_get_size(x_15); +x_17 = lean_unsigned_to_nat(0u); +x_18 = lean_nat_dec_lt(x_17, x_16); +x_19 = lean_array_size(x_10); +lean_inc(x_10); +x_20 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__2(x_19, x_14, x_10); x_21 = lean_array_get_size(x_20); -x_22 = l_Array_filterMapM___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__3(x_20, x_18, x_21); +x_22 = l_Array_filterMapM___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__3(x_20, x_17, x_21); lean_dec(x_21); lean_dec(x_20); x_23 = l_Array_toPArray_x27___rarg(x_22); @@ -2229,117 +2265,114 @@ lean_dec(x_29); x_30 = !lean_is_exclusive(x_28); if (x_30 == 0) { -lean_object* x_31; +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; x_31 = lean_ctor_get(x_28, 1); lean_dec(x_31); lean_ctor_set(x_28, 1, x_23); -if (x_19 == 0) -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -lean_dec(x_17); -lean_dec(x_16); x_32 = lean_ctor_get(x_8, 2); lean_inc(x_32); lean_dec(x_8); x_33 = lean_ctor_get(x_32, 0); lean_inc(x_33); -x_34 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -lean_ctor_set(x_26, 1, x_34); -x_35 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_35, 0, x_26); -lean_ctor_set(x_35, 1, x_32); -lean_ctor_set(x_35, 2, x_33); -lean_ctor_set(x_35, 3, x_11); -x_36 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_1); -lean_ctor_set(x_36, 2, x_2); +x_34 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_19, x_14, x_10); +if (x_18 == 0) +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +lean_dec(x_16); +lean_dec(x_15); +x_35 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +lean_ctor_set(x_26, 1, x_35); +x_36 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_36, 0, x_26); +lean_ctor_set(x_36, 1, x_32); +lean_ctor_set(x_36, 2, x_33); +lean_ctor_set(x_36, 3, x_34); +x_37 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_1); +lean_ctor_set(x_37, 2, x_2); lean_ctor_set(x_6, 1, x_5); -lean_ctor_set(x_6, 0, x_36); +lean_ctor_set(x_6, 0, x_37); return x_6; } else { -lean_object* x_37; lean_object* x_38; uint8_t x_39; -x_37 = lean_ctor_get(x_8, 2); -lean_inc(x_37); -lean_dec(x_8); -x_38 = lean_ctor_get(x_37, 0); -lean_inc(x_38); -x_39 = lean_nat_dec_le(x_17, x_17); -if (x_39 == 0) +uint8_t x_38; +x_38 = lean_nat_dec_le(x_16, x_16); +if (x_38 == 0) { -lean_object* x_40; lean_object* x_41; lean_object* x_42; -lean_dec(x_17); +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_dec(x_16); -x_40 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -lean_ctor_set(x_26, 1, x_40); -x_41 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_41, 0, x_26); -lean_ctor_set(x_41, 1, x_37); -lean_ctor_set(x_41, 2, x_38); -lean_ctor_set(x_41, 3, x_11); -x_42 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_1); -lean_ctor_set(x_42, 2, x_2); +lean_dec(x_15); +x_39 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +lean_ctor_set(x_26, 1, x_39); +x_40 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_40, 0, x_26); +lean_ctor_set(x_40, 1, x_32); +lean_ctor_set(x_40, 2, x_33); +lean_ctor_set(x_40, 3, x_34); +x_41 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_1); +lean_ctor_set(x_41, 2, x_2); lean_ctor_set(x_6, 1, x_5); -lean_ctor_set(x_6, 0, x_42); +lean_ctor_set(x_6, 0, x_41); return x_6; } else { -size_t x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_43 = lean_usize_of_nat(x_17); -lean_dec(x_17); -x_44 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -x_45 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_16, x_15, x_43, x_44); +size_t x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_42 = lean_usize_of_nat(x_16); lean_dec(x_16); -lean_ctor_set(x_26, 1, x_45); -x_46 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_46, 0, x_26); -lean_ctor_set(x_46, 1, x_37); -lean_ctor_set(x_46, 2, x_38); -lean_ctor_set(x_46, 3, x_11); -x_47 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_47, 0, x_46); -lean_ctor_set(x_47, 1, x_1); -lean_ctor_set(x_47, 2, x_2); +x_43 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +x_44 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__6(x_15, x_14, x_42, x_43); +lean_dec(x_15); +lean_ctor_set(x_26, 1, x_44); +x_45 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_45, 0, x_26); +lean_ctor_set(x_45, 1, x_32); +lean_ctor_set(x_45, 2, x_33); +lean_ctor_set(x_45, 3, x_34); +x_46 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_46, 0, x_45); +lean_ctor_set(x_46, 1, x_1); +lean_ctor_set(x_46, 2, x_2); lean_ctor_set(x_6, 1, x_5); -lean_ctor_set(x_6, 0, x_47); +lean_ctor_set(x_6, 0, x_46); return x_6; } } } else { -uint8_t x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get_uint8(x_28, sizeof(void*)*2); -x_49 = lean_ctor_get(x_28, 0); -lean_inc(x_49); +uint8_t 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_uint8(x_28, sizeof(void*)*2); +x_48 = lean_ctor_get(x_28, 0); +lean_inc(x_48); lean_dec(x_28); -x_50 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_50, 0, x_49); -lean_ctor_set(x_50, 1, x_23); -lean_ctor_set_uint8(x_50, sizeof(void*)*2, x_48); -if (x_19 == 0) +x_49 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_23); +lean_ctor_set_uint8(x_49, sizeof(void*)*2, x_47); +x_50 = lean_ctor_get(x_8, 2); +lean_inc(x_50); +lean_dec(x_8); +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_19, x_14, x_10); +if (x_18 == 0) { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -lean_dec(x_17); +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_dec(x_16); -x_51 = lean_ctor_get(x_8, 2); -lean_inc(x_51); -lean_dec(x_8); -x_52 = lean_ctor_get(x_51, 0); -lean_inc(x_52); +lean_dec(x_15); x_53 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -lean_ctor_set(x_26, 6, x_50); +lean_ctor_set(x_26, 6, x_49); lean_ctor_set(x_26, 1, x_53); x_54 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_54, 0, x_26); -lean_ctor_set(x_54, 1, x_51); -lean_ctor_set(x_54, 2, x_52); -lean_ctor_set(x_54, 3, x_11); +lean_ctor_set(x_54, 1, x_50); +lean_ctor_set(x_54, 2, x_51); +lean_ctor_set(x_54, 3, x_52); x_55 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_55, 0, x_54); lean_ctor_set(x_55, 1, x_1); @@ -2350,55 +2383,50 @@ return x_6; } else { -lean_object* x_56; lean_object* x_57; uint8_t x_58; -x_56 = lean_ctor_get(x_8, 2); -lean_inc(x_56); -lean_dec(x_8); -x_57 = lean_ctor_get(x_56, 0); -lean_inc(x_57); -x_58 = lean_nat_dec_le(x_17, x_17); -if (x_58 == 0) +uint8_t x_56; +x_56 = lean_nat_dec_le(x_16, x_16); +if (x_56 == 0) { -lean_object* x_59; lean_object* x_60; lean_object* x_61; -lean_dec(x_17); +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_dec(x_16); -x_59 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -lean_ctor_set(x_26, 6, x_50); -lean_ctor_set(x_26, 1, x_59); -x_60 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_60, 0, x_26); -lean_ctor_set(x_60, 1, x_56); -lean_ctor_set(x_60, 2, x_57); -lean_ctor_set(x_60, 3, x_11); -x_61 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_61, 0, x_60); -lean_ctor_set(x_61, 1, x_1); -lean_ctor_set(x_61, 2, x_2); +lean_dec(x_15); +x_57 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +lean_ctor_set(x_26, 6, x_49); +lean_ctor_set(x_26, 1, x_57); +x_58 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_58, 0, x_26); +lean_ctor_set(x_58, 1, x_50); +lean_ctor_set(x_58, 2, x_51); +lean_ctor_set(x_58, 3, x_52); +x_59 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_59, 0, x_58); +lean_ctor_set(x_59, 1, x_1); +lean_ctor_set(x_59, 2, x_2); lean_ctor_set(x_6, 1, x_5); -lean_ctor_set(x_6, 0, x_61); +lean_ctor_set(x_6, 0, x_59); return x_6; } else { -size_t x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_62 = lean_usize_of_nat(x_17); -lean_dec(x_17); -x_63 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -x_64 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_16, x_15, x_62, x_63); +size_t x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_60 = lean_usize_of_nat(x_16); lean_dec(x_16); -lean_ctor_set(x_26, 6, x_50); -lean_ctor_set(x_26, 1, x_64); -x_65 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_65, 0, x_26); -lean_ctor_set(x_65, 1, x_56); -lean_ctor_set(x_65, 2, x_57); -lean_ctor_set(x_65, 3, x_11); -x_66 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_66, 0, x_65); -lean_ctor_set(x_66, 1, x_1); -lean_ctor_set(x_66, 2, x_2); +x_61 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +x_62 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__6(x_15, x_14, x_60, x_61); +lean_dec(x_15); +lean_ctor_set(x_26, 6, x_49); +lean_ctor_set(x_26, 1, x_62); +x_63 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_63, 0, x_26); +lean_ctor_set(x_63, 1, x_50); +lean_ctor_set(x_63, 2, x_51); +lean_ctor_set(x_63, 3, x_52); +x_64 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_64, 0, x_63); +lean_ctor_set(x_64, 1, x_1); +lean_ctor_set(x_64, 2, x_2); lean_ctor_set(x_6, 1, x_5); -lean_ctor_set(x_6, 0, x_66); +lean_ctor_set(x_6, 0, x_64); return x_6; } } @@ -2406,139 +2434,135 @@ return x_6; } 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; uint8_t x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_67 = lean_ctor_get(x_26, 6); -x_68 = lean_ctor_get(x_26, 0); -x_69 = lean_ctor_get(x_26, 2); -x_70 = lean_ctor_get(x_26, 3); -x_71 = lean_ctor_get(x_26, 4); -x_72 = lean_ctor_get(x_26, 5); -x_73 = lean_ctor_get(x_26, 7); -lean_inc(x_73); -lean_inc(x_67); -lean_inc(x_72); +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; +x_65 = lean_ctor_get(x_26, 6); +x_66 = lean_ctor_get(x_26, 0); +x_67 = lean_ctor_get(x_26, 2); +x_68 = lean_ctor_get(x_26, 3); +x_69 = lean_ctor_get(x_26, 4); +x_70 = lean_ctor_get(x_26, 5); +x_71 = lean_ctor_get(x_26, 7); lean_inc(x_71); +lean_inc(x_65); lean_inc(x_70); lean_inc(x_69); lean_inc(x_68); +lean_inc(x_67); +lean_inc(x_66); lean_dec(x_26); -x_74 = lean_ctor_get_uint8(x_67, sizeof(void*)*2); -x_75 = lean_ctor_get(x_67, 0); -lean_inc(x_75); -if (lean_is_exclusive(x_67)) { - lean_ctor_release(x_67, 0); - lean_ctor_release(x_67, 1); - x_76 = x_67; +x_72 = lean_ctor_get_uint8(x_65, sizeof(void*)*2); +x_73 = lean_ctor_get(x_65, 0); +lean_inc(x_73); +if (lean_is_exclusive(x_65)) { + lean_ctor_release(x_65, 0); + lean_ctor_release(x_65, 1); + x_74 = x_65; } else { - lean_dec_ref(x_67); - x_76 = lean_box(0); + lean_dec_ref(x_65); + x_74 = lean_box(0); } -if (lean_is_scalar(x_76)) { - x_77 = lean_alloc_ctor(0, 2, 1); +if (lean_is_scalar(x_74)) { + x_75 = lean_alloc_ctor(0, 2, 1); } else { - x_77 = x_76; + x_75 = x_74; } -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_23); -lean_ctor_set_uint8(x_77, sizeof(void*)*2, x_74); -if (x_19 == 0) +lean_ctor_set(x_75, 0, x_73); +lean_ctor_set(x_75, 1, x_23); +lean_ctor_set_uint8(x_75, sizeof(void*)*2, x_72); +x_76 = lean_ctor_get(x_8, 2); +lean_inc(x_76); +lean_dec(x_8); +x_77 = lean_ctor_get(x_76, 0); +lean_inc(x_77); +x_78 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_19, x_14, x_10); +if (x_18 == 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_dec(x_17); +lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_dec(x_16); -x_78 = lean_ctor_get(x_8, 2); -lean_inc(x_78); -lean_dec(x_8); -x_79 = lean_ctor_get(x_78, 0); -lean_inc(x_79); -x_80 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -x_81 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_81, 0, x_68); -lean_ctor_set(x_81, 1, x_80); -lean_ctor_set(x_81, 2, x_69); -lean_ctor_set(x_81, 3, x_70); -lean_ctor_set(x_81, 4, x_71); -lean_ctor_set(x_81, 5, x_72); -lean_ctor_set(x_81, 6, x_77); -lean_ctor_set(x_81, 7, x_73); -x_82 = lean_alloc_ctor(0, 4, 0); +lean_dec(x_15); +x_79 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +x_80 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_80, 0, x_66); +lean_ctor_set(x_80, 1, x_79); +lean_ctor_set(x_80, 2, x_67); +lean_ctor_set(x_80, 3, x_68); +lean_ctor_set(x_80, 4, x_69); +lean_ctor_set(x_80, 5, x_70); +lean_ctor_set(x_80, 6, x_75); +lean_ctor_set(x_80, 7, x_71); +x_81 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_81, 1, x_76); +lean_ctor_set(x_81, 2, x_77); +lean_ctor_set(x_81, 3, x_78); +x_82 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_82, 0, x_81); -lean_ctor_set(x_82, 1, x_78); -lean_ctor_set(x_82, 2, x_79); -lean_ctor_set(x_82, 3, x_11); -x_83 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_83, 0, x_82); -lean_ctor_set(x_83, 1, x_1); -lean_ctor_set(x_83, 2, x_2); +lean_ctor_set(x_82, 1, x_1); +lean_ctor_set(x_82, 2, x_2); lean_ctor_set(x_6, 1, x_5); -lean_ctor_set(x_6, 0, x_83); +lean_ctor_set(x_6, 0, x_82); return x_6; } else { -lean_object* x_84; lean_object* x_85; uint8_t x_86; -x_84 = lean_ctor_get(x_8, 2); -lean_inc(x_84); -lean_dec(x_8); -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -x_86 = lean_nat_dec_le(x_17, x_17); -if (x_86 == 0) +uint8_t x_83; +x_83 = lean_nat_dec_le(x_16, x_16); +if (x_83 == 0) { -lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; -lean_dec(x_17); +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_dec(x_16); -x_87 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -x_88 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_88, 0, x_68); -lean_ctor_set(x_88, 1, x_87); -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_77); -lean_ctor_set(x_88, 7, x_73); -x_89 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_89, 0, x_88); -lean_ctor_set(x_89, 1, x_84); -lean_ctor_set(x_89, 2, x_85); -lean_ctor_set(x_89, 3, x_11); -x_90 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_90, 0, x_89); -lean_ctor_set(x_90, 1, x_1); -lean_ctor_set(x_90, 2, x_2); +lean_dec(x_15); +x_84 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +x_85 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_85, 0, x_66); +lean_ctor_set(x_85, 1, x_84); +lean_ctor_set(x_85, 2, x_67); +lean_ctor_set(x_85, 3, x_68); +lean_ctor_set(x_85, 4, x_69); +lean_ctor_set(x_85, 5, x_70); +lean_ctor_set(x_85, 6, x_75); +lean_ctor_set(x_85, 7, x_71); +x_86 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_76); +lean_ctor_set(x_86, 2, x_77); +lean_ctor_set(x_86, 3, x_78); +x_87 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_87, 0, x_86); +lean_ctor_set(x_87, 1, x_1); +lean_ctor_set(x_87, 2, x_2); lean_ctor_set(x_6, 1, x_5); -lean_ctor_set(x_6, 0, x_90); +lean_ctor_set(x_6, 0, x_87); return x_6; } else { -size_t 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_usize_of_nat(x_17); -lean_dec(x_17); -x_92 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -x_93 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_16, x_15, x_91, x_92); +size_t x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_88 = lean_usize_of_nat(x_16); lean_dec(x_16); -x_94 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_94, 0, x_68); -lean_ctor_set(x_94, 1, x_93); -lean_ctor_set(x_94, 2, x_69); -lean_ctor_set(x_94, 3, x_70); -lean_ctor_set(x_94, 4, x_71); -lean_ctor_set(x_94, 5, x_72); -lean_ctor_set(x_94, 6, x_77); -lean_ctor_set(x_94, 7, x_73); -x_95 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_95, 0, x_94); -lean_ctor_set(x_95, 1, x_84); -lean_ctor_set(x_95, 2, x_85); -lean_ctor_set(x_95, 3, x_11); -x_96 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_96, 0, x_95); -lean_ctor_set(x_96, 1, x_1); -lean_ctor_set(x_96, 2, x_2); +x_89 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +x_90 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__6(x_15, x_14, x_88, x_89); +lean_dec(x_15); +x_91 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_91, 0, x_66); +lean_ctor_set(x_91, 1, x_90); +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_75); +lean_ctor_set(x_91, 7, x_71); +x_92 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_92, 0, x_91); +lean_ctor_set(x_92, 1, x_76); +lean_ctor_set(x_92, 2, x_77); +lean_ctor_set(x_92, 3, x_78); +x_93 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_93, 0, x_92); +lean_ctor_set(x_93, 1, x_1); +lean_ctor_set(x_93, 2, x_2); lean_ctor_set(x_6, 1, x_5); -lean_ctor_set(x_6, 0, x_96); +lean_ctor_set(x_6, 0, x_93); return x_6; } } @@ -2546,233 +2570,229 @@ return x_6; } else { -lean_object* x_97; lean_object* x_98; +lean_object* x_94; lean_object* x_95; lean_free_object(x_6); lean_dec(x_8); -x_97 = lean_ctor_get(x_9, 0); -lean_inc(x_97); +x_94 = lean_ctor_get(x_9, 0); +lean_inc(x_94); lean_dec(x_9); -x_98 = lean_ctor_get(x_97, 1); -lean_inc(x_98); -lean_dec(x_97); -x_3 = x_98; -x_4 = x_11; +x_95 = lean_ctor_get(x_94, 1); +lean_inc(x_95); +lean_dec(x_94); +x_3 = x_95; +x_4 = x_10; goto _start; } } else { -lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_100 = lean_ctor_get(x_6, 0); -x_101 = lean_ctor_get(x_6, 1); -lean_inc(x_101); -lean_inc(x_100); +lean_object* x_97; lean_object* x_98; lean_object* x_99; +x_97 = lean_ctor_get(x_6, 0); +x_98 = lean_ctor_get(x_6, 1); +lean_inc(x_98); +lean_inc(x_97); lean_dec(x_6); -x_102 = lean_ctor_get(x_100, 1); -lean_inc(x_102); -x_103 = lean_array_push(x_4, x_102); -if (lean_obj_tag(x_101) == 0) +lean_inc(x_97); +x_99 = lean_array_push(x_4, x_97); +if (lean_obj_tag(x_98) == 0) { -lean_object* x_104; lean_object* x_105; size_t x_106; size_t 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; uint8_t x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; +lean_object* x_100; lean_object* x_101; size_t x_102; size_t x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; uint8_t x_107; size_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; 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_inc(x_2); -x_104 = l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go(x_2); -x_105 = l_Lean_Language_SnapshotTree_getAll(x_104); -x_106 = lean_array_size(x_105); -x_107 = 0; -lean_inc(x_105); -x_108 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__1(x_106, x_107, x_105); -x_109 = lean_array_get_size(x_108); -x_110 = lean_unsigned_to_nat(0u); -x_111 = lean_nat_dec_lt(x_110, x_109); -x_112 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__2(x_106, x_107, x_105); -x_113 = lean_array_get_size(x_112); -x_114 = l_Array_filterMapM___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__3(x_112, x_110, x_113); -lean_dec(x_113); -lean_dec(x_112); -x_115 = l_Array_toPArray_x27___rarg(x_114); +x_100 = l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go(x_2); +x_101 = l_Lean_Language_SnapshotTree_getAll(x_100); +x_102 = lean_array_size(x_101); +x_103 = 0; +x_104 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__1(x_102, x_103, x_101); +x_105 = lean_array_get_size(x_104); +x_106 = lean_unsigned_to_nat(0u); +x_107 = lean_nat_dec_lt(x_106, x_105); +x_108 = lean_array_size(x_99); +lean_inc(x_99); +x_109 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__2(x_108, x_103, x_99); +x_110 = lean_array_get_size(x_109); +x_111 = l_Array_filterMapM___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__3(x_109, x_106, x_110); +lean_dec(x_110); +lean_dec(x_109); +x_112 = l_Array_toPArray_x27___rarg(x_111); +lean_dec(x_111); +x_113 = lean_ctor_get(x_97, 4); +lean_inc(x_113); +x_114 = l_Lean_Language_SnapshotTask_get___rarg(x_113); +x_115 = lean_ctor_get(x_114, 1); +lean_inc(x_115); lean_dec(x_114); -x_116 = lean_ctor_get(x_100, 4); +x_116 = lean_ctor_get(x_115, 6); lean_inc(x_116); -x_117 = l_Lean_Language_SnapshotTask_get___rarg(x_116); -x_118 = lean_ctor_get(x_117, 1); +x_117 = lean_ctor_get(x_115, 0); +lean_inc(x_117); +x_118 = lean_ctor_get(x_115, 2); lean_inc(x_118); -lean_dec(x_117); -x_119 = lean_ctor_get(x_118, 6); +x_119 = lean_ctor_get(x_115, 3); lean_inc(x_119); -x_120 = lean_ctor_get(x_118, 0); +x_120 = lean_ctor_get(x_115, 4); lean_inc(x_120); -x_121 = lean_ctor_get(x_118, 2); +x_121 = lean_ctor_get(x_115, 5); lean_inc(x_121); -x_122 = lean_ctor_get(x_118, 3); +x_122 = lean_ctor_get(x_115, 7); lean_inc(x_122); -x_123 = lean_ctor_get(x_118, 4); -lean_inc(x_123); -x_124 = lean_ctor_get(x_118, 5); -lean_inc(x_124); -x_125 = lean_ctor_get(x_118, 7); -lean_inc(x_125); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - lean_ctor_release(x_118, 2); - lean_ctor_release(x_118, 3); - lean_ctor_release(x_118, 4); - lean_ctor_release(x_118, 5); - lean_ctor_release(x_118, 6); - lean_ctor_release(x_118, 7); - x_126 = x_118; +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); + lean_ctor_release(x_115, 7); + x_123 = x_115; } else { - lean_dec_ref(x_118); - x_126 = lean_box(0); + lean_dec_ref(x_115); + x_123 = lean_box(0); } -x_127 = lean_ctor_get_uint8(x_119, sizeof(void*)*2); -x_128 = lean_ctor_get(x_119, 0); -lean_inc(x_128); -if (lean_is_exclusive(x_119)) { - lean_ctor_release(x_119, 0); - lean_ctor_release(x_119, 1); - x_129 = x_119; +x_124 = lean_ctor_get_uint8(x_116, sizeof(void*)*2); +x_125 = lean_ctor_get(x_116, 0); +lean_inc(x_125); +if (lean_is_exclusive(x_116)) { + lean_ctor_release(x_116, 0); + lean_ctor_release(x_116, 1); + x_126 = x_116; } else { - lean_dec_ref(x_119); - x_129 = lean_box(0); + lean_dec_ref(x_116); + x_126 = lean_box(0); } -if (lean_is_scalar(x_129)) { - x_130 = lean_alloc_ctor(0, 2, 1); +if (lean_is_scalar(x_126)) { + x_127 = lean_alloc_ctor(0, 2, 1); } else { - x_130 = x_129; + x_127 = x_126; } -lean_ctor_set(x_130, 0, x_128); -lean_ctor_set(x_130, 1, x_115); -lean_ctor_set_uint8(x_130, sizeof(void*)*2, x_127); -if (x_111 == 0) +lean_ctor_set(x_127, 0, x_125); +lean_ctor_set(x_127, 1, x_112); +lean_ctor_set_uint8(x_127, sizeof(void*)*2, x_124); +x_128 = lean_ctor_get(x_97, 2); +lean_inc(x_128); +lean_dec(x_97); +x_129 = lean_ctor_get(x_128, 0); +lean_inc(x_129); +x_130 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_108, x_103, x_99); +if (x_107 == 0) { -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_dec(x_109); -lean_dec(x_108); -x_131 = lean_ctor_get(x_100, 2); -lean_inc(x_131); -lean_dec(x_100); -x_132 = lean_ctor_get(x_131, 0); -lean_inc(x_132); -x_133 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -if (lean_is_scalar(x_126)) { - x_134 = lean_alloc_ctor(0, 8, 0); +lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +lean_dec(x_105); +lean_dec(x_104); +x_131 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +if (lean_is_scalar(x_123)) { + x_132 = lean_alloc_ctor(0, 8, 0); } else { - x_134 = x_126; -} -lean_ctor_set(x_134, 0, x_120); -lean_ctor_set(x_134, 1, x_133); -lean_ctor_set(x_134, 2, x_121); -lean_ctor_set(x_134, 3, x_122); -lean_ctor_set(x_134, 4, x_123); -lean_ctor_set(x_134, 5, x_124); -lean_ctor_set(x_134, 6, x_130); -lean_ctor_set(x_134, 7, x_125); -x_135 = lean_alloc_ctor(0, 4, 0); + x_132 = x_123; +} +lean_ctor_set(x_132, 0, x_117); +lean_ctor_set(x_132, 1, x_131); +lean_ctor_set(x_132, 2, x_118); +lean_ctor_set(x_132, 3, x_119); +lean_ctor_set(x_132, 4, x_120); +lean_ctor_set(x_132, 5, x_121); +lean_ctor_set(x_132, 6, x_127); +lean_ctor_set(x_132, 7, x_122); +x_133 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_133, 0, x_132); +lean_ctor_set(x_133, 1, x_128); +lean_ctor_set(x_133, 2, x_129); +lean_ctor_set(x_133, 3, x_130); +x_134 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_134, 0, x_133); +lean_ctor_set(x_134, 1, x_1); +lean_ctor_set(x_134, 2, x_2); +x_135 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_135, 0, x_134); -lean_ctor_set(x_135, 1, x_131); -lean_ctor_set(x_135, 2, x_132); -lean_ctor_set(x_135, 3, x_103); -x_136 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_136, 0, x_135); -lean_ctor_set(x_136, 1, x_1); -lean_ctor_set(x_136, 2, x_2); -x_137 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_137, 0, x_136); -lean_ctor_set(x_137, 1, x_5); -return x_137; +lean_ctor_set(x_135, 1, x_5); +return x_135; } else { -lean_object* x_138; lean_object* x_139; uint8_t x_140; -x_138 = lean_ctor_get(x_100, 2); -lean_inc(x_138); -lean_dec(x_100); -x_139 = lean_ctor_get(x_138, 0); -lean_inc(x_139); -x_140 = lean_nat_dec_le(x_109, x_109); -if (x_140 == 0) +uint8_t x_136; +x_136 = lean_nat_dec_le(x_105, x_105); +if (x_136 == 0) { -lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; -lean_dec(x_109); -lean_dec(x_108); -x_141 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -if (lean_is_scalar(x_126)) { - x_142 = lean_alloc_ctor(0, 8, 0); +lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; +lean_dec(x_105); +lean_dec(x_104); +x_137 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +if (lean_is_scalar(x_123)) { + x_138 = lean_alloc_ctor(0, 8, 0); } else { - x_142 = x_126; -} -lean_ctor_set(x_142, 0, x_120); -lean_ctor_set(x_142, 1, x_141); -lean_ctor_set(x_142, 2, x_121); -lean_ctor_set(x_142, 3, x_122); -lean_ctor_set(x_142, 4, x_123); -lean_ctor_set(x_142, 5, x_124); -lean_ctor_set(x_142, 6, x_130); -lean_ctor_set(x_142, 7, x_125); -x_143 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_143, 0, x_142); -lean_ctor_set(x_143, 1, x_138); -lean_ctor_set(x_143, 2, x_139); -lean_ctor_set(x_143, 3, x_103); -x_144 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_144, 0, x_143); -lean_ctor_set(x_144, 1, x_1); -lean_ctor_set(x_144, 2, x_2); -x_145 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_145, 0, x_144); -lean_ctor_set(x_145, 1, x_5); -return x_145; + x_138 = x_123; +} +lean_ctor_set(x_138, 0, x_117); +lean_ctor_set(x_138, 1, x_137); +lean_ctor_set(x_138, 2, x_118); +lean_ctor_set(x_138, 3, x_119); +lean_ctor_set(x_138, 4, x_120); +lean_ctor_set(x_138, 5, x_121); +lean_ctor_set(x_138, 6, x_127); +lean_ctor_set(x_138, 7, x_122); +x_139 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_139, 0, x_138); +lean_ctor_set(x_139, 1, x_128); +lean_ctor_set(x_139, 2, x_129); +lean_ctor_set(x_139, 3, x_130); +x_140 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_140, 0, x_139); +lean_ctor_set(x_140, 1, x_1); +lean_ctor_set(x_140, 2, x_2); +x_141 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_141, 0, x_140); +lean_ctor_set(x_141, 1, x_5); +return x_141; } else { -size_t 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; -x_146 = lean_usize_of_nat(x_109); -lean_dec(x_109); -x_147 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; -x_148 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_108, x_107, x_146, x_147); -lean_dec(x_108); -if (lean_is_scalar(x_126)) { - x_149 = lean_alloc_ctor(0, 8, 0); +size_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; +x_142 = lean_usize_of_nat(x_105); +lean_dec(x_105); +x_143 = l_Lean_Elab_Frontend_elabCommandAtFrontend___closed__4; +x_144 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__6(x_104, x_103, x_142, x_143); +lean_dec(x_104); +if (lean_is_scalar(x_123)) { + x_145 = lean_alloc_ctor(0, 8, 0); } else { - x_149 = x_126; -} -lean_ctor_set(x_149, 0, x_120); -lean_ctor_set(x_149, 1, x_148); -lean_ctor_set(x_149, 2, x_121); -lean_ctor_set(x_149, 3, x_122); -lean_ctor_set(x_149, 4, x_123); -lean_ctor_set(x_149, 5, x_124); -lean_ctor_set(x_149, 6, x_130); -lean_ctor_set(x_149, 7, x_125); -x_150 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_150, 0, x_149); -lean_ctor_set(x_150, 1, x_138); -lean_ctor_set(x_150, 2, x_139); -lean_ctor_set(x_150, 3, x_103); -x_151 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_151, 0, x_150); -lean_ctor_set(x_151, 1, x_1); -lean_ctor_set(x_151, 2, x_2); -x_152 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_152, 0, x_151); -lean_ctor_set(x_152, 1, x_5); -return x_152; + x_145 = x_123; +} +lean_ctor_set(x_145, 0, x_117); +lean_ctor_set(x_145, 1, x_144); +lean_ctor_set(x_145, 2, x_118); +lean_ctor_set(x_145, 3, x_119); +lean_ctor_set(x_145, 4, x_120); +lean_ctor_set(x_145, 5, x_121); +lean_ctor_set(x_145, 6, x_127); +lean_ctor_set(x_145, 7, x_122); +x_146 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_146, 0, x_145); +lean_ctor_set(x_146, 1, x_128); +lean_ctor_set(x_146, 2, x_129); +lean_ctor_set(x_146, 3, x_130); +x_147 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_147, 0, x_146); +lean_ctor_set(x_147, 1, x_1); +lean_ctor_set(x_147, 2, x_2); +x_148 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_148, 0, x_147); +lean_ctor_set(x_148, 1, x_5); +return x_148; } } } else { -lean_object* x_153; lean_object* x_154; -lean_dec(x_100); -x_153 = lean_ctor_get(x_101, 0); -lean_inc(x_153); -lean_dec(x_101); -x_154 = lean_ctor_get(x_153, 1); -lean_inc(x_154); -lean_dec(x_153); -x_3 = x_154; -x_4 = x_103; +lean_object* x_149; lean_object* x_150; +lean_dec(x_97); +x_149 = lean_ctor_get(x_98, 0); +lean_inc(x_149); +lean_dec(x_98); +x_150 = lean_ctor_get(x_149, 1); +lean_inc(x_150); +lean_dec(x_149); +x_3 = x_150; +x_4 = x_99; goto _start; } } @@ -2826,7 +2846,19 @@ lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5___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_Lean_Elab_IO_processCommandsIncrementally_go___spec__5___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_6 = l_Array_mapMUnsafe_map___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__5(x_4, x_5, x_3); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__6___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; @@ -2834,7 +2866,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_Elab_IO_processCommandsIncrementally_go___spec__5(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_IO_processCommandsIncrementally_go___spec__6(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } diff --git a/stage0/stdlib/Lean/Elab/Inductive.c b/stage0/stdlib/Lean/Elab/Inductive.c index 1f22aede29b0..90fdb9e5deb5 100644 --- a/stage0/stdlib/Lean/Elab/Inductive.c +++ b/stage0/stdlib/Lean/Elab/Inductive.c @@ -85,6 +85,7 @@ static lean_object* l_Lean_Elab_Command_accLevelAtCtor___closed__8; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__2; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__6(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__5(lean_object*, lean_object*); lean_object* l_Lean_indentD(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_resetMaskAt___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___lambda__1___closed__1; @@ -987,7 +988,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_co LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__12(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkIndFVar2Const(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkHeader___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_List_bindTR_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___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_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___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_List_mapM_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___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*, lean_object*, lean_object*, lean_object*); @@ -1327,7 +1327,7 @@ x_4 = lean_alloc_closure((void*)(l_Lean_Elab_Command_checkValidInductiveModifier lean_closure_set(x_4, 0, x_3); lean_closure_set(x_4, 1, x_1); lean_closure_set(x_4, 2, x_2); -x_5 = lean_ctor_get_uint8(x_3, sizeof(void*)*2 + 1); +x_5 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 1); lean_dec(x_3); if (x_5 == 0) { @@ -1397,7 +1397,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___rarg___lam _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_5 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_1, 2); x_6 = lean_array_get_size(x_5); x_7 = lean_unsigned_to_nat(0u); x_8 = lean_nat_dec_eq(x_6, x_7); @@ -1453,7 +1453,7 @@ x_5 = lean_alloc_closure((void*)(l_Lean_Elab_Command_checkValidCtorModifier___ra lean_closure_set(x_5, 0, x_1); lean_closure_set(x_5, 1, x_2); lean_closure_set(x_5, 2, x_3); -x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); +x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); lean_dec(x_1); if (x_6 == 0) { @@ -1571,7 +1571,7 @@ x_4 = lean_alloc_closure((void*)(l_Lean_Elab_Command_checkValidCtorModifier___ra lean_closure_set(x_4, 0, x_3); lean_closure_set(x_4, 1, x_1); lean_closure_set(x_4, 2, x_2); -x_5 = lean_ctor_get_uint8(x_3, sizeof(void*)*2 + 1); +x_5 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 1); lean_dec(x_3); if (x_5 == 0) { @@ -1650,20 +1650,22 @@ return x_2; static lean_object* _init_l_Lean_Elab_Command_instInhabitedCtorView___closed__2() { _start: { -lean_object* x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; x_1 = lean_box(0); -x_2 = 0; +x_2 = lean_box(0); x_3 = 0; x_4 = 0; -x_5 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; -x_6 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -lean_ctor_set_uint8(x_6, sizeof(void*)*2, x_2); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 1, x_3); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 2, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 3, x_3); -return x_6; +x_5 = 0; +x_6 = l_Lean_Elab_Command_instInhabitedCtorView___closed__1; +x_7 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_7, 0, x_2); +lean_ctor_set(x_7, 1, x_1); +lean_ctor_set(x_7, 2, x_6); +lean_ctor_set_uint8(x_7, sizeof(void*)*3, x_3); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 1, x_4); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 2, x_5); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 3, x_4); +return x_7; } } static lean_object* _init_l_Lean_Elab_Command_instInhabitedCtorView___closed__3() { @@ -3022,7 +3024,7 @@ lean_inc(x_16); lean_dec(x_15); x_26 = lean_ctor_get(x_16, 2); lean_inc(x_26); -x_27 = lean_ctor_get_uint8(x_26, sizeof(void*)*2 + 3); +x_27 = lean_ctor_get_uint8(x_26, sizeof(void*)*3 + 3); lean_dec(x_26); if (x_27 == 0) { @@ -3132,7 +3134,7 @@ lean_dec(x_14); x_16 = lean_ctor_get(x_15, 2); lean_inc(x_16); lean_dec(x_15); -x_17 = lean_ctor_get_uint8(x_16, sizeof(void*)*2 + 3); +x_17 = lean_ctor_get_uint8(x_16, sizeof(void*)*3 + 3); lean_dec(x_16); x_18 = lean_box(0); x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1(x_17, x_1, x_12, x_13, x_18, x_2, x_3, x_4, x_5, x_6, x_7, x_8); @@ -26131,7 +26133,7 @@ return x_36; } } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__5(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__5(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -26620,7 +26622,7 @@ lean_inc(x_25); lean_dec(x_23); x_26 = lean_array_to_list(x_19); x_27 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__3___closed__1; -x_28 = l_List_bindTR_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__5(x_24, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__5(x_24, x_27); x_29 = l_List_appendTR___rarg(x_26, x_28); x_30 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams_go(x_3, x_4, x_5, x_7, x_29, x_8, x_9, x_10, x_11, x_25); return x_30; @@ -27791,7 +27793,7 @@ lean_dec(x_31); x_33 = lean_ctor_get(x_14, 2); lean_inc(x_33); lean_dec(x_14); -x_34 = lean_ctor_get(x_33, 1); +x_34 = lean_ctor_get(x_33, 2); lean_inc(x_34); lean_dec(x_33); x_35 = 0; @@ -31271,7 +31273,7 @@ x_16 = lean_ctor_get(x_2, 5); lean_inc(x_16); x_17 = lean_ctor_get(x_2, 2); lean_inc(x_17); -x_18 = lean_ctor_get_uint8(x_17, sizeof(void*)*2 + 3); +x_18 = lean_ctor_get_uint8(x_17, sizeof(void*)*3 + 3); lean_dec(x_17); x_19 = lean_ctor_get(x_2, 0); lean_inc(x_19); @@ -35639,7 +35641,7 @@ lean_inc(x_15); x_16 = lean_ctor_get(x_14, 2); lean_inc(x_16); lean_dec(x_14); -x_17 = lean_ctor_get(x_16, 1); +x_17 = lean_ctor_get(x_16, 2); lean_inc(x_17); lean_dec(x_16); x_18 = 1; diff --git a/stage0/stdlib/Lean/Elab/LetRec.c b/stage0/stdlib/Lean/Elab/LetRec.c index 89af18c5d592..a6f984161b6a 100644 --- a/stage0/stdlib/Lean/Elab/LetRec.c +++ b/stage0/stdlib/Lean/Elab/LetRec.c @@ -26,6 +26,7 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__ lean_object* l_Lean_MapDeclarationExtension_insert___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__18___closed__4; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___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_EXPORT lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7___lambda__7___boxed(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_mkAppN(lean_object*, lean_object*); @@ -70,14 +71,11 @@ lean_object* l_Lean_replaceRef(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabLetRec__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__19___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___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_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__18___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__2___boxed(lean_object**); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); lean_object* l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__22___closed__2; @@ -116,6 +114,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabLetRec lean_object* l_List_appendTR___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__27(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_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__22___closed__6; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__1; size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__20___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_expandOptDocComment_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__1___closed__2; @@ -131,6 +130,7 @@ lean_object* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lea lean_object* l_Array_unzip___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__1___lambda__1___boxed(lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofSyntax(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___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_object*, lean_object*); static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__22___closed__3; lean_object* l_Lean_Elab_Term_expandOptType(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -145,14 +145,15 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_ static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__18___lambda__2___closed__4; static lean_object* l_Lean_Elab_expandOptDocComment_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__1___closed__4; lean_object* l_outOfBounds___rarg(lean_object*); +lean_object* l_Lean_Elab_Term_mkTermInfo(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_EXPORT lean_object* l___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Term_expandDeclId___spec__6(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_Elab_expandOptDocComment_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__26(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_addDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__6___boxed(lean_object*, 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*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__2___boxed(lean_object**); lean_object* l_List_forM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7___lambda__3___closed__3; lean_object* l_Lean_Syntax_getOptional_x3f(lean_object*); @@ -166,6 +167,7 @@ lean_object* l_Lean_Name_append(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_getDeclName_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__27___lambda__1___closed__1; static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7___lambda__4___closed__4; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__3; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__27___lambda__4___closed__3; extern lean_object* l_Lean_instInhabitedExpr; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -175,6 +177,7 @@ static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean LEAN_EXPORT lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getSepArgs(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___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_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___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* l_Lean_Name_str___override(lean_object*, lean_object*); @@ -183,15 +186,17 @@ static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_Le lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7___lambda__3___closed__5; uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__2; lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_mkFreshExprMVarImpl(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___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*); uint8_t l_Lean_Syntax_isIdent(lean_object*); lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__9(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_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___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_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___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*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabLetRec__1___closed__1; static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__18___lambda__2___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Term_elabLetRec_declRange__1___closed__4; static lean_object* l_Lean_Elab_expandOptDocComment_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Std_Format_defWidth; LEAN_EXPORT lean_object* l___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift(lean_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_LetRec_0__Lean_Elab_Term_withAuxLocalDecls_loop___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -225,8 +230,8 @@ static lean_object* l___regBuiltin_Lean_Elab_Term_elabLetRec_declRange__1___clos LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__21(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7___lambda__3___closed__4; lean_object* l_Lean_Elab_Term_addLocalVarInfo(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_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___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*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__20(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___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_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__12___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_addDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__6(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_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__18___lambda__1___boxed(lean_object*); @@ -260,7 +265,9 @@ lean_object* lean_nat_sub(lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__18___closed__5; +lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7___lambda__3___closed__2; +lean_object* l_Lean_Elab_Term_withInfoContext_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_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__27___lambda__5___closed__10; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__21___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_LetRec_0__Lean_Elab_Term_withAuxLocalDecls_loop(lean_object*); @@ -318,7 +325,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_LetRec_ static lean_object* l___regBuiltin_Lean_Elab_Term_elabLetRec__1___closed__6; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___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_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___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_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__27___lambda__5___closed__7; static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__18___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_LetRec_0__Lean_Elab_Term_withAuxLocalDecls_loop___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*, lean_object*); @@ -332,7 +339,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_El LEAN_EXPORT lean_object* l___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__18___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__27___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* l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___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_Elab_elabTerminationHints___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__7___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -681,237 +687,146 @@ return x_56; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___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_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___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) { _start: { -lean_object* x_9; uint8_t 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 = 0; -x_11 = l_Lean_Syntax_getPos_x3f(x_1, x_10); -x_12 = l_Lean_Syntax_getTailPos_x3f(x_1, x_10); -if (lean_obj_tag(x_11) == 0) +uint8_t x_9; lean_object* x_10; +x_9 = 0; +x_10 = l_Lean_Syntax_getRange_x3f(x_1, x_9); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_unsigned_to_nat(0u); -lean_inc(x_9); -x_14 = l_Lean_FileMap_toPosition(x_9, x_13); -lean_inc(x_14); -x_15 = l_Lean_FileMap_leanPosToLspPos(x_9, x_14); -if (lean_obj_tag(x_12) == 0) +lean_object* x_11; lean_object* x_12; +lean_dec(x_6); +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_8); +return x_12; +} +else { -uint8_t x_16; -lean_dec(x_9); -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) +uint8_t x_13; +x_13 = !lean_is_exclusive(x_10); +if (x_13 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_15, 1); -x_18 = lean_ctor_get(x_15, 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_10, 0); +x_15 = lean_ctor_get(x_6, 1); +lean_inc(x_15); +lean_dec(x_6); +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_inc(x_15); +x_17 = l_Lean_FileMap_toPosition(x_15, x_16); +lean_dec(x_16); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_dec(x_14); +lean_inc(x_15); +x_19 = l_Lean_FileMap_toPosition(x_15, x_18); lean_dec(x_18); lean_inc(x_17); -lean_inc(x_14); -x_19 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_19, 0, x_14); -lean_ctor_set(x_19, 1, x_17); -lean_ctor_set(x_19, 2, x_14); -lean_ctor_set(x_19, 3, x_17); -lean_ctor_set(x_15, 1, x_8); -lean_ctor_set(x_15, 0, x_19); -return x_15; -} -else +x_20 = l_Lean_FileMap_leanPosToLspPos(x_15, x_17); +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) { -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_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, 1); +x_23 = lean_ctor_get(x_20, 0); +lean_dec(x_23); +lean_inc(x_19); +x_24 = l_Lean_FileMap_leanPosToLspPos(x_15, x_19); lean_dec(x_15); -lean_inc(x_20); -lean_inc(x_14); -x_21 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_21, 0, x_14); -lean_ctor_set(x_21, 1, x_20); -lean_ctor_set(x_21, 2, x_14); -lean_ctor_set(x_21, 3, 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_8); -return x_22; -} +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_26, 0, x_17); +lean_ctor_set(x_26, 1, x_22); +lean_ctor_set(x_26, 2, x_19); +lean_ctor_set(x_26, 3, x_25); +lean_ctor_set(x_10, 0, x_26); +lean_ctor_set(x_20, 1, x_8); +lean_ctor_set(x_20, 0, x_10); +return x_20; } else { -uint8_t x_23; -x_23 = !lean_is_exclusive(x_15); -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 = lean_ctor_get(x_15, 1); -x_25 = lean_ctor_get(x_15, 0); -lean_dec(x_25); -x_26 = lean_ctor_get(x_12, 0); -lean_inc(x_26); -lean_dec(x_12); -lean_inc(x_9); -x_27 = l_Lean_FileMap_toPosition(x_9, x_26); -lean_dec(x_26); +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_27 = lean_ctor_get(x_20, 1); lean_inc(x_27); -x_28 = l_Lean_FileMap_leanPosToLspPos(x_9, x_27); -lean_dec(x_9); +lean_dec(x_20); +lean_inc(x_19); +x_28 = l_Lean_FileMap_leanPosToLspPos(x_15, x_19); +lean_dec(x_15); x_29 = lean_ctor_get(x_28, 1); lean_inc(x_29); lean_dec(x_28); x_30 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_30, 0, x_14); -lean_ctor_set(x_30, 1, x_24); -lean_ctor_set(x_30, 2, x_27); +lean_ctor_set(x_30, 0, x_17); +lean_ctor_set(x_30, 1, x_27); +lean_ctor_set(x_30, 2, x_19); lean_ctor_set(x_30, 3, x_29); -lean_ctor_set(x_15, 1, x_8); -lean_ctor_set(x_15, 0, x_30); -return x_15; +lean_ctor_set(x_10, 0, x_30); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_10); +lean_ctor_set(x_31, 1, x_8); +return x_31; +} } 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_15, 1); -lean_inc(x_31); -lean_dec(x_15); -x_32 = lean_ctor_get(x_12, 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; lean_object* x_44; lean_object* x_45; +x_32 = lean_ctor_get(x_10, 0); lean_inc(x_32); -lean_dec(x_12); -lean_inc(x_9); -x_33 = l_Lean_FileMap_toPosition(x_9, x_32); +lean_dec(x_10); +x_33 = lean_ctor_get(x_6, 1); +lean_inc(x_33); +lean_dec(x_6); +x_34 = lean_ctor_get(x_32, 0); +lean_inc(x_34); +lean_inc(x_33); +x_35 = l_Lean_FileMap_toPosition(x_33, x_34); +lean_dec(x_34); +x_36 = lean_ctor_get(x_32, 1); +lean_inc(x_36); lean_dec(x_32); lean_inc(x_33); -x_34 = l_Lean_FileMap_leanPosToLspPos(x_9, x_33); -lean_dec(x_9); -x_35 = lean_ctor_get(x_34, 1); +x_37 = l_Lean_FileMap_toPosition(x_33, x_36); +lean_dec(x_36); lean_inc(x_35); -lean_dec(x_34); -x_36 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_36, 0, x_14); -lean_ctor_set(x_36, 1, x_31); -lean_ctor_set(x_36, 2, x_33); -lean_ctor_set(x_36, 3, 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; -} -} -} -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_11, 0); -lean_inc(x_38); -lean_dec(x_11); -lean_inc(x_9); -x_39 = l_Lean_FileMap_toPosition(x_9, x_38); -lean_dec(x_38); +x_38 = l_Lean_FileMap_leanPosToLspPos(x_33, x_35); +x_39 = lean_ctor_get(x_38, 1); lean_inc(x_39); -x_40 = l_Lean_FileMap_leanPosToLspPos(x_9, x_39); -if (lean_obj_tag(x_12) == 0) -{ -uint8_t x_41; -lean_dec(x_9); -x_41 = !lean_is_exclusive(x_40); -if (x_41 == 0) -{ -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_40, 1); -x_43 = lean_ctor_get(x_40, 0); -lean_dec(x_43); -lean_inc(x_42); -lean_inc(x_39); -x_44 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_44, 0, x_39); -lean_ctor_set(x_44, 1, x_42); -lean_ctor_set(x_44, 2, x_39); -lean_ctor_set(x_44, 3, x_42); -lean_ctor_set(x_40, 1, x_8); -lean_ctor_set(x_40, 0, x_44); -return x_40; -} -else -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_40, 1); -lean_inc(x_45); -lean_dec(x_40); -lean_inc(x_45); -lean_inc(x_39); -x_46 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_46, 0, x_39); -lean_ctor_set(x_46, 1, x_45); -lean_ctor_set(x_46, 2, x_39); -lean_ctor_set(x_46, 3, 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_8); -return x_47; -} -} -else -{ -uint8_t x_48; -x_48 = !lean_is_exclusive(x_40); -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; -x_49 = lean_ctor_get(x_40, 1); -x_50 = lean_ctor_get(x_40, 0); -lean_dec(x_50); -x_51 = lean_ctor_get(x_12, 0); -lean_inc(x_51); -lean_dec(x_12); -lean_inc(x_9); -x_52 = l_Lean_FileMap_toPosition(x_9, x_51); -lean_dec(x_51); -lean_inc(x_52); -x_53 = l_Lean_FileMap_leanPosToLspPos(x_9, x_52); -lean_dec(x_9); -x_54 = lean_ctor_get(x_53, 1); -lean_inc(x_54); -lean_dec(x_53); -x_55 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_55, 0, x_39); -lean_ctor_set(x_55, 1, x_49); -lean_ctor_set(x_55, 2, x_52); -lean_ctor_set(x_55, 3, x_54); -lean_ctor_set(x_40, 1, x_8); -lean_ctor_set(x_40, 0, x_55); -return x_40; +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); } -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_40, 1); -lean_inc(x_56); -lean_dec(x_40); -x_57 = lean_ctor_get(x_12, 0); -lean_inc(x_57); -lean_dec(x_12); -lean_inc(x_9); -x_58 = l_Lean_FileMap_toPosition(x_9, x_57); -lean_dec(x_57); -lean_inc(x_58); -x_59 = l_Lean_FileMap_leanPosToLspPos(x_9, x_58); -lean_dec(x_9); -x_60 = lean_ctor_get(x_59, 1); -lean_inc(x_60); -lean_dec(x_59); -x_61 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_61, 0, x_39); -lean_ctor_set(x_61, 1, x_56); -lean_ctor_set(x_61, 2, x_58); -lean_ctor_set(x_61, 3, x_60); -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_8); -return x_62; +lean_inc(x_37); +x_41 = l_Lean_FileMap_leanPosToLspPos(x_33, x_37); +lean_dec(x_33); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +x_43 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_43, 0, x_35); +lean_ctor_set(x_43, 1, x_39); +lean_ctor_set(x_43, 2, x_37); +lean_ctor_set(x_43, 3, x_42); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +if (lean_is_scalar(x_40)) { + x_45 = lean_alloc_ctor(0, 2, 0); +} else { + x_45 = x_40; } +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_8); +return x_45; } } } @@ -1358,42 +1273,97 @@ return x_116; LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___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; uint8_t x_15; +lean_object* x_11; lean_object* x_12; lean_inc(x_8); -x_11 = l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5(x_2, 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_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -lean_inc(x_8); -x_14 = l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) +if (lean_obj_tag(x_12) == 0) { -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_ctor_set(x_14, 1, x_16); -lean_ctor_set(x_14, 0, x_12); -x_18 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__6(x_1, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_17); +uint8_t x_13; lean_dec(x_8); +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 = lean_box(0); +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 = 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; } +} else { 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_ctor_get(x_14, 1); -lean_inc(x_20); +x_19 = lean_ctor_get(x_11, 1); lean_inc(x_19); -lean_dec(x_14); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_12); -lean_ctor_set(x_21, 1, x_19); -x_22 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__6(x_1, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_20); +lean_dec(x_11); +x_20 = lean_ctor_get(x_12, 0); +lean_inc(x_20); +lean_dec(x_12); +lean_inc(x_8); +x_21 = l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_19); +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_20); lean_dec(x_8); -return x_22; +lean_dec(x_1); +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 = lean_box(0); +lean_ctor_set(x_21, 0, x_25); +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 = 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_26); +return x_28; +} +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +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); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_20); +lean_ctor_set(x_31, 1, x_30); +x_32 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__6(x_1, x_31, x_4, x_5, x_6, x_7, x_8, x_9, x_29); +lean_dec(x_8); +return x_32; +} } } } @@ -6417,11 +6387,11 @@ lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___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_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___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) { _start: { lean_object* x_9; -x_9 = l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); @@ -7388,7 +7358,44 @@ return x_22; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___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) { +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("MutualDef", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("body", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__1; +x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___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) { +_start: +{ +lean_object* x_11; uint8_t x_12; lean_object* x_13; +x_11 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__3; +x_12 = 0; +lean_inc(x_2); +x_13 = l_Lean_Elab_Term_mkTermInfo(x_11, x_1, x_3, x_2, x_2, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___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; @@ -7406,7 +7413,7 @@ x_16 = l_Std_Range_forIn_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_ lean_dec(x_2); 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_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; x_17 = lean_ctor_get(x_16, 1); lean_inc(x_17); lean_dec(x_16); @@ -7418,17 +7425,26 @@ lean_dec(x_3); x_20 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_20, 0, x_5); x_21 = lean_box(0); +lean_inc(x_19); x_22 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__1), 11, 4); lean_closure_set(x_22, 0, x_19); lean_closure_set(x_22, 1, x_20); lean_closure_set(x_22, 2, x_21); lean_closure_set(x_22, 3, x_4); -x_23 = l_Lean_Elab_Term_withDeclName___rarg(x_18, x_22, x_6, x_7, x_8, x_9, x_10, x_11, x_17); -return x_23; +lean_inc(x_19); +x_23 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___boxed), 10, 2); +lean_closure_set(x_23, 0, x_19); +lean_closure_set(x_23, 1, x_21); +x_24 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withInfoContext_x27), 10, 3); +lean_closure_set(x_24, 0, x_19); +lean_closure_set(x_24, 1, x_22); +lean_closure_set(x_24, 2, x_23); +x_25 = l_Lean_Elab_Term_withDeclName___rarg(x_18, x_24, x_6, x_7, x_8, x_9, x_10, x_11, x_17); +return x_25; } else { -uint8_t x_24; +uint8_t x_26; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -7438,23 +7454,23 @@ 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) +x_26 = !lean_is_exclusive(x_16); +if (x_26 == 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_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_16, 0); +x_28 = lean_ctor_get(x_16, 1); +lean_inc(x_28); +lean_inc(x_27); 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; +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; } } } @@ -7492,7 +7508,7 @@ x_18 = lean_array_get_size(x_17); lean_inc(x_18); x_19 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_19, 0, x_18); -x_20 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___boxed), 12, 3); +x_20 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__3___boxed), 12, 3); lean_closure_set(x_20, 0, x_17); lean_closure_set(x_20, 1, x_18); lean_closure_set(x_20, 2, x_13); @@ -7578,11 +7594,25 @@ lean_dec(x_1); return x_16; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___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_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___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) { +_start: +{ +lean_object* x_11; +x_11 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___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); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___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_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___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 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___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_1); return x_13; } @@ -7769,7 +7799,7 @@ return x_57; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___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) { _start: { lean_object* x_18; uint8_t x_19; @@ -7992,7 +8022,7 @@ lean_dec(x_21); x_24 = lean_array_get_size(x_1); x_25 = lean_mk_empty_array_with_capacity(x_24); x_26 = lean_unsigned_to_nat(0u); -x_27 = l_Array_mapIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__2(x_1, x_2, x_3, x_20, x_22, x_1, x_24, x_26, lean_box(0), x_25, x_4, x_5, x_6, x_7, x_8, x_9, x_23); +x_27 = l_Array_mapFinIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__2(x_1, x_2, x_3, x_20, x_22, x_1, x_24, x_26, lean_box(0), x_25, x_4, x_5, x_6, x_7, x_8, x_9, x_23); lean_dec(x_8); lean_dec(x_6); lean_dec(x_4); @@ -8141,7 +8171,7 @@ lean_dec(x_2); return x_15; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__2___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___spec__2___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -8162,7 +8192,7 @@ lean_object* x_17 = _args[16]; _start: { lean_object* x_18; -x_18 = l_Array_mapIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___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 = l_Array_mapFinIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___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); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); @@ -9106,6 +9136,12 @@ l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLet lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__27___lambda__5___closed__10); l_Std_Range_forIn_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__1___closed__1 = _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__1___closed__1(); lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__1___closed__1); +l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__1); +l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__2 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__2(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__2); +l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__3 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__3(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__2___closed__3); l___regBuiltin_Lean_Elab_Term_elabLetRec__1___closed__1 = _init_l___regBuiltin_Lean_Elab_Term_elabLetRec__1___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_elabLetRec__1___closed__1); l___regBuiltin_Lean_Elab_Term_elabLetRec__1___closed__2 = _init_l___regBuiltin_Lean_Elab_Term_elabLetRec__1___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/MutualDef.c b/stage0/stdlib/Lean/Elab/MutualDef.c index c30e4edeaa12..b7748f032502 100644 --- a/stage0/stdlib/Lean/Elab/MutualDef.c +++ b/stage0/stdlib/Lean/Elab/MutualDef.c @@ -23,6 +23,8 @@ lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabMutualDef___spec__5(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkSorry(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__8___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_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__3; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__12; static lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__3___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_levelMVarToParam(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -44,7 +46,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getAl LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at_Lean_Elab_Term_elabMutualDef___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_mapMUnsafe_map___at_Lean_LocalContext_getFVars___spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkKinds(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkFreeVarMap___spec__5___rarg___closed__3; static lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___closed__3; lean_object* l_Lean_MapDeclarationExtension_insert___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -79,7 +80,6 @@ static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkKinds static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__3___closed__8; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__5___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__6___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_Elab_instInhabitedDefViewElabHeader___closed__3; -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10; static lean_object* l_Lean_Elab_instInhabitedDefViewElabHeader___closed__6; LEAN_EXPORT lean_object* l_Array_erase___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___spec__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_processDeriving___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -96,30 +96,30 @@ static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeader LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_merge(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkBodyTask(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_MutualDef___hyg_6346____closed__3; -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__7; lean_object* l_Lean_Elab_Command_runTermElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__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___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___closed__2; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___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_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__6; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___closed__5; extern lean_object* l_Lean_declRangeExt; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__2___closed__5; static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosureFor___spec__2(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_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___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_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___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_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__4___closed__2; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__2___closed__1; static lean_object* l_Nat_foldM_loop___at_Lean_Elab_Term_MutualClosure_pushMain___spec__1___closed__1; 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*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_linter_unusedSectionVars; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__4; extern lean_object* l_Lean_Elab_Tactic_instInhabitedTacticParsedSnapshot; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__8___boxed(lean_object**); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__5(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* l_Lean_Language_Snapshot_Diagnostics_ofMessageLog(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__13; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_getMax_x3f___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_pickMaxFVar_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromises___at_Lean_Elab_Term_elabMutualDef_go___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -152,9 +152,8 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_Mutua LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_processDeriving(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__11; lean_object* l_Lean_MessageData_joinSep(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__3___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__3___boxed(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_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__11; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__5___rarg___lambda__2(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__2___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_isAppOfArity(lean_object*, lean_object*, lean_object*); @@ -167,7 +166,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_clean static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__4___rarg___closed__1; lean_object* l_Lean_Elab_logException___at_Lean_Elab_Command_elabCommand___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__9; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef___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*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures(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_Syntax_getId(lean_object*); @@ -175,7 +173,7 @@ static lean_object* l_Nat_foldM_loop___at_Lean_Elab_Term_MutualClosure_pushMain_ lean_object* l_Lean_Elab_Term_elabTermEnsuringType(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_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___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_object* l_Lean_Expr_sort___override(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___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_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___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* 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*); @@ -199,15 +197,15 @@ lean_object* lean_mk_array(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___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*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__5(lean_object*); -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__4___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__2(lean_object*, lean_object*, size_t, size_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); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_deprecated_oldSectionVars; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkModifiers___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosureFor___spec__3(lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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*); +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__3___closed__1; uint8_t l_Array_contains___at___private_Lean_Class_0__Lean_checkOutParam___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArgs(lean_object*); @@ -228,7 +226,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_Replacement_apply___lamb static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___closed__5; 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_Elab_shareCommonPreDefs(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); lean_object* l_Lean_Expr_bvar___override(lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__18(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -238,12 +235,12 @@ static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0_ lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_levelMVarToParamTypesPreDecls___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___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__12___boxed(lean_object**); -lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__3___closed__2; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getPendingMVarErrorMessage___closed__1; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__11___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__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_object*); lean_object* l_Lean_Syntax_TSepArray_getElems___rarg(lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__14; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMutualDef___spec__12(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__9; @@ -270,8 +267,8 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_MutualClosur LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_Command_elabMutualDef___spec__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_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__12___lambda__1___boxed(lean_object**); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___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*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__4(lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6___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_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_MutualClosure_main___spec__3(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_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*); @@ -282,7 +279,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_MutualDef___hyg_6307____closed__6; LEAN_EXPORT uint8_t l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_isExample(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__5___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__6(lean_object*, lean_object*, size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, 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*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__4(lean_object*, 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_MutualDef___hyg_6346____closed__2; @@ -311,15 +308,16 @@ static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfN static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___lambda__2___closed__5; static lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__5; uint8_t l_Lean_MapDeclarationExtension_contains___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__5; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars___spec__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__1___closed__3; lean_object* l_Lean_RBNode_findCore___at_Lean_Meta_mkGeneralizationForbiddenSet_visit___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___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*, lean_object*, lean_object*); uint8_t l_List_any___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___lambda__2(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_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__4(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_Array_mapMUnsafe_map___at_Lean_Elab_Term_MutualClosure_main___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_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___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* l_List_head_x21___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__12___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*); @@ -345,25 +343,29 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__2___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_levelMVarToParamHeaders(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Core_getAndEmptyMessageLog___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__5; static lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___closed__5; LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___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*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___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_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___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_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_levelMVarToParamHeaders_process(lean_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_MutualDef_0__Lean_Elab_Term_declValToTerm(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Elab_DefKind_isExample(uint8_t); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_levelMVarToParamHeaders___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_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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*); static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__1; lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Intro_0__Lean_Meta_introNImp___spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_instantiateMVarsAtLetRecToLift___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_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FVarId_findDecl_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabMutualDef___spec__10___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_MutualDef___hyg_6307____closed__4; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___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_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476_(lean_object*); lean_object* l_Lean_Elab_Term_elabBindersEx___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_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___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_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__1; +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkLetRecsToLiftTypes(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_index(lean_object*); @@ -379,8 +381,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_FixPoint_run___boxed(lea static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_processDeriving___spec__1___closed__1; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__4___closed__3; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Term_elabMutualDef_go___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__3; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__3___closed__5; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___closed__6; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkModifiers___closed__2; @@ -394,11 +394,11 @@ LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_MutualDef_0_ static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__3___closed__2; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_getBodyTerm_x3f___closed__2; lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___boxed(lean_object**); LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_Term_elabMutualDef_go___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_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__3___closed__3; LEAN_EXPORT lean_object* l_Lean_RBNode_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_pushNewVars___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___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*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__7; lean_object* lean_io_promise_resolve(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___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_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_collectUsed___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -412,7 +412,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Mutua LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_fixpoint(lean_object*); lean_object* l_Lean_Elab_Term_expandWhereDeclsOpt(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getPendingMVarErrorMessage___closed__4; -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_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_MutualDef_0__Lean_Elab_Term_check___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_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -429,6 +428,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDe LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___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___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___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_Array_reverse___rarg(lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__12; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_levelMVarToParamHeaders_process___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*); uint8_t l_List_elem___at_Lean_addAliasEntry___spec__16(lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___lambda__1(lean_object*, size_t, lean_object*); @@ -453,6 +453,7 @@ static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_Mu LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosureFor___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_getDeclarationSelectionRef(lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_find___at_Lean_Elab_Term_MutualClosure_isApplicable___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__7; LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___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___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkModifiers___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_realizeGlobalConstNoOverload(lean_object*, lean_object*, lean_object*, lean_object*); @@ -486,6 +487,7 @@ lean_object* lean_nat_div(lean_object*, lean_object*); lean_object* lean_io_add_heartbeats(uint64_t, lean_object*); lean_object* l_Lean_mkHole(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_collectUsed___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabMutualDef___spec__10___lambda__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___lambda__2___closed__4; LEAN_EXPORT uint8_t l_List_mapTR_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getPendingMVarErrorMessage___spec__1___lambda__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -502,6 +504,7 @@ lean_object* l_Lean_registerTraceClass(lean_object*, uint8_t, lean_object*, lean LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosureFor___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_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___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_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___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_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___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* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__13(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_sequenceMap___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at_Lean_Elab_Term_elabMutualDef___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -518,7 +521,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Mutua static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__4___closed__4; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__5; lean_object* l_Lean_CollectFVars_State_addDependencies(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15; LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_Term_MutualClosure_insertReplacementForLetRecs___spec__1(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Term_MutualClosure_isApplicable___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMutualDef___spec__13(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); @@ -541,25 +543,25 @@ lean_object* l_Lean_Meta_check(lean_object*, lean_object*, lean_object*, lean_ob static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef___spec__11(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_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8___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_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__4; -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__7(lean_object*, lean_object*, size_t, size_t, 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_FVarId_getDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_outOfBounds___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__15___boxed(lean_object**); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__10; LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___at_Lean_Elab_Command_elabMutualDef___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___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_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_MutualDef___hyg_6346_(lean_object*); +lean_object* l_Lean_Elab_Term_mkTermInfo(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* l_Array_indexOfAux___at_Lean_LocalContext_erase___spec__3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__7(lean_object*, lean_object*, lean_object*, size_t, 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_MutualDef_0__Lean_Elab_Term_withFunLocalDecls(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__4(lean_object*, 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_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8; lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__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*); static lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___closed__1; @@ -572,6 +574,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabH LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars___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_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_Replacement_apply___lambda__1___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__11; static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__5___closed__3; LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___spec__5(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_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__18___lambda__1___closed__2; @@ -581,7 +584,6 @@ lean_object* l_Lean_Syntax_getOptional_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_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* lean_st_mk_ref(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_updateUsedVarsOf___lambda__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Term_elabMutualDef_go___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_isExample___spec__1(lean_object*, size_t, size_t); LEAN_EXPORT uint8_t l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__4___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -593,7 +595,6 @@ LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Term_MutualClosure_mai static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__2___closed__4; LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_Term_MutualClosure_main___spec__4(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_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___closed__2; -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___lambda__2(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___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_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Term_elabMutualDef___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -607,7 +608,6 @@ lean_object* l_Lean_Elab_instantiateMVarsAtPreDecls(lean_object*, lean_object*, lean_object* l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__1___closed__1; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___lambda__2___closed__6; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_levelMVarToParamHeaders_process___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_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_pushLocalDecl(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*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__4___closed__4; @@ -618,14 +618,13 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabF uint8_t l_Lean_Syntax_isMissing(lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__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___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___closed__2; -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___closed__1; static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__5___closed__4; extern lean_object* l_Lean_levelZero; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5___closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___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_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__1___boxed(lean_object**); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__13; @@ -637,7 +636,7 @@ LEAN_EXPORT lean_object* l_Lean_RBNode_fold___at___private_Lean_Elab_MutualDef_0 lean_object* l_Lean_Elab_InfoTree_substitute(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkModifiers___lambda__2___closed__2; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_getBodyTerm_x3f___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkFreeVarMap___spec__5(lean_object*); @@ -690,7 +689,6 @@ static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__ static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__3___closed__3; static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_MutualDef___hyg_6307____closed__5; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_MutualClosure_main___spec__2(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__2; lean_object* l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_erase___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___spec__2(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); @@ -711,6 +709,7 @@ extern lean_object* l_Lean_Elab_instInhabitedDefView; static lean_object* l_Lean_Elab_Command_elabMutualDef___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMutualDef___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__9; uint8_t l_Lean_Syntax_isIdent(lean_object*); lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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*); @@ -728,6 +727,7 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabMutualDef_ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__7; lean_object* l_Lean_Expr_appFn_x21(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_Command_elabMutualDef___spec__9___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*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__6; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__2(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_getScope___rarg(lean_object*, lean_object*); @@ -746,6 +746,7 @@ lean_object* l_Lean_Elab_Term_withAutoBoundImplicitForbiddenPred___rarg(lean_obj extern lean_object* l_Std_Format_defWidth; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__6___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_instInhabitedDefViewElabHeader___closed__2; +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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* l_Lean_Meta_getZetaDeltaFVarIds___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go___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*); @@ -760,6 +761,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualD lean_object* l_Lean_MVarId_assign___at_Lean_Elab_Term_exprToSyntax___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_Array_foldlMUnsafe_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_pickMaxFVar_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___closed__6; +lean_object* lean_mk_thunk(lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_getBodyTerm_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_isApplicable___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_getKindForLetRecs___boxed(lean_object*); @@ -786,7 +788,6 @@ lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__8; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__4___closed__1; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__12; extern lean_object* l_Lean_Elab_TerminationHints_none; LEAN_EXPORT lean_object* l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__4(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*, lean_object*); @@ -798,6 +799,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_colle LEAN_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__8___lambda__1___boxed(lean_object**); lean_object* l_Lean_Elab_Command_mkDefView(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_getFVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Term_elabMutualDef_go___spec__8(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_Array_mapMUnsafe_map___at_Lean_Elab_Term_MutualClosure_main___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_Elab_MutualDef_0__Lean_Elab_Term_collectUsed___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -805,6 +807,7 @@ lean_object* l_Lean_LocalDecl_userName(lean_object*); lean_object* l_Lean_Syntax_node4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___closed__1; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_registerFailedToInferDefTypeInfo___closed__2; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__8; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___closed__4; extern lean_object* l_Lean_Elab_instTypeNameDefsParsedSnapshot; @@ -814,19 +817,18 @@ LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_E static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_MutualDef___hyg_6307____closed__1; LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___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_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_MutualClosure_main___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_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__8; static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__3___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__3___closed__4; +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkFreeVarMap___spec__5___rarg___closed__1; static lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___lambda__2___closed__2; lean_object* l_Lean_FileMap_leanPosToLspPos(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__2(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___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_elabModifiers___at_Lean_Elab_Command_elabMutualDef___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* l_Lean_Elab_TerminationHints_rememberExtraParams(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__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_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__6; LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromises___at_Lean_Elab_Term_elabMutualDef_go___spec__15(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_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Nat_foldM_loop___at_Lean_Elab_Term_MutualClosure_pushMain___spec__1___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*, lean_object*, lean_object*); @@ -866,6 +868,7 @@ lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Term_elabMutualDef___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_CollectMVars_visit(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__11; static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__3; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5___closed__1; @@ -895,12 +898,12 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDe LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__10(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_Term_elabMutualDef_go___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_isTracingEnabledFor___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___spec__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506_(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__6___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_Elab_Command_elabMutualDef(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureFor___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); 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*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withFunLocalDecls_loop___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*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__13; LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_pushLetRecs(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__2; @@ -911,6 +914,7 @@ static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDe LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__12___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_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Term_elabMutualDef_go___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__3(lean_object*, size_t, size_t); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_registerFailedToInferDefTypeInfo___closed__1; @@ -928,6 +932,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_El static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getFunName___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_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___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*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3; LEAN_EXPORT lean_object* l_Nat_foldM_loop___at_Lean_Elab_Term_MutualClosure_pushMain___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_Nat_foldM_loop___at_Lean_Elab_Term_MutualClosure_pushMain___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*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); @@ -960,6 +965,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__5___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_modifyUsedFVars(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addTrace___at_Lean_Elab_addPreDefinitions___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_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__10; lean_object* l_Lean_LocalDecl_type(lean_object*); uint64_t lean_uint64_xor(uint64_t, uint64_t); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkModifiers___lambda__1___closed__2; @@ -982,7 +988,6 @@ static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfN LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_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_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__6; -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__12; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef___spec__7(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_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef___spec__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_object* l_Lean_LocalContext_get_x21(lean_object*, lean_object*); @@ -1003,8 +1008,8 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDe LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__3(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_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__18___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_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__3___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_Term_withInfoContext_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_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___lambda__2___closed__3; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__9; lean_object* l_List_iotaTR(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__11___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*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__2___closed__1; @@ -1039,7 +1044,7 @@ LEAN_EXPORT lean_object* l_Lean_RBNode_fold___at___private_Lean_Elab_MutualDef_0 LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__6(size_t, size_t, 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_object* l_Lean_Elab_Term_withAuxDecl___rarg(lean_object*, lean_object*, 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_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(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_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_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*, lean_object*); static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_MutualDef___hyg_6346____closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__15___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*); @@ -1058,7 +1063,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualD static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkFreeVarMap___spec__5___rarg___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_fixpoint___boxed(lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__6___closed__1; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__1; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_isMultiConstant_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_modifyUsedFVars___boxed(lean_object*, lean_object*, lean_object*); @@ -1066,10 +1070,13 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_clean lean_object* l_Lean_Meta_removeUnused(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Name_quickCmp(lean_object*, lean_object*); uint8_t l_Lean_Syntax_hasMissing(lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__5___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__6___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_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosureFor___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___boxed(lean_object**); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8; +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10; lean_object* l_Lean_getDelayedMVarRoot___rarg(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Term_instInhabitedLetRecToLift; size_t lean_usize_add(size_t, size_t); @@ -1094,25 +1101,27 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutual lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvar___override(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_array_size(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef___spec__6(lean_object*, 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_MutualDef_0__Lean_Elab_Term_getPendingMVarErrorMessage___closed__3; -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__14; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__6___boxed(lean_object**); static lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_FixPoint_run(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__5___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_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__5(lean_object*, lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5(lean_object*, lean_object*, size_t, size_t, size_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_getUsedFVarsMap(lean_object*); lean_object* l_Lean_Language_SnapshotTask_get___rarg(lean_object*); uint8_t l_Lean_Elab_Modifiers_isNonrec(lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkKinds___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___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_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___closed__6; +static lean_object* l_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___closed__1; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withUsed___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*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__1___rarg___lambda__2(lean_object*, size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__2___closed__4; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_isExample___spec__1___boxed(lean_object*, lean_object*, lean_object*); @@ -1138,6 +1147,7 @@ static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_Mu LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__2(lean_object*, size_t, size_t); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_processDeriving___spec__1___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkFreeVarMap___spec__5___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkFreeVarMap___spec__6___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__6; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___lambda__1___closed__9; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___lambda__1___closed__7; lean_object* lean_string_append(lean_object*, lean_object*); @@ -1154,9 +1164,9 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualD LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__11___lambda__1___boxed(lean_object**); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___boxed(lean_object**); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__3___rarg___lambda__3(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7(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_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__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_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__3(size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__4___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_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__13(lean_object*, size_t, size_t); @@ -1175,6 +1185,7 @@ uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__3___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__11___boxed(lean_object**); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__7; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_resetModified___boxed(lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_cleanupOfNat___lambda__2___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_isExample___boxed(lean_object*); @@ -1193,6 +1204,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualD static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___lambda__2___closed__9; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___rarg___boxed__const__1; +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__3(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_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__4___rarg___lambda__4(lean_object*, size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -1214,15 +1226,13 @@ lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabSyntax___spec__10(le LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_fixLevelParams(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_Term_expandWhereDecls(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___lambda__4___closed__5; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___closed__2; -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabTerminationHints___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_declValToTerminationHint___spec__1___lambda__6___closed__1; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_getFVars___closed__3; -static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__11; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__3(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_getUsedFVarsMap___rarg(lean_object*); uint8_t l_Lean_Elab_Modifiers_isPartial(lean_object*); @@ -1253,6 +1263,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_Mutua LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__6; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars___spec__5(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__9; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_processDeriving___spec__2(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_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withHeaderSecVars_collectUsed___spec__7(lean_object*, lean_object*, size_t, 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_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9___closed__4; @@ -1284,20 +1295,22 @@ return x_2; static lean_object* _init_l_Lean_Elab_instInhabitedDefViewElabHeader___closed__2() { _start: { -lean_object* x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; x_1 = lean_box(0); -x_2 = 0; +x_2 = lean_box(0); x_3 = 0; x_4 = 0; -x_5 = l_Lean_Elab_instInhabitedDefViewElabHeader___closed__1; -x_6 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -lean_ctor_set_uint8(x_6, sizeof(void*)*2, x_2); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 1, x_3); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 2, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 3, x_3); -return x_6; +x_5 = 0; +x_6 = l_Lean_Elab_instInhabitedDefViewElabHeader___closed__1; +x_7 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_7, 0, x_2); +lean_ctor_set(x_7, 1, x_1); +lean_ctor_set(x_7, 2, x_6); +lean_ctor_set_uint8(x_7, sizeof(void*)*3, x_3); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 1, x_4); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 2, x_5); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 3, x_4); +return x_7; } } static lean_object* _init_l_Lean_Elab_instInhabitedDefViewElabHeader___closed__3() { @@ -1473,11 +1486,11 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check _start: { lean_object* x_11; uint8_t x_19; -x_19 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); +x_19 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); if (x_19 == 0) { uint8_t x_20; -x_20 = lean_ctor_get_uint8(x_2, sizeof(void*)*2 + 1); +x_20 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 1); if (x_20 == 0) { lean_object* x_21; lean_object* x_22; @@ -1496,7 +1509,7 @@ goto block_18; else { uint8_t x_24; -x_24 = lean_ctor_get_uint8(x_2, sizeof(void*)*2 + 1); +x_24 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 1); if (x_24 == 0) { lean_object* x_25; @@ -1560,11 +1573,11 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check _start: { lean_object* x_10; uint8_t x_18; -x_18 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); +x_18 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); if (x_18 == 0) { uint8_t x_19; -x_19 = lean_ctor_get_uint8(x_2, sizeof(void*)*2 + 3); +x_19 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 3); if (x_19 == 0) { lean_object* x_20; lean_object* x_21; @@ -1583,7 +1596,7 @@ goto block_17; else { uint8_t x_23; -x_23 = lean_ctor_get_uint8(x_2, sizeof(void*)*2 + 3); +x_23 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 3); if (x_23 == 0) { lean_object* x_24; @@ -2147,7 +2160,7 @@ return x_15; else { uint8_t x_16; -x_16 = lean_ctor_get_uint8(x_12, sizeof(void*)*2 + 3); +x_16 = lean_ctor_get_uint8(x_12, sizeof(void*)*3 + 3); if (x_16 == 0) { lean_object* x_17; lean_object* x_18; @@ -2205,7 +2218,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check lean_object* x_11; lean_object* x_12; uint8_t x_13; x_11 = lean_ctor_get(x_2, 0); x_12 = lean_ctor_get(x_11, 2); -x_13 = lean_ctor_get_uint8(x_12, sizeof(void*)*2 + 1); +x_13 = lean_ctor_get_uint8(x_12, sizeof(void*)*3 + 1); if (x_13 == 0) { lean_object* x_14; lean_object* x_15; @@ -2286,7 +2299,7 @@ else { lean_object* x_16; uint8_t x_17; x_16 = lean_ctor_get(x_11, 2); -x_17 = lean_ctor_get_uint8(x_16, sizeof(void*)*2 + 1); +x_17 = lean_ctor_get_uint8(x_16, sizeof(void*)*3 + 1); if (x_17 == 0) { lean_object* x_18; lean_object* x_19; @@ -2426,7 +2439,7 @@ else { lean_object* x_15; uint8_t x_16; x_15 = lean_ctor_get(x_10, 2); -x_16 = lean_ctor_get_uint8(x_15, sizeof(void*)*2 + 3); +x_16 = lean_ctor_get_uint8(x_15, sizeof(void*)*3 + 3); if (x_16 == 0) { lean_object* x_17; lean_object* x_18; @@ -8118,7 +8131,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Mutua lean_object* x_25; lean_object* x_26; lean_object* x_27; x_25 = lean_ctor_get(x_1, 2); lean_inc(x_25); -x_26 = lean_ctor_get(x_25, 1); +x_26 = lean_ctor_get(x_25, 2); lean_inc(x_26); lean_dec(x_25); lean_inc(x_23); @@ -21632,7 +21645,130 @@ return x_48; } } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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 = 1; +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_12 = l_Lean_Elab_Term_elabTermEnsuringType(x_1, x_2, x_11, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_13; lean_object* x_14; uint8_t x_15; uint8_t x_16; lean_object* x_17; +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 = 1; +x_16 = 0; +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_17 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_15, x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_14); +if (lean_obj_tag(x_17) == 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); +x_19 = l_Lean_Elab_Term_instantiateMVarsProfiling(x_13, x_6, x_7, x_8, x_9, x_18); +return x_19; +} +else +{ +uint8_t x_20; +lean_dec(x_13); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +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; +} +} +} +else +{ +uint8_t 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); +x_24 = !lean_is_exclusive(x_12); +if (x_24 == 0) +{ +return x_12; +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_12, 0); +x_26 = lean_ctor_get(x_12, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_12); +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; +} +} +} +} +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("body", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__5; +x_2 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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; uint8_t x_12; lean_object* x_13; +x_11 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__2; +x_12 = 0; +lean_inc(x_2); +x_13 = l_Lean_Elab_Term_mkTermInfo(x_11, x_1, x_3, x_2, x_2, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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; @@ -21642,7 +21778,7 @@ lean_ctor_set(x_10, 1, x_9); return x_10; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__1() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__1() { _start: { lean_object* x_1; @@ -21650,7 +21786,7 @@ x_1 = l_Lean_Elab_Term_linter_unusedSectionVars; return x_1; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__2() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__2() { _start: { lean_object* x_1; @@ -21658,16 +21794,16 @@ x_1 = lean_mk_string_unchecked("automatically included section variable(s) unuse return x_1; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__2; +x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__2; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__4() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__4() { _start: { lean_object* x_1; @@ -21675,16 +21811,16 @@ x_1 = lean_mk_string_unchecked("':\n ", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__4; +x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__4; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__6() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__6() { _start: { lean_object* x_1; @@ -21692,26 +21828,26 @@ x_1 = lean_mk_string_unchecked("\n ", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__7() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__6; +x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___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_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__7; +x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__7; x_2 = l_Lean_MessageData_ofFormat(x_1); return x_2; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__9() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__9() { _start: { lean_object* x_1; @@ -21719,16 +21855,16 @@ x_1 = lean_mk_string_unchecked("\nconsider restructuring your `variable` declara return x_1; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__9; +x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__9; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__11() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__11() { _start: { lean_object* x_1; @@ -21736,26 +21872,26 @@ x_1 = lean_mk_string_unchecked(" ", 1, 1); return x_1; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__12() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__11; +x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___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_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__12; +x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__12; x_2 = l_Lean_MessageData_ofFormat(x_1); return x_2; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__14() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__14() { _start: { lean_object* x_1; @@ -21763,16 +21899,16 @@ x_1 = lean_mk_string_unchecked(" in theorem ...", 15, 15); return x_1; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__14; +x_1 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__14; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_object* x_17, lean_object* x_18, lean_object* x_19) { +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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, 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_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; @@ -21798,119 +21934,101 @@ lean_dec(x_24); lean_dec(x_21); 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; uint8_t x_33; uint8_t x_34; uint8_t x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; uint8_t x_41; uint8_t x_42; uint8_t x_43; uint8_t x_44; lean_object* x_45; uint8_t x_46; uint8_t x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; +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; uint8_t x_35; uint8_t x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; uint8_t x_43; uint8_t x_44; uint8_t x_45; uint8_t x_46; lean_object* x_47; uint8_t x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; x_27 = lean_ctor_get(x_26, 1); lean_inc(x_27); lean_dec(x_26); x_28 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_28, 0, x_12); x_29 = lean_box(0); -x_30 = lean_ctor_get(x_13, 0); -lean_inc(x_30); -x_31 = lean_ctor_get(x_13, 1); -lean_inc(x_31); -x_32 = lean_ctor_get(x_13, 2); +lean_inc(x_4); +x_30 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__1), 10, 3); +lean_closure_set(x_30, 0, x_4); +lean_closure_set(x_30, 1, x_28); +lean_closure_set(x_30, 2, x_29); +lean_inc(x_4); +x_31 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___boxed), 10, 2); +lean_closure_set(x_31, 0, x_4); +lean_closure_set(x_31, 1, x_29); +x_32 = lean_ctor_get(x_13, 0); lean_inc(x_32); -x_33 = lean_ctor_get_uint8(x_13, sizeof(void*)*9); -x_34 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 1); -x_35 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 2); -x_36 = lean_ctor_get(x_13, 3); -lean_inc(x_36); -x_37 = lean_ctor_get(x_13, 4); -lean_inc(x_37); -x_38 = lean_ctor_get(x_13, 5); +x_33 = lean_ctor_get(x_13, 1); +lean_inc(x_33); +x_34 = lean_ctor_get(x_13, 2); +lean_inc(x_34); +x_35 = lean_ctor_get_uint8(x_13, sizeof(void*)*9); +x_36 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 1); +x_37 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 2); +x_38 = lean_ctor_get(x_13, 3); lean_inc(x_38); -x_39 = lean_ctor_get(x_13, 6); +x_39 = lean_ctor_get(x_13, 4); lean_inc(x_39); -x_40 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 3); -x_41 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 4); -x_42 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 5); -x_43 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 6); -x_44 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 7); -x_45 = lean_ctor_get(x_13, 7); -lean_inc(x_45); -x_46 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 8); -x_47 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 9); -x_48 = lean_alloc_ctor(0, 9, 10); -lean_ctor_set(x_48, 0, x_30); -lean_ctor_set(x_48, 1, x_31); -lean_ctor_set(x_48, 2, x_32); -lean_ctor_set(x_48, 3, x_36); -lean_ctor_set(x_48, 4, x_37); -lean_ctor_set(x_48, 5, x_38); -lean_ctor_set(x_48, 6, x_39); -lean_ctor_set(x_48, 7, x_45); -lean_ctor_set(x_48, 8, x_4); -lean_ctor_set_uint8(x_48, sizeof(void*)*9, x_33); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 1, x_34); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 2, x_35); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 3, x_40); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 4, x_41); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 5, x_42); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 6, x_43); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 7, x_44); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 8, x_46); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 9, x_47); -x_49 = 1; +x_40 = lean_ctor_get(x_13, 5); +lean_inc(x_40); +x_41 = lean_ctor_get(x_13, 6); +lean_inc(x_41); +x_42 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 3); +x_43 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 4); +x_44 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 5); +x_45 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 6); +x_46 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 7); +x_47 = lean_ctor_get(x_13, 7); +lean_inc(x_47); +x_48 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 8); +x_49 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 9); +x_50 = lean_alloc_ctor(0, 9, 10); +lean_ctor_set(x_50, 0, x_32); +lean_ctor_set(x_50, 1, x_33); +lean_ctor_set(x_50, 2, x_34); +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_41); +lean_ctor_set(x_50, 7, x_47); +lean_ctor_set(x_50, 8, x_5); +lean_ctor_set_uint8(x_50, sizeof(void*)*9, x_35); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 1, x_36); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 2, x_37); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 3, x_42); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 4, x_43); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 5, x_44); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 6, x_45); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 7, x_46); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 8, x_48); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 9, x_49); lean_inc(x_18); lean_inc(x_17); lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); -lean_inc(x_48); -x_50 = l_Lean_Elab_Term_elabTermEnsuringType(x_5, x_28, x_49, x_49, x_29, x_48, x_14, x_15, x_16, x_17, x_18, x_27); -if (lean_obj_tag(x_50) == 0) +x_51 = l_Lean_Elab_Term_withInfoContext_x27(x_4, x_30, x_31, x_50, x_14, x_15, x_16, x_17, x_18, x_27); +if (lean_obj_tag(x_51) == 0) { -lean_object* x_51; lean_object* x_52; uint8_t x_53; uint8_t x_54; lean_object* x_55; -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_50, 1); +lean_object* x_52; lean_object* x_53; uint8_t x_54; uint8_t x_55; uint8_t x_56; lean_object* x_57; +x_52 = lean_ctor_get(x_51, 0); lean_inc(x_52); -lean_dec(x_50); -x_53 = 1; +x_53 = lean_ctor_get(x_51, 1); +lean_inc(x_53); +lean_dec(x_51); x_54 = 0; -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -x_55 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_53, x_54, x_48, x_14, x_15, x_16, x_17, x_18, x_52); -if (lean_obj_tag(x_55) == 0) -{ -lean_object* x_56; lean_object* x_57; -x_56 = lean_ctor_get(x_55, 1); -lean_inc(x_56); -lean_dec(x_55); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -x_57 = l_Lean_Elab_Term_instantiateMVarsProfiling(x_51, x_15, x_16, x_17, x_18, x_56); +x_55 = 1; +x_56 = 1; +x_57 = l_Lean_Meta_mkLambdaFVars(x_11, x_52, x_54, x_55, x_54, x_56, x_15, x_16, x_17, x_18, x_53); if (lean_obj_tag(x_57) == 0) { -lean_object* x_58; lean_object* x_59; uint8_t x_60; lean_object* x_61; -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 = 1; -x_61 = l_Lean_Meta_mkLambdaFVars(x_11, x_58, x_54, x_49, x_54, x_60, x_15, x_16, x_17, x_18, x_59); -if (lean_obj_tag(x_61) == 0) -{ -uint8_t x_62; -x_62 = !lean_is_exclusive(x_61); -if (x_62 == 0) +uint8_t x_58; +x_58 = !lean_is_exclusive(x_57); +if (x_58 == 0) { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; -x_63 = lean_ctor_get(x_61, 0); -x_64 = lean_ctor_get(x_61, 1); -x_65 = lean_ctor_get(x_17, 2); -lean_inc(x_65); -x_66 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__1; -x_67 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_65, x_66); -lean_dec(x_65); -if (x_67 == 0) +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_57, 0); +x_60 = lean_ctor_get(x_57, 1); +x_61 = lean_ctor_get(x_17, 2); +lean_inc(x_61); +x_62 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__1; +x_63 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_61, x_62); +lean_dec(x_61); +if (x_63 == 0) { lean_dec(x_18); lean_dec(x_17); @@ -21919,39 +22037,39 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -return x_61; +return x_57; } else { -uint8_t x_68; -x_68 = l_Lean_Expr_hasSorry(x_6); -if (x_68 == 0) +uint8_t x_64; +x_64 = l_Lean_Expr_hasSorry(x_6); +if (x_64 == 0) { -uint8_t x_69; -x_69 = l_Lean_Expr_hasSorry(x_63); -if (x_69 == 0) +uint8_t x_65; +x_65 = l_Lean_Expr_hasSorry(x_59); +if (x_65 == 0) { -lean_object* x_70; lean_object* x_71; -lean_free_object(x_61); -x_70 = lean_array_get_size(x_7); +lean_object* x_66; lean_object* x_67; +lean_free_object(x_57); +x_66 = lean_array_get_size(x_7); lean_inc(x_15); -x_71 = l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__3(x_8, x_7, x_6, x_63, x_7, x_22, x_70, x_13, x_14, x_15, x_16, x_17, x_18, x_64); -lean_dec(x_70); -if (lean_obj_tag(x_71) == 0) +x_67 = l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__3(x_8, x_7, x_6, x_59, x_7, x_22, x_66, x_13, x_14, x_15, x_16, x_17, x_18, x_60); +lean_dec(x_66); +if (lean_obj_tag(x_67) == 0) { -uint8_t x_72; -x_72 = !lean_is_exclusive(x_71); -if (x_72 == 0) +uint8_t x_68; +x_68 = !lean_is_exclusive(x_67); +if (x_68 == 0) { -lean_object* x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; -x_73 = lean_ctor_get(x_71, 0); -x_74 = lean_ctor_get(x_71, 1); -x_75 = lean_array_get_size(x_73); -x_76 = lean_nat_dec_lt(x_22, x_75); -lean_dec(x_75); -if (x_76 == 0) +lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; +x_69 = lean_ctor_get(x_67, 0); +x_70 = lean_ctor_get(x_67, 1); +x_71 = lean_array_get_size(x_69); +x_72 = lean_nat_dec_lt(x_22, x_71); +lean_dec(x_71); +if (x_72 == 0) { -lean_dec(x_73); +lean_dec(x_69); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -21959,86 +22077,86 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -lean_ctor_set(x_71, 0, x_63); -return x_71; +lean_ctor_set(x_67, 0, x_59); +return x_67; } 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; 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; uint8_t x_95; -lean_free_object(x_71); -x_77 = lean_ctor_get(x_9, 0); -x_78 = l_Lean_MessageData_ofName(x_10); -x_79 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3; -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_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5; +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; uint8_t x_91; +lean_free_object(x_67); +x_73 = lean_ctor_get(x_9, 0); +x_74 = l_Lean_MessageData_ofName(x_10); +x_75 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3; +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_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___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 = lean_array_to_list(x_69); +x_80 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8; +lean_inc(x_79); +x_81 = l_Lean_MessageData_joinSep(x_79, x_80); x_82 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_82, 0, x_80); +lean_ctor_set(x_82, 0, x_78); lean_ctor_set(x_82, 1, x_81); -x_83 = lean_array_to_list(x_73); -x_84 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8; -lean_inc(x_83); -x_85 = l_Lean_MessageData_joinSep(x_83, x_84); -x_86 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_86, 0, x_82); -lean_ctor_set(x_86, 1, x_85); -x_87 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10; -x_88 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_88, 0, x_86); -lean_ctor_set(x_88, 1, x_87); -x_89 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13; -x_90 = l_Lean_MessageData_joinSep(x_83, x_89); -x_91 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_91, 0, x_88); -lean_ctor_set(x_91, 1, x_90); -x_92 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15; -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_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_66, x_77, x_93, x_13, x_14, x_15, x_16, x_17, x_18, x_74); +x_83 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10; +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 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13; +x_86 = l_Lean_MessageData_joinSep(x_79, x_85); +x_87 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_87, 0, x_84); +lean_ctor_set(x_87, 1, x_86); +x_88 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15; +x_89 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_89, 0, x_87); +lean_ctor_set(x_89, 1, x_88); +x_90 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_62, x_73, x_89, x_13, x_14, x_15, x_16, x_17, x_18, x_70); lean_dec(x_18); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); -x_95 = !lean_is_exclusive(x_94); -if (x_95 == 0) +x_91 = !lean_is_exclusive(x_90); +if (x_91 == 0) { -lean_object* x_96; -x_96 = lean_ctor_get(x_94, 0); -lean_dec(x_96); -lean_ctor_set(x_94, 0, x_63); -return x_94; +lean_object* x_92; +x_92 = lean_ctor_get(x_90, 0); +lean_dec(x_92); +lean_ctor_set(x_90, 0, x_59); +return x_90; } else { -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 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_98, 0, x_63); -lean_ctor_set(x_98, 1, x_97); -return x_98; +lean_object* x_93; lean_object* x_94; +x_93 = lean_ctor_get(x_90, 1); +lean_inc(x_93); +lean_dec(x_90); +x_94 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_59); +lean_ctor_set(x_94, 1, x_93); +return x_94; } } } else { -lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; -x_99 = lean_ctor_get(x_71, 0); -x_100 = lean_ctor_get(x_71, 1); -lean_inc(x_100); -lean_inc(x_99); -lean_dec(x_71); -x_101 = lean_array_get_size(x_99); -x_102 = lean_nat_dec_lt(x_22, x_101); -lean_dec(x_101); -if (x_102 == 0) +lean_object* x_95; lean_object* x_96; lean_object* x_97; uint8_t x_98; +x_95 = lean_ctor_get(x_67, 0); +x_96 = lean_ctor_get(x_67, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_67); +x_97 = lean_array_get_size(x_95); +x_98 = lean_nat_dec_lt(x_22, x_97); +lean_dec(x_97); +if (x_98 == 0) { -lean_object* x_103; -lean_dec(x_99); +lean_object* x_99; +lean_dec(x_95); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22046,75 +22164,75 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_103 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_103, 0, x_63); -lean_ctor_set(x_103, 1, x_100); -return x_103; -} -else -{ -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; -x_104 = lean_ctor_get(x_9, 0); -x_105 = l_Lean_MessageData_ofName(x_10); -x_106 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3; -x_107 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_107, 0, x_106); -lean_ctor_set(x_107, 1, x_105); -x_108 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5; +x_99 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_99, 0, x_59); +lean_ctor_set(x_99, 1, x_96); +return x_99; +} +else +{ +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; +x_100 = lean_ctor_get(x_9, 0); +x_101 = l_Lean_MessageData_ofName(x_10); +x_102 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3; +x_103 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_103, 0, x_102); +lean_ctor_set(x_103, 1, x_101); +x_104 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5; +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 = lean_array_to_list(x_95); +x_107 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8; +lean_inc(x_106); +x_108 = l_Lean_MessageData_joinSep(x_106, x_107); x_109 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_109, 0, x_107); +lean_ctor_set(x_109, 0, x_105); lean_ctor_set(x_109, 1, x_108); -x_110 = lean_array_to_list(x_99); -x_111 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8; -lean_inc(x_110); -x_112 = l_Lean_MessageData_joinSep(x_110, x_111); -x_113 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_113, 0, x_109); -lean_ctor_set(x_113, 1, x_112); -x_114 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10; -x_115 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_115, 0, x_113); -lean_ctor_set(x_115, 1, x_114); -x_116 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13; -x_117 = l_Lean_MessageData_joinSep(x_110, x_116); -x_118 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_118, 0, x_115); -lean_ctor_set(x_118, 1, x_117); -x_119 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15; -x_120 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_120, 0, x_118); -lean_ctor_set(x_120, 1, x_119); -x_121 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_66, x_104, x_120, x_13, x_14, x_15, x_16, x_17, x_18, x_100); +x_110 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10; +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_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13; +x_113 = l_Lean_MessageData_joinSep(x_106, x_112); +x_114 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_114, 0, x_111); +lean_ctor_set(x_114, 1, x_113); +x_115 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15; +x_116 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_116, 0, x_114); +lean_ctor_set(x_116, 1, x_115); +x_117 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_62, x_100, x_116, x_13, x_14, x_15, x_16, x_17, x_18, x_96); lean_dec(x_18); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); -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; +x_118 = lean_ctor_get(x_117, 1); +lean_inc(x_118); +if (lean_is_exclusive(x_117)) { + lean_ctor_release(x_117, 0); + lean_ctor_release(x_117, 1); + x_119 = x_117; } else { - lean_dec_ref(x_121); - x_123 = lean_box(0); + lean_dec_ref(x_117); + x_119 = lean_box(0); } -if (lean_is_scalar(x_123)) { - x_124 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_119)) { + x_120 = lean_alloc_ctor(0, 2, 0); } else { - x_124 = x_123; + x_120 = x_119; } -lean_ctor_set(x_124, 0, x_63); -lean_ctor_set(x_124, 1, x_122); -return x_124; +lean_ctor_set(x_120, 0, x_59); +lean_ctor_set(x_120, 1, x_118); +return x_120; } } } else { -uint8_t x_125; -lean_dec(x_63); +uint8_t x_121; +lean_dec(x_59); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22122,23 +22240,23 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_125 = !lean_is_exclusive(x_71); -if (x_125 == 0) +x_121 = !lean_is_exclusive(x_67); +if (x_121 == 0) { -return x_71; +return x_67; } else { -lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_126 = lean_ctor_get(x_71, 0); -x_127 = lean_ctor_get(x_71, 1); -lean_inc(x_127); -lean_inc(x_126); -lean_dec(x_71); -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_122; lean_object* x_123; lean_object* x_124; +x_122 = lean_ctor_get(x_67, 0); +x_123 = lean_ctor_get(x_67, 1); +lean_inc(x_123); +lean_inc(x_122); +lean_dec(x_67); +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; } } } @@ -22151,7 +22269,7 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -return x_61; +return x_57; } } else @@ -22163,26 +22281,26 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -return x_61; +return x_57; } } } else { -lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; uint8_t x_133; -x_129 = lean_ctor_get(x_61, 0); -x_130 = lean_ctor_get(x_61, 1); -lean_inc(x_130); -lean_inc(x_129); -lean_dec(x_61); -x_131 = lean_ctor_get(x_17, 2); -lean_inc(x_131); -x_132 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__1; -x_133 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_131, x_132); -lean_dec(x_131); -if (x_133 == 0) +lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; uint8_t x_129; +x_125 = lean_ctor_get(x_57, 0); +x_126 = lean_ctor_get(x_57, 1); +lean_inc(x_126); +lean_inc(x_125); +lean_dec(x_57); +x_127 = lean_ctor_get(x_17, 2); +lean_inc(x_127); +x_128 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__1; +x_129 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_127, x_128); +lean_dec(x_127); +if (x_129 == 0) { -lean_object* x_134; +lean_object* x_130; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22190,48 +22308,48 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_134 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_134, 0, x_129); -lean_ctor_set(x_134, 1, x_130); -return x_134; +x_130 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_130, 0, x_125); +lean_ctor_set(x_130, 1, x_126); +return x_130; } else { -uint8_t x_135; -x_135 = l_Lean_Expr_hasSorry(x_6); -if (x_135 == 0) +uint8_t x_131; +x_131 = l_Lean_Expr_hasSorry(x_6); +if (x_131 == 0) { -uint8_t x_136; -x_136 = l_Lean_Expr_hasSorry(x_129); -if (x_136 == 0) +uint8_t x_132; +x_132 = l_Lean_Expr_hasSorry(x_125); +if (x_132 == 0) { -lean_object* x_137; lean_object* x_138; -x_137 = lean_array_get_size(x_7); +lean_object* x_133; lean_object* x_134; +x_133 = lean_array_get_size(x_7); lean_inc(x_15); -x_138 = l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__3(x_8, x_7, x_6, x_129, x_7, x_22, x_137, x_13, x_14, x_15, x_16, x_17, x_18, x_130); -lean_dec(x_137); -if (lean_obj_tag(x_138) == 0) +x_134 = l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__3(x_8, x_7, x_6, x_125, x_7, x_22, x_133, x_13, x_14, x_15, x_16, x_17, x_18, x_126); +lean_dec(x_133); +if (lean_obj_tag(x_134) == 0) { -lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; uint8_t x_143; -x_139 = lean_ctor_get(x_138, 0); -lean_inc(x_139); -x_140 = lean_ctor_get(x_138, 1); -lean_inc(x_140); -if (lean_is_exclusive(x_138)) { - lean_ctor_release(x_138, 0); - lean_ctor_release(x_138, 1); - x_141 = x_138; +lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; uint8_t x_139; +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_138); - x_141 = lean_box(0); + lean_dec_ref(x_134); + x_137 = lean_box(0); } -x_142 = lean_array_get_size(x_139); -x_143 = lean_nat_dec_lt(x_22, x_142); -lean_dec(x_142); -if (x_143 == 0) +x_138 = lean_array_get_size(x_135); +x_139 = lean_nat_dec_lt(x_22, x_138); +lean_dec(x_138); +if (x_139 == 0) { -lean_object* x_144; -lean_dec(x_139); +lean_object* x_140; +lean_dec(x_135); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22239,79 +22357,79 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -if (lean_is_scalar(x_141)) { - x_144 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_137)) { + x_140 = lean_alloc_ctor(0, 2, 0); } else { - x_144 = x_141; + x_140 = x_137; } -lean_ctor_set(x_144, 0, x_129); -lean_ctor_set(x_144, 1, x_140); -return x_144; +lean_ctor_set(x_140, 0, x_125); +lean_ctor_set(x_140, 1, x_136); +return x_140; } 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; 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_dec(x_141); -x_145 = lean_ctor_get(x_9, 0); -x_146 = l_Lean_MessageData_ofName(x_10); -x_147 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3; -x_148 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_148, 0, x_147); -lean_ctor_set(x_148, 1, x_146); -x_149 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5; +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_dec(x_137); +x_141 = lean_ctor_get(x_9, 0); +x_142 = l_Lean_MessageData_ofName(x_10); +x_143 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3; +x_144 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_144, 0, x_143); +lean_ctor_set(x_144, 1, x_142); +x_145 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5; +x_146 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_146, 0, x_144); +lean_ctor_set(x_146, 1, x_145); +x_147 = lean_array_to_list(x_135); +x_148 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8; +lean_inc(x_147); +x_149 = l_Lean_MessageData_joinSep(x_147, x_148); x_150 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_150, 0, x_148); +lean_ctor_set(x_150, 0, x_146); lean_ctor_set(x_150, 1, x_149); -x_151 = lean_array_to_list(x_139); -x_152 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8; -lean_inc(x_151); -x_153 = l_Lean_MessageData_joinSep(x_151, x_152); -x_154 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_154, 0, x_150); -lean_ctor_set(x_154, 1, x_153); -x_155 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10; -x_156 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_156, 0, x_154); -lean_ctor_set(x_156, 1, x_155); -x_157 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13; -x_158 = l_Lean_MessageData_joinSep(x_151, x_157); -x_159 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_159, 0, x_156); -lean_ctor_set(x_159, 1, x_158); -x_160 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15; -x_161 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_161, 0, x_159); -lean_ctor_set(x_161, 1, x_160); -x_162 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_132, x_145, x_161, x_13, x_14, x_15, x_16, x_17, x_18, x_140); +x_151 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10; +x_152 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_152, 0, x_150); +lean_ctor_set(x_152, 1, x_151); +x_153 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13; +x_154 = l_Lean_MessageData_joinSep(x_147, x_153); +x_155 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_155, 0, x_152); +lean_ctor_set(x_155, 1, x_154); +x_156 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15; +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_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_128, x_141, x_157, x_13, x_14, x_15, x_16, x_17, x_18, x_136); lean_dec(x_18); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); -x_163 = lean_ctor_get(x_162, 1); -lean_inc(x_163); -if (lean_is_exclusive(x_162)) { - lean_ctor_release(x_162, 0); - lean_ctor_release(x_162, 1); - x_164 = x_162; +x_159 = lean_ctor_get(x_158, 1); +lean_inc(x_159); +if (lean_is_exclusive(x_158)) { + lean_ctor_release(x_158, 0); + lean_ctor_release(x_158, 1); + x_160 = x_158; } else { - lean_dec_ref(x_162); - x_164 = lean_box(0); + lean_dec_ref(x_158); + x_160 = lean_box(0); } -if (lean_is_scalar(x_164)) { - x_165 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_160)) { + x_161 = lean_alloc_ctor(0, 2, 0); } else { - x_165 = x_164; + x_161 = x_160; } -lean_ctor_set(x_165, 0, x_129); -lean_ctor_set(x_165, 1, x_163); -return x_165; +lean_ctor_set(x_161, 0, x_125); +lean_ctor_set(x_161, 1, x_159); +return x_161; } } else { -lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; -lean_dec(x_129); +lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; +lean_dec(x_125); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22319,47 +22437,31 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_166 = lean_ctor_get(x_138, 0); -lean_inc(x_166); -x_167 = lean_ctor_get(x_138, 1); -lean_inc(x_167); -if (lean_is_exclusive(x_138)) { - lean_ctor_release(x_138, 0); - lean_ctor_release(x_138, 1); - x_168 = x_138; +x_162 = lean_ctor_get(x_134, 0); +lean_inc(x_162); +x_163 = lean_ctor_get(x_134, 1); +lean_inc(x_163); +if (lean_is_exclusive(x_134)) { + lean_ctor_release(x_134, 0); + lean_ctor_release(x_134, 1); + x_164 = x_134; } else { - lean_dec_ref(x_138); - x_168 = lean_box(0); + lean_dec_ref(x_134); + x_164 = lean_box(0); } -if (lean_is_scalar(x_168)) { - x_169 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_164)) { + x_165 = lean_alloc_ctor(1, 2, 0); } else { - x_169 = x_168; -} -lean_ctor_set(x_169, 0, x_166); -lean_ctor_set(x_169, 1, x_167); -return x_169; -} + x_165 = x_164; } -else -{ -lean_object* x_170; -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_10); -x_170 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_170, 0, x_129); -lean_ctor_set(x_170, 1, x_130); -return x_170; +lean_ctor_set(x_165, 0, x_162); +lean_ctor_set(x_165, 1, x_163); +return x_165; } } else { -lean_object* x_171; +lean_object* x_166; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22367,17 +22469,15 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_171 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_171, 0, x_129); -lean_ctor_set(x_171, 1, x_130); -return x_171; -} -} +x_166 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_166, 0, x_125); +lean_ctor_set(x_166, 1, x_126); +return x_166; } } else { -uint8_t x_172; +lean_object* x_167; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22385,93 +22485,47 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_172 = !lean_is_exclusive(x_61); -if (x_172 == 0) -{ -return x_61; +x_167 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_167, 0, x_125); +lean_ctor_set(x_167, 1, x_126); +return x_167; } -else -{ -lean_object* x_173; lean_object* x_174; lean_object* x_175; -x_173 = lean_ctor_get(x_61, 0); -x_174 = lean_ctor_get(x_61, 1); -lean_inc(x_174); -lean_inc(x_173); -lean_dec(x_61); -x_175 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_175, 0, x_173); -lean_ctor_set(x_175, 1, x_174); -return x_175; } } } else { -uint8_t x_176; +uint8_t x_168; 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_11); lean_dec(x_10); -x_176 = !lean_is_exclusive(x_57); -if (x_176 == 0) +x_168 = !lean_is_exclusive(x_57); +if (x_168 == 0) { return x_57; } else { -lean_object* x_177; lean_object* x_178; lean_object* x_179; -x_177 = lean_ctor_get(x_57, 0); -x_178 = lean_ctor_get(x_57, 1); -lean_inc(x_178); -lean_inc(x_177); +lean_object* x_169; lean_object* x_170; lean_object* x_171; +x_169 = lean_ctor_get(x_57, 0); +x_170 = lean_ctor_get(x_57, 1); +lean_inc(x_170); +lean_inc(x_169); lean_dec(x_57); -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 -{ -uint8_t x_180; -lean_dec(x_51); -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_11); -lean_dec(x_10); -x_180 = !lean_is_exclusive(x_55); -if (x_180 == 0) -{ -return x_55; -} -else -{ -lean_object* x_181; lean_object* x_182; lean_object* x_183; -x_181 = lean_ctor_get(x_55, 0); -x_182 = lean_ctor_get(x_55, 1); -lean_inc(x_182); -lean_inc(x_181); -lean_dec(x_55); -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; +x_171 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_171, 0, x_169); +lean_ctor_set(x_171, 1, x_170); +return x_171; } } } else { -uint8_t x_184; -lean_dec(x_48); +uint8_t x_172; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22480,29 +22534,29 @@ lean_dec(x_14); lean_dec(x_13); lean_dec(x_11); lean_dec(x_10); -x_184 = !lean_is_exclusive(x_50); -if (x_184 == 0) +x_172 = !lean_is_exclusive(x_51); +if (x_172 == 0) { -return x_50; +return x_51; } else { -lean_object* x_185; lean_object* x_186; lean_object* x_187; -x_185 = lean_ctor_get(x_50, 0); -x_186 = lean_ctor_get(x_50, 1); -lean_inc(x_186); -lean_inc(x_185); -lean_dec(x_50); -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_173; lean_object* x_174; lean_object* x_175; +x_173 = lean_ctor_get(x_51, 0); +x_174 = lean_ctor_get(x_51, 1); +lean_inc(x_174); +lean_inc(x_173); +lean_dec(x_51); +x_175 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_175, 0, x_173); +lean_ctor_set(x_175, 1, x_174); +return x_175; } } } else { -uint8_t x_188; +uint8_t x_176; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22514,28 +22568,28 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_5); lean_dec(x_4); -x_188 = !lean_is_exclusive(x_26); -if (x_188 == 0) +x_176 = !lean_is_exclusive(x_26); +if (x_176 == 0) { return x_26; } else { -lean_object* x_189; lean_object* x_190; lean_object* x_191; -x_189 = lean_ctor_get(x_26, 0); -x_190 = lean_ctor_get(x_26, 1); -lean_inc(x_190); -lean_inc(x_189); +lean_object* x_177; lean_object* x_178; lean_object* x_179; +x_177 = lean_ctor_get(x_26, 0); +x_178 = lean_ctor_get(x_26, 1); +lean_inc(x_178); +lean_inc(x_177); lean_dec(x_26); -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; +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; } } } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_object* x_17, lean_object* x_18, lean_object* x_19) { +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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, 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_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; @@ -22561,119 +22615,101 @@ lean_dec(x_24); lean_dec(x_21); 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; uint8_t x_33; uint8_t x_34; uint8_t x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; uint8_t x_41; uint8_t x_42; uint8_t x_43; uint8_t x_44; lean_object* x_45; uint8_t x_46; uint8_t x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; +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; uint8_t x_35; uint8_t x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; uint8_t x_43; uint8_t x_44; uint8_t x_45; uint8_t x_46; lean_object* x_47; uint8_t x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; x_27 = lean_ctor_get(x_26, 1); lean_inc(x_27); lean_dec(x_26); x_28 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_28, 0, x_12); x_29 = lean_box(0); -x_30 = lean_ctor_get(x_13, 0); -lean_inc(x_30); -x_31 = lean_ctor_get(x_13, 1); -lean_inc(x_31); -x_32 = lean_ctor_get(x_13, 2); +lean_inc(x_4); +x_30 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__1), 10, 3); +lean_closure_set(x_30, 0, x_4); +lean_closure_set(x_30, 1, x_28); +lean_closure_set(x_30, 2, x_29); +lean_inc(x_4); +x_31 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___boxed), 10, 2); +lean_closure_set(x_31, 0, x_4); +lean_closure_set(x_31, 1, x_29); +x_32 = lean_ctor_get(x_13, 0); lean_inc(x_32); -x_33 = lean_ctor_get_uint8(x_13, sizeof(void*)*9); -x_34 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 1); -x_35 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 2); -x_36 = lean_ctor_get(x_13, 3); -lean_inc(x_36); -x_37 = lean_ctor_get(x_13, 4); -lean_inc(x_37); -x_38 = lean_ctor_get(x_13, 5); +x_33 = lean_ctor_get(x_13, 1); +lean_inc(x_33); +x_34 = lean_ctor_get(x_13, 2); +lean_inc(x_34); +x_35 = lean_ctor_get_uint8(x_13, sizeof(void*)*9); +x_36 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 1); +x_37 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 2); +x_38 = lean_ctor_get(x_13, 3); lean_inc(x_38); -x_39 = lean_ctor_get(x_13, 6); +x_39 = lean_ctor_get(x_13, 4); lean_inc(x_39); -x_40 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 3); -x_41 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 4); -x_42 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 5); -x_43 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 6); -x_44 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 7); -x_45 = lean_ctor_get(x_13, 7); -lean_inc(x_45); -x_46 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 8); -x_47 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 9); -x_48 = lean_alloc_ctor(0, 9, 10); -lean_ctor_set(x_48, 0, x_30); -lean_ctor_set(x_48, 1, x_31); -lean_ctor_set(x_48, 2, x_32); -lean_ctor_set(x_48, 3, x_36); -lean_ctor_set(x_48, 4, x_37); -lean_ctor_set(x_48, 5, x_38); -lean_ctor_set(x_48, 6, x_39); -lean_ctor_set(x_48, 7, x_45); -lean_ctor_set(x_48, 8, x_4); -lean_ctor_set_uint8(x_48, sizeof(void*)*9, x_33); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 1, x_34); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 2, x_35); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 3, x_40); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 4, x_41); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 5, x_42); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 6, x_43); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 7, x_44); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 8, x_46); -lean_ctor_set_uint8(x_48, sizeof(void*)*9 + 9, x_47); -x_49 = 1; +x_40 = lean_ctor_get(x_13, 5); +lean_inc(x_40); +x_41 = lean_ctor_get(x_13, 6); +lean_inc(x_41); +x_42 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 3); +x_43 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 4); +x_44 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 5); +x_45 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 6); +x_46 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 7); +x_47 = lean_ctor_get(x_13, 7); +lean_inc(x_47); +x_48 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 8); +x_49 = lean_ctor_get_uint8(x_13, sizeof(void*)*9 + 9); +x_50 = lean_alloc_ctor(0, 9, 10); +lean_ctor_set(x_50, 0, x_32); +lean_ctor_set(x_50, 1, x_33); +lean_ctor_set(x_50, 2, x_34); +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_41); +lean_ctor_set(x_50, 7, x_47); +lean_ctor_set(x_50, 8, x_5); +lean_ctor_set_uint8(x_50, sizeof(void*)*9, x_35); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 1, x_36); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 2, x_37); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 3, x_42); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 4, x_43); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 5, x_44); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 6, x_45); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 7, x_46); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 8, x_48); +lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 9, x_49); lean_inc(x_18); lean_inc(x_17); lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); -lean_inc(x_48); -x_50 = l_Lean_Elab_Term_elabTermEnsuringType(x_5, x_28, x_49, x_49, x_29, x_48, x_14, x_15, x_16, x_17, x_18, x_27); -if (lean_obj_tag(x_50) == 0) +x_51 = l_Lean_Elab_Term_withInfoContext_x27(x_4, x_30, x_31, x_50, x_14, x_15, x_16, x_17, x_18, x_27); +if (lean_obj_tag(x_51) == 0) { -lean_object* x_51; lean_object* x_52; uint8_t x_53; uint8_t x_54; lean_object* x_55; -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_50, 1); +lean_object* x_52; lean_object* x_53; uint8_t x_54; uint8_t x_55; uint8_t x_56; lean_object* x_57; +x_52 = lean_ctor_get(x_51, 0); lean_inc(x_52); -lean_dec(x_50); -x_53 = 1; +x_53 = lean_ctor_get(x_51, 1); +lean_inc(x_53); +lean_dec(x_51); x_54 = 0; -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -x_55 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_53, x_54, x_48, x_14, x_15, x_16, x_17, x_18, x_52); -if (lean_obj_tag(x_55) == 0) -{ -lean_object* x_56; lean_object* x_57; -x_56 = lean_ctor_get(x_55, 1); -lean_inc(x_56); -lean_dec(x_55); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -x_57 = l_Lean_Elab_Term_instantiateMVarsProfiling(x_51, x_15, x_16, x_17, x_18, x_56); +x_55 = 1; +x_56 = 1; +x_57 = l_Lean_Meta_mkLambdaFVars(x_11, x_52, x_54, x_55, x_54, x_56, x_15, x_16, x_17, x_18, x_53); if (lean_obj_tag(x_57) == 0) { -lean_object* x_58; lean_object* x_59; uint8_t x_60; lean_object* x_61; -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 = 1; -x_61 = l_Lean_Meta_mkLambdaFVars(x_11, x_58, x_54, x_49, x_54, x_60, x_15, x_16, x_17, x_18, x_59); -if (lean_obj_tag(x_61) == 0) -{ -uint8_t x_62; -x_62 = !lean_is_exclusive(x_61); -if (x_62 == 0) +uint8_t x_58; +x_58 = !lean_is_exclusive(x_57); +if (x_58 == 0) { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; -x_63 = lean_ctor_get(x_61, 0); -x_64 = lean_ctor_get(x_61, 1); -x_65 = lean_ctor_get(x_17, 2); -lean_inc(x_65); -x_66 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__1; -x_67 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_65, x_66); -lean_dec(x_65); -if (x_67 == 0) +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_57, 0); +x_60 = lean_ctor_get(x_57, 1); +x_61 = lean_ctor_get(x_17, 2); +lean_inc(x_61); +x_62 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__1; +x_63 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_61, x_62); +lean_dec(x_61); +if (x_63 == 0) { lean_dec(x_18); lean_dec(x_17); @@ -22682,39 +22718,39 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -return x_61; +return x_57; } else { -uint8_t x_68; -x_68 = l_Lean_Expr_hasSorry(x_6); -if (x_68 == 0) +uint8_t x_64; +x_64 = l_Lean_Expr_hasSorry(x_6); +if (x_64 == 0) { -uint8_t x_69; -x_69 = l_Lean_Expr_hasSorry(x_63); -if (x_69 == 0) +uint8_t x_65; +x_65 = l_Lean_Expr_hasSorry(x_59); +if (x_65 == 0) { -lean_object* x_70; lean_object* x_71; -lean_free_object(x_61); -x_70 = lean_array_get_size(x_7); +lean_object* x_66; lean_object* x_67; +lean_free_object(x_57); +x_66 = lean_array_get_size(x_7); lean_inc(x_15); -x_71 = l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__8(x_8, x_7, x_6, x_63, x_7, x_22, x_70, x_13, x_14, x_15, x_16, x_17, x_18, x_64); -lean_dec(x_70); -if (lean_obj_tag(x_71) == 0) +x_67 = l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__8(x_8, x_7, x_6, x_59, x_7, x_22, x_66, x_13, x_14, x_15, x_16, x_17, x_18, x_60); +lean_dec(x_66); +if (lean_obj_tag(x_67) == 0) { -uint8_t x_72; -x_72 = !lean_is_exclusive(x_71); -if (x_72 == 0) +uint8_t x_68; +x_68 = !lean_is_exclusive(x_67); +if (x_68 == 0) { -lean_object* x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; -x_73 = lean_ctor_get(x_71, 0); -x_74 = lean_ctor_get(x_71, 1); -x_75 = lean_array_get_size(x_73); -x_76 = lean_nat_dec_lt(x_22, x_75); -lean_dec(x_75); -if (x_76 == 0) +lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; +x_69 = lean_ctor_get(x_67, 0); +x_70 = lean_ctor_get(x_67, 1); +x_71 = lean_array_get_size(x_69); +x_72 = lean_nat_dec_lt(x_22, x_71); +lean_dec(x_71); +if (x_72 == 0) { -lean_dec(x_73); +lean_dec(x_69); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22722,86 +22758,86 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -lean_ctor_set(x_71, 0, x_63); -return x_71; +lean_ctor_set(x_67, 0, x_59); +return x_67; } 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; 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; uint8_t x_95; -lean_free_object(x_71); -x_77 = lean_ctor_get(x_9, 0); -x_78 = l_Lean_MessageData_ofName(x_10); -x_79 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3; -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_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5; +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; uint8_t x_91; +lean_free_object(x_67); +x_73 = lean_ctor_get(x_9, 0); +x_74 = l_Lean_MessageData_ofName(x_10); +x_75 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3; +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_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___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 = lean_array_to_list(x_69); +x_80 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8; +lean_inc(x_79); +x_81 = l_Lean_MessageData_joinSep(x_79, x_80); x_82 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_82, 0, x_80); +lean_ctor_set(x_82, 0, x_78); lean_ctor_set(x_82, 1, x_81); -x_83 = lean_array_to_list(x_73); -x_84 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8; -lean_inc(x_83); -x_85 = l_Lean_MessageData_joinSep(x_83, x_84); -x_86 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_86, 0, x_82); -lean_ctor_set(x_86, 1, x_85); -x_87 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10; -x_88 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_88, 0, x_86); -lean_ctor_set(x_88, 1, x_87); -x_89 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13; -x_90 = l_Lean_MessageData_joinSep(x_83, x_89); -x_91 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_91, 0, x_88); -lean_ctor_set(x_91, 1, x_90); -x_92 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15; -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_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_66, x_77, x_93, x_13, x_14, x_15, x_16, x_17, x_18, x_74); +x_83 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10; +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 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13; +x_86 = l_Lean_MessageData_joinSep(x_79, x_85); +x_87 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_87, 0, x_84); +lean_ctor_set(x_87, 1, x_86); +x_88 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15; +x_89 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_89, 0, x_87); +lean_ctor_set(x_89, 1, x_88); +x_90 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_62, x_73, x_89, x_13, x_14, x_15, x_16, x_17, x_18, x_70); lean_dec(x_18); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); -x_95 = !lean_is_exclusive(x_94); -if (x_95 == 0) +x_91 = !lean_is_exclusive(x_90); +if (x_91 == 0) { -lean_object* x_96; -x_96 = lean_ctor_get(x_94, 0); -lean_dec(x_96); -lean_ctor_set(x_94, 0, x_63); -return x_94; +lean_object* x_92; +x_92 = lean_ctor_get(x_90, 0); +lean_dec(x_92); +lean_ctor_set(x_90, 0, x_59); +return x_90; } else { -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 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_98, 0, x_63); -lean_ctor_set(x_98, 1, x_97); -return x_98; +lean_object* x_93; lean_object* x_94; +x_93 = lean_ctor_get(x_90, 1); +lean_inc(x_93); +lean_dec(x_90); +x_94 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_59); +lean_ctor_set(x_94, 1, x_93); +return x_94; } } } else { -lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; -x_99 = lean_ctor_get(x_71, 0); -x_100 = lean_ctor_get(x_71, 1); -lean_inc(x_100); -lean_inc(x_99); -lean_dec(x_71); -x_101 = lean_array_get_size(x_99); -x_102 = lean_nat_dec_lt(x_22, x_101); -lean_dec(x_101); -if (x_102 == 0) +lean_object* x_95; lean_object* x_96; lean_object* x_97; uint8_t x_98; +x_95 = lean_ctor_get(x_67, 0); +x_96 = lean_ctor_get(x_67, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_67); +x_97 = lean_array_get_size(x_95); +x_98 = lean_nat_dec_lt(x_22, x_97); +lean_dec(x_97); +if (x_98 == 0) { -lean_object* x_103; -lean_dec(x_99); +lean_object* x_99; +lean_dec(x_95); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22809,75 +22845,75 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_103 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_103, 0, x_63); -lean_ctor_set(x_103, 1, x_100); -return x_103; -} -else -{ -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; -x_104 = lean_ctor_get(x_9, 0); -x_105 = l_Lean_MessageData_ofName(x_10); -x_106 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3; -x_107 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_107, 0, x_106); -lean_ctor_set(x_107, 1, x_105); -x_108 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5; +x_99 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_99, 0, x_59); +lean_ctor_set(x_99, 1, x_96); +return x_99; +} +else +{ +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; +x_100 = lean_ctor_get(x_9, 0); +x_101 = l_Lean_MessageData_ofName(x_10); +x_102 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3; +x_103 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_103, 0, x_102); +lean_ctor_set(x_103, 1, x_101); +x_104 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5; +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 = lean_array_to_list(x_95); +x_107 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8; +lean_inc(x_106); +x_108 = l_Lean_MessageData_joinSep(x_106, x_107); x_109 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_109, 0, x_107); +lean_ctor_set(x_109, 0, x_105); lean_ctor_set(x_109, 1, x_108); -x_110 = lean_array_to_list(x_99); -x_111 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8; -lean_inc(x_110); -x_112 = l_Lean_MessageData_joinSep(x_110, x_111); -x_113 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_113, 0, x_109); -lean_ctor_set(x_113, 1, x_112); -x_114 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10; -x_115 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_115, 0, x_113); -lean_ctor_set(x_115, 1, x_114); -x_116 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13; -x_117 = l_Lean_MessageData_joinSep(x_110, x_116); -x_118 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_118, 0, x_115); -lean_ctor_set(x_118, 1, x_117); -x_119 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15; -x_120 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_120, 0, x_118); -lean_ctor_set(x_120, 1, x_119); -x_121 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_66, x_104, x_120, x_13, x_14, x_15, x_16, x_17, x_18, x_100); +x_110 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10; +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_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13; +x_113 = l_Lean_MessageData_joinSep(x_106, x_112); +x_114 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_114, 0, x_111); +lean_ctor_set(x_114, 1, x_113); +x_115 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15; +x_116 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_116, 0, x_114); +lean_ctor_set(x_116, 1, x_115); +x_117 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_62, x_100, x_116, x_13, x_14, x_15, x_16, x_17, x_18, x_96); lean_dec(x_18); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); -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; +x_118 = lean_ctor_get(x_117, 1); +lean_inc(x_118); +if (lean_is_exclusive(x_117)) { + lean_ctor_release(x_117, 0); + lean_ctor_release(x_117, 1); + x_119 = x_117; } else { - lean_dec_ref(x_121); - x_123 = lean_box(0); + lean_dec_ref(x_117); + x_119 = lean_box(0); } -if (lean_is_scalar(x_123)) { - x_124 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_119)) { + x_120 = lean_alloc_ctor(0, 2, 0); } else { - x_124 = x_123; + x_120 = x_119; } -lean_ctor_set(x_124, 0, x_63); -lean_ctor_set(x_124, 1, x_122); -return x_124; +lean_ctor_set(x_120, 0, x_59); +lean_ctor_set(x_120, 1, x_118); +return x_120; } } } else { -uint8_t x_125; -lean_dec(x_63); +uint8_t x_121; +lean_dec(x_59); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22885,23 +22921,23 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_125 = !lean_is_exclusive(x_71); -if (x_125 == 0) +x_121 = !lean_is_exclusive(x_67); +if (x_121 == 0) { -return x_71; +return x_67; } else { -lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_126 = lean_ctor_get(x_71, 0); -x_127 = lean_ctor_get(x_71, 1); -lean_inc(x_127); -lean_inc(x_126); -lean_dec(x_71); -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_122; lean_object* x_123; lean_object* x_124; +x_122 = lean_ctor_get(x_67, 0); +x_123 = lean_ctor_get(x_67, 1); +lean_inc(x_123); +lean_inc(x_122); +lean_dec(x_67); +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; } } } @@ -22914,7 +22950,7 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -return x_61; +return x_57; } } else @@ -22926,26 +22962,26 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -return x_61; +return x_57; } } } else { -lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; uint8_t x_133; -x_129 = lean_ctor_get(x_61, 0); -x_130 = lean_ctor_get(x_61, 1); -lean_inc(x_130); -lean_inc(x_129); -lean_dec(x_61); -x_131 = lean_ctor_get(x_17, 2); -lean_inc(x_131); -x_132 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__1; -x_133 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_131, x_132); -lean_dec(x_131); -if (x_133 == 0) +lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; uint8_t x_129; +x_125 = lean_ctor_get(x_57, 0); +x_126 = lean_ctor_get(x_57, 1); +lean_inc(x_126); +lean_inc(x_125); +lean_dec(x_57); +x_127 = lean_ctor_get(x_17, 2); +lean_inc(x_127); +x_128 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__1; +x_129 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_127, x_128); +lean_dec(x_127); +if (x_129 == 0) { -lean_object* x_134; +lean_object* x_130; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -22953,48 +22989,48 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_134 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_134, 0, x_129); -lean_ctor_set(x_134, 1, x_130); -return x_134; +x_130 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_130, 0, x_125); +lean_ctor_set(x_130, 1, x_126); +return x_130; } else { -uint8_t x_135; -x_135 = l_Lean_Expr_hasSorry(x_6); -if (x_135 == 0) +uint8_t x_131; +x_131 = l_Lean_Expr_hasSorry(x_6); +if (x_131 == 0) { -uint8_t x_136; -x_136 = l_Lean_Expr_hasSorry(x_129); -if (x_136 == 0) +uint8_t x_132; +x_132 = l_Lean_Expr_hasSorry(x_125); +if (x_132 == 0) { -lean_object* x_137; lean_object* x_138; -x_137 = lean_array_get_size(x_7); +lean_object* x_133; lean_object* x_134; +x_133 = lean_array_get_size(x_7); lean_inc(x_15); -x_138 = l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__8(x_8, x_7, x_6, x_129, x_7, x_22, x_137, x_13, x_14, x_15, x_16, x_17, x_18, x_130); -lean_dec(x_137); -if (lean_obj_tag(x_138) == 0) +x_134 = l_Array_filterMapM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__8(x_8, x_7, x_6, x_125, x_7, x_22, x_133, x_13, x_14, x_15, x_16, x_17, x_18, x_126); +lean_dec(x_133); +if (lean_obj_tag(x_134) == 0) { -lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; uint8_t x_143; -x_139 = lean_ctor_get(x_138, 0); -lean_inc(x_139); -x_140 = lean_ctor_get(x_138, 1); -lean_inc(x_140); -if (lean_is_exclusive(x_138)) { - lean_ctor_release(x_138, 0); - lean_ctor_release(x_138, 1); - x_141 = x_138; +lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; uint8_t x_139; +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_138); - x_141 = lean_box(0); + lean_dec_ref(x_134); + x_137 = lean_box(0); } -x_142 = lean_array_get_size(x_139); -x_143 = lean_nat_dec_lt(x_22, x_142); -lean_dec(x_142); -if (x_143 == 0) +x_138 = lean_array_get_size(x_135); +x_139 = lean_nat_dec_lt(x_22, x_138); +lean_dec(x_138); +if (x_139 == 0) { -lean_object* x_144; -lean_dec(x_139); +lean_object* x_140; +lean_dec(x_135); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -23002,79 +23038,79 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -if (lean_is_scalar(x_141)) { - x_144 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_137)) { + x_140 = lean_alloc_ctor(0, 2, 0); } else { - x_144 = x_141; + x_140 = x_137; } -lean_ctor_set(x_144, 0, x_129); -lean_ctor_set(x_144, 1, x_140); -return x_144; +lean_ctor_set(x_140, 0, x_125); +lean_ctor_set(x_140, 1, x_136); +return x_140; } 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; 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_dec(x_141); -x_145 = lean_ctor_get(x_9, 0); -x_146 = l_Lean_MessageData_ofName(x_10); -x_147 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3; -x_148 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_148, 0, x_147); -lean_ctor_set(x_148, 1, x_146); -x_149 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5; +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_dec(x_137); +x_141 = lean_ctor_get(x_9, 0); +x_142 = l_Lean_MessageData_ofName(x_10); +x_143 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3; +x_144 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_144, 0, x_143); +lean_ctor_set(x_144, 1, x_142); +x_145 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5; +x_146 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_146, 0, x_144); +lean_ctor_set(x_146, 1, x_145); +x_147 = lean_array_to_list(x_135); +x_148 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8; +lean_inc(x_147); +x_149 = l_Lean_MessageData_joinSep(x_147, x_148); x_150 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_150, 0, x_148); +lean_ctor_set(x_150, 0, x_146); lean_ctor_set(x_150, 1, x_149); -x_151 = lean_array_to_list(x_139); -x_152 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8; -lean_inc(x_151); -x_153 = l_Lean_MessageData_joinSep(x_151, x_152); -x_154 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_154, 0, x_150); -lean_ctor_set(x_154, 1, x_153); -x_155 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10; -x_156 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_156, 0, x_154); -lean_ctor_set(x_156, 1, x_155); -x_157 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13; -x_158 = l_Lean_MessageData_joinSep(x_151, x_157); -x_159 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_159, 0, x_156); -lean_ctor_set(x_159, 1, x_158); -x_160 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15; -x_161 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_161, 0, x_159); -lean_ctor_set(x_161, 1, x_160); -x_162 = l_Lean_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_132, x_145, x_161, x_13, x_14, x_15, x_16, x_17, x_18, x_140); +x_151 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10; +x_152 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_152, 0, x_150); +lean_ctor_set(x_152, 1, x_151); +x_153 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13; +x_154 = l_Lean_MessageData_joinSep(x_147, x_153); +x_155 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_155, 0, x_152); +lean_ctor_set(x_155, 1, x_154); +x_156 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15; +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_Linter_logLint___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__5(x_128, x_141, x_157, x_13, x_14, x_15, x_16, x_17, x_18, x_136); lean_dec(x_18); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); -x_163 = lean_ctor_get(x_162, 1); -lean_inc(x_163); -if (lean_is_exclusive(x_162)) { - lean_ctor_release(x_162, 0); - lean_ctor_release(x_162, 1); - x_164 = x_162; +x_159 = lean_ctor_get(x_158, 1); +lean_inc(x_159); +if (lean_is_exclusive(x_158)) { + lean_ctor_release(x_158, 0); + lean_ctor_release(x_158, 1); + x_160 = x_158; } else { - lean_dec_ref(x_162); - x_164 = lean_box(0); + lean_dec_ref(x_158); + x_160 = lean_box(0); } -if (lean_is_scalar(x_164)) { - x_165 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_160)) { + x_161 = lean_alloc_ctor(0, 2, 0); } else { - x_165 = x_164; + x_161 = x_160; } -lean_ctor_set(x_165, 0, x_129); -lean_ctor_set(x_165, 1, x_163); -return x_165; +lean_ctor_set(x_161, 0, x_125); +lean_ctor_set(x_161, 1, x_159); +return x_161; } } else { -lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; -lean_dec(x_129); +lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; +lean_dec(x_125); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -23082,47 +23118,31 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_166 = lean_ctor_get(x_138, 0); -lean_inc(x_166); -x_167 = lean_ctor_get(x_138, 1); -lean_inc(x_167); -if (lean_is_exclusive(x_138)) { - lean_ctor_release(x_138, 0); - lean_ctor_release(x_138, 1); - x_168 = x_138; +x_162 = lean_ctor_get(x_134, 0); +lean_inc(x_162); +x_163 = lean_ctor_get(x_134, 1); +lean_inc(x_163); +if (lean_is_exclusive(x_134)) { + lean_ctor_release(x_134, 0); + lean_ctor_release(x_134, 1); + x_164 = x_134; } else { - lean_dec_ref(x_138); - x_168 = lean_box(0); + lean_dec_ref(x_134); + x_164 = lean_box(0); } -if (lean_is_scalar(x_168)) { - x_169 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_164)) { + x_165 = lean_alloc_ctor(1, 2, 0); } else { - x_169 = x_168; -} -lean_ctor_set(x_169, 0, x_166); -lean_ctor_set(x_169, 1, x_167); -return x_169; -} + x_165 = x_164; } -else -{ -lean_object* x_170; -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_10); -x_170 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_170, 0, x_129); -lean_ctor_set(x_170, 1, x_130); -return x_170; +lean_ctor_set(x_165, 0, x_162); +lean_ctor_set(x_165, 1, x_163); +return x_165; } } else { -lean_object* x_171; +lean_object* x_166; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -23130,17 +23150,15 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_171 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_171, 0, x_129); -lean_ctor_set(x_171, 1, x_130); -return x_171; -} -} +x_166 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_166, 0, x_125); +lean_ctor_set(x_166, 1, x_126); +return x_166; } } else { -uint8_t x_172; +lean_object* x_167; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -23148,93 +23166,47 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_10); -x_172 = !lean_is_exclusive(x_61); -if (x_172 == 0) -{ -return x_61; +x_167 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_167, 0, x_125); +lean_ctor_set(x_167, 1, x_126); +return x_167; } -else -{ -lean_object* x_173; lean_object* x_174; lean_object* x_175; -x_173 = lean_ctor_get(x_61, 0); -x_174 = lean_ctor_get(x_61, 1); -lean_inc(x_174); -lean_inc(x_173); -lean_dec(x_61); -x_175 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_175, 0, x_173); -lean_ctor_set(x_175, 1, x_174); -return x_175; } } } else { -uint8_t x_176; +uint8_t x_168; 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_11); lean_dec(x_10); -x_176 = !lean_is_exclusive(x_57); -if (x_176 == 0) +x_168 = !lean_is_exclusive(x_57); +if (x_168 == 0) { return x_57; } else { -lean_object* x_177; lean_object* x_178; lean_object* x_179; -x_177 = lean_ctor_get(x_57, 0); -x_178 = lean_ctor_get(x_57, 1); -lean_inc(x_178); -lean_inc(x_177); +lean_object* x_169; lean_object* x_170; lean_object* x_171; +x_169 = lean_ctor_get(x_57, 0); +x_170 = lean_ctor_get(x_57, 1); +lean_inc(x_170); +lean_inc(x_169); lean_dec(x_57); -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 -{ -uint8_t x_180; -lean_dec(x_51); -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_11); -lean_dec(x_10); -x_180 = !lean_is_exclusive(x_55); -if (x_180 == 0) -{ -return x_55; -} -else -{ -lean_object* x_181; lean_object* x_182; lean_object* x_183; -x_181 = lean_ctor_get(x_55, 0); -x_182 = lean_ctor_get(x_55, 1); -lean_inc(x_182); -lean_inc(x_181); -lean_dec(x_55); -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; +x_171 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_171, 0, x_169); +lean_ctor_set(x_171, 1, x_170); +return x_171; } } } else { -uint8_t x_184; -lean_dec(x_48); +uint8_t x_172; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -23243,29 +23215,29 @@ lean_dec(x_14); lean_dec(x_13); lean_dec(x_11); lean_dec(x_10); -x_184 = !lean_is_exclusive(x_50); -if (x_184 == 0) +x_172 = !lean_is_exclusive(x_51); +if (x_172 == 0) { -return x_50; +return x_51; } else { -lean_object* x_185; lean_object* x_186; lean_object* x_187; -x_185 = lean_ctor_get(x_50, 0); -x_186 = lean_ctor_get(x_50, 1); -lean_inc(x_186); -lean_inc(x_185); -lean_dec(x_50); -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_173; lean_object* x_174; lean_object* x_175; +x_173 = lean_ctor_get(x_51, 0); +x_174 = lean_ctor_get(x_51, 1); +lean_inc(x_174); +lean_inc(x_173); +lean_dec(x_51); +x_175 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_175, 0, x_173); +lean_ctor_set(x_175, 1, x_174); +return x_175; } } } else { -uint8_t x_188; +uint8_t x_176; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -23277,28 +23249,28 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_5); lean_dec(x_4); -x_188 = !lean_is_exclusive(x_26); -if (x_188 == 0) +x_176 = !lean_is_exclusive(x_26); +if (x_176 == 0) { return x_26; } else { -lean_object* x_189; lean_object* x_190; lean_object* x_191; -x_189 = lean_ctor_get(x_26, 0); -x_190 = lean_ctor_get(x_26, 1); -lean_inc(x_190); -lean_inc(x_189); +lean_object* x_177; lean_object* x_178; lean_object* x_179; +x_177 = lean_ctor_get(x_26, 0); +x_178 = lean_ctor_get(x_26, 1); +lean_inc(x_178); +lean_inc(x_177); lean_dec(x_26); -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; +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; } } } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_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; lean_object* x_21; @@ -23310,7 +23282,7 @@ lean_inc(x_17); x_18 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_18, 0, x_17); lean_inc(x_16); -x_19 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__3___boxed), 19, 10); +x_19 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___boxed), 19, 10); lean_closure_set(x_19, 0, x_1); lean_closure_set(x_19, 1, x_2); lean_closure_set(x_19, 2, x_17); @@ -23326,7 +23298,7 @@ x_21 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Term_addAutoBoundImplic return x_21; } } -static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___closed__1() { +static lean_object* _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___closed__1() { _start: { lean_object* x_1; @@ -23334,7 +23306,7 @@ x_1 = l_Lean_Elab_Term_deprecated_oldSectionVars; return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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) { _start: { lean_object* x_16; @@ -23364,7 +23336,7 @@ goto block_27; else { lean_object* x_32; uint8_t x_33; -x_32 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___closed__1; +x_32 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___closed__1; x_33 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_28, x_32); lean_dec(x_28); if (x_33 == 0) @@ -23372,11 +23344,11 @@ 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_inc(x_5); lean_inc(x_3); -x_34 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4), 15, 7); +x_34 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6), 15, 7); lean_closure_set(x_34, 0, x_2); lean_closure_set(x_34, 1, x_3); -lean_closure_set(x_34, 2, x_4); -lean_closure_set(x_34, 3, x_17); +lean_closure_set(x_34, 2, x_17); +lean_closure_set(x_34, 3, x_4); lean_closure_set(x_34, 4, x_5); lean_closure_set(x_34, 5, x_6); lean_closure_set(x_34, 6, x_7); @@ -23411,12 +23383,12 @@ x_22 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_22, 0, x_21); x_23 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; lean_inc(x_20); -x_24 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___boxed), 19, 10); +x_24 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___boxed), 19, 10); lean_closure_set(x_24, 0, x_2); lean_closure_set(x_24, 1, x_3); lean_closure_set(x_24, 2, x_21); -lean_closure_set(x_24, 3, x_4); -lean_closure_set(x_24, 4, x_17); +lean_closure_set(x_24, 3, x_17); +lean_closure_set(x_24, 4, x_4); lean_closure_set(x_24, 5, x_20); lean_closure_set(x_24, 6, x_23); lean_closure_set(x_24, 7, x_5); @@ -23463,7 +23435,7 @@ return x_43; } } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_11; uint8_t x_12; @@ -23698,7 +23670,7 @@ lean_inc(x_18); x_19 = lean_ctor_get(x_6, 2); lean_inc(x_19); lean_inc(x_7); -x_20 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___boxed), 15, 8); +x_20 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___boxed), 15, 8); lean_closure_set(x_20, 0, x_8); lean_closure_set(x_20, 1, x_6); lean_closure_set(x_20, 2, x_3); @@ -23721,7 +23693,7 @@ x_24 = lean_ctor_get(x_10, 8); lean_dec(x_24); lean_ctor_set(x_10, 8, x_9); x_25 = lean_box(0); -x_26 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(x_18, x_22, x_10, x_11, x_12, x_13, x_25, x_15, x_16, x_17); +x_26 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(x_18, x_22, x_10, x_11, x_12, x_13, x_25, x_15, x_16, x_17); return x_26; } else @@ -23775,7 +23747,7 @@ lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 7, x_41); lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 8, x_43); lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 9, x_44); x_46 = lean_box(0); -x_47 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(x_18, x_22, x_45, x_11, x_12, x_13, x_46, x_15, x_16, x_17); +x_47 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(x_18, x_22, x_45, x_11, x_12, x_13, x_46, x_15, x_16, x_17); return x_47; } } @@ -23893,7 +23865,7 @@ lean_inc(x_18); x_19 = lean_ctor_get(x_6, 2); lean_inc(x_19); lean_inc(x_7); -x_20 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___boxed), 15, 8); +x_20 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___boxed), 15, 8); lean_closure_set(x_20, 0, x_8); lean_closure_set(x_20, 1, x_6); lean_closure_set(x_20, 2, x_3); @@ -23916,7 +23888,7 @@ x_24 = lean_ctor_get(x_10, 8); lean_dec(x_24); lean_ctor_set(x_10, 8, x_9); x_25 = lean_box(0); -x_26 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(x_18, x_22, x_10, x_11, x_12, x_13, x_25, x_15, x_16, x_17); +x_26 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(x_18, x_22, x_10, x_11, x_12, x_13, x_25, x_15, x_16, x_17); return x_26; } else @@ -23970,7 +23942,7 @@ lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 7, x_41); lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 8, x_43); lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 9, x_44); x_46 = lean_box(0); -x_47 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(x_18, x_22, x_45, x_11, x_12, x_13, x_46, x_15, x_16, x_17); +x_47 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(x_18, x_22, x_45, x_11, x_12, x_13, x_46, x_15, x_16, x_17); return x_47; } } @@ -24574,7 +24546,7 @@ lean_inc(x_18); x_19 = lean_ctor_get(x_6, 2); lean_inc(x_19); lean_inc(x_7); -x_20 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___boxed), 15, 8); +x_20 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___boxed), 15, 8); lean_closure_set(x_20, 0, x_8); lean_closure_set(x_20, 1, x_6); lean_closure_set(x_20, 2, x_3); @@ -24597,7 +24569,7 @@ x_24 = lean_ctor_get(x_10, 8); lean_dec(x_24); lean_ctor_set(x_10, 8, x_9); x_25 = lean_box(0); -x_26 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(x_18, x_22, x_10, x_11, x_12, x_13, x_25, x_15, x_16, x_17); +x_26 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(x_18, x_22, x_10, x_11, x_12, x_13, x_25, x_15, x_16, x_17); return x_26; } else @@ -24651,7 +24623,7 @@ lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 7, x_41); lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 8, x_43); lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 9, x_44); x_46 = lean_box(0); -x_47 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(x_18, x_22, x_45, x_11, x_12, x_13, x_46, x_15, x_16, x_17); +x_47 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(x_18, x_22, x_45, x_11, x_12, x_13, x_46, x_15, x_16, x_17); return x_47; } } @@ -24769,7 +24741,7 @@ lean_inc(x_18); x_19 = lean_ctor_get(x_6, 2); lean_inc(x_19); lean_inc(x_7); -x_20 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___boxed), 15, 8); +x_20 = lean_alloc_closure((void*)(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___boxed), 15, 8); lean_closure_set(x_20, 0, x_8); lean_closure_set(x_20, 1, x_6); lean_closure_set(x_20, 2, x_3); @@ -24792,7 +24764,7 @@ x_24 = lean_ctor_get(x_10, 8); lean_dec(x_24); lean_ctor_set(x_10, 8, x_9); x_25 = lean_box(0); -x_26 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(x_18, x_22, x_10, x_11, x_12, x_13, x_25, x_15, x_16, x_17); +x_26 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(x_18, x_22, x_10, x_11, x_12, x_13, x_25, x_15, x_16, x_17); return x_26; } else @@ -24846,7 +24818,7 @@ lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 7, x_41); lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 8, x_43); lean_ctor_set_uint8(x_45, sizeof(void*)*9 + 9, x_44); x_46 = lean_box(0); -x_47 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(x_18, x_22, x_45, x_11, x_12, x_13, x_46, x_15, x_16, x_17); +x_47 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__8(x_18, x_22, x_45, x_11, x_12, x_13, x_46, x_15, x_16, x_17); return x_47; } } @@ -27155,11 +27127,25 @@ lean_dec(x_1); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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); @@ -27170,7 +27156,7 @@ lean_dec(x_2); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -27193,7 +27179,7 @@ lean_object* x_19 = _args[18]; _start: { lean_object* x_20; -x_20 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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, x_17, x_18, x_19); +x_20 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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, x_15, x_16, x_17, x_18, x_19); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -27204,7 +27190,7 @@ lean_dec(x_1); return x_20; } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__3___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -27227,7 +27213,7 @@ lean_object* x_19 = _args[18]; _start: { lean_object* x_20; -x_20 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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, x_17, x_18, x_19); +x_20 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__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, x_14, x_15, x_16, x_17, x_18, x_19); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -27238,20 +27224,20 @@ lean_dec(x_1); return x_20; } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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) { _start: { lean_object* x_16; -x_16 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__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, x_14, x_15); +x_16 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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); lean_dec(x_8); return x_16; } } -LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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: { lean_object* x_11; -x_11 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___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_7); return x_11; } @@ -37385,11 +37371,11 @@ x_14 = !lean_is_exclusive(x_1); 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_21; -x_15 = lean_ctor_get(x_1, 1); +x_15 = lean_ctor_get(x_1, 2); lean_dec(x_15); x_16 = lean_ctor_get(x_2, 2); lean_inc(x_16); -lean_ctor_set(x_1, 1, x_16); +lean_ctor_set(x_1, 2, x_16); x_17 = lean_ctor_get(x_2, 4); x_18 = lean_ctor_get(x_2, 10); lean_inc(x_18); @@ -37411,41 +37397,44 @@ return x_21; } else { -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_32; lean_object* x_33; +lean_object* x_22; lean_object* x_23; uint8_t x_24; uint8_t x_25; uint8_t 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; x_22 = lean_ctor_get(x_1, 0); -x_23 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); -x_24 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); -x_25 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 2); -x_26 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); +x_23 = lean_ctor_get(x_1, 1); +x_24 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); +x_25 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); +x_26 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 2); +x_27 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); +lean_inc(x_23); lean_inc(x_22); lean_dec(x_1); -x_27 = lean_ctor_get(x_2, 2); -lean_inc(x_27); -x_28 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_28, 0, x_22); -lean_ctor_set(x_28, 1, x_27); -lean_ctor_set_uint8(x_28, sizeof(void*)*2, x_23); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 1, x_24); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 2, x_25); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 3, x_26); -x_29 = lean_ctor_get(x_2, 4); -x_30 = lean_ctor_get(x_2, 10); +x_28 = lean_ctor_get(x_2, 2); +lean_inc(x_28); +x_29 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_29, 0, x_22); +lean_ctor_set(x_29, 1, x_23); +lean_ctor_set(x_29, 2, x_28); +lean_ctor_set_uint8(x_29, sizeof(void*)*3, x_24); +lean_ctor_set_uint8(x_29, sizeof(void*)*3 + 1, x_25); +lean_ctor_set_uint8(x_29, sizeof(void*)*3 + 2, x_26); +lean_ctor_set_uint8(x_29, sizeof(void*)*3 + 3, x_27); +x_30 = lean_ctor_get(x_2, 4); +x_31 = lean_ctor_get(x_2, 10); +lean_inc(x_31); lean_inc(x_30); -lean_inc(x_29); -x_31 = lean_alloc_ctor(0, 7, 1); -lean_ctor_set(x_31, 0, x_3); -lean_ctor_set(x_31, 1, x_13); -lean_ctor_set(x_31, 2, x_28); -lean_ctor_set(x_31, 3, x_29); -lean_ctor_set(x_31, 4, x_4); -lean_ctor_set(x_31, 5, x_5); -lean_ctor_set(x_31, 6, x_30); -lean_ctor_set_uint8(x_31, sizeof(void*)*7, x_7); -x_32 = lean_array_push(x_6, 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_12); -return x_33; +x_32 = lean_alloc_ctor(0, 7, 1); +lean_ctor_set(x_32, 0, x_3); +lean_ctor_set(x_32, 1, x_13); +lean_ctor_set(x_32, 2, x_29); +lean_ctor_set(x_32, 3, x_30); +lean_ctor_set(x_32, 4, x_4); +lean_ctor_set(x_32, 5, x_5); +lean_ctor_set(x_32, 6, x_31); +lean_ctor_set_uint8(x_32, sizeof(void*)*7, x_7); +x_33 = lean_array_push(x_6, 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_12); +return x_34; } } } @@ -37996,7 +37985,7 @@ lean_dec(x_5); x_7 = lean_ctor_get(x_6, 2); lean_inc(x_7); lean_dec(x_6); -x_8 = lean_ctor_get_uint8(x_7, sizeof(void*)*2 + 3); +x_8 = lean_ctor_get_uint8(x_7, sizeof(void*)*3 + 3); lean_dec(x_7); if (x_8 == 0) { @@ -38076,7 +38065,7 @@ lean_dec(x_5); x_7 = lean_ctor_get(x_6, 2); lean_inc(x_7); lean_dec(x_6); -x_8 = lean_ctor_get_uint8(x_7, sizeof(void*)*2 + 1); +x_8 = lean_ctor_get_uint8(x_7, sizeof(void*)*3 + 1); lean_dec(x_7); if (x_8 == 0) { @@ -38101,6 +38090,20 @@ return x_13; } } } +static lean_object* _init_l_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___closed__1() { +_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___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___closed__10; +x_3 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; +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; +} +} LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs(lean_object* x_1) { _start: { @@ -38111,99 +38114,105 @@ x_4 = lean_unsigned_to_nat(0u); x_5 = lean_nat_dec_lt(x_4, x_3); if (x_5 == 0) { -uint8_t x_32; -x_32 = 0; -x_6 = x_32; -goto block_31; +uint8_t x_35; +x_35 = 0; +x_6 = x_35; +goto block_34; } else { -size_t x_33; size_t x_34; uint8_t x_35; -x_33 = 0; -x_34 = lean_usize_of_nat(x_3); -x_35 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__3(x_1, x_33, x_34); -x_6 = x_35; -goto block_31; +size_t x_36; size_t x_37; uint8_t x_38; +x_36 = 0; +x_37 = lean_usize_of_nat(x_3); +x_38 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__3(x_1, x_36, x_37); +x_6 = x_38; +goto block_34; } -block_31: +block_34: { lean_object* x_7; if (x_5 == 0) { -lean_object* x_21; -x_21 = lean_box(0); -x_7 = x_21; -goto block_20; +lean_object* x_23; +x_23 = lean_box(0); +x_7 = x_23; +goto block_22; } else { -size_t x_22; size_t x_23; uint8_t x_24; -x_22 = 0; -x_23 = lean_usize_of_nat(x_3); -x_24 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__2(x_1, x_22, x_23); -if (x_24 == 0) +size_t x_24; size_t x_25; uint8_t x_26; +x_24 = 0; +x_25 = lean_usize_of_nat(x_3); +x_26 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__2(x_1, x_24, x_25); +if (x_26 == 0) { -lean_object* x_25; -x_25 = lean_box(0); -x_7 = x_25; -goto block_20; +lean_object* x_27; +x_27 = lean_box(0); +x_7 = x_27; +goto block_22; } else { -uint8_t x_26; uint8_t x_27; uint8_t x_28; lean_object* x_29; lean_object* x_30; +uint8_t x_28; lean_object* x_29; uint8_t x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; lean_dec(x_3); -x_26 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__1(x_1, x_22, x_23); -x_27 = 0; -x_28 = 0; -x_29 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; -x_30 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_30, 0, x_2); -lean_ctor_set(x_30, 1, x_29); -lean_ctor_set_uint8(x_30, sizeof(void*)*2, x_27); -lean_ctor_set_uint8(x_30, sizeof(void*)*2 + 1, x_6); -lean_ctor_set_uint8(x_30, sizeof(void*)*2 + 2, x_28); -lean_ctor_set_uint8(x_30, sizeof(void*)*2 + 3, x_26); -return x_30; +x_28 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__1(x_1, x_24, x_25); +x_29 = l_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___closed__1; +x_30 = 0; +x_31 = 0; +x_32 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; +x_33 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_33, 0, x_29); +lean_ctor_set(x_33, 1, x_2); +lean_ctor_set(x_33, 2, x_32); +lean_ctor_set_uint8(x_33, sizeof(void*)*3, x_30); +lean_ctor_set_uint8(x_33, sizeof(void*)*3 + 1, x_6); +lean_ctor_set_uint8(x_33, sizeof(void*)*3 + 2, x_31); +lean_ctor_set_uint8(x_33, sizeof(void*)*3 + 3, x_28); +return x_33; } } -block_20: +block_22: { lean_dec(x_7); if (x_5 == 0) { -uint8_t x_8; uint8_t x_9; uint8_t x_10; lean_object* x_11; lean_object* x_12; +lean_object* x_8; uint8_t x_9; uint8_t x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_dec(x_3); -x_8 = 0; -x_9 = 2; -x_10 = 0; -x_11 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; -x_12 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_12, 0, x_2); -lean_ctor_set(x_12, 1, x_11); -lean_ctor_set_uint8(x_12, sizeof(void*)*2, x_8); -lean_ctor_set_uint8(x_12, sizeof(void*)*2 + 1, x_6); -lean_ctor_set_uint8(x_12, sizeof(void*)*2 + 2, x_9); -lean_ctor_set_uint8(x_12, sizeof(void*)*2 + 3, x_10); -return x_12; +x_8 = l_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___closed__1; +x_9 = 0; +x_10 = 2; +x_11 = 0; +x_12 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; +x_13 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_13, 0, x_8); +lean_ctor_set(x_13, 1, x_2); +lean_ctor_set(x_13, 2, x_12); +lean_ctor_set_uint8(x_13, sizeof(void*)*3, x_9); +lean_ctor_set_uint8(x_13, sizeof(void*)*3 + 1, x_6); +lean_ctor_set_uint8(x_13, sizeof(void*)*3 + 2, x_10); +lean_ctor_set_uint8(x_13, sizeof(void*)*3 + 3, x_11); +return x_13; } else { -size_t x_13; size_t x_14; uint8_t x_15; uint8_t x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; -x_13 = 0; -x_14 = lean_usize_of_nat(x_3); +size_t x_14; size_t x_15; uint8_t x_16; lean_object* x_17; uint8_t x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; +x_14 = 0; +x_15 = lean_usize_of_nat(x_3); lean_dec(x_3); -x_15 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__1(x_1, x_13, x_14); -x_16 = 0; -x_17 = 2; -x_18 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; -x_19 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_19, 0, x_2); -lean_ctor_set(x_19, 1, x_18); -lean_ctor_set_uint8(x_19, sizeof(void*)*2, x_16); -lean_ctor_set_uint8(x_19, sizeof(void*)*2 + 1, x_6); -lean_ctor_set_uint8(x_19, sizeof(void*)*2 + 2, x_17); -lean_ctor_set_uint8(x_19, sizeof(void*)*2 + 3, x_15); -return x_19; +x_16 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__1(x_1, x_14, x_15); +x_17 = l_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___closed__1; +x_18 = 0; +x_19 = 2; +x_20 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; +x_21 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_21, 0, x_17); +lean_ctor_set(x_21, 1, x_2); +lean_ctor_set(x_21, 2, x_20); +lean_ctor_set_uint8(x_21, sizeof(void*)*3, x_18); +lean_ctor_set_uint8(x_21, sizeof(void*)*3 + 1, x_6); +lean_ctor_set_uint8(x_21, sizeof(void*)*3 + 2, x_19); +lean_ctor_set_uint8(x_21, sizeof(void*)*3 + 3, x_16); +return x_21; } } } @@ -42906,237 +42915,146 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Term_elabMutualDef_go___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_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Term_elabMutualDef_go___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) { _start: { -lean_object* x_9; uint8_t 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 = 0; -x_11 = l_Lean_Syntax_getPos_x3f(x_1, x_10); -x_12 = l_Lean_Syntax_getTailPos_x3f(x_1, x_10); -if (lean_obj_tag(x_11) == 0) +uint8_t x_9; lean_object* x_10; +x_9 = 0; +x_10 = l_Lean_Syntax_getRange_x3f(x_1, x_9); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_unsigned_to_nat(0u); -lean_inc(x_9); -x_14 = l_Lean_FileMap_toPosition(x_9, x_13); -lean_inc(x_14); -x_15 = l_Lean_FileMap_leanPosToLspPos(x_9, x_14); -if (lean_obj_tag(x_12) == 0) +lean_object* x_11; lean_object* x_12; +lean_dec(x_6); +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_8); +return x_12; +} +else { -uint8_t x_16; -lean_dec(x_9); -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) +uint8_t x_13; +x_13 = !lean_is_exclusive(x_10); +if (x_13 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_15, 1); -x_18 = lean_ctor_get(x_15, 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_10, 0); +x_15 = lean_ctor_get(x_6, 1); +lean_inc(x_15); +lean_dec(x_6); +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_inc(x_15); +x_17 = l_Lean_FileMap_toPosition(x_15, x_16); +lean_dec(x_16); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_dec(x_14); +lean_inc(x_15); +x_19 = l_Lean_FileMap_toPosition(x_15, x_18); lean_dec(x_18); lean_inc(x_17); -lean_inc(x_14); -x_19 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_19, 0, x_14); -lean_ctor_set(x_19, 1, x_17); -lean_ctor_set(x_19, 2, x_14); -lean_ctor_set(x_19, 3, x_17); -lean_ctor_set(x_15, 1, x_8); -lean_ctor_set(x_15, 0, x_19); -return x_15; -} -else +x_20 = l_Lean_FileMap_leanPosToLspPos(x_15, x_17); +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) { -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_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, 1); +x_23 = lean_ctor_get(x_20, 0); +lean_dec(x_23); +lean_inc(x_19); +x_24 = l_Lean_FileMap_leanPosToLspPos(x_15, x_19); lean_dec(x_15); -lean_inc(x_20); -lean_inc(x_14); -x_21 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_21, 0, x_14); -lean_ctor_set(x_21, 1, x_20); -lean_ctor_set(x_21, 2, x_14); -lean_ctor_set(x_21, 3, 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_8); -return x_22; -} +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_26, 0, x_17); +lean_ctor_set(x_26, 1, x_22); +lean_ctor_set(x_26, 2, x_19); +lean_ctor_set(x_26, 3, x_25); +lean_ctor_set(x_10, 0, x_26); +lean_ctor_set(x_20, 1, x_8); +lean_ctor_set(x_20, 0, x_10); +return x_20; } else { -uint8_t x_23; -x_23 = !lean_is_exclusive(x_15); -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 = lean_ctor_get(x_15, 1); -x_25 = lean_ctor_get(x_15, 0); -lean_dec(x_25); -x_26 = lean_ctor_get(x_12, 0); -lean_inc(x_26); -lean_dec(x_12); -lean_inc(x_9); -x_27 = l_Lean_FileMap_toPosition(x_9, x_26); -lean_dec(x_26); +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_27 = lean_ctor_get(x_20, 1); lean_inc(x_27); -x_28 = l_Lean_FileMap_leanPosToLspPos(x_9, x_27); -lean_dec(x_9); +lean_dec(x_20); +lean_inc(x_19); +x_28 = l_Lean_FileMap_leanPosToLspPos(x_15, x_19); +lean_dec(x_15); x_29 = lean_ctor_get(x_28, 1); lean_inc(x_29); lean_dec(x_28); x_30 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_30, 0, x_14); -lean_ctor_set(x_30, 1, x_24); -lean_ctor_set(x_30, 2, x_27); +lean_ctor_set(x_30, 0, x_17); +lean_ctor_set(x_30, 1, x_27); +lean_ctor_set(x_30, 2, x_19); lean_ctor_set(x_30, 3, x_29); -lean_ctor_set(x_15, 1, x_8); -lean_ctor_set(x_15, 0, x_30); -return x_15; +lean_ctor_set(x_10, 0, x_30); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_10); +lean_ctor_set(x_31, 1, x_8); +return x_31; +} } 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_15, 1); -lean_inc(x_31); -lean_dec(x_15); -x_32 = lean_ctor_get(x_12, 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; lean_object* x_44; lean_object* x_45; +x_32 = lean_ctor_get(x_10, 0); lean_inc(x_32); -lean_dec(x_12); -lean_inc(x_9); -x_33 = l_Lean_FileMap_toPosition(x_9, x_32); +lean_dec(x_10); +x_33 = lean_ctor_get(x_6, 1); +lean_inc(x_33); +lean_dec(x_6); +x_34 = lean_ctor_get(x_32, 0); +lean_inc(x_34); +lean_inc(x_33); +x_35 = l_Lean_FileMap_toPosition(x_33, x_34); +lean_dec(x_34); +x_36 = lean_ctor_get(x_32, 1); +lean_inc(x_36); lean_dec(x_32); lean_inc(x_33); -x_34 = l_Lean_FileMap_leanPosToLspPos(x_9, x_33); -lean_dec(x_9); -x_35 = lean_ctor_get(x_34, 1); +x_37 = l_Lean_FileMap_toPosition(x_33, x_36); +lean_dec(x_36); lean_inc(x_35); -lean_dec(x_34); -x_36 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_36, 0, x_14); -lean_ctor_set(x_36, 1, x_31); -lean_ctor_set(x_36, 2, x_33); -lean_ctor_set(x_36, 3, 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; -} -} -} -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_11, 0); -lean_inc(x_38); -lean_dec(x_11); -lean_inc(x_9); -x_39 = l_Lean_FileMap_toPosition(x_9, x_38); -lean_dec(x_38); -lean_inc(x_39); -x_40 = l_Lean_FileMap_leanPosToLspPos(x_9, x_39); -if (lean_obj_tag(x_12) == 0) -{ -uint8_t x_41; -lean_dec(x_9); -x_41 = !lean_is_exclusive(x_40); -if (x_41 == 0) -{ -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_40, 1); -x_43 = lean_ctor_get(x_40, 0); -lean_dec(x_43); -lean_inc(x_42); -lean_inc(x_39); -x_44 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_44, 0, x_39); -lean_ctor_set(x_44, 1, x_42); -lean_ctor_set(x_44, 2, x_39); -lean_ctor_set(x_44, 3, x_42); -lean_ctor_set(x_40, 1, x_8); -lean_ctor_set(x_40, 0, x_44); -return x_40; -} -else -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_40, 1); -lean_inc(x_45); -lean_dec(x_40); -lean_inc(x_45); +x_38 = l_Lean_FileMap_leanPosToLspPos(x_33, x_35); +x_39 = lean_ctor_get(x_38, 1); lean_inc(x_39); -x_46 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_46, 0, x_39); -lean_ctor_set(x_46, 1, x_45); -lean_ctor_set(x_46, 2, x_39); -lean_ctor_set(x_46, 3, 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_8); -return x_47; -} -} -else -{ -uint8_t x_48; -x_48 = !lean_is_exclusive(x_40); -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; -x_49 = lean_ctor_get(x_40, 1); -x_50 = lean_ctor_get(x_40, 0); -lean_dec(x_50); -x_51 = lean_ctor_get(x_12, 0); -lean_inc(x_51); -lean_dec(x_12); -lean_inc(x_9); -x_52 = l_Lean_FileMap_toPosition(x_9, x_51); -lean_dec(x_51); -lean_inc(x_52); -x_53 = l_Lean_FileMap_leanPosToLspPos(x_9, x_52); -lean_dec(x_9); -x_54 = lean_ctor_get(x_53, 1); -lean_inc(x_54); -lean_dec(x_53); -x_55 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_55, 0, x_39); -lean_ctor_set(x_55, 1, x_49); -lean_ctor_set(x_55, 2, x_52); -lean_ctor_set(x_55, 3, x_54); -lean_ctor_set(x_40, 1, x_8); -lean_ctor_set(x_40, 0, x_55); -return x_40; +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); } -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_40, 1); -lean_inc(x_56); -lean_dec(x_40); -x_57 = lean_ctor_get(x_12, 0); -lean_inc(x_57); -lean_dec(x_12); -lean_inc(x_9); -x_58 = l_Lean_FileMap_toPosition(x_9, x_57); -lean_dec(x_57); -lean_inc(x_58); -x_59 = l_Lean_FileMap_leanPosToLspPos(x_9, x_58); -lean_dec(x_9); -x_60 = lean_ctor_get(x_59, 1); -lean_inc(x_60); -lean_dec(x_59); -x_61 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_61, 0, x_39); -lean_ctor_set(x_61, 1, x_56); -lean_ctor_set(x_61, 2, x_58); -lean_ctor_set(x_61, 3, x_60); -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_8); -return x_62; +lean_inc(x_37); +x_41 = l_Lean_FileMap_leanPosToLspPos(x_33, x_37); +lean_dec(x_33); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +x_43 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_43, 0, x_35); +lean_ctor_set(x_43, 1, x_39); +lean_ctor_set(x_43, 2, x_37); +lean_ctor_set(x_43, 3, x_42); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +if (lean_is_scalar(x_40)) { + x_45 = lean_alloc_ctor(0, 2, 0); +} else { + x_45 = x_40; } +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_8); +return x_45; } } } @@ -43580,6 +43498,122 @@ return x_116; } } } +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___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) { +_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; +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); +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 = lean_box(2); +x_17 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_mkTacTask___closed__10; +x_18 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +lean_ctor_set(x_18, 2, x_15); +lean_inc(x_9); +x_19 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Term_elabMutualDef_go___spec__8(x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_18); +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_9); +lean_dec(x_3); +lean_dec(x_1); +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 = lean_box(0); +lean_ctor_set(x_19, 0, x_23); +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 = 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; +} +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +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); +x_29 = l_Lean_Elab_getDeclarationSelectionRef(x_1); +lean_inc(x_9); +x_30 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Term_elabMutualDef_go___spec__8(x_29, x_5, x_6, x_7, x_8, x_9, x_10, x_27); +lean_dec(x_29); +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +if (lean_obj_tag(x_31) == 0) +{ +uint8_t x_32; +lean_dec(x_28); +lean_dec(x_9); +lean_dec(x_3); +x_32 = !lean_is_exclusive(x_30); +if (x_32 == 0) +{ +lean_object* x_33; lean_object* x_34; +x_33 = lean_ctor_get(x_30, 0); +lean_dec(x_33); +x_34 = lean_box(0); +lean_ctor_set(x_30, 0, x_34); +return x_30; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_30, 1); +lean_inc(x_35); +lean_dec(x_30); +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 +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_38 = lean_ctor_get(x_30, 1); +lean_inc(x_38); +lean_dec(x_30); +x_39 = lean_ctor_get(x_31, 0); +lean_inc(x_39); +lean_dec(x_31); +x_40 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_40, 0, x_28); +lean_ctor_set(x_40, 1, x_39); +x_41 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9(x_3, x_40, x_5, x_6, x_7, x_8, x_9, x_10, x_38); +lean_dec(x_9); +return x_41; +} +} +} +} static lean_object* _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__1() { _start: { @@ -43600,68 +43634,34 @@ x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___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_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___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) { _start: { -lean_object* x_10; lean_object* x_11; uint8_t x_12; -lean_inc(x_2); -x_10 = l_Lean_Syntax_getKind(x_2); -x_11 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__2; -x_12 = lean_name_eq(x_10, x_11); -lean_dec(x_10); -if (x_12 == 0) -{ -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_inc(x_7); -x_13 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Term_elabMutualDef_go___spec__8(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -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_getDeclarationSelectionRef(x_2); -lean_inc(x_7); -x_17 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Term_elabMutualDef_go___spec__8(x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_15); -lean_dec(x_16); -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 = lean_ctor_get(x_17, 1); -lean_ctor_set(x_17, 1, x_19); -lean_ctor_set(x_17, 0, x_14); -x_21 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9(x_1, x_17, x_3, x_4, x_5, x_6, x_7, x_8, x_20); -lean_dec(x_7); -return x_21; -} -else +lean_object* x_11; lean_object* x_12; uint8_t x_13; +lean_inc(x_3); +x_11 = l_Lean_Syntax_getKind(x_3); +x_12 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___closed__2; +x_13 = lean_name_eq(x_11, x_12); +lean_dec(x_11); +if (x_13 == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -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(0, 2, 0); -lean_ctor_set(x_24, 0, x_14); -lean_ctor_set(x_24, 1, x_22); -x_25 = l_Lean_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__9(x_1, x_24, x_3, x_4, x_5, x_6, x_7, x_8, x_23); -lean_dec(x_7); -return x_25; -} +lean_object* x_14; lean_object* x_15; +x_14 = lean_box(0); +x_15 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___lambda__1(x_3, x_2, x_1, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_15; } else { -lean_object* x_26; lean_object* x_27; -lean_dec(x_7); +lean_object* x_16; lean_object* x_17; +lean_dec(x_8); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -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_9); -return x_27; +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_10); +return x_17; } } } @@ -43709,7 +43709,7 @@ uint8_t x_20; x_20 = !lean_is_exclusive(x_4); 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; size_t x_32; size_t x_33; +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; size_t x_34; size_t x_35; x_21 = lean_ctor_get(x_4, 2); lean_dec(x_21); x_22 = lean_ctor_get(x_4, 1); @@ -43727,51 +43727,61 @@ lean_dec(x_24); x_28 = lean_ctor_get(x_27, 1); lean_inc(x_28); lean_dec(x_27); -x_29 = lean_ctor_get(x_14, 0); +x_29 = lean_ctor_get(x_14, 2); lean_inc(x_29); +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +lean_dec(x_29); +x_31 = lean_ctor_get(x_14, 0); +lean_inc(x_31); lean_dec(x_14); lean_inc(x_9); -x_30 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7(x_28, x_29, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -x_31 = lean_ctor_get(x_30, 1); -lean_inc(x_31); -lean_dec(x_30); -x_32 = 1; -x_33 = lean_usize_add(x_3, x_32); -x_3 = x_33; -x_11 = x_31; +x_32 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7(x_28, x_30, x_31, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); +x_34 = 1; +x_35 = lean_usize_add(x_3, x_34); +x_3 = x_35; +x_11 = x_33; goto _start; } 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; size_t x_44; size_t x_45; +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; size_t x_48; size_t x_49; lean_dec(x_4); -x_35 = lean_array_fget(x_15, x_16); -x_36 = lean_unsigned_to_nat(1u); -x_37 = lean_nat_add(x_16, x_36); +x_37 = lean_array_fget(x_15, x_16); +x_38 = lean_unsigned_to_nat(1u); +x_39 = lean_nat_add(x_16, x_38); lean_dec(x_16); -x_38 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_38, 0, x_15); -lean_ctor_set(x_38, 1, x_37); -lean_ctor_set(x_38, 2, x_17); -x_39 = lean_ctor_get(x_35, 1); -lean_inc(x_39); -lean_dec(x_35); -x_40 = lean_ctor_get(x_39, 1); -lean_inc(x_40); -lean_dec(x_39); -x_41 = lean_ctor_get(x_14, 0); +x_40 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_40, 0, x_15); +lean_ctor_set(x_40, 1, x_39); +lean_ctor_set(x_40, 2, x_17); +x_41 = lean_ctor_get(x_37, 1); lean_inc(x_41); +lean_dec(x_37); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +x_43 = lean_ctor_get(x_14, 2); +lean_inc(x_43); +x_44 = lean_ctor_get(x_43, 0); +lean_inc(x_44); +lean_dec(x_43); +x_45 = lean_ctor_get(x_14, 0); +lean_inc(x_45); lean_dec(x_14); lean_inc(x_9); -x_42 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7(x_40, x_41, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -x_43 = lean_ctor_get(x_42, 1); -lean_inc(x_43); -lean_dec(x_42); -x_44 = 1; -x_45 = lean_usize_add(x_3, x_44); -x_3 = x_45; -x_4 = x_38; -x_11 = x_43; +x_46 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7(x_42, x_44, x_45, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_47 = lean_ctor_get(x_46, 1); +lean_inc(x_47); +lean_dec(x_46); +x_48 = 1; +x_49 = lean_usize_add(x_3, x_48); +x_3 = x_49; +x_4 = x_40; +x_11 = x_47; goto _start; } } @@ -44516,7 +44526,7 @@ if (x_33 == 0) { lean_object* x_36; uint8_t x_37; lean_dec(x_31); -x_36 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___closed__1; +x_36 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___closed__1; x_37 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_30, x_36); lean_dec(x_30); if (x_37 == 0) @@ -44546,7 +44556,7 @@ x_41 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_elabMutualDef_go___spec__5(x_1 if (x_41 == 0) { lean_object* x_42; uint8_t x_43; -x_42 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___closed__1; +x_42 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___closed__1; x_43 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_30, x_42); lean_dec(x_30); if (x_43 == 0) @@ -45293,11 +45303,11 @@ lean_dec(x_4); return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Term_elabMutualDef_go___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_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Term_elabMutualDef_go___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) { _start: { lean_object* x_9; -x_9 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Term_elabMutualDef_go___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Term_elabMutualDef_go___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); @@ -45321,17 +45331,31 @@ lean_dec(x_3); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___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, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___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_10; -x_10 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_object* x_12; +x_12 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__7___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_5); lean_dec(x_4); -lean_dec(x_3); -return x_10; +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___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, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Term_elabMutualDef_go___spec__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_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_11; } } LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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_object* x_11) { @@ -48733,142 +48757,147 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(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) { _start: { -uint8_t x_10; uint8_t x_11; -x_10 = l_Lean_Syntax_isNone(x_1); -x_11 = l_Lean_Syntax_isNone(x_2); -if (x_10 == 0) -{ +uint8_t x_11; uint8_t x_12; +x_11 = l_Lean_Syntax_isNone(x_1); +x_12 = l_Lean_Syntax_isNone(x_2); if (x_11 == 0) { -uint8_t x_12; lean_object* x_13; lean_object* x_14; -x_12 = 1; -x_13 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_13, 0, x_3); -lean_ctor_set(x_13, 1, x_6); -lean_ctor_set_uint8(x_13, sizeof(void*)*2, x_4); -lean_ctor_set_uint8(x_13, sizeof(void*)*2 + 1, x_12); -lean_ctor_set_uint8(x_13, sizeof(void*)*2 + 2, x_5); -lean_ctor_set_uint8(x_13, sizeof(void*)*2 + 3, 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_9); -return x_14; +if (x_12 == 0) +{ +uint8_t x_13; lean_object* x_14; lean_object* x_15; +x_13 = 1; +x_14 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_14, 0, x_3); +lean_ctor_set(x_14, 1, x_4); +lean_ctor_set(x_14, 2, x_7); +lean_ctor_set_uint8(x_14, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 1, x_13); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_14, sizeof(void*)*3 + 3, 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_10); +return x_15; } else { -uint8_t x_15; uint8_t x_16; lean_object* x_17; lean_object* x_18; -x_15 = 1; -x_16 = 0; -x_17 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_17, 0, x_3); -lean_ctor_set(x_17, 1, x_6); -lean_ctor_set_uint8(x_17, sizeof(void*)*2, x_4); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 1, x_15); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 2, x_5); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 3, 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_9); -return x_18; +uint8_t x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; +x_16 = 1; +x_17 = 0; +x_18 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_18, 0, x_3); +lean_ctor_set(x_18, 1, x_4); +lean_ctor_set(x_18, 2, x_7); +lean_ctor_set_uint8(x_18, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 1, x_16); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 3, 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_10); +return x_19; } } else { -if (x_11 == 0) +if (x_12 == 0) { -uint8_t x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; -x_19 = 0; -x_20 = 1; -x_21 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_21, 0, x_3); -lean_ctor_set(x_21, 1, x_6); -lean_ctor_set_uint8(x_21, sizeof(void*)*2, x_4); -lean_ctor_set_uint8(x_21, sizeof(void*)*2 + 1, x_19); -lean_ctor_set_uint8(x_21, sizeof(void*)*2 + 2, x_5); -lean_ctor_set_uint8(x_21, sizeof(void*)*2 + 3, 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_9); -return x_22; +uint8_t x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; +x_20 = 0; +x_21 = 1; +x_22 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_22, 0, x_3); +lean_ctor_set(x_22, 1, x_4); +lean_ctor_set(x_22, 2, x_7); +lean_ctor_set_uint8(x_22, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 1, x_20); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 3, 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_10); +return x_23; } else { -uint8_t x_23; lean_object* x_24; lean_object* x_25; -x_23 = 0; -x_24 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_24, 0, x_3); -lean_ctor_set(x_24, 1, x_6); -lean_ctor_set_uint8(x_24, sizeof(void*)*2, x_4); -lean_ctor_set_uint8(x_24, sizeof(void*)*2 + 1, x_23); -lean_ctor_set_uint8(x_24, sizeof(void*)*2 + 2, x_5); -lean_ctor_set_uint8(x_24, sizeof(void*)*2 + 3, 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_9); -return x_25; +uint8_t x_24; lean_object* x_25; lean_object* x_26; +x_24 = 0; +x_25 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_25, 0, x_3); +lean_ctor_set(x_25, 1, x_4); +lean_ctor_set(x_25, 2, x_7); +lean_ctor_set_uint8(x_25, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_25, sizeof(void*)*3 + 1, x_24); +lean_ctor_set_uint8(x_25, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_25, sizeof(void*)*3 + 3, 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_10); +return x_26; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(lean_object* x_1, lean_object* x_2, 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, lean_object* x_10) { _start: { -lean_object* x_10; -x_10 = l_Lean_Syntax_getOptional_x3f(x_5); -if (lean_obj_tag(x_10) == 0) +lean_object* x_11; +x_11 = l_Lean_Syntax_getOptional_x3f(x_6); +if (lean_obj_tag(x_11) == 0) { -lean_object* x_11; lean_object* x_12; -x_11 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; -x_12 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(x_1, x_2, x_3, x_6, x_4, x_11, x_7, x_8, x_9); -lean_dec(x_7); -return x_12; +lean_object* x_12; lean_object* x_13; +x_12 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___closed__1; +x_13 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_7, x_5, x_12, x_8, x_9, x_10); +lean_dec(x_8); +return x_13; } 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); -lean_inc(x_7); -x_14 = l_Lean_Elab_elabDeclAttrs___at_Lean_Elab_Command_elabMutualDef___spec__2(x_13, x_7, x_8, x_9); -lean_dec(x_13); -if (lean_obj_tag(x_14) == 0) +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_11, 0); +lean_inc(x_14); +lean_dec(x_11); +lean_inc(x_8); +x_15 = l_Lean_Elab_elabDeclAttrs___at_Lean_Elab_Command_elabMutualDef___spec__2(x_14, x_8, x_9, x_10); +lean_dec(x_14); +if (lean_obj_tag(x_15) == 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; lean_object* x_18; +x_16 = lean_ctor_get(x_15, 0); lean_inc(x_16); -lean_dec(x_14); -x_17 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(x_1, x_2, x_3, x_6, x_4, x_15, x_7, x_8, x_16); -lean_dec(x_7); -return x_17; +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +x_18 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_7, x_5, x_16, x_8, x_9, x_17); +lean_dec(x_8); +return x_18; } else { -uint8_t x_18; -lean_dec(x_7); +uint8_t x_19; +lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); -x_18 = !lean_is_exclusive(x_14); -if (x_18 == 0) +x_19 = !lean_is_exclusive(x_15); +if (x_19 == 0) { -return x_14; +return x_15; } 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_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_15, 0); +x_21 = lean_ctor_get(x_15, 1); +lean_inc(x_21); 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; +lean_dec(x_15); +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; } } } @@ -48931,77 +48960,78 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___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_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___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) { _start: { -lean_object* x_10; -x_10 = l_Lean_Syntax_getOptional_x3f(x_5); -if (lean_obj_tag(x_10) == 0) +lean_object* x_11; +x_11 = l_Lean_Syntax_getOptional_x3f(x_6); +if (lean_obj_tag(x_11) == 0) { -uint8_t x_11; lean_object* x_12; -x_11 = 0; -x_12 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(x_1, x_2, x_6, x_3, x_4, x_11, x_7, x_8, x_9); -return x_12; +uint8_t x_12; lean_object* x_13; +x_12 = 0; +x_13 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(x_1, x_2, x_3, x_7, x_4, x_5, x_12, x_8, x_9, x_10); +return x_13; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_13 = lean_ctor_get(x_10, 0); -lean_inc(x_13); -lean_dec(x_10); -lean_inc(x_13); -x_14 = l_Lean_Syntax_getKind(x_13); -x_15 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__2; -x_16 = lean_name_eq(x_14, x_15); -if (x_16 == 0) +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_14 = lean_ctor_get(x_11, 0); +lean_inc(x_14); +lean_dec(x_11); +lean_inc(x_14); +x_15 = l_Lean_Syntax_getKind(x_14); +x_16 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__2; +x_17 = lean_name_eq(x_15, x_16); +if (x_17 == 0) { -lean_object* x_17; uint8_t x_18; -x_17 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__4; -x_18 = lean_name_eq(x_14, x_17); -lean_dec(x_14); -if (x_18 == 0) +lean_object* x_18; uint8_t x_19; +x_18 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__4; +x_19 = lean_name_eq(x_15, x_18); +lean_dec(x_15); +if (x_19 == 0) { -lean_object* x_19; lean_object* x_20; uint8_t x_21; -lean_dec(x_6); -x_19 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__6; -x_20 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualDef___spec__7(x_13, x_19, x_7, x_8, x_9); -lean_dec(x_13); -x_21 = !lean_is_exclusive(x_20); -if (x_21 == 0) +lean_object* x_20; lean_object* x_21; uint8_t x_22; +lean_dec(x_7); +lean_dec(x_3); +x_20 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__6; +x_21 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualDef___spec__7(x_14, x_20, x_8, x_9, x_10); +lean_dec(x_14); +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) { -return x_20; +return x_21; } 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_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_24); lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_20); -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_dec(x_21); +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_25; lean_object* x_26; -lean_dec(x_13); -x_25 = 1; -x_26 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(x_1, x_2, x_6, x_3, x_4, x_25, x_7, x_8, x_9); -return x_26; +uint8_t x_26; lean_object* x_27; +lean_dec(x_14); +x_26 = 1; +x_27 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(x_1, x_2, x_3, x_7, x_4, x_5, x_26, x_8, x_9, x_10); +return x_27; } } else { -uint8_t x_27; lean_object* x_28; +uint8_t x_28; lean_object* x_29; +lean_dec(x_15); lean_dec(x_14); -lean_dec(x_13); -x_27 = 2; -x_28 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(x_1, x_2, x_6, x_3, x_4, x_27, x_7, x_8, x_9); -return x_28; +x_28 = 2; +x_29 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(x_1, x_2, x_3, x_7, x_4, x_5, x_28, x_8, x_9, x_10); +return x_29; } } } @@ -49083,7 +49113,7 @@ if (lean_obj_tag(x_18) == 0) { lean_object* x_20; lean_object* x_21; x_20 = lean_box(0); -x_21 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(x_12, x_14, x_19, x_8, x_10, x_20, x_2, x_3, x_4); +x_21 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(x_12, x_14, x_1, x_19, x_8, x_10, x_20, x_2, x_3, x_4); lean_dec(x_10); lean_dec(x_8); lean_dec(x_14); @@ -49110,7 +49140,7 @@ x_26 = lean_ctor_get(x_24, 1); lean_inc(x_26); lean_dec(x_24); lean_ctor_set(x_18, 0, x_25); -x_27 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(x_12, x_14, x_19, x_8, x_10, x_18, x_2, x_3, x_26); +x_27 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(x_12, x_14, x_1, x_19, x_8, x_10, x_18, x_2, x_3, x_26); lean_dec(x_10); lean_dec(x_8); lean_dec(x_14); @@ -49126,6 +49156,7 @@ lean_dec(x_12); lean_dec(x_10); lean_dec(x_8); lean_dec(x_2); +lean_dec(x_1); x_28 = !lean_is_exclusive(x_24); if (x_28 == 0) { @@ -49165,7 +49196,7 @@ lean_inc(x_35); lean_dec(x_33); x_36 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_36, 0, x_34); -x_37 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(x_12, x_14, x_19, x_8, x_10, x_36, x_2, x_3, x_35); +x_37 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(x_12, x_14, x_1, x_19, x_8, x_10, x_36, x_2, x_3, x_35); lean_dec(x_10); lean_dec(x_8); lean_dec(x_14); @@ -49180,6 +49211,7 @@ lean_dec(x_12); lean_dec(x_10); lean_dec(x_8); 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); @@ -49750,6 +49782,7 @@ lean_ctor_set(x_25, 1, x_43); x_44 = lean_array_fget(x_1, x_10); x_45 = l_Lean_Syntax_getArg(x_44, x_18); lean_inc(x_13); +lean_inc(x_45); x_46 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_45, x_13, x_14, x_15); if (lean_obj_tag(x_46) == 0) { @@ -50047,6 +50080,7 @@ lean_ctor_set(x_99, 2, x_35); x_100 = lean_array_fget(x_1, x_10); x_101 = l_Lean_Syntax_getArg(x_100, x_18); lean_inc(x_13); +lean_inc(x_101); x_102 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_101, x_13, x_14, x_15); if (lean_obj_tag(x_102) == 0) { @@ -50393,6 +50427,7 @@ lean_ctor_set(x_160, 2, x_153); x_161 = lean_array_fget(x_1, x_10); x_162 = l_Lean_Syntax_getArg(x_161, x_18); lean_inc(x_13); +lean_inc(x_162); x_163 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_162, x_13, x_14, x_15); if (lean_obj_tag(x_163) == 0) { @@ -50756,6 +50791,7 @@ lean_ctor_set(x_224, 2, x_216); x_225 = lean_array_fget(x_1, x_10); x_226 = l_Lean_Syntax_getArg(x_225, x_18); lean_inc(x_13); +lean_inc(x_226); x_227 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_226, x_13, x_14, x_15); if (lean_obj_tag(x_227) == 0) { @@ -51135,6 +51171,7 @@ lean_ctor_set(x_291, 2, x_282); x_292 = lean_array_fget(x_1, x_10); x_293 = l_Lean_Syntax_getArg(x_292, x_18); lean_inc(x_13); +lean_inc(x_293); x_294 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_293, x_13, x_14, x_15); if (lean_obj_tag(x_294) == 0) { @@ -51434,48 +51471,55 @@ return x_341; } } } -LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabMutualDef___spec__10(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabMutualDef___spec__10___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; uint8_t x_4; -lean_inc(x_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); -x_4 = !lean_is_exclusive(x_2); -if (x_4 == 0) +uint8_t x_3; +x_3 = !lean_is_exclusive(x_1); +if (x_3 == 0) { -lean_object* x_5; size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; -x_5 = lean_ctor_get(x_2, 1); -x_6 = lean_array_size(x_5); -x_7 = 0; -x_8 = l_Array_mapMUnsafe_map___at_Lean_Elab_instToSnapshotTreeDefsParsedSnapshot___spec__1(x_6, x_7, x_5); -lean_ctor_set(x_2, 1, x_8); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_3); -lean_ctor_set(x_9, 1, x_2); -return x_9; +lean_object* x_4; size_t x_5; size_t x_6; lean_object* x_7; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_array_size(x_4); +x_6 = 0; +x_7 = l_Array_mapMUnsafe_map___at_Lean_Elab_instToSnapshotTreeDefsParsedSnapshot___spec__1(x_5, x_6, x_4); +lean_ctor_set(x_1, 1, x_7); +return x_1; } else { -lean_object* x_10; lean_object* x_11; size_t x_12; size_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_10 = lean_ctor_get(x_2, 0); -x_11 = lean_ctor_get(x_2, 1); -lean_inc(x_11); -lean_inc(x_10); -lean_dec(x_2); -x_12 = lean_array_size(x_11); -x_13 = 0; -x_14 = l_Array_mapMUnsafe_map___at_Lean_Elab_instToSnapshotTreeDefsParsedSnapshot___spec__1(x_12, x_13, x_11); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_10); -lean_ctor_set(x_15, 1, x_14); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_3); -lean_ctor_set(x_16, 1, x_15); -return x_16; +lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; +x_8 = lean_ctor_get(x_1, 0); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +lean_inc(x_8); +lean_dec(x_1); +x_10 = lean_array_size(x_9); +x_11 = 0; +x_12 = l_Array_mapMUnsafe_map___at_Lean_Elab_instToSnapshotTreeDefsParsedSnapshot___spec__1(x_10, x_11, x_9); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_8); +lean_ctor_set(x_13, 1, x_12); +return x_13; +} } } +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabMutualDef___spec__10(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_inc(x_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); +x_4 = lean_alloc_closure((void*)(l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabMutualDef___spec__10___lambda__1___boxed), 2, 1); +lean_closure_set(x_4, 0, x_2); +x_5 = lean_mk_thunk(x_4); +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_3); +lean_ctor_set(x_6, 1, x_5); +return x_6; +} } LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMutualDef___spec__12(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: @@ -52044,51 +52088,51 @@ lean_dec(x_1); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___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_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___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) { _start: { -uint8_t x_10; uint8_t x_11; lean_object* x_12; -x_10 = lean_unbox(x_4); -lean_dec(x_4); +uint8_t x_11; uint8_t x_12; lean_object* x_13; x_11 = lean_unbox(x_5); lean_dec(x_5); -x_12 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(x_1, x_2, x_3, x_10, x_11, x_6, x_7, x_8, x_9); +x_12 = lean_unbox(x_6); +lean_dec(x_6); +x_13 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_11, x_12, x_7, x_8, x_9, x_10); +lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); lean_dec(x_2); lean_dec(x_1); -return x_12; +return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___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_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___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) { _start: { -uint8_t x_10; uint8_t x_11; lean_object* x_12; -x_10 = lean_unbox(x_4); -lean_dec(x_4); -x_11 = lean_unbox(x_6); -lean_dec(x_6); -x_12 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(x_1, x_2, x_3, x_10, x_5, x_11, x_7, x_8, x_9); -lean_dec(x_8); +uint8_t x_11; uint8_t x_12; lean_object* x_13; +x_11 = lean_unbox(x_5); lean_dec(x_5); +x_12 = lean_unbox(x_7); +lean_dec(x_7); +x_13 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_11, x_6, x_12, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_6); lean_dec(x_2); lean_dec(x_1); -return x_12; +return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___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_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___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) { _start: { -uint8_t x_10; lean_object* x_11; -x_10 = lean_unbox(x_3); -lean_dec(x_3); -x_11 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(x_1, x_2, x_10, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_5); +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_4); lean_dec(x_4); +x_12 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3(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_6); +lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); -return x_11; +return x_12; } } LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { @@ -52097,7 +52141,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMu lean_object* x_5; x_5 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_1, x_2, x_3, x_4); lean_dec(x_3); -lean_dec(x_1); return x_5; } } @@ -52143,6 +52186,15 @@ lean_dec(x_1); return x_16; } } +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabMutualDef___spec__10___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Elab_Command_elabMutualDef___spec__10___lambda__1(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMutualDef___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) { _start: { @@ -52208,7 +52260,7 @@ lean_dec(x_2); return x_9; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__1() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -52218,27 +52270,27 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__2() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__1; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__1; x_2 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__5___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__3() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__2; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__2; x_2 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_getBodyTerm_x3f___closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__4() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__4() { _start: { lean_object* x_1; @@ -52246,17 +52298,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__5() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__3; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__4; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__3; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__6() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__6() { _start: { lean_object* x_1; @@ -52264,47 +52316,47 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__7() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__5; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__6; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__5; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__8() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__7; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__7; x_2 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders_getBodyTerm_x3f___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__9() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__8; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__8; x_2 = l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__5___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__10() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__9; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__9; x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__12___lambda__2___closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__11() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__11() { _start: { lean_object* x_1; @@ -52312,33 +52364,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__12() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__10; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__11; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__10; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__11; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__13() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__12; -x_2 = lean_unsigned_to_nat(16476u); +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__12; +x_2 = lean_unsigned_to_nat(16506u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506_(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_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___closed__2; x_3 = 0; -x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__13; +x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__13; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -52821,34 +52873,38 @@ l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Ela lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__1); l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__2 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__2(); lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__2); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__3); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__4 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__4(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__4); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__5); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__6 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__6(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__6); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__7 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__7(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__7); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__8); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__9 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__9(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__9); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__10); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__11 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__11(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__11); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__12 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__12(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__12); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__13); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__14 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__14(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__14); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__2___closed__15); -l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___closed__1 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___closed__1(); -lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__5___closed__1); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__1 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__1); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__2 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__2); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__3); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__4 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__4(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__4); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__5); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__6 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__6(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__6); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__7 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__7(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__7); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__8); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__9 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__9(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__9); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__10); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__11 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__11(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__11); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__12 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__12(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__12); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__13); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__14 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__14(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__14); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__4___closed__15); +l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___closed__1 = _init_l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___closed__1(); +lean_mark_persistent(l_Lean_Core_withRestoreOrSaveFull___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__13___lambda__7___closed__1); l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__18___lambda__1___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__18___lambda__1___closed__1(); lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__18___lambda__1___closed__1); l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__18___lambda__1___closed__2 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues___spec__18___lambda__1___closed__2(); @@ -52908,6 +52964,8 @@ l_Nat_foldM_loop___at_Lean_Elab_Term_MutualClosure_pushMain___spec__1___closed__ lean_mark_persistent(l_Nat_foldM_loop___at_Lean_Elab_Term_MutualClosure_pushMain___spec__1___closed__3); l_Nat_foldM_loop___at_Lean_Elab_Term_MutualClosure_pushMain___spec__1___closed__4 = _init_l_Nat_foldM_loop___at_Lean_Elab_Term_MutualClosure_pushMain___spec__1___closed__4(); lean_mark_persistent(l_Nat_foldM_loop___at_Lean_Elab_Term_MutualClosure_pushMain___spec__1___closed__4); +l_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___closed__1 = _init_l_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___closed__1(); +lean_mark_persistent(l_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___closed__1); l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_processDeriving___spec__1___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_processDeriving___spec__1___closed__1(); lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_processDeriving___spec__1___closed__1); l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_processDeriving___spec__1___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_processDeriving___spec__1___closed__2(); @@ -52994,33 +53052,33 @@ l_Lean_Elab_Command_elabMutualDef___lambda__3___closed__4 = _init_l_Lean_Elab_Co lean_mark_persistent(l_Lean_Elab_Command_elabMutualDef___lambda__3___closed__4); l_Lean_Elab_Command_elabMutualDef___lambda__3___closed__5 = _init_l_Lean_Elab_Command_elabMutualDef___lambda__3___closed__5(); lean_mark_persistent(l_Lean_Elab_Command_elabMutualDef___lambda__3___closed__5); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__1); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__2); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__3(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__3); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__4(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__4); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__5(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__5); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__6(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__6); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__7 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__7(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__7); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__8 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__8(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__8); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__9 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__9(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__9); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__10 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__10(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__10); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__11 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__11(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__11); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__12 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__12(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__12); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__13 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__13(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476____closed__13); -if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16476_(lean_io_mk_world()); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__1); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__2); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__3); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__4(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__4); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__5(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__5); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__6(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__6); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__7 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__7(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__7); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__8 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__8(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__8); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__9 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__9(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__9); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__10 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__10(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__10); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__11 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__11(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__11); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__12 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__12(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__12); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__13 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__13(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506____closed__13); +if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_MutualDef___hyg_16506_(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/ParseImportsFast.c b/stage0/stdlib/Lean/Elab/ParseImportsFast.c index c8420f76784d..4d9535dc6060 100644 --- a/stage0/stdlib/Lean/Elab/ParseImportsFast.c +++ b/stage0/stdlib/Lean/Elab/ParseImportsFast.c @@ -35,6 +35,7 @@ static lean_object* l_Lean_ParseImports_instInhabitedState___closed__1; LEAN_EXPORT lean_object* l_Lean_ParseImports_moduleIdent_parse(uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParseImports_isIdRestFast___boxed(lean_object*); extern uint32_t l_Lean_idBeginEscape; +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParseImports_keywordCore_go___at_Lean_ParseImports_main___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParseImports_many___at_Lean_ParseImports_main___spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParseImports_keywordCore_go___at_Lean_ParseImports_preludeOpt___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -83,7 +84,6 @@ LEAN_EXPORT lean_object* l_Lean_ParseImports_many(lean_object*, lean_object*, le LEAN_EXPORT lean_object* l_Lean_ParseImports_keyword(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParseImports_State_mkEOIError___closed__2; LEAN_EXPORT lean_object* l_Lean_ParseImports_State_mkEOIError(lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); lean_object* l_IO_FS_readFile(lean_object*, lean_object*); uint8_t l_Lean_isLetterLike(uint32_t); LEAN_EXPORT lean_object* l_Lean_ParseImports_moduleIdent_parse___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -4366,7 +4366,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_10); lean_ctor_set(x_17, 1, x_16); x_18 = l_Lean_parseImports_x27___closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -4550,7 +4550,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_4); lean_ctor_set(x_15, 1, x_14); x_16 = l_Lean_parseImports_x27___closed__1; -x_17 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -4641,7 +4641,7 @@ x_10 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_10, 0, x_9); lean_ctor_set(x_10, 1, x_8); x_11 = l_Lean_parseImports_x27___closed__1; -x_12 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); +x_12 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_10, x_11); x_13 = l_Lean_Json_mkObj(x_12); return x_13; } diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Basic.c b/stage0/stdlib/Lean/Elab/PreDefinition/Basic.c index 8ec45e86bfc0..aa73562eaad2 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Basic.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Basic.c @@ -324,7 +324,6 @@ LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_checkCodomainsLev LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_fixLevelParams___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_ensureNoRecFn(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___closed__1; lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_compileDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -403,20 +402,22 @@ return x_2; static lean_object* _init_l_Lean_Elab_instInhabitedPreDefinition___closed__2() { _start: { -lean_object* x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; x_1 = lean_box(0); -x_2 = 0; +x_2 = lean_box(0); x_3 = 0; x_4 = 0; -x_5 = l_Lean_Elab_instInhabitedPreDefinition___closed__1; -x_6 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -lean_ctor_set_uint8(x_6, sizeof(void*)*2, x_2); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 1, x_3); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 2, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 3, x_3); -return x_6; +x_5 = 0; +x_6 = l_Lean_Elab_instInhabitedPreDefinition___closed__1; +x_7 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_7, 0, x_2); +lean_ctor_set(x_7, 1, x_1); +lean_ctor_set(x_7, 2, x_6); +lean_ctor_set_uint8(x_7, sizeof(void*)*3, x_3); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 1, x_4); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 2, x_5); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 3, x_4); +return x_7; } } static lean_object* _init_l_Lean_Elab_instInhabitedPreDefinition___closed__3() { @@ -2919,7 +2920,7 @@ lean_inc(x_16); x_17 = lean_ctor_get(x_15, 2); lean_inc(x_17); lean_dec(x_15); -x_18 = lean_ctor_get(x_17, 1); +x_18 = lean_ctor_get(x_17, 2); lean_inc(x_18); lean_dec(x_17); lean_inc(x_11); @@ -3468,7 +3469,7 @@ lean_ctor_set(x_11, 0, x_8); lean_ctor_set(x_11, 1, x_9); lean_ctor_set(x_11, 2, x_10); x_12 = lean_ctor_get(x_1, 2); -x_13 = lean_ctor_get_uint8(x_12, sizeof(void*)*2 + 3); +x_13 = lean_ctor_get_uint8(x_12, sizeof(void*)*3 + 3); x_14 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_14, 0, x_11); lean_ctor_set_uint8(x_14, sizeof(void*)*1, x_13); @@ -3558,7 +3559,7 @@ if (x_3 == 0) { lean_object* x_4; uint8_t x_5; x_4 = lean_ctor_get(x_1, 2); -x_5 = lean_ctor_get_uint8(x_4, sizeof(void*)*2 + 1); +x_5 = lean_ctor_get_uint8(x_4, sizeof(void*)*3 + 1); if (x_5 == 0) { uint8_t x_6; @@ -7133,7 +7134,7 @@ if (lean_obj_tag(x_23) == 0) lean_object* x_24; uint8_t x_25; x_24 = lean_ctor_get(x_1, 2); lean_inc(x_24); -x_25 = lean_ctor_get_uint8(x_24, sizeof(void*)*2 + 1); +x_25 = lean_ctor_get_uint8(x_24, sizeof(void*)*3 + 1); lean_dec(x_24); if (x_25 == 0) { @@ -7523,7 +7524,7 @@ x_40 = lean_ctor_get(x_17, 5); lean_inc(x_40); x_41 = lean_ctor_get(x_17, 2); lean_inc(x_41); -x_42 = lean_ctor_get_uint8(x_41, sizeof(void*)*2 + 3); +x_42 = lean_ctor_get_uint8(x_41, sizeof(void*)*3 + 3); lean_dec(x_41); x_43 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_43, 0, x_39); @@ -7553,7 +7554,7 @@ lean_ctor_set(x_50, 1, x_48); lean_ctor_set(x_50, 2, x_49); x_51 = lean_ctor_get(x_17, 2); lean_inc(x_51); -x_52 = lean_ctor_get_uint8(x_51, sizeof(void*)*2 + 3); +x_52 = lean_ctor_get_uint8(x_51, sizeof(void*)*3 + 3); lean_dec(x_51); if (x_52 == 0) { @@ -7630,7 +7631,7 @@ x_79 = lean_alloc_ctor(2, 0, 4); lean_ctor_set_uint32(x_79, 0, x_78); x_80 = lean_ctor_get(x_17, 2); lean_inc(x_80); -x_81 = lean_ctor_get_uint8(x_80, sizeof(void*)*2 + 3); +x_81 = lean_ctor_get_uint8(x_80, sizeof(void*)*3 + 3); lean_dec(x_80); if (x_81 == 0) { @@ -7846,7 +7847,7 @@ x_134 = lean_ctor_get(x_111, 5); lean_inc(x_134); x_135 = lean_ctor_get(x_111, 2); lean_inc(x_135); -x_136 = lean_ctor_get_uint8(x_135, sizeof(void*)*2 + 3); +x_136 = lean_ctor_get_uint8(x_135, sizeof(void*)*3 + 3); lean_dec(x_135); x_137 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_137, 0, x_133); @@ -7876,7 +7877,7 @@ lean_ctor_set(x_144, 1, x_142); lean_ctor_set(x_144, 2, x_143); x_145 = lean_ctor_get(x_111, 2); lean_inc(x_145); -x_146 = lean_ctor_get_uint8(x_145, sizeof(void*)*2 + 3); +x_146 = lean_ctor_get_uint8(x_145, sizeof(void*)*3 + 3); lean_dec(x_145); if (x_146 == 0) { @@ -7953,7 +7954,7 @@ x_173 = lean_alloc_ctor(2, 0, 4); lean_ctor_set_uint32(x_173, 0, x_172); x_174 = lean_ctor_get(x_111, 2); lean_inc(x_174); -x_175 = lean_ctor_get_uint8(x_174, sizeof(void*)*2 + 3); +x_175 = lean_ctor_get_uint8(x_174, sizeof(void*)*3 + 3); lean_dec(x_174); if (x_175 == 0) { @@ -9431,25 +9432,6 @@ return x_17; } } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___closed__1() { -_start: -{ -lean_object* x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_1 = lean_box(0); -x_2 = 0; -x_3 = 0; -x_4 = 2; -x_5 = l___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_getLevelParamsPreDecls___closed__4; -x_6 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -lean_ctor_set_uint8(x_6, sizeof(void*)*2, x_2); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 1, x_3); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 2, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 3, x_3); -return x_6; -} -} LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { _start: { @@ -9485,7 +9467,7 @@ lean_closure_set(x_16, 1, x_1); x_17 = lean_replace_expr(x_16, x_12); lean_dec(x_12); lean_dec(x_16); -x_18 = l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___closed__1; +x_18 = l_Lean_Elab_instInhabitedPreDefinition___closed__2; lean_ctor_set(x_7, 5, x_17); lean_ctor_set(x_7, 3, x_15); lean_ctor_set(x_7, 2, x_18); @@ -9523,7 +9505,7 @@ lean_closure_set(x_32, 1, x_1); x_33 = lean_replace_expr(x_32, x_28); lean_dec(x_28); lean_dec(x_32); -x_34 = l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___closed__1; +x_34 = l_Lean_Elab_instInhabitedPreDefinition___closed__2; x_35 = lean_alloc_ctor(0, 7, 1); lean_ctor_set(x_35, 0, x_23); lean_ctor_set(x_35, 1, x_25); @@ -13518,8 +13500,6 @@ l_Lean_Elab_addAndCompileUnsafe___boxed__const__1 = _init_l_Lean_Elab_addAndComp lean_mark_persistent(l_Lean_Elab_addAndCompileUnsafe___boxed__const__1); l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___lambda__1___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___lambda__1___closed__1(); lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___lambda__1___closed__1); -l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___closed__1(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Elab_addAndCompilePartialRec___spec__2___closed__1); l_Lean_Elab_ensureNoRecFn___lambda__1___closed__1 = _init_l_Lean_Elab_ensureNoRecFn___lambda__1___closed__1(); lean_mark_persistent(l_Lean_Elab_ensureNoRecFn___lambda__1___closed__1); l_Lean_Elab_ensureNoRecFn___lambda__1___closed__2 = _init_l_Lean_Elab_ensureNoRecFn___lambda__1___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Main.c b/stage0/stdlib/Lean/Elab/PreDefinition/Main.c index 1718b6022d6f..8bad5ff25bbd 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Main.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Main.c @@ -12911,7 +12911,7 @@ lean_ctor_set(x_18, 1, x_16); lean_ctor_set(x_18, 2, x_17); x_19 = lean_ctor_get(x_14, 2); lean_inc(x_19); -x_20 = lean_ctor_get_uint8(x_19, sizeof(void*)*2 + 3); +x_20 = lean_ctor_get_uint8(x_19, sizeof(void*)*3 + 3); lean_dec(x_19); x_21 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_21, 0, x_18); @@ -16700,7 +16700,7 @@ x_5 = lean_array_uget(x_1, x_2); x_6 = lean_ctor_get(x_5, 2); lean_inc(x_6); lean_dec(x_5); -x_7 = lean_ctor_get_uint8(x_6, sizeof(void*)*2 + 3); +x_7 = lean_ctor_get_uint8(x_6, sizeof(void*)*3 + 3); lean_dec(x_6); if (x_7 == 0) { @@ -18613,7 +18613,7 @@ if (lean_obj_tag(x_28) == 0) lean_object* x_29; uint8_t x_30; x_29 = lean_ctor_get(x_25, 2); lean_inc(x_29); -x_30 = lean_ctor_get_uint8(x_29, sizeof(void*)*2 + 1); +x_30 = lean_ctor_get_uint8(x_29, sizeof(void*)*3 + 1); lean_dec(x_29); if (x_30 == 0) { diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/BRecOn.c b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/BRecOn.c index 57cfbf73de8f..30aa1081783f 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/BRecOn.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/BRecOn.c @@ -19,6 +19,7 @@ lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___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_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__10___boxed(lean_object*); lean_object* l_Lean_Meta_inferArgumentTypesN(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_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___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_Elab_Structural_mkBrecOnApp(lean_object*, lean_object*, 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_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__4(lean_object*); @@ -38,6 +39,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_getMatcherInfo_x3f___at___private_Lean_Elab static lean_object* l_Lean_Elab_Structural_mkBrecOnApp___lambda__2___closed__5; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Structural_mkBRecOnConst___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_mkBRecOnConst___lambda__5(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_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___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_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__27(lean_object*, lean_object*, lean_object*, lean_object*, 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_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___lambda__5___closed__4; lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); @@ -54,6 +56,7 @@ lean_object* l_Lean_Elab_Structural_IndGroupInfo_numMotives(lean_object*); uint8_t l_Lean_Exception_isInterrupt(lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___closed__7; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__39___lambda__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___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_isExprDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaBoundedTelescope___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__38___rarg(lean_object*, 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___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -62,6 +65,7 @@ lean_object* l_Lean_Elab_Structural_RecArgInfo_pickIndicesMajor(lean_object*, le static lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__3___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___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*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_inferBRecOnFTypes___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_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___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_EXPORT lean_object* l_Lean_Elab_Structural_mkBRecOnConst___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Structural_mkBRecOnF___spec__1___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_findIdx_x3f_loop___rarg(lean_object*, lean_object*, lean_object*); @@ -80,7 +84,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at___privat static lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__5___closed__1; static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___lambda__5___closed__3; uint8_t lean_usize_dec_eq(size_t, size_t); -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__2; lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__13(lean_object*); static lean_object* l_Lean_Elab_Structural_searchPProd___rarg___closed__4; @@ -88,8 +91,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Structural_inferBRecOnFTypes___lambda__1(le lean_object* l_Lean_replaceRef(lean_object*, lean_object*); uint8_t l_Array_contains___at_Lean_Elab_Structural_RecArgInfo_pickIndicesMajor___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__12(lean_object*); -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__2; -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__5; +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__35___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__40___boxed(lean_object*); lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); @@ -103,8 +105,10 @@ extern lean_object* l_Lean_casesOnSuffix; lean_object* l_Lean_Meta_Match_MatcherInfo_arity(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__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_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__3(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__4; LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__13___rarg(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_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___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_environment_find(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getMatcherInfo_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -126,6 +130,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0 LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__43(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__40___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__22___lambda__1(lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__5; lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps___spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -137,18 +142,15 @@ LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_ lean_object* l_Lean_stringToMessageData(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__31___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___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_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12(lean_object*); LEAN_EXPORT uint8_t l_Array_getIdx_x3f___at_Lean_Elab_Structural_mkBrecOnApp___spec__6___lambda__1(lean_object*, lean_object*); uint8_t l___private_Lean_Util_Trace_0__Lean_checkTraceOption(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___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_getConstInfoInduct___at_Lean_Elab_Structural_mkBRecOnConst___spec__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___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_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11___rarg(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_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__7___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__7___closed__2; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__9(size_t, size_t, lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___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*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___rarg___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___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___lambda__5___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_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*); @@ -157,7 +159,6 @@ LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structur LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__26___boxed(lean_object*); extern lean_object* l_Lean_Elab_Structural_instInhabitedRecArgInfo; static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4___closed__7; -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Structural_mkBRecOnF___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 double l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__37___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__31___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -167,14 +168,13 @@ static lean_object* l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Str LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___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_Lean_Elab_Structural_searchPProd___rarg___closed__2; extern lean_object* l_instInhabitedPUnit; -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___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*); static lean_object* l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__14___closed__1; +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___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_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__36___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_Elab_Structural_mkBRecOnMotive___spec__1___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Structural_IndGroupInst_brecOn(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_throwToBelowFailed___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__10(lean_object*, lean_object*, 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_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___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*); static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelow___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_isTypeCorrect(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -191,20 +191,18 @@ static lean_object* l_Lean_Elab_Structural_mkBrecOnApp___lambda__2___closed__9; lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_lambdaTelescopeImp___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_String_toNat_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__21___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__14___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_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__22(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, 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_withLocalDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__41(lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__33___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_mkBRecOnF___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_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__39___lambda__2___closed__4; 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_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___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_st_ref_take(lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLetDeclImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__41___rarg___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_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___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_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__1; -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___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_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___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 lean_object* l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___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*); uint8_t lean_expr_eqv(lean_object*, lean_object*); @@ -218,7 +216,7 @@ static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lea static lean_object* l_Lean_Elab_Structural_searchPProd___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__39(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*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__41___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__1; +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8(lean_object*); lean_object* l_Lean_Meta_PProdN_proj(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_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*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_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_object*); @@ -226,6 +224,7 @@ static lean_object* l_Lean_Elab_Structural_mkBrecOnApp___lambda__2___closed__7; LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__29___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_mkBRecOnConst___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___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_object*); +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___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*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_throwToBelowFailed___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_getIdx_x3f___at_Lean_Elab_Structural_mkBrecOnApp___spec__6___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__7(lean_object*); @@ -235,10 +234,12 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefi LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__28___boxed(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*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLocalDeclImp___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_getPrefix(lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__13___boxed(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_Lean_isTracingEnabledFor___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__35___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__2; lean_object* l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___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_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__23(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*, lean_object*); @@ -258,6 +259,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_mkBr LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__1(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_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__22___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__17(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___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_throwToBelowFailed___spec__1___rarg(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_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___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*); @@ -286,7 +288,9 @@ static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lea extern lean_object* l_Lean_instInhabitedExpr; LEAN_EXPORT lean_object* l_Lean_Elab_Structural_inferBRecOnFTypes(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___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_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___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_EXPORT lean_object* l_Lean_Elab_Structural_mkBRecOnConst___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__43___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___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_List_lengthTRAux___rarg(lean_object*, lean_object*); @@ -301,7 +305,6 @@ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__22___closed__2; lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_PrettyPrinter_Delaborator_returnsPi___spec__1___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_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__24(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___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_Meta_withLocalDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___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*); static lean_object* l_Lean_Elab_Structural_inferBRecOnFTypes___closed__2; LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__40___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -309,10 +312,12 @@ static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lea static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__9___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__19(lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__5___closed__2; +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__2; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__5___closed__1; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__3___closed__1; lean_object* l_Lean_Meta_PProdN_packLambdas(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +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*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__9(lean_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_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___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_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps___spec__1___boxed(lean_object*, lean_object*, lean_object*); @@ -325,24 +330,19 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinitio LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___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*, lean_object*); static lean_object* l_Lean_Elab_Structural_mkBrecOnApp___lambda__2___closed__1; extern lean_object* l_Lean_Meta_instMonadMetaM; -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__2; static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__19___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__1; LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__8(lean_object*); static lean_object* l_Lean_Elab_Structural_searchPProd___rarg___closed__5; LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__22___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_Elab_Structural_mkBrecOnApp___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___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*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_forallTelescopeCompatibleAux___spec__15___rarg(lean_object*, uint8_t, 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_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__37___rarg___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_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___closed__6; -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__2; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__39___lambda__3___closed__4; lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__11___boxed(lean_object*); -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__3; extern lean_object* l_Lean_inheritedTraceOptions; static lean_object* l_Lean_Elab_Structural_mkBrecOnApp___lambda__2___closed__8; lean_object* l_Lean_MessageData_ofExpr(lean_object*); @@ -352,9 +352,9 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefi LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___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_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__7___closed__3; LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Structural_mkBrecOnApp___spec__4(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___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*); double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__26(lean_object*); -static lean_object* l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; lean_object* l_Array_extract___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__39___lambda__2___closed__1; LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__9___boxed(lean_object*); @@ -365,17 +365,16 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Structural_mkBRecOnMotive___lambda__1(lean_ static lean_object* l_Lean_Elab_Structural_mkBrecOnApp___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__33___rarg(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_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__21___rarg(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_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___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_addTrace___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__37___rarg(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_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__39___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_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__14___closed__2; lean_object* l_Lean_Expr_replaceFVars(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__3___closed__2; -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__34___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_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelow(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_zetaReduce___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Structural_inferBRecOnFTypes___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_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___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*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4___closed__2; @@ -391,7 +390,6 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinitio LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__6(lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_Elab_Structural_mkBRecOnMotive___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_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_inferBRecOnFTypes___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_getConstInfo___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__3___closed__1; LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -419,12 +417,11 @@ static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lea 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_Meta_withLocalDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__42(lean_object*, lean_object*); lean_object* l_Lean_Meta_MatcherApp_toExpr(lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__32(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* l_Lean_Meta_zetaReduce___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___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_EXPORT lean_object* l_Lean_Meta_lambdaBoundedTelescope___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___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_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11___rarg___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_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___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* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___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*, lean_object*); @@ -435,6 +432,7 @@ static lean_object* l_Lean_Elab_Structural_mkBrecOnApp___lambda__2___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___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_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__27___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*); static lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__7___rarg___closed__3; +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__2; static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4___closed__8; LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Structural_mkBRecOnConst___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__37(lean_object*); @@ -454,23 +452,18 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0 LEAN_EXPORT lean_object* l_Lean_Elab_Structural_searchPProd___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___lambda__1___boxed(lean_object**); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___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_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__2; LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__8___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___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_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__16___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); -static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__4; static lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__7___rarg___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___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_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__26___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_ensureNoRecFn(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_throwToBelowFailed___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedName; -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___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*, 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_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__9___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4(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_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_throwToBelowFailed___rarg___closed__1; @@ -486,8 +479,8 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Structural_searchPProd(lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAux___rarg(lean_object*, lean_object*, lean_object*, uint8_t, 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*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_Elab_Structural_mkBRecOnMotive___spec__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___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_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___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_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___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_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__7___boxed(lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Structural_mkBRecOnConst___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -513,7 +506,6 @@ lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint LEAN_EXPORT lean_object* l_Lean_Meta_getMatcherInfo_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux(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_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__16(lean_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_getIdx_x3f___at_Lean_Elab_Structural_mkBrecOnApp___spec__6___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___closed__3; @@ -521,14 +513,13 @@ uint8_t l_Lean_Exception_isRuntime(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_inferBRecOnFTypes___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_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___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_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__18(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*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___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_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__39___lambda__3___boxed(lean_object**); static lean_object* l_Lean_Elab_Structural_mkBrecOnApp___lambda__2___closed__11; -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_panic___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__7___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__19___boxed(lean_object*); lean_object* l_Lean_InductiveVal_numCtors(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaBoundedTelescope___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__38___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__3; static lean_object* l_Lean_Elab_Structural_mkBRecOnF___lambda__2___closed__1; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___closed__5; @@ -539,7 +530,7 @@ lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(lean_ LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__43___rarg(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_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4___closed__9; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__39___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_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__2; lean_object* l_ReaderT_instMonad___rarg(lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4___closed__4; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__33___boxed(lean_object*); @@ -2805,218 +2796,7 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__9(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; size_t x_8; size_t x_9; uint8_t x_10; -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 = 1; -x_9 = lean_usize_add(x_2, x_8); -x_10 = !lean_is_exclusive(x_5); -if (x_10 == 0) -{ -lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = lean_ctor_get(x_5, 0); -x_12 = 0; -x_13 = lean_box(x_12); -lean_ctor_set(x_5, 0, x_13); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_11); -lean_ctor_set(x_14, 1, x_5); -x_15 = lean_array_uset(x_7, x_2, x_14); -x_2 = x_9; -x_3 = x_15; -goto _start; -} -else -{ -lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_17 = lean_ctor_get(x_5, 0); -x_18 = lean_ctor_get(x_5, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_5); -x_19 = 0; -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_18); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_17); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_array_uset(x_7, x_2, x_22); -x_2 = x_9; -x_3 = x_23; -goto _start; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11___rarg___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_array_push(x_1, x_5); -x_12 = l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11___rarg(x_2, x_3, x_4, x_11, x_6, x_7, x_8, x_9, x_10); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11___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; uint8_t x_12; -x_10 = lean_array_get_size(x_4); -x_11 = lean_array_get_size(x_1); -x_12 = lean_nat_dec_lt(x_10, x_11); -lean_dec(x_11); -if (x_12 == 0) -{ -lean_object* x_13; -lean_dec(x_10); -lean_dec(x_3); -lean_dec(x_1); -x_13 = lean_apply_6(x_2, x_4, x_5, x_6, x_7, x_8, x_9); -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; -x_14 = lean_array_fget(x_1, x_10); -lean_dec(x_10); -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 0); -lean_inc(x_16); -lean_dec(x_14); -x_17 = lean_ctor_get(x_15, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_dec(x_15); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_19 = lean_apply_6(x_18, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; uint8_t 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 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11___rarg___lambda__1), 10, 4); -lean_closure_set(x_22, 0, x_4); -lean_closure_set(x_22, 1, x_1); -lean_closure_set(x_22, 2, x_2); -lean_closure_set(x_22, 3, x_3); -x_23 = 0; -x_24 = lean_unbox(x_17); -lean_dec(x_17); -x_25 = l_Lean_Meta_withLocalDecl___at_Lean_Meta_forallTelescopeCompatibleAux___spec__15___rarg(x_16, x_24, x_20, x_22, x_23, x_5, x_6, x_7, x_8, x_21); -return x_25; -} -else -{ -uint8_t x_26; -lean_dec(x_17); -lean_dec(x_16); -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_19); -if (x_26 == 0) -{ -return x_19; -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_19, 0); -x_28 = lean_ctor_get(x_19, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_19); -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_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11___rarg), 9, 0); -return x_2; -} -} -static lean_object* _init_l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___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_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___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 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; -x_10 = l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__11___rarg(x_2, x_3, x_1, x_9, x_4, x_5, x_6, x_7, x_8); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg), 8, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___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: -{ -size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_array_size(x_2); -x_10 = 0; -x_11 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__9(x_9, x_10, x_2); -x_12 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDeclsD___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg), 8, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___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_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___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; @@ -3024,7 +2804,7 @@ x_10 = lean_apply_7(x_1, x_2, x_3, x_5, x_6, x_7, x_8, x_9); return x_10; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__1() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__1() { _start: { lean_object* x_1; @@ -3032,16 +2812,16 @@ x_1 = lean_mk_string_unchecked("not type correct!", 17, 17); return x_1; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__2() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__1; +x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___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_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___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; @@ -3086,7 +2866,7 @@ lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean x_20 = lean_ctor_get(x_15, 1); lean_inc(x_20); lean_dec(x_15); -x_21 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__2; +x_21 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__2; x_22 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(x_4, x_21, x_6, x_7, x_8, x_9, x_20); x_23 = lean_ctor_get(x_22, 1); lean_inc(x_23); @@ -3138,7 +2918,7 @@ return x_30; } } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__1() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__1() { _start: { lean_object* x_1; @@ -3146,7 +2926,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Meta_PProdN_packLambdas), 7, 0); return x_1; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__2() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__2() { _start: { lean_object* x_1; @@ -3154,16 +2934,16 @@ x_1 = lean_mk_string_unchecked("initial belowDict for ", 22, 22); return x_1; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__3() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__2; +x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__2; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__4() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__4() { _start: { lean_object* x_1; @@ -3171,21 +2951,21 @@ x_1 = lean_mk_string_unchecked(":", 1, 1); return x_1; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__5() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__4; +x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__4; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___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_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___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; x_13 = l_Lean_instInhabitedExpr; -x_14 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__1; +x_14 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__1; lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -3217,7 +2997,7 @@ x_24 = lean_ctor_get(x_21, 1); lean_inc(x_24); lean_dec(x_21); x_25 = lean_box(0); -x_26 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2(x_20, x_6, x_7, x_5, x_25, x_8, x_9, x_10, x_11, x_24); +x_26 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2(x_20, x_6, x_7, x_5, x_25, x_8, x_9, x_10, x_11, x_24); return x_26; } else @@ -3235,11 +3015,11 @@ x_30 = lean_array_to_list(x_7); x_31 = lean_box(0); x_32 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_30, x_31); x_33 = l_Lean_MessageData_ofList(x_32); -x_34 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__3; +x_34 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__3; lean_ctor_set_tag(x_21, 7); lean_ctor_set(x_21, 1, x_33); lean_ctor_set(x_21, 0, x_34); -x_35 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__5; +x_35 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__5; x_36 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_36, 0, x_21); lean_ctor_set(x_36, 1, x_35); @@ -3259,7 +3039,7 @@ lean_inc(x_42); x_43 = lean_ctor_get(x_41, 1); lean_inc(x_43); lean_dec(x_41); -x_44 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2(x_20, x_6, x_7, x_5, x_42, x_8, x_9, x_10, x_11, x_43); +x_44 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2(x_20, x_6, x_7, x_5, x_42, x_8, x_9, x_10, x_11, x_43); lean_dec(x_42); return x_44; } @@ -3274,11 +3054,11 @@ x_46 = lean_array_to_list(x_7); x_47 = lean_box(0); x_48 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_46, x_47); x_49 = l_Lean_MessageData_ofList(x_48); -x_50 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__3; +x_50 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__3; 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_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__5; +x_52 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__5; x_53 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_53, 0, x_51); lean_ctor_set(x_53, 1, x_52); @@ -3298,7 +3078,7 @@ lean_inc(x_59); x_60 = lean_ctor_get(x_58, 1); lean_inc(x_60); lean_dec(x_58); -x_61 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2(x_20, x_6, x_7, x_5, x_59, x_8, x_9, x_10, x_11, x_60); +x_61 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2(x_20, x_6, x_7, x_5, x_59, x_8, x_9, x_10, x_11, x_60); lean_dec(x_59); return x_61; } @@ -3336,7 +3116,7 @@ return x_65; } } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__1() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -3345,20 +3125,20 @@ x_2 = l_Lean_Level_ofNat(x_1); return x_2; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__2() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__1; +x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__1; x_2 = l_Lean_Expr_sort___override(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___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, lean_object* x_7, lean_object* x_8, lean_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___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___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, lean_object* x_7, lean_object* x_8, 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; size_t x_21; size_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; size_t x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_15 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__2; +x_15 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__2; x_16 = lean_mk_array(x_1, x_15); x_17 = lean_array_get_size(x_2); x_18 = lean_unsigned_to_nat(0u); @@ -3385,18 +3165,18 @@ lean_inc(x_29); x_30 = lean_ctor_get(x_28, 1); lean_inc(x_30); lean_dec(x_28); -x_31 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___boxed), 12, 6); +x_31 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___boxed), 12, 6); lean_closure_set(x_31, 0, x_3); lean_closure_set(x_31, 1, x_2); lean_closure_set(x_31, 2, x_4); lean_closure_set(x_31, 3, x_5); lean_closure_set(x_31, 4, x_6); lean_closure_set(x_31, 5, x_7); -x_32 = l_Lean_Meta_withLocalDeclsD___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg(x_8, x_29, x_31, x_10, x_11, x_12, x_13, x_30); +x_32 = l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(x_8, x_29, x_31, x_10, x_11, x_12, x_13, x_30); return x_32; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__1() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__1() { _start: { lean_object* x_1; @@ -3404,16 +3184,16 @@ x_1 = lean_mk_string_unchecked("numMotives: ", 12, 12); return x_1; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__2() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__1; +x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___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, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___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, 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; lean_object* x_21; lean_object* x_22; @@ -3457,7 +3237,7 @@ x_29 = lean_ctor_get(x_26, 1); lean_inc(x_29); lean_dec(x_26); x_30 = lean_box(0); -x_31 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4(x_25, x_23, x_5, x_21, x_19, x_6, x_7, x_8, x_30, x_10, x_11, x_12, x_13, x_29); +x_31 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4(x_25, x_23, x_5, x_21, x_19, x_6, x_7, x_8, x_30, x_10, x_11, x_12, x_13, x_29); return x_31; } else @@ -3475,7 +3255,7 @@ x_35 = l___private_Init_Data_Repr_0__Nat_reprFast(x_25); 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_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__2; +x_38 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__2; lean_ctor_set_tag(x_26, 7); lean_ctor_set(x_26, 1, x_37); lean_ctor_set(x_26, 0, x_38); @@ -3490,7 +3270,7 @@ lean_inc(x_42); x_43 = lean_ctor_get(x_41, 1); lean_inc(x_43); lean_dec(x_41); -x_44 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4(x_25, x_23, x_5, x_21, x_19, x_6, x_7, x_8, x_42, x_10, x_11, x_12, x_13, x_43); +x_44 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4(x_25, x_23, x_5, x_21, x_19, x_6, x_7, x_8, x_42, x_10, x_11, x_12, x_13, x_43); lean_dec(x_42); return x_44; } @@ -3505,7 +3285,7 @@ x_46 = l___private_Init_Data_Repr_0__Nat_reprFast(x_25); 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 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__2; +x_49 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__2; x_50 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_50, 0, x_49); lean_ctor_set(x_50, 1, x_48); @@ -3520,7 +3300,7 @@ lean_inc(x_54); x_55 = lean_ctor_get(x_53, 1); lean_inc(x_55); lean_dec(x_53); -x_56 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4(x_25, x_23, x_5, x_21, x_19, x_6, x_7, x_8, x_54, x_10, x_11, x_12, x_13, x_55); +x_56 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4(x_25, x_23, x_5, x_21, x_19, x_6, x_7, x_8, x_54, x_10, x_11, x_12, x_13, x_55); lean_dec(x_54); return x_56; } @@ -3560,7 +3340,7 @@ return x_60; } } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___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_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___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) { _start: { lean_object* x_8; uint8_t x_9; @@ -3585,7 +3365,7 @@ return x_12; } } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__1() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__1() { _start: { lean_object* x_1; @@ -3593,16 +3373,16 @@ x_1 = lean_mk_string_unchecked("unexpected 'below' type", 23, 23); return x_1; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__2() { +static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__1; +x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___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, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___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, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { if (lean_obj_tag(x_8) == 5) @@ -3634,7 +3414,7 @@ lean_inc(x_8); lean_inc(x_5); lean_inc(x_2); lean_inc(x_9); -x_22 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___boxed), 14, 8); +x_22 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___boxed), 14, 8); lean_closure_set(x_22, 0, x_9); lean_closure_set(x_22, 1, x_2); lean_closure_set(x_22, 2, x_5); @@ -3673,7 +3453,7 @@ x_29 = lean_ctor_get(x_26, 1); lean_inc(x_29); lean_dec(x_26); x_30 = lean_box(0); -x_31 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__6(x_22, x_30, x_11, x_12, x_13, x_14, x_29); +x_31 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__6(x_22, x_30, x_11, x_12, x_13, x_14, x_29); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); @@ -3692,7 +3472,7 @@ x_33 = lean_ctor_get(x_26, 1); x_34 = lean_ctor_get(x_26, 0); lean_dec(x_34); x_35 = l_Lean_indentExpr(x_6); -x_36 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__2; +x_36 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__2; lean_ctor_set_tag(x_26, 7); lean_ctor_set(x_26, 1, x_35); lean_ctor_set(x_26, 0, x_36); @@ -3706,7 +3486,7 @@ lean_inc(x_40); x_41 = lean_ctor_get(x_39, 1); lean_inc(x_41); lean_dec(x_39); -x_42 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__6(x_22, x_40, x_11, x_12, x_13, x_14, x_41); +x_42 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__6(x_22, x_40, x_11, x_12, x_13, x_14, x_41); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); @@ -3722,7 +3502,7 @@ x_43 = lean_ctor_get(x_26, 1); lean_inc(x_43); lean_dec(x_26); x_44 = l_Lean_indentExpr(x_6); -x_45 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__2; +x_45 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__2; x_46 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_46, 0, x_45); lean_ctor_set(x_46, 1, x_44); @@ -3736,7 +3516,7 @@ lean_inc(x_50); x_51 = lean_ctor_get(x_49, 1); lean_inc(x_51); lean_dec(x_49); -x_52 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__6(x_22, x_50, x_11, x_12, x_13, x_14, x_51); +x_52 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__6(x_22, x_50, x_11, x_12, x_13, x_14, x_51); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); @@ -3753,17 +3533,17 @@ lean_object* x_53; lean_object* x_54; lean_dec(x_22); lean_dec(x_6); x_53 = lean_box(0); -x_54 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5(x_9, x_2, x_5, x_8, x_3, x_7, x_4, x_1, x_53, x_11, x_12, x_13, x_14, x_15); +x_54 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5(x_9, x_2, x_5, x_8, x_3, x_7, x_4, x_1, x_53, x_11, x_12, x_13, x_14, x_15); return x_54; } } } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg), 15, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg), 15, 0); return x_2; } } @@ -3780,7 +3560,7 @@ x_18 = lean_unsigned_to_nat(1u); x_19 = lean_nat_sub(x_15, x_18); lean_dec(x_15); lean_inc(x_1); -x_20 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg(x_2, x_3, x_4, x_5, x_6, x_1, x_7, x_1, x_17, x_19, x_9, x_10, x_11, x_12, x_13); +x_20 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg(x_2, x_3, x_4, x_5, x_6, x_1, x_7, x_1, x_17, x_19, x_9, x_10, x_11, x_12, x_13); return x_20; } } @@ -3828,7 +3608,7 @@ lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean x_25 = lean_ctor_get(x_19, 1); lean_inc(x_25); lean_dec(x_19); -x_26 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__2; +x_26 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__2; lean_inc(x_8); x_27 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(x_8, x_26, x_10, x_11, x_12, x_13, x_25); x_28 = lean_ctor_get(x_27, 0); @@ -4128,70 +3908,58 @@ lean_dec(x_3); return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___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; -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_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__9(x_4, x_5, x_3); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___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_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___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_object* x_9) { _start: { lean_object* x_10; -x_10 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_4); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___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_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___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) { _start: { lean_object* x_11; -x_11 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___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); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___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_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___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: { lean_object* x_13; -x_13 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___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 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___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_4); lean_dec(x_2); lean_dec(x_1); return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___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_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___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) { _start: { lean_object* x_15; -x_15 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___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); +x_15 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___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_9); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___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_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___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) { _start: { lean_object* x_15; -x_15 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__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, x_14); +x_15 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__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, x_14); lean_dec(x_9); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___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_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___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) { _start: { lean_object* x_8; -x_8 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__6(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); @@ -8785,6 +8553,15 @@ static lean_object* _init_l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_El _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_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__2() { +_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); @@ -8851,7 +8628,7 @@ x_40 = l_outOfBounds___rarg(x_39); if (x_37 == 0) { lean_object* x_41; lean_object* x_42; -x_41 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_41 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_42 = l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__14(x_4, x_38, x_41, x_7, x_8, x_9, x_10, x_11, x_12, x_13); if (lean_obj_tag(x_42) == 0) { @@ -8870,7 +8647,7 @@ x_48 = l_Array_ofSubarray___rarg(x_30); lean_dec(x_30); x_49 = l_Array_ofSubarray___rarg(x_32); lean_dec(x_32); -x_50 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; +x_50 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__2; x_51 = lean_alloc_ctor(0, 10, 0); lean_ctor_set(x_51, 0, x_5); lean_ctor_set(x_51, 1, x_45); @@ -8904,7 +8681,7 @@ x_58 = l_Array_ofSubarray___rarg(x_30); lean_dec(x_30); x_59 = l_Array_ofSubarray___rarg(x_32); lean_dec(x_32); -x_60 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; +x_60 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__2; x_61 = lean_alloc_ctor(0, 10, 0); lean_ctor_set(x_61, 0, x_5); lean_ctor_set(x_61, 1, x_55); @@ -8958,7 +8735,7 @@ return x_67; else { lean_object* x_68; lean_object* x_69; -x_68 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_68 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_69 = l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__15(x_4, x_38, x_68, x_7, x_8, x_9, x_10, x_11, x_12, x_13); if (lean_obj_tag(x_69) == 0) { @@ -9073,7 +8850,7 @@ lean_dec(x_2); if (x_37 == 0) { lean_object* x_95; lean_object* x_96; -x_95 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_95 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_96 = l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__16(x_4, x_93, x_95, x_7, x_8, x_9, x_10, x_11, x_12, x_13); if (lean_obj_tag(x_96) == 0) { @@ -9092,7 +8869,7 @@ x_102 = l_Array_ofSubarray___rarg(x_30); lean_dec(x_30); x_103 = l_Array_ofSubarray___rarg(x_32); lean_dec(x_32); -x_104 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; +x_104 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__2; x_105 = lean_alloc_ctor(0, 10, 0); lean_ctor_set(x_105, 0, x_5); lean_ctor_set(x_105, 1, x_99); @@ -9126,7 +8903,7 @@ x_112 = l_Array_ofSubarray___rarg(x_30); lean_dec(x_30); x_113 = l_Array_ofSubarray___rarg(x_32); lean_dec(x_32); -x_114 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; +x_114 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__2; x_115 = lean_alloc_ctor(0, 10, 0); lean_ctor_set(x_115, 0, x_5); lean_ctor_set(x_115, 1, x_109); @@ -9180,7 +8957,7 @@ return x_121; else { lean_object* x_122; lean_object* x_123; -x_122 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_122 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_123 = l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__17(x_4, x_93, x_122, x_7, x_8, x_9, x_10, x_11, x_12, x_13); if (lean_obj_tag(x_123) == 0) { @@ -26022,7 +25799,7 @@ lean_ctor_set(x_23, 1, x_22); lean_ctor_set_float(x_23, sizeof(void*)*2, x_20); lean_ctor_set_float(x_23, sizeof(void*)*2 + 8, x_20); lean_ctor_set_uint8(x_23, sizeof(void*)*2 + 16, x_21); -x_24 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_24 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_25 = lean_alloc_ctor(9, 3, 0); lean_ctor_set(x_25, 0, x_23); lean_ctor_set(x_25, 1, x_12); @@ -26084,7 +25861,7 @@ 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_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_46 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_47 = lean_alloc_ctor(9, 3, 0); lean_ctor_set(x_47, 0, x_45); lean_ctor_set(x_47, 1, x_12); @@ -26167,7 +25944,7 @@ 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_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_69 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_70 = lean_alloc_ctor(9, 3, 0); lean_ctor_set(x_70, 0, x_68); lean_ctor_set(x_70, 1, x_12); @@ -26817,7 +26594,7 @@ lean_ctor_set(x_23, 1, x_22); lean_ctor_set_float(x_23, sizeof(void*)*2, x_20); lean_ctor_set_float(x_23, sizeof(void*)*2 + 8, x_20); lean_ctor_set_uint8(x_23, sizeof(void*)*2 + 16, x_21); -x_24 = l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_24 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_25 = lean_alloc_ctor(9, 3, 0); lean_ctor_set(x_25, 0, x_23); lean_ctor_set(x_25, 1, x_12); @@ -26879,7 +26656,7 @@ 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_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_46 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_47 = lean_alloc_ctor(9, 3, 0); lean_ctor_set(x_47, 0, x_45); lean_ctor_set(x_47, 1, x_12); @@ -26962,7 +26739,7 @@ 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_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1; +x_69 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1; x_70 = lean_alloc_ctor(9, 3, 0); lean_ctor_set(x_70, 0, x_68); lean_ctor_set(x_70, 1, x_12); @@ -30414,7 +30191,7 @@ x_17 = lean_ctor_get(x_15, 1); lean_inc(x_17); lean_dec(x_15); x_18 = l_Lean_instInhabitedExpr; -x_19 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__1; +x_19 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__1; x_20 = l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4(x_18, x_19, x_3, x_16, x_4, x_6, x_7, x_8, x_9, x_17); lean_dec(x_16); if (lean_obj_tag(x_20) == 0) @@ -30537,7 +30314,7 @@ x_17 = lean_ctor_get(x_15, 1); lean_inc(x_17); lean_dec(x_15); x_18 = l_Lean_instInhabitedExpr; -x_19 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__1; +x_19 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__1; x_20 = l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4(x_18, x_19, x_4, x_16, x_5, x_7, x_8, x_9, x_10, x_17); lean_dec(x_16); if (lean_obj_tag(x_20) == 0) @@ -31206,248 +30983,216 @@ return x_2; LEAN_EXPORT lean_object* l_Lean_Elab_Structural_inferBRecOnFTypes(lean_object* x_1, lean_object* x_2, 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; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_object* x_9; lean_object* x_10; lean_object* x_57; lean_object* x_58; uint8_t x_59; x_9 = lean_array_get_size(x_2); -x_10 = lean_array_get_size(x_1); -x_11 = lean_unsigned_to_nat(0u); -x_12 = lean_nat_dec_lt(x_11, x_10); -lean_dec(x_10); -x_13 = lean_apply_1(x_3, x_11); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_13); -x_14 = l_Lean_Meta_check(x_13, x_4, x_5, x_6, x_7, x_8); -if (x_12 == 0) -{ -if (lean_obj_tag(x_14) == 0) -{ -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_14, 1); -lean_inc(x_54); -lean_dec(x_14); -x_55 = l_Lean_Elab_Structural_instInhabitedRecArgInfo; -x_56 = l_outOfBounds___rarg(x_55); -x_15 = x_56; -x_16 = x_54; -goto block_53; -} -else -{ -uint8_t x_57; -lean_dec(x_13); -lean_dec(x_9); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -x_57 = !lean_is_exclusive(x_14); -if (x_57 == 0) +x_57 = lean_array_get_size(x_1); +x_58 = lean_unsigned_to_nat(0u); +x_59 = lean_nat_dec_lt(x_58, x_57); +lean_dec(x_57); +if (x_59 == 0) { -return x_14; +lean_object* x_60; lean_object* x_61; +x_60 = l_Lean_Elab_Structural_instInhabitedRecArgInfo; +x_61 = l_outOfBounds___rarg(x_60); +x_10 = x_61; +goto block_56; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_58 = lean_ctor_get(x_14, 0); -x_59 = lean_ctor_get(x_14, 1); -lean_inc(x_59); -lean_inc(x_58); -lean_dec(x_14); -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_62; +x_62 = lean_array_fget(x_1, x_58); +x_10 = x_62; +goto block_56; } -else -{ -if (lean_obj_tag(x_14) == 0) +block_56: { -lean_object* x_61; lean_object* x_62; -x_61 = lean_ctor_get(x_14, 1); -lean_inc(x_61); -lean_dec(x_14); -x_62 = lean_array_fget(x_1, x_11); -x_15 = x_62; -x_16 = x_61; -goto block_53; -} -else +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_10, 5); +lean_inc(x_11); +x_12 = lean_apply_1(x_3, x_11); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_12); +x_13 = l_Lean_Meta_check(x_12, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_13) == 0) { -uint8_t x_63; +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_dec(x_9); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -x_63 = !lean_is_exclusive(x_14); -if (x_63 == 0) -{ -return x_14; -} -else -{ -lean_object* x_64; lean_object* x_65; lean_object* x_66; -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 = 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; -} -} -} -block_53: -{ -lean_object* x_17; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_17 = lean_infer_type(x_13, x_4, x_5, x_6, x_7, x_16); -if (lean_obj_tag(x_17) == 0) +x_15 = lean_infer_type(x_12, x_4, x_5, x_6, x_7, x_14); +if (lean_obj_tag(x_15) == 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_25; uint8_t x_26; lean_object* x_27; -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, 3); -lean_inc(x_20); +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; +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_21 = lean_array_get_size(x_20); -lean_dec(x_20); -x_22 = lean_unsigned_to_nat(1u); -x_23 = lean_nat_add(x_21, x_22); -lean_dec(x_21); -x_24 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_24, 0, x_23); +x_18 = lean_ctor_get(x_10, 3); +lean_inc(x_18); +lean_dec(x_10); +x_19 = lean_array_get_size(x_18); +lean_dec(x_18); +x_20 = lean_unsigned_to_nat(1u); +x_21 = lean_nat_add(x_19, x_20); +lean_dec(x_19); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_21); lean_inc(x_9); -x_25 = lean_alloc_closure((void*)(l_Lean_Elab_Structural_inferBRecOnFTypes___lambda__1___boxed), 8, 1); -lean_closure_set(x_25, 0, x_9); -x_26 = 0; +x_23 = lean_alloc_closure((void*)(l_Lean_Elab_Structural_inferBRecOnFTypes___lambda__1___boxed), 8, 1); +lean_closure_set(x_23, 0, x_9); +x_24 = 0; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_27 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Meta_arrowDomainsN___spec__6___rarg(x_18, x_24, x_25, x_26, x_4, x_5, x_6, x_7, x_19); -if (lean_obj_tag(x_27) == 0) +x_25 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Meta_arrowDomainsN___spec__6___rarg(x_16, x_22, x_23, x_24, x_4, x_5, x_6, x_7, x_17); +if (lean_obj_tag(x_25) == 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; size_t x_35; size_t x_36; lean_object* x_37; uint8_t x_38; -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_Elab_Structural_Positions_numIndices(x_2); -x_31 = l_Lean_Elab_Structural_inferBRecOnFTypes___closed__2; -x_32 = lean_mk_array(x_30, x_31); -x_33 = l_Array_toSubarray___rarg(x_2, x_11, x_9); -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_33); -lean_ctor_set(x_34, 1, x_32); -x_35 = lean_array_size(x_28); -x_36 = 0; -x_37 = l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_inferBRecOnFTypes___spec__2(x_28, x_35, x_36, x_34, x_4, x_5, x_6, x_7, x_29); +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; size_t x_34; size_t x_35; lean_object* x_36; uint8_t x_37; +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_Elab_Structural_Positions_numIndices(x_2); +x_29 = l_Lean_Elab_Structural_inferBRecOnFTypes___closed__2; +x_30 = lean_mk_array(x_28, x_29); +x_31 = lean_unsigned_to_nat(0u); +x_32 = l_Array_toSubarray___rarg(x_2, x_31, x_9); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_30); +x_34 = lean_array_size(x_26); +x_35 = 0; +x_36 = l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_inferBRecOnFTypes___spec__2(x_26, x_34, x_35, x_33, x_4, x_5, x_6, x_7, x_27); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_28); -x_38 = !lean_is_exclusive(x_37); -if (x_38 == 0) +lean_dec(x_26); +x_37 = !lean_is_exclusive(x_36); +if (x_37 == 0) { -lean_object* x_39; lean_object* x_40; -x_39 = lean_ctor_get(x_37, 0); -x_40 = lean_ctor_get(x_39, 1); -lean_inc(x_40); -lean_dec(x_39); -lean_ctor_set(x_37, 0, x_40); -return x_37; +lean_object* x_38; lean_object* x_39; +x_38 = lean_ctor_get(x_36, 0); +x_39 = lean_ctor_get(x_38, 1); +lean_inc(x_39); +lean_dec(x_38); +lean_ctor_set(x_36, 0, x_39); +return x_36; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_41 = lean_ctor_get(x_37, 0); -x_42 = lean_ctor_get(x_37, 1); -lean_inc(x_42); +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_dec(x_37); -x_43 = lean_ctor_get(x_41, 1); -lean_inc(x_43); -lean_dec(x_41); -x_44 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_42); -return x_44; +lean_inc(x_40); +lean_dec(x_36); +x_42 = lean_ctor_get(x_40, 1); +lean_inc(x_42); +lean_dec(x_40); +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; } } else { -uint8_t x_45; +uint8_t x_44; lean_dec(x_9); 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_27); -if (x_45 == 0) +x_44 = !lean_is_exclusive(x_25); +if (x_44 == 0) { -return x_27; +return x_25; } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_46 = lean_ctor_get(x_27, 0); -x_47 = lean_ctor_get(x_27, 1); -lean_inc(x_47); +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_25, 0); +x_46 = lean_ctor_get(x_25, 1); lean_inc(x_46); -lean_dec(x_27); -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_inc(x_45); +lean_dec(x_25); +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 { -uint8_t x_49; -lean_dec(x_15); +uint8_t x_48; +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_2); -x_49 = !lean_is_exclusive(x_17); -if (x_49 == 0) +x_48 = !lean_is_exclusive(x_15); +if (x_48 == 0) { -return x_17; +return x_15; } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_17, 0); -x_51 = lean_ctor_get(x_17, 1); -lean_inc(x_51); +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_dec(x_17); -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_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; +} +} +} +else +{ +uint8_t x_52; +lean_dec(x_12); +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_2); +x_52 = !lean_is_exclusive(x_13); +if (x_52 == 0) +{ +return x_13; +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_13, 0); +x_54 = lean_ctor_get(x_13, 1); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_13); +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; } } } @@ -32557,34 +32302,32 @@ l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition lean_mark_persistent(l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4___closed__8); l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4___closed__9 = _init_l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4___closed__9(); lean_mark_persistent(l_Lean_Elab_Structural_Positions_mapMwith___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__4___closed__9); -l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1 = _init_l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1(); -lean_mark_persistent(l_Lean_Meta_withLocalDecls___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__10___rarg___closed__1); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__1); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__2___closed__2); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__1); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__2); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__3 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__3(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__3); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__4 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__4(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__4); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__5 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__5(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__3___closed__5); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__1); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__2(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__4___closed__2); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__1(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__1); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__2(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___lambda__5___closed__2); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__1(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__1); -l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__2(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__12___rarg___closed__2); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__1); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__2___closed__2); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__1); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__2); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__3 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__3(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__3); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__4 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__4(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__4); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__5 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__5(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__3___closed__5); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__1); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__4___closed__2); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__1(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__1); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__2(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___lambda__5___closed__2); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__1(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__1); +l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__2 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__2(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__8___rarg___closed__2); l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___rarg___closed__1 = _init_l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___rarg___closed__1(); lean_mark_persistent(l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___rarg___closed__1); l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___rarg___closed__2 = _init_l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___rarg___closed__2(); @@ -32613,6 +32356,8 @@ l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Le lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__14___closed__4); l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1 = _init_l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__1); +l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__2 = _init_l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___lambda__2___closed__2); l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___closed__1 = _init_l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___closed__1(); lean_mark_persistent(l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__1___closed__1); l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__22___closed__1 = _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__22___closed__1(); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/FindRecArg.c b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/FindRecArg.c index 97b4a2400d9e..1da398428595 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/FindRecArg.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/FindRecArg.c @@ -135,7 +135,6 @@ static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_tryAllArg LEAN_EXPORT lean_object* l_Lean_Elab_Structural_prettyRecArg___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_Structural_inductiveGroups(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Structural_getRecArgInfo___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__31; LEAN_EXPORT lean_object* l_Lean_Elab_Structural_tryAllArgs___rarg___lambda__4(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* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_tryAllArgs___spec__9___rarg___closed__7; @@ -241,7 +240,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_FindRecA LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_tryAllArgs___spec__8___rarg___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 uint8_t l_Lean_PersistentArray_anyM___at___private_Lean_Elab_PreDefinition_Structural_FindRecArg_0__Lean_Elab_Structural_hasBadIndexDep_x3f___spec__13(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Structural_tryAllArgs___rarg___lambda__4___closed__3; -static lean_object* l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__30; static lean_object* l_Lean_Elab_Structural_prettyParam___closed__2; lean_object* l_Lean_LocalDecl_fvarId(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_tryAllArgs___spec__8___rarg___closed__4; @@ -5278,7 +5276,7 @@ static lean_object* _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___clo _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked(" its type ", 10, 10); +x_1 = lean_mk_string_unchecked("its type ", 9, 9); return x_1; } } @@ -5410,7 +5408,7 @@ static lean_object* _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___clo _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("its type ", 9, 9); +x_1 = lean_mk_string_unchecked(" is an inductive family", 23, 23); return x_1; } } @@ -5427,7 +5425,7 @@ static lean_object* _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___clo _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked(" is an inductive family", 23, 23); +x_1 = lean_mk_string_unchecked("\nand index", 10, 10); return x_1; } } @@ -5444,7 +5442,7 @@ static lean_object* _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___clo _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("\nand index", 10, 10); +x_1 = lean_mk_string_unchecked("\ndepends on the non index", 25, 25); return x_1; } } @@ -5461,7 +5459,7 @@ static lean_object* _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___clo _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("\ndepends on the non index", 25, 25); +x_1 = lean_mk_string_unchecked(" is an inductive family and indices are not variables", 53, 53); return x_1; } } @@ -5478,7 +5476,7 @@ static lean_object* _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___clo _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked(" is an inductive family and indices are not variables", 53, 53); +x_1 = lean_mk_string_unchecked(" is a reflexive inductive, but ", 31, 31); return x_1; } } @@ -5495,7 +5493,7 @@ static lean_object* _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___clo _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked(" is a reflexive inductive, but ", 31, 31); +x_1 = lean_mk_string_unchecked(" does not exist and it is not an inductive predicate", 52, 52); return x_1; } } @@ -5508,23 +5506,6 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__30() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" does not exist and it is not an inductive predicate", 52, 52); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__31() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__30; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} LEAN_EXPORT lean_object* l_Lean_Elab_Structural_getRecArgInfo___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: { @@ -5668,11 +5649,11 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); x_215 = l_Lean_MessageData_ofName(x_30); -x_216 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__19; +x_216 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__4; x_217 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_217, 0, x_216); lean_ctor_set(x_217, 1, x_215); -x_218 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__29; +x_218 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__27; x_219 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_219, 0, x_217); lean_ctor_set(x_219, 1, x_218); @@ -5680,7 +5661,7 @@ x_220 = l_Lean_MessageData_ofName(x_32); x_221 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_221, 0, x_219); lean_ctor_set(x_221, 1, x_220); -x_222 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__31; +x_222 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__29; x_223 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_223, 0, x_221); lean_ctor_set(x_223, 1, x_222); @@ -5855,11 +5836,11 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); x_200 = l_Lean_MessageData_ofName(x_30); -x_201 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__19; +x_201 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__4; x_202 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_202, 0, x_201); lean_ctor_set(x_202, 1, x_200); -x_203 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__27; +x_203 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__25; x_204 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_204, 0, x_202); lean_ctor_set(x_204, 1, x_203); @@ -6172,11 +6153,11 @@ lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; x_144 = lean_ctor_get(x_141, 0); x_145 = lean_ctor_get(x_141, 1); x_146 = l_Lean_MessageData_ofName(x_30); -x_147 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__19; +x_147 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__4; lean_ctor_set_tag(x_141, 7); lean_ctor_set(x_141, 1, x_146); lean_ctor_set(x_141, 0, x_147); -x_148 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__21; +x_148 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__19; x_149 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_149, 0, x_141); lean_ctor_set(x_149, 1, x_148); @@ -6184,7 +6165,7 @@ x_150 = l_Lean_indentExpr(x_14); x_151 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_151, 0, x_149); lean_ctor_set(x_151, 1, x_150); -x_152 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__23; +x_152 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__21; x_153 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_153, 0, x_151); lean_ctor_set(x_153, 1, x_152); @@ -6192,7 +6173,7 @@ x_154 = l_Lean_indentExpr(x_144); 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_Elab_Structural_getRecArgInfo___lambda__1___closed__25; +x_156 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__23; x_157 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_157, 0, x_155); lean_ctor_set(x_157, 1, x_156); @@ -6220,11 +6201,11 @@ lean_inc(x_164); lean_inc(x_163); lean_dec(x_141); x_165 = l_Lean_MessageData_ofName(x_30); -x_166 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__19; +x_166 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__4; x_167 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_167, 0, x_166); lean_ctor_set(x_167, 1, x_165); -x_168 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__21; +x_168 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__19; x_169 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_169, 0, x_167); lean_ctor_set(x_169, 1, x_168); @@ -6232,7 +6213,7 @@ x_170 = l_Lean_indentExpr(x_14); 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_Elab_Structural_getRecArgInfo___lambda__1___closed__23; +x_172 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__21; x_173 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_173, 0, x_171); lean_ctor_set(x_173, 1, x_172); @@ -6240,7 +6221,7 @@ x_174 = l_Lean_indentExpr(x_163); 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 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__25; +x_176 = l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__23; x_177 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_177, 0, x_175); lean_ctor_set(x_177, 1, x_176); @@ -17276,10 +17257,6 @@ l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__28 = _init_l_Lean_Ela lean_mark_persistent(l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__28); l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__29 = _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__29(); lean_mark_persistent(l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__29); -l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__30 = _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__30(); -lean_mark_persistent(l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__30); -l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__31 = _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__31(); -lean_mark_persistent(l_Lean_Elab_Structural_getRecArgInfo___lambda__1___closed__31); l_Lean_Elab_Structural_getRecArgInfo___lambda__2___closed__1 = _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Elab_Structural_getRecArgInfo___lambda__2___closed__1); l_Lean_Elab_Structural_getRecArgInfo___lambda__2___closed__2 = _init_l_Lean_Elab_Structural_getRecArgInfo___lambda__2___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Main.c b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Main.c index 5caddcbec9bc..a63bacb44620 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Main.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Main.c @@ -24,7 +24,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Structural_getMutualFixedPrefix(lean_object lean_object* l_Lean_Elab_Structural_mkBrecOnApp(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_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__3___closed__4; lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLocalContextImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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*, lean_object*); extern lean_object* l_Lean_Elab_instInhabitedPreDefinition; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___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*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_getMutualFixedPrefix___spec__14___lambda__3___closed__2; @@ -44,7 +44,6 @@ static lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_ LEAN_EXPORT lean_object* l_Lean_Meta_visitLambda_visit___at_Lean_Elab_Structural_getMutualFixedPrefix___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_EXPORT lean_object* l_Lean_Meta_withLetDecl___at_Lean_Elab_Structural_getMutualFixedPrefix___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_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__16(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, 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_withLocalDecl___at_Lean_Elab_Structural_getMutualFixedPrefix___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_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_lambdaTelescope___at___private_Lean_Meta_Eqns_0__Lean_Meta_mkSimpleEqThm___spec__1___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -154,6 +153,7 @@ lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_setEnv___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___lambda__5___closed__4; LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___spec__20(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, 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_lambdaBoundedTelescope___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___spec__15___rarg___lambda__1(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_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___spec__26___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -226,7 +226,8 @@ lean_object* l_Lean_Elab_Structural_run___rarg(lean_object*, lean_object*, lean_ LEAN_EXPORT lean_object* l_Lean_Elab_Structural_getMutualFixedPrefix___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ST_Prim_Ref_modifyGetUnsafe___rarg___boxed(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_levelZero; -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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*); +static lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__8; +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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_Elab_abstractNestedProofs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_reportTermArg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedExpr; @@ -278,7 +279,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_forEachExpr_x27_visit___at_Lean_Elab_Struct static lean_object* l_Lean_Elab_Structural_getMutualFixedPrefix___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Structural_structuralRecursion___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_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_getMutualFixedPrefix___spec__14___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___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__3___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_getFixedPrefix(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -415,7 +415,7 @@ uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___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*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___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_Array_foldlMUnsafe_fold___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_inferRecArgPos___spec__8(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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_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_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__13___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__14(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forEachExpr_x27___at_Lean_Elab_Structural_getMutualFixedPrefix___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -425,8 +425,10 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefi static lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__4___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at_Lean_Elab_Structural_getMutualFixedPrefix___spec__13___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__5(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_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_getMutualFixedPrefix___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___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6(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*); +static lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__9; +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6(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* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Split_0__Lean_Meta_Split_generalizeMatchDiscrs___spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_visitLambda_visit___at_Lean_Elab_Structural_getMutualFixedPrefix___spec__6___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_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__4(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*); @@ -434,6 +436,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__ lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_ReaderT_bind___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApp___spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__3(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* l_Lean_MessageData_ofName(lean_object*); lean_object* lean_expr_instantiate1(lean_object*, lean_object*); lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_getFixedPrefix___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -6581,100 +6584,100 @@ return x_31; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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, lean_object* x_8, lean_object* x_9, 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_mapFinIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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, lean_object* x_8, lean_object* x_9, 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; uint8_t x_18; -x_17 = lean_unsigned_to_nat(0u); -x_18 = lean_nat_dec_eq(x_7, x_17); -if (x_18 == 0) +lean_object* x_16; uint8_t x_17; +x_16 = lean_unsigned_to_nat(0u); +x_17 = lean_nat_dec_eq(x_6, x_16); +if (x_17 == 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_unsigned_to_nat(1u); -x_20 = lean_nat_sub(x_7, x_19); -lean_dec(x_7); -x_21 = lean_array_fget(x_6, x_8); -x_22 = lean_ctor_get(x_21, 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_unsigned_to_nat(1u); +x_19 = lean_nat_sub(x_6, x_18); +lean_dec(x_6); +x_20 = lean_array_fget(x_5, x_7); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); -lean_inc(x_23); -lean_dec(x_21); -lean_inc(x_15); +lean_dec(x_20); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -lean_inc(x_5); +lean_inc(x_11); lean_inc(x_4); -lean_inc(x_8); lean_inc(x_3); -x_24 = l_Lean_Elab_Structural_mkBrecOnApp(x_3, x_8, x_4, x_5, x_22, x_23, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_24) == 0) +lean_inc(x_7); +lean_inc(x_1); +x_23 = l_Lean_Elab_Structural_mkBrecOnApp(x_1, x_7, x_3, x_4, x_21, x_22, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_23) == 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_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); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); -x_27 = lean_nat_add(x_8, x_19); -lean_dec(x_8); -x_28 = lean_array_push(x_10, x_25); -x_7 = x_20; -x_8 = x_27; -x_9 = lean_box(0); -x_10 = x_28; -x_16 = x_26; +lean_dec(x_23); +x_26 = lean_nat_add(x_7, x_18); +lean_dec(x_7); +x_27 = lean_array_push(x_9, x_24); +x_6 = x_19; +x_7 = x_26; +x_8 = lean_box(0); +x_9 = x_27; +x_15 = x_25; goto _start; } else { -uint8_t x_30; -lean_dec(x_20); -lean_dec(x_15); +uint8_t x_29; +lean_dec(x_19); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_5); +lean_dec(x_11); +lean_dec(x_9); +lean_dec(x_7); lean_dec(x_4); lean_dec(x_3); -x_30 = !lean_is_exclusive(x_24); -if (x_30 == 0) +lean_dec(x_1); +x_29 = !lean_is_exclusive(x_23); +if (x_29 == 0) { -return x_24; +return x_23; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_24, 0); -x_32 = lean_ctor_get(x_24, 1); -lean_inc(x_32); +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_dec(x_24); -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_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; } } } else { -lean_object* x_34; -lean_dec(x_15); +lean_object* x_33; lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -lean_dec(x_8); +lean_dec(x_11); lean_dec(x_7); -lean_dec(x_5); +lean_dec(x_6); lean_dec(x_4); lean_dec(x_3); -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_10); -lean_ctor_set(x_34, 1, x_16); -return x_34; +lean_dec(x_1); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_9); +lean_ctor_set(x_33, 1, x_15); +return x_33; } } } @@ -7042,113 +7045,113 @@ lean_inc(x_2); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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, size_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___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* 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: { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_17 = lean_array_get_size(x_1); -x_18 = lean_mk_empty_array_with_capacity(x_17); -x_19 = lean_unsigned_to_nat(0u); -lean_inc(x_15); -lean_inc(x_14); +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_array_get_size(x_1); +x_16 = lean_mk_empty_array_with_capacity(x_15); +x_17 = lean_unsigned_to_nat(0u); lean_inc(x_13); lean_inc(x_12); -x_20 = l_Array_mapIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__10(x_2, x_3, x_4, x_5, x_6, x_1, x_17, x_19, lean_box(0), x_18, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_20) == 0) +lean_inc(x_11); +lean_inc(x_10); +x_18 = l_Array_mapFinIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__10(x_2, x_1, x_3, x_4, x_1, x_15, x_17, lean_box(0), x_16, x_9, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_21; lean_object* x_22; size_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 = lean_array_size(x_21); -x_24 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__11(x_7, x_23, x_8, x_21, x_11, x_12, x_13, x_14, x_15, x_22); -lean_dec(x_15); -lean_dec(x_14); +lean_object* x_19; lean_object* x_20; size_t 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_array_size(x_19); +x_22 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__11(x_5, x_21, x_6, x_19, x_9, x_10, x_11, x_12, x_13, x_20); lean_dec(x_13); lean_dec(x_12); -if (lean_obj_tag(x_24) == 0) +lean_dec(x_11); +lean_dec(x_10); +if (lean_obj_tag(x_22) == 0) { -uint8_t x_25; -x_25 = !lean_is_exclusive(x_24); -if (x_25 == 0) +uint8_t x_23; +x_23 = !lean_is_exclusive(x_22); +if (x_23 == 0) { -lean_object* x_26; lean_object* x_27; size_t x_28; lean_object* x_29; -x_26 = lean_ctor_get(x_24, 0); -x_27 = l_Array_zip___rarg(x_9, x_26); -lean_dec(x_26); -x_28 = lean_array_size(x_27); -x_29 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__12(x_28, x_8, x_27); -lean_ctor_set(x_24, 0, x_29); -return x_24; +lean_object* x_24; lean_object* x_25; size_t x_26; lean_object* x_27; +x_24 = lean_ctor_get(x_22, 0); +x_25 = l_Array_zip___rarg(x_7, x_24); +lean_dec(x_24); +x_26 = lean_array_size(x_25); +x_27 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__12(x_26, x_6, x_25); +lean_ctor_set(x_22, 0, x_27); +return x_22; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; size_t x_33; lean_object* x_34; lean_object* x_35; -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_Array_zip___rarg(x_9, x_30); -lean_dec(x_30); -x_33 = lean_array_size(x_32); -x_34 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__12(x_33, x_8, 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_31); -return x_35; +lean_object* x_28; lean_object* x_29; lean_object* x_30; size_t x_31; lean_object* x_32; lean_object* x_33; +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 = l_Array_zip___rarg(x_7, x_28); +lean_dec(x_28); +x_31 = lean_array_size(x_30); +x_32 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__12(x_31, x_6, 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_29); +return x_33; } } else { -uint8_t x_36; -x_36 = !lean_is_exclusive(x_24); -if (x_36 == 0) +uint8_t x_34; +x_34 = !lean_is_exclusive(x_22); +if (x_34 == 0) { -return x_24; +return x_22; } else { -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; +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; } } } else { -uint8_t x_40; -lean_dec(x_15); -lean_dec(x_14); +uint8_t x_38; lean_dec(x_13); lean_dec(x_12); -lean_dec(x_7); -x_40 = !lean_is_exclusive(x_20); -if (x_40 == 0) +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_5); +x_38 = !lean_is_exclusive(x_18); +if (x_38 == 0) { -return x_20; +return x_18; } else { -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; +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_18, 0); +x_40 = lean_ctor_get(x_18, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_18); +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; } } } @@ -7201,7 +7204,6 @@ lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_4); -lean_inc(x_3); x_21 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__9(x_3, x_4, x_20, x_5, x_19, x_12, x_13, x_14, x_15, x_16, x_17); if (lean_obj_tag(x_21) == 0) { @@ -7225,9 +7227,8 @@ 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_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(x_7, x_3, x_1, x_4, x_8, x_22, x_9, x_5, x_10, x_28, x_12, x_13, x_14, x_15, x_16, x_27); +x_29 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(x_7, x_4, x_8, x_22, x_9, x_5, x_10, x_28, x_12, x_13, x_14, x_15, x_16, x_27); lean_dec(x_12); -lean_dec(x_3); return x_29; } else @@ -7259,10 +7260,9 @@ lean_inc(x_41); x_42 = lean_ctor_get(x_40, 1); lean_inc(x_42); lean_dec(x_40); -x_43 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(x_7, x_3, x_1, x_4, x_8, x_22, x_9, x_5, x_10, x_41, x_12, x_13, x_14, x_15, x_16, x_42); +x_43 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(x_7, x_4, x_8, x_22, x_9, x_5, x_10, x_41, x_12, x_13, x_14, x_15, x_16, x_42); lean_dec(x_12); lean_dec(x_41); -lean_dec(x_3); return x_43; } else @@ -7290,10 +7290,9 @@ lean_inc(x_54); x_55 = lean_ctor_get(x_53, 1); lean_inc(x_55); lean_dec(x_53); -x_56 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(x_7, x_3, x_1, x_4, x_8, x_22, x_9, x_5, x_10, x_54, x_12, x_13, x_14, x_15, x_16, x_55); +x_56 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(x_7, x_4, x_8, x_22, x_9, x_5, x_10, x_54, x_12, x_13, x_14, x_15, x_16, x_55); lean_dec(x_12); lean_dec(x_54); -lean_dec(x_3); return x_56; } } @@ -7310,7 +7309,6 @@ lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); lean_dec(x_4); -lean_dec(x_3); x_57 = !lean_is_exclusive(x_21); if (x_57 == 0) { @@ -7739,7 +7737,7 @@ static lean_object* _init_l___private_Lean_Elab_PreDefinition_Structural_Main_0_ _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("positions: ", 11, 11); +x_1 = lean_mk_string_unchecked("assignments of type formers of ", 31, 31); return x_1; } } @@ -7752,92 +7750,126 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* 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_object* x_11, lean_object* x_12, lean_object* x_13) { +static lean_object* _init_l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__8() { _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; lean_object* x_21; uint8_t x_22; -x_14 = l_Lean_InductiveVal_numTypeFormers(x_1); -x_15 = l_Array_range(x_14); -x_16 = l_Lean_Elab_Structural_instInhabitedRecArgInfo; -x_17 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__1; -x_18 = l_Lean_Elab_Structural_Positions_groupAndSort___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__4(x_16, x_17, x_2, x_15); -x_19 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__5; -x_20 = l_Lean_isTracingEnabledFor___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApp___spec__2(x_19, x_8, x_9, x_10, x_11, x_12, x_13); -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_1; +x_1 = lean_mk_string_unchecked(" to functions: ", 15, 15); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__9() { +_start: { -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_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__5(x_2, x_3, x_4, x_19, x_18, x_5, x_6, x_24, x_8, x_9, x_10, x_11, x_12, x_23); -return x_25; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__8; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* 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_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; lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_15 = l_Lean_InductiveVal_numTypeFormers(x_1); +x_16 = l_Array_range(x_15); +x_17 = l_Lean_Elab_Structural_instInhabitedRecArgInfo; +x_18 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__1; +x_19 = l_Lean_Elab_Structural_Positions_groupAndSort___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__4(x_17, x_18, x_2, x_16); +x_20 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__5; +x_21 = l_Lean_isTracingEnabledFor___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApp___spec__2(x_20, 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; +lean_dec(x_7); +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_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__5(x_2, x_3, x_4, x_20, x_19, x_5, x_6, x_25, x_9, x_10, x_11, x_12, x_13, x_24); +return x_26; } else { -uint8_t x_26; -x_26 = !lean_is_exclusive(x_20); -if (x_26 == 0) +uint8_t x_27; +x_27 = !lean_is_exclusive(x_21); +if (x_27 == 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; -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 = lean_array_to_list(x_18); -x_30 = lean_box(0); -x_31 = l_List_mapTR_loop___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__16(x_29, x_30); -x_32 = l_Lean_MessageData_ofList(x_31); -x_33 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__7; -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 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__3___closed__4; -x_35 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_35, 0, x_20); -lean_ctor_set(x_35, 1, x_34); -x_36 = l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApp___spec__3(x_19, x_35, x_8, x_9, x_10, x_11, x_12, x_27); -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___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__5(x_2, x_3, x_4, x_19, x_18, x_5, x_6, x_37, x_8, x_9, x_10, x_11, x_12, x_38); -lean_dec(x_37); -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; 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_28 = lean_ctor_get(x_21, 1); +x_29 = lean_ctor_get(x_21, 0); +lean_dec(x_29); +x_30 = l_Lean_MessageData_ofName(x_7); +x_31 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__7; +lean_ctor_set_tag(x_21, 7); +lean_ctor_set(x_21, 1, x_30); +lean_ctor_set(x_21, 0, x_31); +x_32 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__9; +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_21); +lean_ctor_set(x_33, 1, x_32); +lean_inc(x_19); +x_34 = lean_array_to_list(x_19); +x_35 = lean_box(0); +x_36 = l_List_mapTR_loop___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__16(x_34, x_35); +x_37 = l_Lean_MessageData_ofList(x_36); +x_38 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_38, 0, x_33); +lean_ctor_set(x_38, 1, x_37); +x_39 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__3___closed__4; +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___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApp___spec__3(x_20, x_40, x_9, x_10, x_11, x_12, x_13, x_28); +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_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__5(x_2, x_3, x_4, x_20, x_19, x_5, x_6, x_42, x_9, x_10, x_11, x_12, x_13, x_43); +lean_dec(x_42); +return x_44; } 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; -x_40 = lean_ctor_get(x_20, 1); -lean_inc(x_40); -lean_dec(x_20); -lean_inc(x_18); -x_41 = lean_array_to_list(x_18); -x_42 = lean_box(0); -x_43 = l_List_mapTR_loop___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__16(x_41, x_42); -x_44 = l_Lean_MessageData_ofList(x_43); -x_45 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__7; -x_46 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_44); -x_47 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__3___closed__4; +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_45 = lean_ctor_get(x_21, 1); +lean_inc(x_45); +lean_dec(x_21); +x_46 = l_Lean_MessageData_ofName(x_7); +x_47 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__7; x_48 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_48, 0, x_46); -lean_ctor_set(x_48, 1, x_47); -x_49 = l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApp___spec__3(x_19, x_48, x_8, x_9, x_10, x_11, x_12, 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_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__5(x_2, x_3, x_4, x_19, x_18, x_5, x_6, x_50, x_8, x_9, x_10, x_11, x_12, x_51); -lean_dec(x_50); -return x_52; +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_46); +x_49 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__9; +x_50 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +lean_inc(x_19); +x_51 = lean_array_to_list(x_19); +x_52 = lean_box(0); +x_53 = l_List_mapTR_loop___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__16(x_51, x_52); +x_54 = l_Lean_MessageData_ofList(x_53); +x_55 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_55, 0, x_50); +lean_ctor_set(x_55, 1, x_54); +x_56 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__3___closed__4; +x_57 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +x_58 = l_Lean_addTrace___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApp___spec__3(x_20, x_57, x_9, x_10, x_11, x_12, x_13, x_45); +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_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__5(x_2, x_3, x_4, x_20, x_19, x_5, x_6, x_59, x_9, x_10, x_11, x_12, x_13, x_60); +lean_dec(x_59); +return x_61; } } } @@ -8386,6 +8418,7 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); +lean_inc(x_21); x_22 = l_Lean_Meta_isInductivePredicate(x_21, x_5, x_6, x_7, x_8, x_19); if (lean_obj_tag(x_22) == 0) { @@ -8402,7 +8435,7 @@ 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_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6(x_18, x_3, x_13, x_11, x_2, x_1, x_26, x_4, x_5, x_6, x_7, x_8, x_25); +x_27 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6(x_18, x_3, x_13, x_11, x_2, x_1, x_21, x_26, x_4, x_5, x_6, x_7, x_8, x_25); lean_dec(x_1); lean_dec(x_13); lean_dec(x_18); @@ -8411,6 +8444,7 @@ return x_27; else { lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +lean_dec(x_21); lean_dec(x_18); lean_dec(x_3); x_28 = lean_ctor_get(x_22, 1); @@ -8467,6 +8501,7 @@ return x_39; else { uint8_t x_40; +lean_dec(x_21); lean_dec(x_18); lean_dec(x_15); lean_dec(x_13); @@ -8680,16 +8715,15 @@ x_14 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_ return x_14; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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_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_mapFinIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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_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_Array_mapIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__10(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_6); +lean_object* x_16; +x_16 = l_Array_mapFinIdxM_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___spec__10(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_10); +lean_dec(x_5); lean_dec(x_2); -lean_dec(x_1); -return x_17; +return x_16; } } LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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) { @@ -8730,20 +8764,18 @@ lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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: { -size_t x_17; lean_object* x_18; -x_17 = lean_unbox_usize(x_8); -lean_dec(x_8); -x_18 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_17, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_11); -lean_dec(x_10); +size_t x_15; lean_object* x_16; +x_15 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_16 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__2(x_1, x_2, x_3, x_4, x_5, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); lean_dec(x_9); -lean_dec(x_3); -lean_dec(x_2); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_1); -return x_18; +return x_16; } } LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__3___boxed(lean_object** _args) { @@ -8806,18 +8838,18 @@ lean_dec(x_2); return x_16; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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_object* x_13) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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_object* x_13, lean_object* x_14) { _start: { -size_t x_14; lean_object* x_15; -x_14 = lean_unbox_usize(x_4); +size_t x_15; lean_object* x_16; +x_15 = lean_unbox_usize(x_4); lean_dec(x_4); -x_15 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6(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); -lean_dec(x_7); +x_16 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6(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_8); lean_dec(x_6); lean_dec(x_3); lean_dec(x_1); -return x_15; +return x_16; } } LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___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) { @@ -15918,6 +15950,10 @@ l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elim lean_mark_persistent(l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__6); l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__7 = _init_l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__7(); lean_mark_persistent(l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__7); +l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__8 = _init_l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__8(); +lean_mark_persistent(l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__8); +l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__9 = _init_l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__9(); +lean_mark_persistent(l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__6___closed__9); l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__8___closed__1 = _init_l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__8___closed__1(); lean_mark_persistent(l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__8___closed__1); l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__8___closed__2 = _init_l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimMutualRecursion___lambda__8___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/SmartUnfolding.c b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/SmartUnfolding.c index b98f3ad63761..e3f05672380d 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/SmartUnfolding.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/SmartUnfolding.c @@ -17,6 +17,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_addS LEAN_EXPORT lean_object* l_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___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_lambdaBoundedTelescope___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__8___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, 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*); +lean_object* lean_mk_empty_array_with_capacity(lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaBoundedTelescope___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__8___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -67,6 +68,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at_Lean_Elab_Structural_addSm LEAN_EXPORT lean_object* l_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_levelZero; extern lean_object* l_Lean_instInhabitedExpr; +static lean_object* l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); @@ -3467,20 +3469,31 @@ return x_10; static lean_object* _init_l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__1() { _start: { -lean_object* x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +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_Elab_Structural_addSmartUnfoldingDefAux___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; x_1 = lean_box(0); -x_2 = 0; +x_2 = lean_box(0); x_3 = 0; -x_4 = 2; -x_5 = l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__1___lambda__2___closed__1; -x_6 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -lean_ctor_set_uint8(x_6, sizeof(void*)*2, x_2); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 1, x_3); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 2, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 3, x_3); -return x_6; +x_4 = 0; +x_5 = 0; +x_6 = l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__1; +x_7 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_7, 0, x_2); +lean_ctor_set(x_7, 1, x_1); +lean_ctor_set(x_7, 2, x_6); +lean_ctor_set_uint8(x_7, sizeof(void*)*3, x_3); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 1, x_4); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 2, x_5); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 3, x_4); +return x_7; } } LEAN_EXPORT lean_object* l_Lean_Elab_Structural_addSmartUnfoldingDefAux(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { @@ -3530,7 +3543,7 @@ lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; x_25 = lean_ctor_get(x_15, 0); x_26 = l_Lean_Meta_smartUnfoldingSuffix; x_27 = l_Lean_Name_str___override(x_11, x_26); -x_28 = l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__1; +x_28 = l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__2; lean_ctor_set(x_1, 5, x_25); lean_ctor_set(x_1, 3, x_27); lean_ctor_set(x_1, 2, x_28); @@ -3547,7 +3560,7 @@ lean_inc(x_29); lean_dec(x_15); x_31 = l_Lean_Meta_smartUnfoldingSuffix; x_32 = l_Lean_Name_str___override(x_11, x_31); -x_33 = l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__1; +x_33 = l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__2; lean_ctor_set(x_1, 5, x_29); lean_ctor_set(x_1, 3, x_32); lean_ctor_set(x_1, 2, x_33); @@ -3606,7 +3619,7 @@ if (lean_is_exclusive(x_15)) { } x_42 = l_Lean_Meta_smartUnfoldingSuffix; x_43 = l_Lean_Name_str___override(x_11, x_42); -x_44 = l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__1; +x_44 = l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__2; x_45 = lean_alloc_ctor(0, 7, 1); lean_ctor_set(x_45, 0, x_8); lean_ctor_set(x_45, 1, x_10); @@ -3864,6 +3877,8 @@ l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__9___lambda__3___closed__6); l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__1 = _init_l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__1(); lean_mark_persistent(l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__1); +l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__2 = _init_l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__2(); +lean_mark_persistent(l_Lean_Elab_Structural_addSmartUnfoldingDefAux___closed__2); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/WF/GuessLex.c b/stage0/stdlib/Lean/Elab/PreDefinition/WF/GuessLex.c index deb8496e4a93..0be97e0a6bbf 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/WF/GuessLex.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/WF/GuessLex.c @@ -63,7 +63,6 @@ LEAN_EXPORT uint8_t l_Lean_Expr_hasAnyFVar_visit___at_Lean_Elab_WF_GuessLex_mayO LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_WF_GuessLex_explainMutualFailure___spec__9___boxed(lean_object**); static lean_object* l_Lean_Elab_WF_guessLex___closed__1; static lean_object* l_Lean_Elab_WF_GuessLex_collectRecCalls___lambda__5___closed__1; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___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* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_RecCallCache_prettyEntry(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_WF_GuessLex_explainMutualFailure___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*); @@ -73,6 +72,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_exp LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__24(lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_filterSubsumed___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_collectHeaders___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___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*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_GuessLexRel_toNatRel___closed__17; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__32___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Elab_WF_GuessLex_mkProdElem___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -102,6 +102,7 @@ lean_object* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, l static lean_object* l___private_Lean_Elab_PreDefinition_WF_GuessLex_0__Lean_Elab_WF_GuessLex_reprGuessLexRel____x40_Lean_Elab_PreDefinition_WF_GuessLex___hyg_4223____closed__5; lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getMatcherInfo_x3f___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__2___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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_Lean_Elab_WF_GuessLex_RecCallWithContext_posString___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__25___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_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_WF_GuessLex_withRecApps_loop___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*); @@ -236,9 +237,9 @@ LEAN_EXPORT lean_object* l_Lean_Meta_lambdaBoundedTelescope___at_Lean_Elab_WF_Gu LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_withRecApps___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* l_Array_mapMUnsafe_map___at_Lean_Meta_MatcherApp_inferMatchType___spec__9(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___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*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__5(lean_object*, 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_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___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*); static lean_object* l___private_Lean_Elab_PreDefinition_WF_GuessLex_0__Lean_Elab_WF_GuessLex_reprGuessLexRel____x40_Lean_Elab_PreDefinition_WF_GuessLex___hyg_4223____closed__25; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_WF_GuessLex_formatTable___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_Array_mapMUnsafe_map___at_Lean_Elab_WF_GuessLex_explainMutualFailure___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -296,7 +297,6 @@ lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_logAt___at_Lean_Elab_Term_reportUnsolvedGoals___spec__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_GuessLexRel_toNatRel___closed__20; LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_withRecApps_containsRecFn(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___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*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_collectRecCalls___lambda__2___closed__3; size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_explainMutualFailure___spec__12___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -324,6 +324,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_withRecApps_loop___rarg___lambd LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_formatTable(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_WF_GuessLex_generateCombinations_x3f_go___spec__2___boxed(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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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_EXPORT lean_object* l_panic___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__10___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_WF_GuessLex_0__Lean_Elab_WF_GuessLex_reprGuessLexRel____x40_Lean_Elab_PreDefinition_WF_GuessLex___hyg_4223____boxed(lean_object*, lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); @@ -340,10 +341,10 @@ lean_object* lean_nat_to_int(lean_object*); lean_object* l_Lean_MessageData_ofSyntax(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_WF_GuessLex_generateMeasures___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_collectRecCalls___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, 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_WF_GuessLex_toTerminationArguments(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__3___rarg___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_WF_GuessLex_filterSubsumed___lambda__2___closed__4; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_guessLex___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_solve_go___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__9(lean_object*, lean_object*); @@ -365,7 +366,6 @@ lean_object* l_Lean_Name_getPrefix(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_WF_GuessLex_explainNonMutualFailure___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_Elab_WF_GuessLex_naryVarNames_freshen___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__25___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*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1(uint8_t, 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_throwError___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__18___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_isNatCmp___closed__5; static lean_object* l_Lean_Elab_WF_GuessLex_collectRecCalls___lambda__2___closed__4; @@ -431,7 +431,6 @@ lean_object* lean_st_mk_ref(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__12___rarg(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_Lean_throwError___at_Lean_Elab_WF_guessLex___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___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_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_mayOmitSizeOf___closed__8; lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); @@ -451,6 +450,7 @@ static lean_object* l___private_Lean_Elab_PreDefinition_WF_GuessLex_0__Lean_Elab static lean_object* l_Lean_Elab_WF_GuessLex_GuessLexRel_toNatRel___closed__27; static lean_object* l_Lean_Elab_WF_guessLex___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_evalRecCall___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_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_WF_GuessLex_explainMutualFailure___spec__11(lean_object*, lean_object*, 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_WF_GuessLex_complexMeasures___boxed(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_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__11___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -461,7 +461,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_guessLex___s extern lean_object* l_Lean_instInhabitedExpr; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10___lambda__1(lean_object*, 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_Elab_WF_GuessLex_withRecApps_processApp(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__1___rarg___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*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_explainNonMutualFailure___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_isNatCmp(lean_object*); @@ -520,6 +519,7 @@ lean_object* l_Lean_LocalContext_setUserName(lean_object*, lean_object*, lean_ob LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_WF_GuessLex_solve_go___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_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_withRecApps___rarg___closed__7; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_WF_GuessLex_evalRecCall___spec__3___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_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_reportTermArgs___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* l_Lean_Meta_saveState___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_WF_guessLex___spec__6(size_t, size_t, lean_object*); @@ -531,13 +531,12 @@ LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_WF_GuessLex_s LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_WF_GuessLex_evalRecCall___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_mayOmitSizeOf___closed__6; LEAN_EXPORT lean_object* l_Lean_Expr_hasAnyFVar_visit___at_Lean_Elab_WF_GuessLex_mayOmitSizeOf___spec__1___boxed(lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_withRecApps_containsRecFn___rarg(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_loop___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__17___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_Std_Range_forIn_x27_loop___at_Lean_Elab_WF_GuessLex_formatTable___spec__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_Lean_Elab_WF_guessLex___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_WF_GuessLex_explainMutualFailure___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___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*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___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*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_guessLex___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_WF_GuessLex_evalRecCall___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_instInhabitedMeasure; @@ -570,7 +569,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_showInferredTerminationBy; lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_WF_GuessLex_explainMutualFailure___spec__8___boxed(lean_object**); LEAN_EXPORT uint8_t l_Lean_Elab_WF_GuessLex_GuessLexRel_ofNat(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__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_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_WF_GuessLex_formatTable___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_List_forIn_loop___at_Lean_Elab_WF_GuessLex_evalRecCall___spec__3___lambda__8___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__31___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -600,7 +598,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_GuessLexRel_noConfusion(lean_ob LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_evalRecCall(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_WF_guessLex___lambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_solve_go___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_WF_GuessLex_evalRecCall___spec__3___closed__4; static size_t l_Lean_Elab_WF_GuessLex_generateMeasures___closed__3; @@ -648,6 +645,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_com static lean_object* l_Lean_Elab_WF_GuessLex_withRecApps___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_WF_guessLex___spec__3___boxed(lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__11(lean_object*, lean_object*, 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_WF_GuessLex_GuessLexRel_toNatRel___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_withUserNames___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_Meta_getMatcherInfo_x3f___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -668,7 +666,7 @@ lean_object* l_Lean_Elab_Term_TermElabM_run___rarg(lean_object*, lean_object*, l LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_Measure_toString(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_WF_guessLex___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__1___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*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10(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_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10(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_Elab_WF_GuessLex_GuessLexRel_toNatRel___closed__26; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_solve_go___spec__1___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getLocalInstances(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -695,6 +693,7 @@ static lean_object* l_Lean_Elab_WF_GuessLex_filterSubsumed___lambda__2___closed_ LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_solve_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_solve_go___at_Lean_Elab_WF_guessLex___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_StateRefT_x27_lift(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__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*); uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__8(lean_object*, lean_object*); lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); @@ -706,7 +705,6 @@ static lean_object* l_Lean_Elab_WF_GuessLex_withRecApps___rarg___lambda__1___clo LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__8___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_List_forM___at_Lean_Elab_WF_GuessLex_evalRecCall___spec__1___closed__2; 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_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___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_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_SavedLocalContext_run___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_type(lean_object*); lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_evalTactic_handleEx___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -754,7 +752,6 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_WF_GuessLex_wi LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10___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_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__25___rarg(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*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_WF_GuessLex_evalRecCall___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_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__12(lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_GuessLexRel_toNatRel___closed__15; LEAN_EXPORT lean_object* l_Array_isEqvAux___at_Lean_Elab_WF_GuessLex_filterSubsumed___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -770,6 +767,7 @@ static lean_object* l_Lean_Elab_WF_GuessLex_isNatCmp___closed__4; lean_object* l_Array_ofSubarray___rarg(lean_object*); LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_simpleMeasures___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10___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_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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*); static lean_object* l_Lean_Elab_WF_GuessLex_explainFailure___closed__5; LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_explainMutualFailure(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -779,6 +777,8 @@ static lean_object* l___private_Lean_Elab_PreDefinition_WF_GuessLex_0__Lean_Elab LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__18___boxed(lean_object*, lean_object*); static lean_object* l_List_forM___at_Lean_Elab_WF_GuessLex_evalRecCall___spec__1___closed__1; static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__21___rarg___lambda__2___closed__2; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___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_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_withRecApps_processApp___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_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_instDecidableEqGuessLexRel___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_WF_GuessLex_filterSubsumed___spec__6(lean_object*); @@ -789,6 +789,7 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_WF_GuessLex_withRecApp static lean_object* l_Lean_Elab_WF_GuessLex_explainFailure___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_filterSubsumed___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_withRecApps_loop___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_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1(uint8_t, 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_lambdaBoundedTelescope___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__28(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_inspectCall(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_sub(size_t, size_t); @@ -860,7 +861,6 @@ uint8_t l_Lean_isAuxRecursorWithSuffix(lean_object*, lean_object*, lean_object*) lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_WF_GuessLex_naryVarNames_freshen___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_evalRecCall___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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_EXPORT lean_object* l_panic___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__13(lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_GuessLex_evalRecCall___lambda__3___closed__1; LEAN_EXPORT uint8_t l_Lean_Elab_WF_GuessLex_instDecidableEqGuessLexRel(uint8_t, uint8_t); @@ -896,6 +896,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_SavedLocalContext_run(lean_obje static lean_object* l_Lean_Elab_WF_GuessLex_instInhabitedMeasure___closed__1; static lean_object* l_Lean_Elab_WF_GuessLex_RecCallWithContext_posString___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_WF_GuessLex_solve___at_Lean_Elab_WF_guessLex___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___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_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__22(lean_object*, lean_object*); uint8_t l_Lean_Expr_isFVar(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_WF_GuessLex_formatTable___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -928,7 +929,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_com LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_instMonad___rarg(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_explainMutualFailure___spec__12___closed__10; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__31(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_isEqvAux___at_Lean_Elab_WF_GuessLex_filterSubsumed___spec__2(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_WF_GuessLex_withRecApps_loop___spec__30___rarg(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*, lean_object*); @@ -3455,7 +3455,7 @@ return x_56; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1(uint8_t 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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1(uint8_t 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_13; @@ -3506,7 +3506,7 @@ return x_21; } } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -3515,7 +3515,7 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___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) { _start: { lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; size_t x_18; lean_object* x_19; size_t x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; @@ -3539,7 +3539,7 @@ x_22 = lean_box(x_4); x_23 = lean_box_usize(x_18); x_24 = lean_box_usize(x_20); lean_inc(x_14); -x_25 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1___boxed), 12, 7); +x_25 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1___boxed), 12, 7); lean_closure_set(x_25, 0, x_22); lean_closure_set(x_25, 1, x_5); lean_closure_set(x_25, 2, x_14); @@ -3550,7 +3550,7 @@ lean_closure_set(x_25, 6, x_21); if (x_16 == 0) { lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_26 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_27 = l_outOfBounds___rarg(x_26); x_28 = l_Lean_Elab_WF_GuessLex_withUserNames___rarg(x_14, x_27, x_25, x_7, x_8, x_9, x_10, x_11); lean_dec(x_14); @@ -3566,7 +3566,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__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: { lean_object* x_15; uint8_t x_16; @@ -3586,7 +3586,7 @@ x_21 = lean_box(x_4); lean_inc(x_7); lean_inc(x_3); lean_inc(x_2); -x_22 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___boxed), 11, 4); +x_22 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___boxed), 11, 4); lean_closure_set(x_22, 0, x_2); lean_closure_set(x_22, 1, x_3); lean_closure_set(x_22, 2, x_7); @@ -3674,7 +3674,7 @@ x_10 = lean_unsigned_to_nat(1u); x_11 = lean_nat_dec_lt(x_10, x_9); x_12 = lean_mk_empty_array_with_capacity(x_9); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2(x_1, x_2, x_3, x_11, x_1, x_9, x_13, lean_box(0), x_12, x_4, x_5, x_6, x_7, x_8); +x_14 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2(x_1, x_2, x_3, x_11, x_1, x_9, x_13, lean_box(0), x_12, x_4, x_5, x_6, x_7, x_8); return x_14; } } @@ -3718,7 +3718,7 @@ lean_dec(x_3); return x_16; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___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) { _start: { uint8_t x_13; size_t x_14; size_t x_15; lean_object* x_16; @@ -3728,32 +3728,32 @@ x_14 = lean_unbox_usize(x_5); lean_dec(x_5); x_15 = lean_unbox_usize(x_6); lean_dec(x_6); -x_16 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1(x_13, x_2, x_3, x_4, x_14, x_15, x_7, x_8, x_9, x_10, x_11, x_12); +x_16 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__1(x_13, x_2, x_3, x_4, x_14, x_15, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_4); lean_dec(x_3); return x_16; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___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) { _start: { uint8_t x_12; lean_object* x_13; x_12 = lean_unbox(x_4); lean_dec(x_4); -x_13 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2(x_1, x_2, x_3, x_12, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_13 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2(x_1, x_2, x_3, x_12, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_6); lean_dec(x_3); lean_dec(x_2); return x_13; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___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, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___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, lean_object* x_14) { _start: { uint8_t x_15; lean_object* x_16; x_15 = lean_unbox(x_4); lean_dec(x_4); -x_16 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__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); +x_16 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__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_1); return x_16; @@ -18292,7 +18292,7 @@ lean_closure_set(x_27, 6, x_1); if (x_24 == 0) { lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_28 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_28 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_29 = l_outOfBounds___rarg(x_28); x_30 = lean_alloc_closure((void*)(l_Lean_Elab_WF_GuessLex_withUserNames___rarg___boxed), 8, 3); lean_closure_set(x_30, 0, x_22); @@ -18466,140 +18466,140 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10(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_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___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, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -uint8_t x_14; -x_14 = lean_usize_dec_lt(x_7, x_6); -if (x_14 == 0) +uint8_t x_13; +x_13 = lean_usize_dec_lt(x_6, x_5); +if (x_13 == 0) { -lean_object* x_15; -lean_dec(x_12); +lean_object* x_14; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_2); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_8); -lean_ctor_set(x_15, 1, x_13); -return x_15; +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_16; lean_object* x_17; uint8_t x_18; -x_16 = lean_array_uget(x_5, x_7); -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -x_18 = lean_nat_dec_eq(x_17, x_4); -lean_dec(x_17); -if (x_18 == 0) -{ -size_t x_19; size_t x_20; +lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_15 = lean_array_uget(x_4, x_6); +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +x_17 = lean_nat_dec_eq(x_16, x_3); lean_dec(x_16); -x_19 = 1; -x_20 = lean_usize_add(x_7, x_19); -x_7 = x_20; +if (x_17 == 0) +{ +size_t x_18; size_t x_19; +lean_dec(x_15); +x_18 = 1; +x_19 = lean_usize_add(x_6, x_18); +x_6 = x_19; goto _start; } else { -lean_object* x_22; lean_object* x_23; -x_22 = lean_box(0); -lean_inc(x_12); +lean_object* x_21; lean_object* x_22; +x_21 = lean_box(0); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_2); -x_23 = l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10___lambda__4(x_16, x_2, x_3, x_4, x_8, x_22, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_23) == 0) +lean_inc(x_8); +lean_inc(x_1); +x_22 = l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10___lambda__4(x_15, x_1, x_2, x_3, x_7, x_21, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_22) == 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_23; +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +if (lean_obj_tag(x_23) == 0) { -uint8_t x_25; -lean_dec(x_12); +uint8_t x_24; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_2); -x_25 = !lean_is_exclusive(x_23); -if (x_25 == 0) +lean_dec(x_8); +lean_dec(x_1); +x_24 = !lean_is_exclusive(x_22); +if (x_24 == 0) { -lean_object* x_26; lean_object* x_27; +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_22, 0); +lean_dec(x_25); 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_inc(x_26); +lean_dec(x_23); +lean_ctor_set(x_22, 0, x_26); +return x_22; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_23, 1); +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); -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; +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_31; lean_object* x_32; size_t x_33; size_t x_34; -x_31 = lean_ctor_get(x_23, 1); +lean_object* x_30; lean_object* x_31; size_t x_32; size_t x_33; +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); -x_32 = lean_ctor_get(x_24, 0); -lean_inc(x_32); -lean_dec(x_24); -x_33 = 1; -x_34 = lean_usize_add(x_7, x_33); -x_7 = x_34; -x_8 = x_32; -x_13 = x_31; +x_32 = 1; +x_33 = lean_usize_add(x_6, x_32); +x_6 = x_33; +x_7 = x_31; +x_12 = x_30; goto _start; } } else { -uint8_t x_36; -lean_dec(x_12); +uint8_t x_35; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_2); -x_36 = !lean_is_exclusive(x_23); -if (x_36 == 0) +lean_dec(x_8); +lean_dec(x_1); +x_35 = !lean_is_exclusive(x_22); +if (x_35 == 0) { -return x_23; +return x_22; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_23, 0); -x_38 = lean_ctor_get(x_23, 1); -lean_inc(x_38); +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_22, 0); +x_37 = lean_ctor_get(x_22, 1); lean_inc(x_37); -lean_dec(x_23); -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_inc(x_36); +lean_dec(x_22); +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_mapIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___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, lean_object* x_8, lean_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_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___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, lean_object* x_8, 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; @@ -18619,7 +18619,7 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_2); -x_22 = l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10(x_1, x_2, x_3, x_7, x_4, x_19, x_20, x_21, x_10, x_11, x_12, x_13, x_14); +x_22 = l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10(x_2, x_3, x_7, x_4, x_19, x_20, x_21, x_10, x_11, x_12, x_13, x_14); if (lean_obj_tag(x_22) == 0) { lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; @@ -18693,7 +18693,7 @@ lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_10 = lean_array_get_size(x_1); x_11 = lean_mk_empty_array_with_capacity(x_10); x_12 = lean_unsigned_to_nat(0u); -x_13 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__11(x_1, x_2, x_3, x_4, x_1, x_10, x_12, lean_box(0), x_11, x_5, x_6, x_7, x_8, x_9); +x_13 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__11(x_1, x_2, x_3, x_4, x_1, x_10, x_12, lean_box(0), x_11, x_5, x_6, x_7, x_8, x_9); return x_13; } } @@ -18920,27 +18920,26 @@ lean_dec(x_3); return x_12; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___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_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___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_object* x_11, lean_object* x_12) { _start: { -size_t x_14; size_t x_15; lean_object* x_16; +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 = lean_unbox_usize(x_7); -lean_dec(x_7); -x_16 = l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10(x_1, x_2, x_3, x_4, x_5, x_14, x_15, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_5); +x_15 = l_Array_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__10(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_1); -return x_16; +lean_dec(x_2); +return x_15; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___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_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___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_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; -x_15 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__11(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_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_complexMeasures___spec__11(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_4); lean_dec(x_3); @@ -22629,7 +22628,7 @@ if (x_10 == 0) { lean_object* x_50; lean_object* x_51; lean_dec(x_6); -x_50 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_50 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_51 = l_outOfBounds___rarg(x_50); x_14 = x_51; goto block_49; @@ -22650,7 +22649,7 @@ if (x_12 == 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_dec(x_11); -x_16 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_16 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_17 = l_outOfBounds___rarg(x_16); x_18 = lean_array_get_size(x_17); x_19 = lean_mk_array(x_18, x_5); @@ -22828,7 +22827,7 @@ if (x_50 == 0) { lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; lean_dec(x_12); -x_51 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_51 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_52 = l_outOfBounds___rarg(x_51); x_53 = lean_array_get_size(x_52); x_54 = lean_nat_dec_lt(x_3, x_53); @@ -23094,7 +23093,7 @@ if (x_106 == 0) { lean_object* x_107; lean_object* x_108; lean_object* x_109; uint8_t x_110; lean_dec(x_70); -x_107 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_107 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_108 = l_outOfBounds___rarg(x_107); x_109 = lean_array_get_size(x_108); x_110 = lean_nat_dec_lt(x_3, x_109); @@ -23392,7 +23391,7 @@ if (x_46 == 0) { lean_object* x_47; lean_object* x_48; lean_dec(x_11); -x_47 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_47 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_48 = l_outOfBounds___rarg(x_47); x_15 = x_48; goto block_44; @@ -25867,7 +25866,7 @@ lean_ctor_set(x_7, 2, x_6); if (x_4 == 0) { lean_object* x_15; lean_object* x_16; -x_15 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_15 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_16 = l_outOfBounds___rarg(x_15); x_8 = x_16; goto block_14; @@ -28549,7 +28548,7 @@ lean_ctor_set(x_51, 1, x_29); if (x_32 == 0) { lean_object* x_167; lean_object* x_168; -x_167 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_167 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_168 = l_outOfBounds___rarg(x_167); x_52 = x_168; goto block_166; @@ -28579,7 +28578,7 @@ x_58 = lean_nat_dec_lt(x_18, 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; -x_59 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_59 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_60 = l_outOfBounds___rarg(x_59); x_61 = lean_array_get_size(x_60); lean_dec(x_60); @@ -28693,7 +28692,7 @@ lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean x_85 = lean_array_fget(x_2, x_18); x_86 = lean_array_get_size(x_85); lean_dec(x_85); -x_87 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_87 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_88 = lean_unsigned_to_nat(0u); x_89 = lean_unsigned_to_nat(1u); lean_inc(x_86); @@ -28811,7 +28810,7 @@ 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; lean_object* x_122; lean_object* x_123; lean_dec(x_17); -x_113 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_113 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_114 = l_outOfBounds___rarg(x_113); x_115 = lean_array_get_size(x_114); lean_dec(x_114); @@ -29124,7 +29123,7 @@ lean_ctor_set(x_209, 1, x_187); if (x_190 == 0) { lean_object* x_317; lean_object* x_318; -x_317 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_317 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_318 = l_outOfBounds___rarg(x_317); x_210 = x_318; goto block_316; @@ -29154,7 +29153,7 @@ x_216 = lean_nat_dec_lt(x_18, x_215); if (x_216 == 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; lean_object* x_224; lean_object* x_225; lean_object* x_226; -x_217 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_217 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_218 = l_outOfBounds___rarg(x_217); x_219 = lean_array_get_size(x_218); lean_dec(x_218); @@ -29265,7 +29264,7 @@ lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; x_241 = lean_array_fget(x_2, x_18); x_242 = lean_array_get_size(x_241); lean_dec(x_241); -x_243 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_243 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_244 = lean_unsigned_to_nat(0u); x_245 = lean_unsigned_to_nat(1u); lean_inc(x_242); @@ -29380,7 +29379,7 @@ if (x_266 == 0) { 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_dec(x_17); -x_267 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_267 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_268 = l_outOfBounds___rarg(x_267); x_269 = lean_array_get_size(x_268); lean_dec(x_268); @@ -30232,7 +30231,7 @@ if (x_28 == 0) { lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_dec(x_2); -x_29 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_29 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_30 = l_outOfBounds___rarg(x_29); x_31 = l_Lean_Elab_WF_GuessLex_explainNonMutualFailure(x_30, x_3, x_4, x_5, x_6, x_7, x_8); if (lean_obj_tag(x_31) == 0) @@ -30874,7 +30873,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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) { _start: { lean_object* x_8; @@ -30986,7 +30985,7 @@ return x_31; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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) { _start: { lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; size_t x_19; size_t x_20; lean_object* x_21; lean_object* x_22; @@ -31002,7 +31001,7 @@ x_19 = lean_array_size(x_4); x_20 = 0; lean_inc(x_7); x_21 = l_Array_mapMUnsafe_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__1(x_3, x_5, x_7, x_19, x_20, x_4); -x_22 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__1), 7, 2); +x_22 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__1), 7, 2); lean_closure_set(x_22, 0, x_21); lean_closure_set(x_22, 1, x_7); if (x_18 == 0) @@ -31024,7 +31023,7 @@ return x_26; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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: { lean_object* x_16; uint8_t x_17; @@ -31046,7 +31045,7 @@ lean_dec(x_20); if (x_22 == 0) { lean_object* x_39; lean_object* x_40; -x_39 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_39 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; x_40 = l_outOfBounds___rarg(x_39); x_24 = x_40; goto block_38; @@ -31061,12 +31060,12 @@ goto block_38; block_38: { lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; -x_25 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; +x_25 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1; lean_inc(x_5); lean_inc(x_8); lean_inc(x_3); lean_inc(x_2); -x_26 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__2___boxed), 13, 6); +x_26 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2___lambda__2___boxed), 13, 6); lean_closure_set(x_26, 0, x_2); lean_closure_set(x_26, 1, x_3); lean_closure_set(x_26, 2, x_8); @@ -31157,7 +31156,7 @@ lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_11 = lean_array_get_size(x_1); x_12 = lean_mk_empty_array_with_capacity(x_11); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2(x_1, x_2, x_3, x_4, x_5, x_1, x_11, x_13, lean_box(0), x_12, x_6, x_7, x_8, x_9, x_10); +x_14 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___spec__2(x_1, x_2, x_3, x_4, x_5, x_1, x_11, x_13, lean_box(0), x_12, x_6, x_7, x_8, x_9, x_10); return x_14; } } @@ -31175,11 +31174,11 @@ lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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) { _start: { lean_object* x_14; -x_14 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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); lean_dec(x_8); lean_dec(x_5); lean_dec(x_3); @@ -31187,11 +31186,11 @@ lean_dec(x_2); return x_14; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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, lean_object* x_14, lean_object* x_15) { _start: { lean_object* x_16; -x_16 = l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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 = l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_toTerminationArguments___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); lean_dec(x_6); lean_dec(x_4); lean_dec(x_1); @@ -35204,8 +35203,8 @@ l_Subarray_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__1_ lean_mark_persistent(l_Subarray_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__1___closed__1); l_Subarray_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__1___closed__2 = _init_l_Subarray_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__1___closed__2(); lean_mark_persistent(l_Subarray_forInUnsafe_loop___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__1___closed__2); -l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1 = _init_l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1); +l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_WF_GuessLex_simpleMeasures___spec__2___lambda__2___closed__1); l_Lean_Elab_WF_GuessLex_withRecApps_processRec___rarg___closed__1 = _init_l_Lean_Elab_WF_GuessLex_withRecApps_processRec___rarg___closed__1(); lean_mark_persistent(l_Lean_Elab_WF_GuessLex_withRecApps_processRec___rarg___closed__1); l_Lean_getConstInfo___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__3___rarg___closed__1 = _init_l_Lean_getConstInfo___at_Lean_Elab_WF_GuessLex_withRecApps_loop___spec__3___rarg___closed__1(); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/WF/Main.c b/stage0/stdlib/Lean/Elab/PreDefinition/WF/Main.c index 30022192c2b0..4f5f5d88f089 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/WF/Main.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/WF/Main.c @@ -7087,7 +7087,7 @@ lean_dec(x_33); x_35 = lean_ctor_get(x_15, 2); lean_inc(x_35); lean_dec(x_15); -x_36 = lean_ctor_get(x_35, 1); +x_36 = lean_ctor_get(x_35, 2); lean_inc(x_36); lean_dec(x_35); x_37 = lean_array_get_size(x_36); @@ -7244,7 +7244,7 @@ lean_dec(x_66); x_68 = lean_ctor_get(x_15, 2); lean_inc(x_68); lean_dec(x_15); -x_69 = lean_ctor_get(x_68, 1); +x_69 = lean_ctor_get(x_68, 2); lean_inc(x_69); lean_dec(x_68); x_70 = lean_array_get_size(x_69); diff --git a/stage0/stdlib/Lean/Elab/Quotation.c b/stage0/stdlib/Lean/Elab/Quotation.c index e6ec4af0a445..24d5a2676fae 100644 --- a/stage0/stdlib/Lean/Elab/Quotation.c +++ b/stage0/stdlib/Lean/Elab/Quotation.c @@ -128,13 +128,14 @@ static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_ static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__38; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_elabNoErrorIfUnused(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_of_nat(lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___lambda__1___closed__28; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__7; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__14___closed__6; lean_object* l_Lean_Elab_Term_elabTerm(lean_object*, 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_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__15(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*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quotation___hyg_16962____closed__10; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__27___closed__3; LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -772,7 +773,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quota static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__12___closed__1; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getSepStxFromSplice___closed__9; static lean_object* l_Lean_Elab_Term_Quotation_commandElab__stx__quot_____closed__11; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6440____closed__2; LEAN_EXPORT lean_object* l_Lean_resolveNamespaceCore___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__26___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_Elab_Quotation_0__Lean_Elab_Term_Quotation_deduplicate(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -832,6 +833,7 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_ LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__20___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_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6426____closed__2; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__3___closed__17; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__23___lambda__2___closed__9; static lean_object* l___private_Init_Meta_0__Lean_quoteList___at_Lean_Elab_Term_Quotation_ArrayStxBuilder_build___spec__2___closed__6; 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_365____spec__1(lean_object*, lean_object*); @@ -974,7 +976,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quota lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__13___rarg(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__11___closed__3; static lean_object* l_Lean_Elab_Term_Quotation_mkTuple___closed__12; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_mkSyntaxQuotation___closed__18; lean_object* l_Substring_prevn(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_Quotation_mkTuple___closed__10; @@ -1019,7 +1020,6 @@ static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation_____ static lean_object* l_Lean_Elab_Term_Quotation_getQuotKind___closed__16; lean_object* l_Lean_Syntax_antiquotSpliceKind_x3f(lean_object*); lean_object* l_Array_mkArray1___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot__1____x40_Lean_Elab_Quotation___hyg_6419____closed__3; static lean_object* l_Lean_Elab_Term_Quotation_mkTuple___closed__13; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -21006,7 +21006,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___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) { _start: { lean_object* x_9; uint8_t x_10; @@ -26338,53 +26338,53 @@ return x_36; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___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_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13(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_6) == 2) +if (lean_obj_tag(x_5) == 2) { -lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_7 = lean_ctor_get(x_6, 0); -x_8 = lean_ctor_get(x_6, 1); -x_9 = lean_nat_dec_eq(x_7, x_1); -if (x_9 == 0) +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = lean_ctor_get(x_5, 0); +x_7 = lean_ctor_get(x_5, 1); +x_8 = lean_nat_dec_eq(x_6, x_1); +if (x_8 == 0) { -lean_object* x_10; -x_10 = lean_box(1); -return x_10; +lean_object* x_9; +x_9 = lean_box(1); +return x_9; } else { -uint8_t x_11; -x_11 = lean_nat_dec_eq(x_8, x_2); -if (x_11 == 0) +uint8_t x_10; +x_10 = lean_nat_dec_eq(x_7, x_2); +if (x_10 == 0) { -lean_object* x_12; -x_12 = lean_box(1); -return x_12; +lean_object* x_11; +x_11 = lean_box(1); +return x_11; } else { -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; -x_13 = lean_array_get_size(x_3); -x_14 = lean_mk_empty_array_with_capacity(x_13); -x_15 = lean_unsigned_to_nat(0u); -x_16 = l_Array_mapIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6(x_4, x_5, x_1, x_3, x_13, x_15, lean_box(0), x_14); -x_17 = lean_alloc_closure((void*)(l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__11___boxed), 9, 1); -lean_closure_set(x_17, 0, x_16); -x_18 = 1; -x_19 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set_uint8(x_19, sizeof(void*)*1, x_18); -return x_19; +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; +x_12 = lean_array_get_size(x_3); +x_13 = lean_mk_empty_array_with_capacity(x_12); +x_14 = lean_unsigned_to_nat(0u); +x_15 = l_Array_mapFinIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6(x_4, x_3, x_1, x_3, x_12, x_14, lean_box(0), x_13); +x_16 = lean_alloc_closure((void*)(l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__11___boxed), 9, 1); +lean_closure_set(x_16, 0, x_15); +x_17 = 1; +x_18 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set_uint8(x_18, sizeof(void*)*1, x_17); +return x_18; } } } else { -lean_object* x_20; -x_20 = lean_box(2); -return x_20; +lean_object* x_19; +x_19 = lean_box(2); +return x_19; } } } @@ -34655,6 +34655,7 @@ x_49 = lean_ctor_get(x_20, 0); lean_inc(x_49); lean_dec(x_20); x_50 = l_Lean_Syntax_getNumArgs(x_1); +lean_dec(x_1); x_51 = lean_unsigned_to_nat(1u); x_52 = lean_nat_sub(x_50, x_51); lean_dec(x_50); @@ -34667,12 +34668,11 @@ lean_ctor_set(x_54, 1, x_53); lean_inc(x_2); lean_inc(x_53); lean_inc(x_49); -x_55 = lean_alloc_closure((void*)(l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13___boxed), 6, 5); +x_55 = lean_alloc_closure((void*)(l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13___boxed), 5, 4); lean_closure_set(x_55, 0, x_49); lean_closure_set(x_55, 1, x_53); lean_closure_set(x_55, 2, x_16); lean_closure_set(x_55, 3, x_2); -lean_closure_set(x_55, 4, x_1); x_56 = lean_alloc_closure((void*)(l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__14___boxed), 14, 5); lean_closure_set(x_56, 0, x_49); lean_closure_set(x_56, 1, x_2); @@ -35608,11 +35608,11 @@ x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___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: { lean_object* x_9; -x_9 = l_Array_mapIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Array_mapFinIdxM_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -35904,18 +35904,17 @@ x_8 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___ return x_8; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___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_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13___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_7; -x_7 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_6); +lean_object* x_6; +x_6 = l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__13(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_7; +return x_6; } } LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___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) { diff --git a/stage0/stdlib/Lean/Elab/StructInst.c b/stage0/stdlib/Lean/Elab/StructInst.c index 09b45eca86c1..8bbc4164e26f 100644 --- a/stage0/stdlib/Lean/Elab/StructInst.c +++ b/stage0/stdlib/Lean/Elab/StructInst.c @@ -34,7 +34,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_Stru LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_mkProjStx_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_Elab_Term_StructInst_DefaultFields_tryToSynthesizeDefault_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_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getFieldIdx___lambda__1(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__11; static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev_declRange__1___closed__1; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStructInstAux___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_Term_StructInst_Struct_structName___boxed(lean_object*); @@ -48,7 +47,9 @@ static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___la static lean_object* l_Lean_Elab_Term_StructInst_formatField___closed__4; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_elabStructInst__1___closed__4; +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__5; LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_Term_StructInst_DefaultFields_collectStructNames___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__14; LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___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_mk_empty_array_with_capacity(lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); @@ -69,6 +70,7 @@ LEAN_EXPORT lean_object* l_Lean_MVarId_isAssigned___at_Lean_Elab_Term_StructInst lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Format_joinSep___at_Lean_Elab_Term_StructInst_formatField___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Term_StructInst_DefaultFields_step___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_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__7; LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_Term_StructInst_formatStruct___spec__5(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkCtorHeaderAux___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev__1(lean_object*); @@ -184,7 +186,6 @@ 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_Lean_Elab_Term_StructInst_DefaultFields_mkDefaultValueAux_x3f___lambda__2(lean_object*, lean_object*, lean_object*, 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_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__2; static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___lambda__1___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_toFieldLHS___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_isDefaultMissing_x3f___at_Lean_Elab_Term_StructInst_DefaultFields_allDefaultMissing_go___spec__1___rarg___lambda__2(lean_object*, lean_object*); @@ -227,7 +228,6 @@ LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_StructInst static lean_object* l_List_format___at_Lean_Elab_Term_StructInst_formatStruct___spec__3___closed__1; lean_object* l_Lean_stringToMessageData(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_Struct_structName(lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__8; LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructSource___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___lambda__1___closed__2; uint8_t l___private_Lean_Util_Trace_0__Lean_checkTraceOption(lean_object*, lean_object*, lean_object*); @@ -266,7 +266,6 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at___priv lean_object* l_Lean_getStructureFields(lean_object*, lean_object*); extern lean_object* l_instInhabitedPUnit; lean_object* l_Lean_Meta_project_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__14; lean_object* l_Lean_getDefaultFnForField_x3f(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_isModifyOp_x3f___spec__3___closed__1; static lean_object* l_List_mapM_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_groupFields___spec__6___closed__1; @@ -300,15 +299,12 @@ static lean_object* l_Lean_Elab_Term_StructInst_instInhabitedField___closed__1; lean_object* l_Lean_Meta_mkFreshLevelMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_getFieldValue_x3f(lean_object*, lean_object*); static lean_object* l_List_foldlM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___spec__5___lambda__1___closed__4; -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__13; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStructInstAux___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_Elab_Term_StructInst_instInhabitedField(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNonAtomicExplicitSources___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_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__9; static lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_mkDefaultValueAux_x3f___closed__3; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructSource___spec__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___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_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__7; LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_Term_StructInst_formatField___spec__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_findDefaultMissing_x3f___at_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop___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_addTrace___at_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop___spec__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -334,7 +330,6 @@ LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Term_StructInst_Defaul lean_object* l_Array_contains___at_Lean_findField_x3f___spec__1___boxed(lean_object*, lean_object*); 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*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_groupFields(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__1; LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_groupFields___spec__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* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev_declRange__1___closed__6; @@ -354,6 +349,7 @@ LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_StructInst_0_ lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandParentFields___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* l_Lean_Core_instantiateValueLevelParams(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__10; LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_tryToSynthesizeDefault_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*, lean_object*, lean_object*); lean_object* lean_nat_to_int(lean_object*); lean_object* l_List_findSome_x3f___rarg(lean_object*, lean_object*); @@ -378,6 +374,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_Struct_setParams(lean_objec LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_reduce___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); 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_List_mapM_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_groupFields___spec__6___closed__2; +static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__8; lean_object* l_Lean_Elab_Term_elabTerm___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_StructInst_expandStructInstFieldAbbrev___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Term_StructInst_DefaultFields_allDefaultMissing_go___spec__5___rarg___lambda__4(lean_object*, lean_object*); @@ -393,6 +390,7 @@ lean_object* l_Lean_MessageData_ofFormat(lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_Term_StructInst_DefaultFields_getHierarchyDepth___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Elab_getBetterRef(lean_object*, lean_object*); uint8_t l_Lean_Expr_isMVar(lean_object*); +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructName_throwUnexpectedExpectedType(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_StructInst_Struct_allDefault___closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_groupFields___spec__5___boxed(lean_object*, lean_object*); @@ -451,6 +449,7 @@ LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_StructInst_0 static lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop___lambda__1___closed__2; static lean_object* l_Lean_Elab_Term_StructInst_markDefaultMissing___closed__2; uint8_t l_Lean_Syntax_isMissing(lean_object*); +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__12; static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_toFieldLHS___closed__1; LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop___spec__12(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__22; @@ -492,6 +491,7 @@ static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_StructIns LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_groupFields___spec__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_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandCompositeFields___spec__2(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getSepArgs(lean_object*); +static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__10; lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__24; LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___boxed(lean_object*, lean_object*, lean_object*); @@ -557,6 +557,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_allDefaultMis static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_isModifyOp_x3f___spec__3___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_propagateExpectedType___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_StructInst_formatStruct___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316_(lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__7; static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__5; LEAN_EXPORT lean_object* l_Lean_MVarId_isAssigned___at_Lean_Elab_Term_StructInst_DefaultFields_allDefaultMissing_go___spec__4(lean_object*); @@ -579,6 +580,7 @@ static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructIns static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructSource___spec__2___closed__2; static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___lambda__1___closed__4; extern lean_object* l_Lean_inheritedTraceOptions; +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_Struct_modifyFieldsM(lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); static lean_object* l_List_mapM_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandParentFields___spec__3___closed__1; @@ -639,9 +641,9 @@ LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_StructInst_0 LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_instToFormatFieldStruct; static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_isDefaultMissing_x3f___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__4; static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev_declRange__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstExpectedType__1(lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__4; static lean_object* l_List_foldlM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___spec__5___closed__4; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructSource___spec__2___closed__4; static lean_object* l_List_format___at_Lean_Elab_Term_StructInst_formatStruct___spec__3___closed__2; @@ -662,7 +664,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_isDefaultMiss lean_object* l_Lean_Syntax_SepArray_ofElems(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructName___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_Term_StructInst_elabStructInst(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_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__12; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_instToStringStruct___closed__1; lean_object* lean_environment_main_module(lean_object*); @@ -674,12 +675,12 @@ LEAN_EXPORT lean_object* l_List_findSomeM_x3f___at_Lean_Elab_Term_StructInst_Def LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_Struct_source(lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__14; static lean_object* l_List_mapM_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNumLitFields___spec__3___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_mkProjStx_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* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l_List_foldlM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkFieldMap___spec__10___closed__4; uint8_t l_Lean_isPrivateNameFromImportedModule(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstExpectedType_declRange__1___closed__2; +static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__9; static lean_object* l_List_mapM_loop___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNumLitFields___spec__3___closed__4; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkFieldMap___spec__9(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkCtorHeaderAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -776,7 +777,6 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_StructInst_0 LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_tryToSynthesizeDefault___boxed(lean_object*, lean_object*, lean_object*, 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_StructInst_DefaultFields_isDefaultMissing_x3f(lean_object*); lean_object* l_String_intercalate(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__6; size_t lean_usize_sub(size_t, size_t); lean_object* lean_array_mk(lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_instInhabitedStruct___closed__1; @@ -785,6 +785,7 @@ LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Term_StructInst_Defa LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNonAtomicExplicitSources___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___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__15; LEAN_EXPORT lean_object* l_Lean_MVarId_isAssigned___at_Lean_Elab_Term_StructInst_DefaultFields_allDefaultMissing_go___spec__2(lean_object*); +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__11; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStructInstAux___spec__1___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_isDefaultMissing_x3f___rarg___lambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__12; @@ -813,7 +814,7 @@ LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_StructIn LEAN_EXPORT lean_object* l_List_foldlM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___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_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_allDefaultMissing_go(lean_object*); size_t lean_array_size(lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__10; +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__13; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___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_Elab_Term_StructInst_DefaultFields_reduce(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__23; @@ -822,7 +823,6 @@ static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructIns lean_object* l_instInhabitedOfMonad___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_formatStruct___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_mkDefaultValueAux_x3f___lambda__3___boxed(lean_object*); -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__5; extern lean_object* l_Lean_instInhabitedSyntax; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___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*); @@ -850,10 +850,12 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_Struct_params(lean_object*) LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___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_array_get_size(lean_object*); lean_object* l_panic___at___private_Init_Prelude_0__Lean_assembleParts___spec__1(lean_object*); +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNumLitFields___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_Term_StructInst_throwFailedToElabField___rarg___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_instInhabitedSource; LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_instToStringStruct___lambda__1(lean_object*); +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__8; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop___spec__11(lean_object*, lean_object*, lean_object*, size_t, size_t); static lean_object* l_List_format___at_Lean_Elab_Term_StructInst_formatStruct___spec__3___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_formatStruct(lean_object*); @@ -875,10 +877,10 @@ LEAN_EXPORT lean_object* l_Lean_MVarId_isAssigned___at_Lean_Elab_Term_StructInst LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_404_(uint8_t, uint8_t); static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStructInstAux___spec__5___rarg___closed__2; -static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__3; 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___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructName___boxed(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_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__1; static lean_object* l_Lean_Elab_Term_StructInst_formatStruct___closed__6; static lean_object* l_Lean_Elab_Term_StructInst_FieldVal_toSyntax___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_groupFields___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -902,6 +904,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstExp lean_object* l_Lean_getStructureFieldsFlattened(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_groupFields___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_Expr_mvarId_x21(lean_object*); +static lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__6; static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_elabStructInst_declRange__1___closed__7; lean_object* l_String_toSubstring_x27(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -5079,7 +5082,7 @@ static lean_object* _init_l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_Str _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("modifyOp", 8, 8); +x_1 = lean_mk_string_unchecked("modify", 6, 6); return x_1; } } @@ -5126,7 +5129,7 @@ static lean_object* _init_l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_Str _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("idx", 3, 3); +x_1 = lean_mk_string_unchecked("i", 1, 1); return x_1; } } @@ -5273,26 +5276,26 @@ lean_inc(x_28); x_29 = lean_st_ref_get(x_17, x_18); if (x_24 == 0) { -lean_object* x_171; lean_object* x_172; -x_171 = l_Lean_Elab_Term_StructInst_instInhabitedExplicitSourceInfo; -x_172 = l_outOfBounds___rarg(x_171); -x_30 = x_172; -goto block_170; +lean_object* x_175; lean_object* x_176; +x_175 = l_Lean_Elab_Term_StructInst_instInhabitedExplicitSourceInfo; +x_176 = l_outOfBounds___rarg(x_175); +x_30 = x_176; +goto block_174; } else { -lean_object* x_173; -x_173 = lean_array_fget(x_2, x_19); -x_30 = x_173; -goto block_170; +lean_object* x_177; +x_177 = lean_array_fget(x_2, x_19); +x_30 = x_177; +goto block_174; } -block_170: +block_174: { uint8_t x_31; x_31 = !lean_is_exclusive(x_29); 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; 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; uint8_t x_76; +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; uint8_t x_78; x_32 = lean_ctor_get(x_29, 0); x_33 = lean_ctor_get(x_29, 1); x_34 = lean_ctor_get(x_30, 0); @@ -5311,349 +5314,363 @@ x_38 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyO lean_inc(x_28); lean_inc(x_36); x_39 = l_Lean_addMacroScope(x_36, x_38, x_28); -x_40 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__7; lean_inc(x_3); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_3); +lean_inc(x_3); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_3); +x_42 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__7; lean_inc(x_27); -x_41 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_41, 0, x_27); -lean_ctor_set(x_41, 1, x_40); -lean_ctor_set(x_41, 2, x_39); -lean_ctor_set(x_41, 3, x_3); -x_42 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__4; +x_43 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_43, 0, x_27); +lean_ctor_set(x_43, 1, x_42); +lean_ctor_set(x_43, 2, x_39); +lean_ctor_set(x_43, 3, x_41); +x_44 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__4; lean_inc(x_27); -x_43 = l_Lean_Syntax_node3(x_27, x_42, x_34, x_29, x_41); -x_44 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__10; +x_45 = l_Lean_Syntax_node3(x_27, x_44, x_34, x_29, x_43); +x_46 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__10; lean_inc(x_27); -x_45 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_45, 0, x_27); -lean_ctor_set(x_45, 1, x_44); -x_46 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__13; +x_47 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_47, 0, x_27); +lean_ctor_set(x_47, 1, x_46); +x_48 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__13; lean_inc(x_28); lean_inc(x_36); -x_47 = l_Lean_addMacroScope(x_36, x_46, x_28); -x_48 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__12; +x_49 = l_Lean_addMacroScope(x_36, x_48, x_28); +x_50 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__12; lean_inc(x_3); lean_inc(x_27); -x_49 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_49, 0, x_27); -lean_ctor_set(x_49, 1, x_48); -lean_ctor_set(x_49, 2, x_47); -lean_ctor_set(x_49, 3, x_3); -x_50 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___spec__2___closed__5; -lean_inc(x_27); -x_51 = lean_alloc_ctor(2, 2, 0); +x_51 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_51, 0, x_27); lean_ctor_set(x_51, 1, x_50); -x_52 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__12; +lean_ctor_set(x_51, 2, x_49); +lean_ctor_set(x_51, 3, x_3); +x_52 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___spec__2___closed__5; lean_inc(x_27); x_53 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_53, 0, x_27); lean_ctor_set(x_53, 1, x_52); -x_54 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__10; -lean_inc(x_53); -lean_inc(x_45); +x_54 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__12; lean_inc(x_27); -x_55 = l_Lean_Syntax_node5(x_27, x_54, x_45, x_49, x_51, x_22, x_53); -x_56 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__16; +x_55 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_55, 0, x_27); +lean_ctor_set(x_55, 1, x_54); +x_56 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__10; +lean_inc(x_55); +lean_inc(x_47); lean_inc(x_27); -x_57 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_57, 0, x_27); -lean_ctor_set(x_57, 1, x_56); -x_58 = l_Lean_addMacroScope(x_36, x_4, x_28); +x_57 = l_Lean_Syntax_node5(x_27, x_56, x_47, x_51, x_53, x_22, x_55); +x_58 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__16; lean_inc(x_27); -x_59 = lean_alloc_ctor(3, 4, 0); +x_59 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_59, 0, x_27); -lean_ctor_set(x_59, 1, x_5); -lean_ctor_set(x_59, 2, x_58); -lean_ctor_set(x_59, 3, x_3); -lean_inc(x_6); +lean_ctor_set(x_59, 1, x_58); +x_60 = l_Lean_addMacroScope(x_36, x_4, x_28); lean_inc(x_27); -x_60 = l_Lean_Syntax_node1(x_27, x_6, x_59); -x_61 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__1; +x_61 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_61, 0, x_27); +lean_ctor_set(x_61, 1, x_5); +lean_ctor_set(x_61, 2, x_60); +lean_ctor_set(x_61, 3, x_3); lean_inc(x_6); lean_inc(x_27); -x_62 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_62, 0, x_27); -lean_ctor_set(x_62, 1, x_6); -lean_ctor_set(x_62, 2, x_61); -x_63 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__20; +x_62 = l_Lean_Syntax_node1(x_27, x_6, x_61); +x_63 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__1; +lean_inc(x_6); lean_inc(x_27); -x_64 = lean_alloc_ctor(2, 2, 0); +x_64 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_64, 0, x_27); -lean_ctor_set(x_64, 1, x_63); -x_65 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__19; +lean_ctor_set(x_64, 1, x_6); +lean_ctor_set(x_64, 2, x_63); +x_65 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__20; +lean_inc(x_27); +x_66 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_66, 0, x_27); +lean_ctor_set(x_66, 1, x_65); +x_67 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__19; lean_inc(x_27); -x_66 = l_Lean_Syntax_node4(x_27, x_65, x_60, x_62, x_64, x_7); -x_67 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__17; +x_68 = l_Lean_Syntax_node4(x_27, x_67, x_62, x_64, x_66, x_7); +x_69 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__17; lean_inc(x_27); -x_68 = l_Lean_Syntax_node2(x_27, x_67, x_57, x_66); -x_69 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__15; +x_70 = l_Lean_Syntax_node2(x_27, x_69, x_59, x_68); +x_71 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__15; lean_inc(x_27); -x_70 = l_Lean_Syntax_node3(x_27, x_69, x_45, x_68, x_53); +x_72 = l_Lean_Syntax_node3(x_27, x_71, x_47, x_70, x_55); lean_inc(x_27); -x_71 = l_Lean_Syntax_node2(x_27, x_6, x_55, x_70); -x_72 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__2; -x_73 = l_Lean_Syntax_node2(x_27, x_72, x_43, x_71); +x_73 = l_Lean_Syntax_node2(x_27, x_6, x_57, x_72); +x_74 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__2; +x_75 = l_Lean_Syntax_node2(x_27, x_74, x_45, x_73); lean_inc(x_8); -x_74 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_8, x_12, x_13, x_14, x_15, x_16, x_17, x_33); -x_75 = lean_ctor_get(x_74, 0); -lean_inc(x_75); -x_76 = lean_unbox(x_75); -lean_dec(x_75); -if (x_76 == 0) +x_76 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_8, x_12, x_13, x_14, x_15, x_16, x_17, x_33); +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_77; lean_object* x_78; lean_object* x_79; +lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_dec(x_8); -x_77 = lean_ctor_get(x_74, 1); -lean_inc(x_77); -lean_dec(x_74); -x_78 = lean_box(0); -x_79 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_73, x_9, x_10, x_78, x_12, x_13, x_14, x_15, x_16, x_17, x_77); -return x_79; +x_79 = lean_ctor_get(x_76, 1); +lean_inc(x_79); +lean_dec(x_76); +x_80 = lean_box(0); +x_81 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_75, x_9, x_10, x_80, x_12, x_13, x_14, x_15, x_16, x_17, x_79); +return x_81; } else { -uint8_t x_80; -x_80 = !lean_is_exclusive(x_74); -if (x_80 == 0) +uint8_t x_82; +x_82 = !lean_is_exclusive(x_76); +if (x_82 == 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; lean_object* x_92; lean_object* x_93; -x_81 = lean_ctor_get(x_74, 1); -x_82 = lean_ctor_get(x_74, 0); -lean_dec(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_83 = lean_ctor_get(x_76, 1); +x_84 = lean_ctor_get(x_76, 0); +lean_dec(x_84); lean_inc(x_10); -x_83 = l_Lean_MessageData_ofSyntax(x_10); -x_84 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__22; -lean_ctor_set_tag(x_74, 7); -lean_ctor_set(x_74, 1, x_83); -lean_ctor_set(x_74, 0, x_84); -x_85 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__24; -x_86 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_86, 0, x_74); -lean_ctor_set(x_86, 1, x_85); -lean_inc(x_73); -x_87 = l_Lean_MessageData_ofSyntax(x_73); +x_85 = l_Lean_MessageData_ofSyntax(x_10); +x_86 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__22; +lean_ctor_set_tag(x_76, 7); +lean_ctor_set(x_76, 1, x_85); +lean_ctor_set(x_76, 0, x_86); +x_87 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__24; x_88 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_88, 0, x_86); +lean_ctor_set(x_88, 0, x_76); lean_ctor_set(x_88, 1, x_87); -x_89 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_89, 0, x_88); -lean_ctor_set(x_89, 1, x_84); -x_90 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_8, x_89, x_12, x_13, x_14, x_15, x_16, x_17, x_81); -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___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_73, x_9, x_10, x_91, x_12, x_13, x_14, x_15, x_16, x_17, x_92); -lean_dec(x_91); -return x_93; +lean_inc(x_75); +x_89 = l_Lean_MessageData_ofSyntax(x_75); +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_86); +x_92 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_8, x_91, x_12, x_13, x_14, x_15, x_16, x_17, x_83); +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_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_75, x_9, x_10, x_93, x_12, x_13, x_14, x_15, x_16, x_17, x_94); +lean_dec(x_93); +return x_95; } 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; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; -x_94 = lean_ctor_get(x_74, 1); -lean_inc(x_94); -lean_dec(x_74); +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_96 = lean_ctor_get(x_76, 1); +lean_inc(x_96); +lean_dec(x_76); lean_inc(x_10); -x_95 = l_Lean_MessageData_ofSyntax(x_10); -x_96 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__22; -x_97 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_97, 0, x_96); -lean_ctor_set(x_97, 1, x_95); -x_98 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__24; +x_97 = l_Lean_MessageData_ofSyntax(x_10); +x_98 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__22; x_99 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_99, 0, x_97); -lean_ctor_set(x_99, 1, x_98); -lean_inc(x_73); -x_100 = l_Lean_MessageData_ofSyntax(x_73); +lean_ctor_set(x_99, 0, x_98); +lean_ctor_set(x_99, 1, x_97); +x_100 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__24; 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 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_102, 0, x_101); -lean_ctor_set(x_102, 1, x_96); -x_103 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_8, x_102, x_12, x_13, x_14, x_15, x_16, x_17, x_94); -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 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_73, x_9, x_10, x_104, x_12, x_13, x_14, x_15, x_16, x_17, x_105); -lean_dec(x_104); -return x_106; +lean_inc(x_75); +x_102 = l_Lean_MessageData_ofSyntax(x_75); +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 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_104, 0, x_103); +lean_ctor_set(x_104, 1, x_98); +x_105 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_8, x_104, x_12, x_13, x_14, x_15, x_16, x_17, x_96); +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___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_75, x_9, x_10, x_106, x_12, x_13, x_14, x_15, x_16, x_17, x_107); +lean_dec(x_106); +return x_108; } } } 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; 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; uint8_t x_152; -x_107 = lean_ctor_get(x_29, 0); -x_108 = lean_ctor_get(x_29, 1); -lean_inc(x_108); -lean_inc(x_107); -lean_dec(x_29); -x_109 = lean_ctor_get(x_30, 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; 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; uint8_t x_156; +x_109 = lean_ctor_get(x_29, 0); +x_110 = lean_ctor_get(x_29, 1); +lean_inc(x_110); lean_inc(x_109); +lean_dec(x_29); +x_111 = lean_ctor_get(x_30, 0); +lean_inc(x_111); lean_dec(x_30); -x_110 = lean_ctor_get(x_107, 0); -lean_inc(x_110); -lean_dec(x_107); -x_111 = lean_environment_main_module(x_110); -x_112 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__5; +x_112 = lean_ctor_get(x_109, 0); +lean_inc(x_112); +lean_dec(x_109); +x_113 = lean_environment_main_module(x_112); +x_114 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__5; lean_inc(x_27); -x_113 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_113, 0, x_27); -lean_ctor_set(x_113, 1, x_112); -x_114 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__8; +x_115 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_115, 0, x_27); +lean_ctor_set(x_115, 1, x_114); +x_116 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__8; lean_inc(x_28); -lean_inc(x_111); -x_115 = l_Lean_addMacroScope(x_111, x_114, x_28); -x_116 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__7; +lean_inc(x_113); +x_117 = l_Lean_addMacroScope(x_113, x_116, x_28); lean_inc(x_3); +x_118 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_118, 0, x_116); +lean_ctor_set(x_118, 1, x_3); +lean_inc(x_3); +x_119 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_119, 0, x_118); +lean_ctor_set(x_119, 1, x_3); +x_120 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__7; lean_inc(x_27); -x_117 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_117, 0, x_27); -lean_ctor_set(x_117, 1, x_116); -lean_ctor_set(x_117, 2, x_115); -lean_ctor_set(x_117, 3, x_3); -x_118 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__4; -lean_inc(x_27); -x_119 = l_Lean_Syntax_node3(x_27, x_118, x_109, x_113, x_117); -x_120 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__10; -lean_inc(x_27); -x_121 = lean_alloc_ctor(2, 2, 0); +x_121 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_121, 0, x_27); lean_ctor_set(x_121, 1, x_120); -x_122 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__13; -lean_inc(x_28); -lean_inc(x_111); -x_123 = l_Lean_addMacroScope(x_111, x_122, x_28); -x_124 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__12; -lean_inc(x_3); +lean_ctor_set(x_121, 2, x_117); +lean_ctor_set(x_121, 3, x_119); +x_122 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__4; +lean_inc(x_27); +x_123 = l_Lean_Syntax_node3(x_27, x_122, x_111, x_115, x_121); +x_124 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__10; lean_inc(x_27); -x_125 = lean_alloc_ctor(3, 4, 0); +x_125 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_125, 0, x_27); lean_ctor_set(x_125, 1, x_124); -lean_ctor_set(x_125, 2, x_123); -lean_ctor_set(x_125, 3, x_3); -x_126 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___spec__2___closed__5; -lean_inc(x_27); -x_127 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_127, 0, x_27); -lean_ctor_set(x_127, 1, x_126); -x_128 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__12; +x_126 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__13; +lean_inc(x_28); +lean_inc(x_113); +x_127 = l_Lean_addMacroScope(x_113, x_126, x_28); +x_128 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__12; +lean_inc(x_3); lean_inc(x_27); -x_129 = lean_alloc_ctor(2, 2, 0); +x_129 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_129, 0, x_27); lean_ctor_set(x_129, 1, x_128); -x_130 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__10; -lean_inc(x_129); -lean_inc(x_121); +lean_ctor_set(x_129, 2, x_127); +lean_ctor_set(x_129, 3, x_3); +x_130 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___spec__2___closed__5; lean_inc(x_27); -x_131 = l_Lean_Syntax_node5(x_27, x_130, x_121, x_125, x_127, x_22, x_129); -x_132 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__16; +x_131 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_131, 0, x_27); +lean_ctor_set(x_131, 1, x_130); +x_132 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__12; lean_inc(x_27); x_133 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_133, 0, x_27); lean_ctor_set(x_133, 1, x_132); -x_134 = l_Lean_addMacroScope(x_111, x_4, x_28); +x_134 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__10; +lean_inc(x_133); +lean_inc(x_125); +lean_inc(x_27); +x_135 = l_Lean_Syntax_node5(x_27, x_134, x_125, x_129, x_131, x_22, x_133); +x_136 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__16; lean_inc(x_27); -x_135 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_135, 0, x_27); -lean_ctor_set(x_135, 1, x_5); -lean_ctor_set(x_135, 2, x_134); -lean_ctor_set(x_135, 3, x_3); +x_137 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_137, 0, x_27); +lean_ctor_set(x_137, 1, x_136); +x_138 = l_Lean_addMacroScope(x_113, x_4, x_28); +lean_inc(x_27); +x_139 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_139, 0, x_27); +lean_ctor_set(x_139, 1, x_5); +lean_ctor_set(x_139, 2, x_138); +lean_ctor_set(x_139, 3, x_3); lean_inc(x_6); lean_inc(x_27); -x_136 = l_Lean_Syntax_node1(x_27, x_6, x_135); -x_137 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__1; +x_140 = l_Lean_Syntax_node1(x_27, x_6, x_139); +x_141 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__1; lean_inc(x_6); lean_inc(x_27); -x_138 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_138, 0, x_27); -lean_ctor_set(x_138, 1, x_6); -lean_ctor_set(x_138, 2, x_137); -x_139 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__20; +x_142 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_142, 0, x_27); +lean_ctor_set(x_142, 1, x_6); +lean_ctor_set(x_142, 2, x_141); +x_143 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__20; lean_inc(x_27); -x_140 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_140, 0, x_27); -lean_ctor_set(x_140, 1, x_139); -x_141 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__19; +x_144 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_144, 0, x_27); +lean_ctor_set(x_144, 1, x_143); +x_145 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__19; lean_inc(x_27); -x_142 = l_Lean_Syntax_node4(x_27, x_141, x_136, x_138, x_140, x_7); -x_143 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__17; +x_146 = l_Lean_Syntax_node4(x_27, x_145, x_140, x_142, x_144, x_7); +x_147 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__17; lean_inc(x_27); -x_144 = l_Lean_Syntax_node2(x_27, x_143, x_133, x_142); -x_145 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__15; +x_148 = l_Lean_Syntax_node2(x_27, x_147, x_137, x_146); +x_149 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__15; lean_inc(x_27); -x_146 = l_Lean_Syntax_node3(x_27, x_145, x_121, x_144, x_129); +x_150 = l_Lean_Syntax_node3(x_27, x_149, x_125, x_148, x_133); lean_inc(x_27); -x_147 = l_Lean_Syntax_node2(x_27, x_6, x_131, x_146); -x_148 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__2; -x_149 = l_Lean_Syntax_node2(x_27, x_148, x_119, x_147); +x_151 = l_Lean_Syntax_node2(x_27, x_6, x_135, x_150); +x_152 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__2; +x_153 = l_Lean_Syntax_node2(x_27, x_152, x_123, x_151); lean_inc(x_8); -x_150 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_8, x_12, x_13, x_14, x_15, x_16, x_17, x_108); -x_151 = lean_ctor_get(x_150, 0); -lean_inc(x_151); -x_152 = lean_unbox(x_151); -lean_dec(x_151); -if (x_152 == 0) +x_154 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_8, x_12, x_13, x_14, x_15, x_16, x_17, x_110); +x_155 = lean_ctor_get(x_154, 0); +lean_inc(x_155); +x_156 = lean_unbox(x_155); +lean_dec(x_155); +if (x_156 == 0) { -lean_object* x_153; lean_object* x_154; lean_object* x_155; +lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_dec(x_8); -x_153 = lean_ctor_get(x_150, 1); -lean_inc(x_153); -lean_dec(x_150); -x_154 = lean_box(0); -x_155 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_149, x_9, x_10, x_154, x_12, x_13, x_14, x_15, x_16, x_17, x_153); -return x_155; +x_157 = lean_ctor_get(x_154, 1); +lean_inc(x_157); +lean_dec(x_154); +x_158 = lean_box(0); +x_159 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_153, x_9, x_10, x_158, x_12, x_13, x_14, x_15, x_16, x_17, x_157); +return x_159; } else { -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_156 = lean_ctor_get(x_150, 1); -lean_inc(x_156); -if (lean_is_exclusive(x_150)) { - lean_ctor_release(x_150, 0); - lean_ctor_release(x_150, 1); - x_157 = x_150; +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_160 = lean_ctor_get(x_154, 1); +lean_inc(x_160); +if (lean_is_exclusive(x_154)) { + lean_ctor_release(x_154, 0); + lean_ctor_release(x_154, 1); + x_161 = x_154; } else { - lean_dec_ref(x_150); - x_157 = lean_box(0); + lean_dec_ref(x_154); + x_161 = lean_box(0); } lean_inc(x_10); -x_158 = l_Lean_MessageData_ofSyntax(x_10); -x_159 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__22; -if (lean_is_scalar(x_157)) { - x_160 = lean_alloc_ctor(7, 2, 0); +x_162 = l_Lean_MessageData_ofSyntax(x_10); +x_163 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__22; +if (lean_is_scalar(x_161)) { + x_164 = lean_alloc_ctor(7, 2, 0); } else { - x_160 = x_157; - lean_ctor_set_tag(x_160, 7); + x_164 = x_161; + lean_ctor_set_tag(x_164, 7); } -lean_ctor_set(x_160, 0, x_159); -lean_ctor_set(x_160, 1, x_158); -x_161 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__24; -x_162 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_162, 0, x_160); -lean_ctor_set(x_162, 1, x_161); -lean_inc(x_149); -x_163 = l_Lean_MessageData_ofSyntax(x_149); -x_164 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_164, 0, x_162); -lean_ctor_set(x_164, 1, x_163); -x_165 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_165, 0, x_164); -lean_ctor_set(x_165, 1, x_159); -x_166 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_8, x_165, x_12, x_13, x_14, x_15, x_16, x_17, x_156); -x_167 = lean_ctor_get(x_166, 0); -lean_inc(x_167); -x_168 = lean_ctor_get(x_166, 1); -lean_inc(x_168); -lean_dec(x_166); -x_169 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_149, x_9, x_10, x_167, x_12, x_13, x_14, x_15, x_16, x_17, x_168); -lean_dec(x_167); -return x_169; +lean_ctor_set(x_164, 0, x_163); +lean_ctor_set(x_164, 1, x_162); +x_165 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__24; +x_166 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_166, 0, x_164); +lean_ctor_set(x_166, 1, x_165); +lean_inc(x_153); +x_167 = l_Lean_MessageData_ofSyntax(x_153); +x_168 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_168, 0, x_166); +lean_ctor_set(x_168, 1, x_167); +x_169 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_169, 0, x_168); +lean_ctor_set(x_169, 1, x_163); +x_170 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_8, x_169, x_12, x_13, x_14, x_15, x_16, x_17, x_160); +x_171 = lean_ctor_get(x_170, 0); +lean_inc(x_171); +x_172 = lean_ctor_get(x_170, 1); +lean_inc(x_172); +lean_dec(x_170); +x_173 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_153, x_9, x_10, x_171, x_12, x_13, x_14, x_15, x_16, x_17, x_172); +lean_dec(x_171); +return x_173; } } } @@ -5697,15 +5714,23 @@ return x_1; static lean_object* _init_l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__5() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("modifyOp", 8, 8); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__6() { +_start: +{ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstExpectedType__1___closed__3; x_2 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__4; -x_3 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__6; +x_3 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__5; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__6() { +static lean_object* _init_l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__7() { _start: { lean_object* x_1; @@ -5713,15 +5738,39 @@ x_1 = lean_mk_string_unchecked("\nval: ", 6, 6); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__7() { +static lean_object* _init_l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__6; +x_1 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__7; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } +static lean_object* _init_l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__8; +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_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__9; +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_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___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: { @@ -5790,7 +5839,7 @@ x_46 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkSourcesWi lean_dec(x_45); lean_inc(x_2); x_47 = l_Lean_Syntax_setArg(x_2, x_15, x_46); -x_48 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__5; +x_48 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__6; x_49 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_48, x_6, x_7, x_8, x_9, x_10, x_11, x_25); if (x_36 == 0) { @@ -5853,7 +5902,7 @@ x_67 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyO 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___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__7; +x_69 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__8; x_70 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_70, 0, x_68); lean_ctor_set(x_70, 1, x_69); @@ -5924,7 +5973,7 @@ x_94 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyO x_95 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_95, 0, x_94); lean_ctor_set(x_95, 1, x_93); -x_96 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__7; +x_96 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__8; x_97 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_97, 0, x_95); lean_ctor_set(x_97, 1, x_96); @@ -6000,7 +6049,7 @@ x_130 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkSourcesW lean_dec(x_129); lean_inc(x_2); x_131 = l_Lean_Syntax_setArg(x_2, x_15, x_130); -x_132 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__5; +x_132 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__6; x_133 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_132, x_6, x_7, x_8, x_9, x_10, x_11, x_108); if (x_119 == 0) { @@ -6074,7 +6123,7 @@ x_152 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModify 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_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__7; +x_154 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___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); @@ -6116,20 +6165,20 @@ x_170 = lean_nat_dec_lt(x_13, x_169); lean_dec(x_169); if (x_170 == 0) { -lean_object* x_326; lean_object* x_327; -x_326 = l_Lean_Elab_Term_StructInst_instInhabitedExplicitSourceInfo; -x_327 = l_outOfBounds___rarg(x_326); -x_171 = x_327; -goto block_325; +lean_object* x_328; lean_object* x_329; +x_328 = l_Lean_Elab_Term_StructInst_instInhabitedExplicitSourceInfo; +x_329 = l_outOfBounds___rarg(x_328); +x_171 = x_329; +goto block_327; } else { -lean_object* x_328; -x_328 = lean_array_fget(x_3, x_13); -x_171 = x_328; -goto block_325; +lean_object* x_330; +x_330 = lean_array_fget(x_3, x_13); +x_171 = x_330; +goto block_327; } -block_325: +block_327: { lean_object* x_172; lean_object* x_173; uint8_t x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; uint8_t x_178; x_172 = lean_ctor_get(x_171, 0); @@ -6146,7 +6195,7 @@ x_177 = lean_st_ref_get(x_11, x_12); x_178 = !lean_is_exclusive(x_177); if (x_178 == 0) { -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; uint8_t x_227; +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; uint8_t x_228; x_179 = lean_ctor_get(x_177, 0); x_180 = lean_ctor_get(x_177, 1); x_181 = lean_ctor_get(x_179, 0); @@ -6164,342 +6213,344 @@ lean_inc(x_182); x_185 = l_Lean_addMacroScope(x_182, x_184, x_176); x_186 = lean_box(0); x_187 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__7; +x_188 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__10; lean_inc(x_175); -x_188 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_188, 0, x_175); -lean_ctor_set(x_188, 1, x_187); -lean_ctor_set(x_188, 2, x_185); -lean_ctor_set(x_188, 3, x_186); -x_189 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__4; +x_189 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_189, 0, x_175); +lean_ctor_set(x_189, 1, x_187); +lean_ctor_set(x_189, 2, x_185); +lean_ctor_set(x_189, 3, x_188); +x_190 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__4; lean_inc(x_175); -x_190 = l_Lean_Syntax_node3(x_175, x_189, x_172, x_177, x_188); -x_191 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__10; +x_191 = l_Lean_Syntax_node3(x_175, x_190, x_172, x_177, x_189); +x_192 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__10; lean_inc(x_175); -x_192 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_192, 0, x_175); -lean_ctor_set(x_192, 1, x_191); -x_193 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__13; +x_193 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_193, 0, x_175); +lean_ctor_set(x_193, 1, x_192); +x_194 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__13; lean_inc(x_176); lean_inc(x_182); -x_194 = l_Lean_addMacroScope(x_182, x_193, x_176); -x_195 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__12; +x_195 = l_Lean_addMacroScope(x_182, x_194, x_176); +x_196 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__12; lean_inc(x_175); -x_196 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_196, 0, x_175); -lean_ctor_set(x_196, 1, x_195); -lean_ctor_set(x_196, 2, x_194); -lean_ctor_set(x_196, 3, x_186); -x_197 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___spec__2___closed__5; +x_197 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_197, 0, x_175); +lean_ctor_set(x_197, 1, x_196); +lean_ctor_set(x_197, 2, x_195); +lean_ctor_set(x_197, 3, x_186); +x_198 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___spec__2___closed__5; lean_inc(x_175); -x_198 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_198, 0, x_175); -lean_ctor_set(x_198, 1, x_197); -x_199 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__12; +x_199 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_199, 0, x_175); +lean_ctor_set(x_199, 1, x_198); +x_200 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__12; lean_inc(x_175); -x_200 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_200, 0, x_175); -lean_ctor_set(x_200, 1, x_199); -x_201 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__10; -lean_inc(x_200); -lean_inc(x_192); +x_201 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_201, 0, x_175); +lean_ctor_set(x_201, 1, x_200); +x_202 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__10; +lean_inc(x_201); +lean_inc(x_193); lean_inc(x_175); -x_202 = l_Lean_Syntax_node5(x_175, x_201, x_192, x_196, x_198, x_168, x_200); -x_203 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__16; +x_203 = l_Lean_Syntax_node5(x_175, x_202, x_193, x_197, x_199, x_168, x_201); +x_204 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__16; lean_inc(x_175); -x_204 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_204, 0, x_175); -lean_ctor_set(x_204, 1, x_203); -x_205 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__3; -x_206 = l_Lean_addMacroScope(x_182, x_205, x_176); -x_207 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__2; +x_205 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_205, 0, x_175); +lean_ctor_set(x_205, 1, x_204); +x_206 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__3; +x_207 = l_Lean_addMacroScope(x_182, x_206, x_176); +x_208 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__2; lean_inc(x_175); -x_208 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_208, 0, x_175); -lean_ctor_set(x_208, 1, x_207); -lean_ctor_set(x_208, 2, x_206); -lean_ctor_set(x_208, 3, x_186); -x_209 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__3; +x_209 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_209, 0, x_175); +lean_ctor_set(x_209, 1, x_208); +lean_ctor_set(x_209, 2, x_207); +lean_ctor_set(x_209, 3, x_186); +x_210 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__3; lean_inc(x_175); -x_210 = l_Lean_Syntax_node1(x_175, x_209, x_208); -x_211 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__1; +x_211 = l_Lean_Syntax_node1(x_175, x_210, x_209); +x_212 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__1; lean_inc(x_175); -x_212 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_212, 0, x_175); -lean_ctor_set(x_212, 1, x_209); -lean_ctor_set(x_212, 2, x_211); -x_213 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__20; +x_213 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_213, 0, x_175); +lean_ctor_set(x_213, 1, x_210); +lean_ctor_set(x_213, 2, x_212); +x_214 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__20; lean_inc(x_175); -x_214 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_214, 0, x_175); -lean_ctor_set(x_214, 1, x_213); -x_215 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__19; +x_215 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_215, 0, x_175); +lean_ctor_set(x_215, 1, x_214); +x_216 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__19; lean_inc(x_175); -x_216 = l_Lean_Syntax_node4(x_175, x_215, x_210, x_212, x_214, x_166); -x_217 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__17; +x_217 = l_Lean_Syntax_node4(x_175, x_216, x_211, x_213, x_215, x_166); +x_218 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__17; lean_inc(x_175); -x_218 = l_Lean_Syntax_node2(x_175, x_217, x_204, x_216); -x_219 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__15; +x_219 = l_Lean_Syntax_node2(x_175, x_218, x_205, x_217); +x_220 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__15; lean_inc(x_175); -x_220 = l_Lean_Syntax_node3(x_175, x_219, x_192, x_218, x_200); +x_221 = l_Lean_Syntax_node3(x_175, x_220, x_193, x_219, x_201); lean_inc(x_175); -x_221 = l_Lean_Syntax_node2(x_175, x_209, x_202, x_220); -x_222 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__2; -x_223 = l_Lean_Syntax_node2(x_175, x_222, x_190, x_221); -x_224 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__5; -x_225 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_224, x_6, x_7, x_8, x_9, x_10, x_11, x_180); -x_226 = lean_ctor_get(x_225, 0); -lean_inc(x_226); -x_227 = lean_unbox(x_226); -lean_dec(x_226); -if (x_227 == 0) +x_222 = l_Lean_Syntax_node2(x_175, x_210, x_203, x_221); +x_223 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__2; +x_224 = l_Lean_Syntax_node2(x_175, x_223, x_191, x_222); +x_225 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__6; +x_226 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_225, x_6, x_7, x_8, x_9, x_10, x_11, x_180); +x_227 = lean_ctor_get(x_226, 0); +lean_inc(x_227); +x_228 = lean_unbox(x_227); +lean_dec(x_227); +if (x_228 == 0) { -lean_object* x_228; lean_object* x_229; lean_object* x_230; -x_228 = lean_ctor_get(x_225, 1); -lean_inc(x_228); -lean_dec(x_225); -x_229 = lean_box(0); -x_230 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_223, x_4, x_2, x_229, x_6, x_7, x_8, x_9, x_10, x_11, x_228); -return x_230; +lean_object* x_229; lean_object* x_230; lean_object* x_231; +x_229 = lean_ctor_get(x_226, 1); +lean_inc(x_229); +lean_dec(x_226); +x_230 = lean_box(0); +x_231 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_224, x_4, x_2, x_230, x_6, x_7, x_8, x_9, x_10, x_11, x_229); +return x_231; } else { -uint8_t x_231; -x_231 = !lean_is_exclusive(x_225); -if (x_231 == 0) +uint8_t x_232; +x_232 = !lean_is_exclusive(x_226); +if (x_232 == 0) { -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; -x_232 = lean_ctor_get(x_225, 1); -x_233 = lean_ctor_get(x_225, 0); -lean_dec(x_233); +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_233 = lean_ctor_get(x_226, 1); +x_234 = lean_ctor_get(x_226, 0); +lean_dec(x_234); lean_inc(x_2); -x_234 = l_Lean_MessageData_ofSyntax(x_2); -x_235 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__22; -lean_ctor_set_tag(x_225, 7); -lean_ctor_set(x_225, 1, x_234); -lean_ctor_set(x_225, 0, x_235); -x_236 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__24; -x_237 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_237, 0, x_225); -lean_ctor_set(x_237, 1, x_236); -lean_inc(x_223); -x_238 = l_Lean_MessageData_ofSyntax(x_223); -x_239 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_239, 0, x_237); -lean_ctor_set(x_239, 1, x_238); +x_235 = l_Lean_MessageData_ofSyntax(x_2); +x_236 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__22; +lean_ctor_set_tag(x_226, 7); +lean_ctor_set(x_226, 1, x_235); +lean_ctor_set(x_226, 0, x_236); +x_237 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__24; +x_238 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_238, 0, x_226); +lean_ctor_set(x_238, 1, x_237); +lean_inc(x_224); +x_239 = l_Lean_MessageData_ofSyntax(x_224); x_240 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_240, 0, x_239); -lean_ctor_set(x_240, 1, x_235); -x_241 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_224, x_240, x_6, x_7, x_8, x_9, x_10, x_11, x_232); -x_242 = lean_ctor_get(x_241, 0); -lean_inc(x_242); -x_243 = lean_ctor_get(x_241, 1); +lean_ctor_set(x_240, 0, x_238); +lean_ctor_set(x_240, 1, x_239); +x_241 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_241, 0, x_240); +lean_ctor_set(x_241, 1, x_236); +x_242 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_225, x_241, x_6, x_7, x_8, x_9, x_10, x_11, x_233); +x_243 = lean_ctor_get(x_242, 0); lean_inc(x_243); -lean_dec(x_241); -x_244 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_223, x_4, x_2, x_242, x_6, x_7, x_8, x_9, x_10, x_11, x_243); +x_244 = lean_ctor_get(x_242, 1); +lean_inc(x_244); lean_dec(x_242); -return x_244; +x_245 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_224, x_4, x_2, x_243, x_6, x_7, x_8, x_9, x_10, x_11, x_244); +lean_dec(x_243); +return x_245; } 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; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; -x_245 = lean_ctor_get(x_225, 1); -lean_inc(x_245); -lean_dec(x_225); +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; +x_246 = lean_ctor_get(x_226, 1); +lean_inc(x_246); +lean_dec(x_226); lean_inc(x_2); -x_246 = l_Lean_MessageData_ofSyntax(x_2); -x_247 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__22; -x_248 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_248, 0, x_247); -lean_ctor_set(x_248, 1, x_246); -x_249 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__24; -x_250 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_250, 0, x_248); -lean_ctor_set(x_250, 1, x_249); -lean_inc(x_223); -x_251 = l_Lean_MessageData_ofSyntax(x_223); -x_252 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_252, 0, x_250); -lean_ctor_set(x_252, 1, x_251); +x_247 = l_Lean_MessageData_ofSyntax(x_2); +x_248 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__22; +x_249 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_249, 0, x_248); +lean_ctor_set(x_249, 1, x_247); +x_250 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__24; +x_251 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_251, 0, x_249); +lean_ctor_set(x_251, 1, x_250); +lean_inc(x_224); +x_252 = l_Lean_MessageData_ofSyntax(x_224); x_253 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_253, 0, x_252); -lean_ctor_set(x_253, 1, x_247); -x_254 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_224, x_253, x_6, x_7, x_8, x_9, x_10, x_11, x_245); -x_255 = lean_ctor_get(x_254, 0); -lean_inc(x_255); -x_256 = lean_ctor_get(x_254, 1); +lean_ctor_set(x_253, 0, x_251); +lean_ctor_set(x_253, 1, x_252); +x_254 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_254, 0, x_253); +lean_ctor_set(x_254, 1, x_248); +x_255 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_225, x_254, x_6, x_7, x_8, x_9, x_10, x_11, x_246); +x_256 = lean_ctor_get(x_255, 0); lean_inc(x_256); -lean_dec(x_254); -x_257 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_223, x_4, x_2, x_255, x_6, x_7, x_8, x_9, x_10, x_11, x_256); +x_257 = lean_ctor_get(x_255, 1); +lean_inc(x_257); lean_dec(x_255); -return x_257; +x_258 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_224, x_4, x_2, x_256, x_6, x_7, x_8, x_9, x_10, x_11, x_257); +lean_dec(x_256); +return x_258; } } } else { -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; uint8_t x_307; -x_258 = lean_ctor_get(x_177, 0); -x_259 = lean_ctor_get(x_177, 1); +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; uint8_t x_309; +x_259 = lean_ctor_get(x_177, 0); +x_260 = lean_ctor_get(x_177, 1); +lean_inc(x_260); lean_inc(x_259); -lean_inc(x_258); lean_dec(x_177); -x_260 = lean_ctor_get(x_258, 0); -lean_inc(x_260); -lean_dec(x_258); -x_261 = lean_environment_main_module(x_260); -x_262 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__5; +x_261 = lean_ctor_get(x_259, 0); +lean_inc(x_261); +lean_dec(x_259); +x_262 = lean_environment_main_module(x_261); +x_263 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__5; lean_inc(x_175); -x_263 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_263, 0, x_175); -lean_ctor_set(x_263, 1, x_262); -x_264 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__8; +x_264 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_264, 0, x_175); +lean_ctor_set(x_264, 1, x_263); +x_265 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__8; lean_inc(x_176); -lean_inc(x_261); -x_265 = l_Lean_addMacroScope(x_261, x_264, x_176); -x_266 = lean_box(0); -x_267 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__7; +lean_inc(x_262); +x_266 = l_Lean_addMacroScope(x_262, x_265, x_176); +x_267 = lean_box(0); +x_268 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__7; +x_269 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__10; lean_inc(x_175); -x_268 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_268, 0, x_175); -lean_ctor_set(x_268, 1, x_267); -lean_ctor_set(x_268, 2, x_265); -lean_ctor_set(x_268, 3, x_266); -x_269 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__4; +x_270 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_270, 0, x_175); +lean_ctor_set(x_270, 1, x_268); +lean_ctor_set(x_270, 2, x_266); +lean_ctor_set(x_270, 3, x_269); +x_271 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__4; lean_inc(x_175); -x_270 = l_Lean_Syntax_node3(x_175, x_269, x_172, x_263, x_268); -x_271 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__10; +x_272 = l_Lean_Syntax_node3(x_175, x_271, x_172, x_264, x_270); +x_273 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__10; lean_inc(x_175); -x_272 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_272, 0, x_175); -lean_ctor_set(x_272, 1, x_271); -x_273 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__13; +x_274 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_274, 0, x_175); +lean_ctor_set(x_274, 1, x_273); +x_275 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__13; lean_inc(x_176); -lean_inc(x_261); -x_274 = l_Lean_addMacroScope(x_261, x_273, x_176); -x_275 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__12; -lean_inc(x_175); -x_276 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_276, 0, x_175); -lean_ctor_set(x_276, 1, x_275); -lean_ctor_set(x_276, 2, x_274); -lean_ctor_set(x_276, 3, x_266); -x_277 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___spec__2___closed__5; +lean_inc(x_262); +x_276 = l_Lean_addMacroScope(x_262, x_275, x_176); +x_277 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__12; lean_inc(x_175); -x_278 = lean_alloc_ctor(2, 2, 0); +x_278 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_278, 0, x_175); lean_ctor_set(x_278, 1, x_277); -x_279 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__12; +lean_ctor_set(x_278, 2, x_276); +lean_ctor_set(x_278, 3, x_267); +x_279 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___spec__2___closed__5; lean_inc(x_175); x_280 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_280, 0, x_175); lean_ctor_set(x_280, 1, x_279); -x_281 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__10; -lean_inc(x_280); -lean_inc(x_272); +x_281 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__12; lean_inc(x_175); -x_282 = l_Lean_Syntax_node5(x_175, x_281, x_272, x_276, x_278, x_168, x_280); -x_283 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__16; +x_282 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_282, 0, x_175); +lean_ctor_set(x_282, 1, x_281); +x_283 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__10; +lean_inc(x_282); +lean_inc(x_274); lean_inc(x_175); -x_284 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_284, 0, x_175); -lean_ctor_set(x_284, 1, x_283); -x_285 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__3; -x_286 = l_Lean_addMacroScope(x_261, x_285, x_176); -x_287 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__2; +x_284 = l_Lean_Syntax_node5(x_175, x_283, x_274, x_278, x_280, x_168, x_282); +x_285 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__16; lean_inc(x_175); -x_288 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_288, 0, x_175); -lean_ctor_set(x_288, 1, x_287); -lean_ctor_set(x_288, 2, x_286); -lean_ctor_set(x_288, 3, x_266); -x_289 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__3; +x_286 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_286, 0, x_175); +lean_ctor_set(x_286, 1, x_285); +x_287 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__3; +x_288 = l_Lean_addMacroScope(x_262, x_287, x_176); +x_289 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__2; lean_inc(x_175); -x_290 = l_Lean_Syntax_node1(x_175, x_289, x_288); -x_291 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__1; +x_290 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_290, 0, x_175); +lean_ctor_set(x_290, 1, x_289); +lean_ctor_set(x_290, 2, x_288); +lean_ctor_set(x_290, 3, x_267); +x_291 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__3; lean_inc(x_175); -x_292 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_292, 0, x_175); -lean_ctor_set(x_292, 1, x_289); -lean_ctor_set(x_292, 2, x_291); -x_293 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__20; +x_292 = l_Lean_Syntax_node1(x_175, x_291, x_290); +x_293 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__1; lean_inc(x_175); -x_294 = lean_alloc_ctor(2, 2, 0); +x_294 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_294, 0, x_175); -lean_ctor_set(x_294, 1, x_293); -x_295 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__19; +lean_ctor_set(x_294, 1, x_291); +lean_ctor_set(x_294, 2, x_293); +x_295 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__20; lean_inc(x_175); -x_296 = l_Lean_Syntax_node4(x_175, x_295, x_290, x_292, x_294, x_166); -x_297 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__17; +x_296 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_296, 0, x_175); +lean_ctor_set(x_296, 1, x_295); +x_297 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__19; lean_inc(x_175); -x_298 = l_Lean_Syntax_node2(x_175, x_297, x_284, x_296); -x_299 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__15; +x_298 = l_Lean_Syntax_node4(x_175, x_297, x_292, x_294, x_296, x_166); +x_299 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__17; lean_inc(x_175); -x_300 = l_Lean_Syntax_node3(x_175, x_299, x_272, x_298, x_280); +x_300 = l_Lean_Syntax_node2(x_175, x_299, x_286, x_298); +x_301 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__15; lean_inc(x_175); -x_301 = l_Lean_Syntax_node2(x_175, x_289, x_282, x_300); -x_302 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__2; -x_303 = l_Lean_Syntax_node2(x_175, x_302, x_270, x_301); -x_304 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__5; -x_305 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_304, x_6, x_7, x_8, x_9, x_10, x_11, x_259); -x_306 = lean_ctor_get(x_305, 0); -lean_inc(x_306); -x_307 = lean_unbox(x_306); -lean_dec(x_306); -if (x_307 == 0) -{ -lean_object* x_308; lean_object* x_309; lean_object* x_310; -x_308 = lean_ctor_get(x_305, 1); +x_302 = l_Lean_Syntax_node3(x_175, x_301, x_274, x_300, x_282); +lean_inc(x_175); +x_303 = l_Lean_Syntax_node2(x_175, x_291, x_284, x_302); +x_304 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__2; +x_305 = l_Lean_Syntax_node2(x_175, x_304, x_272, x_303); +x_306 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__6; +x_307 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___spec__1(x_306, x_6, x_7, x_8, x_9, x_10, x_11, x_260); +x_308 = lean_ctor_get(x_307, 0); lean_inc(x_308); -lean_dec(x_305); -x_309 = lean_box(0); -x_310 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_303, x_4, x_2, x_309, x_6, x_7, x_8, x_9, x_10, x_11, x_308); -return x_310; +x_309 = lean_unbox(x_308); +lean_dec(x_308); +if (x_309 == 0) +{ +lean_object* x_310; lean_object* x_311; lean_object* x_312; +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_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_305, x_4, x_2, x_311, x_6, x_7, x_8, x_9, x_10, x_11, x_310); +return x_312; } else { -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; -x_311 = lean_ctor_get(x_305, 1); -lean_inc(x_311); -if (lean_is_exclusive(x_305)) { - lean_ctor_release(x_305, 0); - lean_ctor_release(x_305, 1); - x_312 = x_305; +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; +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_305); - x_312 = lean_box(0); + lean_dec_ref(x_307); + x_314 = lean_box(0); } lean_inc(x_2); -x_313 = l_Lean_MessageData_ofSyntax(x_2); -x_314 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__22; -if (lean_is_scalar(x_312)) { - x_315 = lean_alloc_ctor(7, 2, 0); -} else { - x_315 = x_312; - lean_ctor_set_tag(x_315, 7); -} -lean_ctor_set(x_315, 0, x_314); -lean_ctor_set(x_315, 1, x_313); -x_316 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__24; -x_317 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_317, 0, x_315); -lean_ctor_set(x_317, 1, x_316); -lean_inc(x_303); -x_318 = l_Lean_MessageData_ofSyntax(x_303); +x_315 = l_Lean_MessageData_ofSyntax(x_2); +x_316 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__22; +if (lean_is_scalar(x_314)) { + x_317 = lean_alloc_ctor(7, 2, 0); +} else { + x_317 = x_314; + lean_ctor_set_tag(x_317, 7); +} +lean_ctor_set(x_317, 0, x_316); +lean_ctor_set(x_317, 1, x_315); +x_318 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__24; x_319 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_319, 0, x_317); lean_ctor_set(x_319, 1, x_318); -x_320 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_320, 0, x_319); -lean_ctor_set(x_320, 1, x_314); -x_321 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_304, x_320, x_6, x_7, x_8, x_9, x_10, x_11, x_311); -x_322 = lean_ctor_get(x_321, 0); -lean_inc(x_322); -x_323 = lean_ctor_get(x_321, 1); -lean_inc(x_323); -lean_dec(x_321); -x_324 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_303, x_4, x_2, x_322, x_6, x_7, x_8, x_9, x_10, x_11, x_323); -lean_dec(x_322); -return x_324; +lean_inc(x_305); +x_320 = l_Lean_MessageData_ofSyntax(x_305); +x_321 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_321, 0, x_319); +lean_ctor_set(x_321, 1, x_320); +x_322 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_322, 0, x_321); +lean_ctor_set(x_322, 1, x_316); +x_323 = l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(x_306, x_322, x_6, x_7, x_8, x_9, x_10, x_11, x_313); +x_324 = lean_ctor_get(x_323, 0); +lean_inc(x_324); +x_325 = lean_ctor_get(x_323, 1); +lean_inc(x_325); +lean_dec(x_323); +x_326 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__1(x_305, x_4, x_2, x_324, x_6, x_7, x_8, x_9, x_10, x_11, x_325); +lean_dec(x_324); +return x_326; } } } @@ -37115,7 +37166,7 @@ x_4 = l_Lean_addBuiltinDeclarationRanges(x_2, x_3, x_1); return x_4; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__1() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -37125,37 +37176,37 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__2() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__1; +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__1; x_2 = l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstExpectedType__1___closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__3() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__2; +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__2; x_2 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__4() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__3; +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__3; x_2 = l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstExpectedType__1___closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__5() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__5() { _start: { lean_object* x_1; @@ -37163,17 +37214,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__6() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__4; -x_2 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__5; +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__4; +x_2 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__7() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__7() { _start: { lean_object* x_1; @@ -37181,47 +37232,47 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__8() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__6; -x_2 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__7; +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__6; +x_2 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__9() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__8; +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__8; x_2 = l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__10() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__9; +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__9; x_2 = l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstExpectedType__1___closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__11() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__10; +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__10; x_2 = l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstExpectedType__1___closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__12() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__12() { _start: { lean_object* x_1; @@ -37229,33 +37280,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__13() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__11; -x_2 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__12; +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__11; +x_2 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__14() { +static lean_object* _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__13; -x_2 = lean_unsigned_to_nat(13312u); +x_1 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__13; +x_2 = lean_unsigned_to_nat(13316u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l_List_foldlM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStruct___spec__5___closed__3; x_3 = 0; -x_4 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__14; +x_4 = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__14; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); if (lean_obj_tag(x_5) == 0) { @@ -37263,7 +37314,7 @@ lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = lean_ctor_get(x_5, 1); lean_inc(x_6); lean_dec(x_5); -x_7 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__5; +x_7 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__6; x_8 = l_Lean_registerTraceClass(x_7, x_3, x_4, x_6); return x_8; } @@ -37567,6 +37618,12 @@ l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lam lean_mark_persistent(l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__6); l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__7 = _init_l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__7(); lean_mark_persistent(l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__7); +l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__8 = _init_l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__8(); +lean_mark_persistent(l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__8); +l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__9 = _init_l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__9(); +lean_mark_persistent(l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__9); +l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__10 = _init_l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__10(); +lean_mark_persistent(l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__10); l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___closed__1 = _init_l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___closed__1(); lean_mark_persistent(l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___closed__1); l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___closed__2 = _init_l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___closed__2(); @@ -37916,35 +37973,35 @@ lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_StructInst_elabStructInst_dec if (builtin) {res = l___regBuiltin_Lean_Elab_Term_StructInst_elabStructInst_declRange__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__1 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__1(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__1); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__2 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__2(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__2); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__3 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__3(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__3); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__4 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__4(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__4); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__5 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__5(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__5); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__6 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__6(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__6); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__7 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__7(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__7); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__8 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__8(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__8); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__9 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__9(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__9); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__10 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__10(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__10); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__11 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__11(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__11); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__12 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__12(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__12); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__13 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__13(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__13); -l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__14 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__14(); -lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312____closed__14); -if (builtin) {res = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13312_(lean_io_mk_world()); +}l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__1 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__1(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__1); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__2 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__2(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__2); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__3 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__3(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__3); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__4 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__4(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__4); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__5 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__5(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__5); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__6 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__6(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__6); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__7 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__7(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__7); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__8 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__8(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__8); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__9 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__9(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__9); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__10 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__10(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__10); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__11 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__11(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__11); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__12 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__12(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__12); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__13 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__13(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__13); +l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__14 = _init_l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__14(); +lean_mark_persistent(l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316____closed__14); +if (builtin) {res = l_Lean_Elab_Term_StructInst_initFn____x40_Lean_Elab_StructInst___hyg_13316_(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/Structure.c b/stage0/stdlib/Lean/Elab/Structure.c index 2d79f61f3af5..37b8bfb6f944 100644 --- a/stage0/stdlib/Lean/Elab/Structure.c +++ b/stage0/stdlib/Lean/Elab/Structure.c @@ -27,7 +27,6 @@ lean_object* l_Lean_Elab_Term_levelMVarToParam(lean_object*, lean_object*, lean_ static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___closed__1; lean_object* l_Lean_Name_reprPrec(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__7; LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___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*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2___closed__1; @@ -85,15 +84,13 @@ lean_object* l_Lean_Elab_Command_runTermElabM___rarg(lean_object*, lean_object*, lean_object* l_Lean_Elab_sortDeclLevelParams(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___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_object* l_Lean_throwError___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_declRangeExt; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__11; static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__1; lean_object* l_Lean_Elab_Command_mkResultUniverse(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___spec__1(lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__6; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__1; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__6; lean_object* l_Lean_ConstantInfo_type(lean_object*); @@ -141,8 +138,6 @@ static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__15; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__6(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__13; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022_(lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__1; lean_object* l_Lean_Syntax_getId(lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__19; @@ -172,10 +167,9 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0_ uint8_t lean_usize_dec_eq(size_t, size_t); static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__4; lean_object* l_Lean_Syntax_getArgs(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__3; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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*); static lean_object* l_Lean_Elab_Command_instReprStructFieldInfo___closed__1; lean_object* l_Lean_replaceRef(lean_object*, lean_object*); static uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__3; @@ -193,7 +187,6 @@ static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__L LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabStructure___closed__2; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__1; -lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__20; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__3; LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_containsFieldName(lean_object*, lean_object*); @@ -219,7 +212,6 @@ lean_object* l_Lean_Elab_Term_declareTacticSyntax(lean_object*, lean_object*, le lean_object* l_Lean_RBNode_insert___at_Lean_NameSet_insert___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__1___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__15; LEAN_EXPORT lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -260,6 +252,7 @@ uint8_t lean_string_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__2___boxed(lean_object**); lean_object* l_Lean_Elab_Term_instInhabitedTermElabM(lean_object*); static lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___closed__1; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__2; static lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___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*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -273,7 +266,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Struc lean_object* l_Lean_CollectLevelParams_main(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__9(lean_object*); static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19___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_Structure_0__Lean_Elab_Command_addDefaults___boxed__const__1; lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_GeneralizeTelescope_generalizeTelescopeAux___spec__1___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_appArg_x21(lean_object*); @@ -290,6 +282,7 @@ static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandF static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__11___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984_(lean_object*); lean_object* l_Lean_getStructureFields(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateFieldInfoVal___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__9___rarg(lean_object*); @@ -324,22 +317,19 @@ static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandF size_t lean_usize_of_nat(lean_object*); uint8_t l_Lean_TagDeclarationExtension_isTagged(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInFVars___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_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__1; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_removeUnused___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getResultUniverse___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_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParamFVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__2; lean_object* lean_expr_abstract(lean_object*, lean_object*); lean_object* l_Lean_Meta_withLCtx___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__3___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_Elab_Structure_0__Lean_Elab_Command_processSubfields_go(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___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*, 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_Structure_0__Lean_Elab_Command_addDefaults___spec__2(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_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___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_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__6; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__7___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, 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_Elab_Command_elabStructure___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, 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_Elab_Command_StructFieldKind_noConfusion___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__22; LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -348,7 +338,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structu LEAN_EXPORT uint8_t l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2(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_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__1; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__4; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__6; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__9; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___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_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__12; @@ -360,9 +350,11 @@ static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0_ lean_object* lean_st_ref_take(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInStructure___closed__1; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__9; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__10; lean_object* l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__19; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__3; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__12; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, 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*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); @@ -374,6 +366,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_co lean_object* l_Lean_Elab_getDeclarationSelectionRef(lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017_(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_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* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lean_object*, lean_object*); @@ -391,7 +384,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__1 lean_object* l_Lean_Core_instantiateValueLevelParams(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Elab_Modifiers_isProtected(lean_object*); lean_object* lean_nat_to_int(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__12; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withUsed___rarg(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_Structure_0__Lean_Elab_Command_defaultCtorName___closed__1; @@ -407,7 +399,6 @@ lean_object* l_Lean_getConstInfo___at_Lean_Elab_Term_mkConst___spec__1(lean_obje LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__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___private_Lean_Elab_Structure_0__Lean_Elab_Command_registerStructure___spec__2___closed__1; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_registerStructure(lean_object*, lean_object*); @@ -426,6 +417,7 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0_ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__2(lean_object*, lean_object*, 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* l_Lean_Elab_Command_getRef(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__4; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__13; LEAN_EXPORT lean_object* l_Lean_setReducibilityStatus___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__7; @@ -443,7 +435,7 @@ static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoerc static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__7; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__19; lean_object* l_Lean_Syntax_getKind(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___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_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___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_object* l_Lean_MessageData_ofFormat(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___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*, lean_object*, lean_object*); lean_object* l_Lean_Elab_getBetterRef(lean_object*, lean_object*); @@ -460,6 +452,7 @@ static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_default LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_addCtorFields(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_value(lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__5; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInStructure(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_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__3; 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*); @@ -561,6 +554,7 @@ static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structu static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1___closed__1; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addCtorFields___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_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_Lean_Expr_appFn_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___boxed(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_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -576,7 +570,9 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_el LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__5(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___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*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__2; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__5; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInStructure___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_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___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*); uint8_t lean_name_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -587,10 +583,11 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_ex static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instReprStructFieldKind; static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__7; -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___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_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___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_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUsed___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_throwErrorAt___at_Lean_Elab_Term_processDefDeriving___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_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__11; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___closed__1; lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -605,13 +602,14 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_ lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___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_Elab_Structure_0__Lean_Elab_Command_mkProjections___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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*); static lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__2; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4(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_Structure_0__Lean_Elab_Command_expandFields___spec__5___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*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__6; lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_mkFreshExprMVarImpl(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___lambda__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___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_object*, lean_object*, lean_object*, lean_object*); @@ -627,12 +625,12 @@ static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStr static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__5___closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__2(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___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__12; lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg(lean_object*, uint8_t, 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_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_processOveriddenDefaultValues___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* l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2(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_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__6; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___lambda__4___closed__5; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__3; lean_object* l_Lean_Elab_Term_withAutoBoundImplicitForbiddenPred___rarg(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_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__1; LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -644,8 +642,10 @@ static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure static lean_object* l_Lean_Elab_Command_StructFieldKind_noConfusion___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__2; lean_object* l_panic___at_Lean_mkNoConfusionEnum_mkToCtorIdx___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent___lambda__2___boxed(lean_object**); +static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__4; static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__4; static lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__7___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -656,7 +656,6 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_ LEAN_EXPORT lean_object* l_Lean_Elab_Command_instReprStructFieldInfo; lean_object* l_Lean_Meta_instInhabitedMetaM___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2(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_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__8; lean_object* l_Lean_addDocString_x27___at_Lean_Elab_Term_expandDeclId___spec__8(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_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__13; @@ -674,7 +673,7 @@ LEAN_EXPORT lean_object* l_Lean_ofExceptKernelException___at___private_Lean_Elab static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___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*); uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___closed__2; static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__4; static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__2; @@ -710,7 +709,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___priva static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__3; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__4(lean_object*); static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__2___closed__1; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__14; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___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*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__4; @@ -724,6 +722,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_co LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__2; uint8_t l_Lean_Syntax_isToken(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__10; static lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__2; static lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getResultUniverse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -740,7 +739,6 @@ lean_object* l_Lean_Elab_Term_addAutoBoundImplicits(lean_object*, lean_object*, lean_object* l_Lean_Elab_Term_addLocalVarInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_bindingDomain_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__2; lean_object* l_Lean_mkNoConfusion(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__2; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__11; @@ -756,6 +754,7 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0_ LEAN_EXPORT uint8_t l_Lean_Elab_Command_StructFieldInfo_isSubobject(lean_object*); extern lean_object* l_Lean_NameSet_empty; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___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_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___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_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withParents_go___rarg___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_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___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*); @@ -790,7 +789,6 @@ lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta lean_object* l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__11(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_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__5; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUsed___spec__1(lean_object*, size_t, size_t, 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_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4(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_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -802,25 +800,25 @@ static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFie lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___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_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__1(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_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__1(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* l_Lean_Elab_Term_elabBinders___rarg(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_Structure_0__Lean_Elab_Command_addDefaults___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_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___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_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__14; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_removeUnused___closed__4; lean_object* l_Lean_indentExpr(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParamFVar___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_Elab_Structure_0__Lean_Elab_Command_reduceProjs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__2; uint8_t l_Lean_BinderInfo_isExplicit(uint8_t); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__9; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_updateResultingUniverse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__1___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*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__8; LEAN_EXPORT uint8_t l___private_Lean_Elab_Structure_0__Lean_Elab_Command_levelMVarToParam_levelMVarToParam_x27___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990_(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabStructure___spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2___closed__2; lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); @@ -867,20 +865,22 @@ LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___at___private_Lean_Elab_Stru LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___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_Elab_Command_elabStructure___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__10; -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___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_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___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_Meta_addInstance(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_liftCoreM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__3___closed__1; static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___closed__2; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_failed___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_mkCompositeField___spec__2(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* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); lean_object* l_Lean_Elab_Term_withoutAutoBoundImplicit___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_isPrivateName(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_StructFieldKind_noConfusion(lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__4; static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__3; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_expandOptDeclSig(lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__7; @@ -905,6 +905,7 @@ static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Le LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___lambda__1___boxed(lean_object*); lean_object* l_List_reverse___rarg(lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__7; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy(lean_object*); lean_object* l_Lean_Meta_mkAuxDefinition(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); @@ -943,8 +944,10 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Stru LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2(lean_object*); static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__3; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_339____closed__3; +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__3; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__11; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkToParentName(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___boxed(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*); @@ -953,7 +956,6 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0_ LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___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_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_547____closed__25; static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getNestedProjectionArg___lambda__1___boxed(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*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__17(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -978,7 +980,6 @@ static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandF static lean_object* l_Lean_Elab_Command_instReprStructFieldKind___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__4___rarg___boxed(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_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__4; static lean_object* l_Lean_Elab_Command_elabStructure___closed__6; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectUniversesFromFields_go___spec__2___closed__1; static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20___closed__5; @@ -1021,6 +1022,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_wi LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__3___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_Structure_0__Lean_Elab_Command_updateFieldInfoVal(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Exception_isRuntime(lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__4; static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__8___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___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5(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*); @@ -1031,7 +1033,6 @@ LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_ static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___closed__3; uint8_t l_Lean_Expr_isFVar(lean_object*); uint8_t l_Lean_Expr_isForall(lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__10; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__4___boxed(lean_object**); lean_object* l_Lean_expandMacros(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getStructureFieldsFlattened(lean_object*, lean_object*, uint8_t); @@ -1075,6 +1076,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_co static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7; LEAN_EXPORT lean_object* l_Lean_Linter_logLintIf___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__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_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__18(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_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__8; lean_object* l_Lean_addDecl(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__6___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___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*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -4241,146 +4243,151 @@ return x_32; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, uint8_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_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__1(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_object* x_13, lean_object* x_14) { _start: { -uint8_t x_14; uint8_t x_15; -x_14 = l_Lean_Syntax_isNone(x_1); -x_15 = l_Lean_Syntax_isNone(x_2); -if (x_14 == 0) -{ +uint8_t x_15; uint8_t x_16; +x_15 = l_Lean_Syntax_isNone(x_1); +x_16 = l_Lean_Syntax_isNone(x_2); if (x_15 == 0) { -uint8_t x_16; lean_object* x_17; lean_object* x_18; -x_16 = 1; -x_17 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_17, 0, x_3); -lean_ctor_set(x_17, 1, x_6); -lean_ctor_set_uint8(x_17, sizeof(void*)*2, x_4); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 1, x_16); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 2, x_5); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 3, 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_13); -return x_18; +if (x_16 == 0) +{ +uint8_t x_17; lean_object* x_18; lean_object* x_19; +x_17 = 1; +x_18 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_18, 0, x_3); +lean_ctor_set(x_18, 1, x_4); +lean_ctor_set(x_18, 2, x_7); +lean_ctor_set_uint8(x_18, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 1, x_17); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_18, sizeof(void*)*3 + 3, 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_14); +return x_19; } else { -uint8_t x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; -x_19 = 1; -x_20 = 0; -x_21 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_21, 0, x_3); -lean_ctor_set(x_21, 1, x_6); -lean_ctor_set_uint8(x_21, sizeof(void*)*2, x_4); -lean_ctor_set_uint8(x_21, sizeof(void*)*2 + 1, x_19); -lean_ctor_set_uint8(x_21, sizeof(void*)*2 + 2, x_5); -lean_ctor_set_uint8(x_21, sizeof(void*)*2 + 3, 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_13); -return x_22; +uint8_t x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; +x_20 = 1; +x_21 = 0; +x_22 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_22, 0, x_3); +lean_ctor_set(x_22, 1, x_4); +lean_ctor_set(x_22, 2, x_7); +lean_ctor_set_uint8(x_22, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 1, x_20); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_22, sizeof(void*)*3 + 3, 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_14); +return x_23; } } else { -if (x_15 == 0) +if (x_16 == 0) { -uint8_t x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; -x_23 = 0; -x_24 = 1; -x_25 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_25, 0, x_3); -lean_ctor_set(x_25, 1, x_6); -lean_ctor_set_uint8(x_25, sizeof(void*)*2, x_4); -lean_ctor_set_uint8(x_25, sizeof(void*)*2 + 1, x_23); -lean_ctor_set_uint8(x_25, sizeof(void*)*2 + 2, x_5); -lean_ctor_set_uint8(x_25, sizeof(void*)*2 + 3, 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_13); -return x_26; +uint8_t x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; +x_24 = 0; +x_25 = 1; +x_26 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_26, 0, x_3); +lean_ctor_set(x_26, 1, x_4); +lean_ctor_set(x_26, 2, x_7); +lean_ctor_set_uint8(x_26, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_26, sizeof(void*)*3 + 1, x_24); +lean_ctor_set_uint8(x_26, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_26, sizeof(void*)*3 + 3, 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_14); +return x_27; } else { -uint8_t x_27; lean_object* x_28; lean_object* x_29; -x_27 = 0; -x_28 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_28, 0, x_3); -lean_ctor_set(x_28, 1, x_6); -lean_ctor_set_uint8(x_28, sizeof(void*)*2, x_4); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 1, x_27); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 2, x_5); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 3, 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_13); -return x_29; +uint8_t x_28; lean_object* x_29; lean_object* x_30; +x_28 = 0; +x_29 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_29, 0, x_3); +lean_ctor_set(x_29, 1, x_4); +lean_ctor_set(x_29, 2, x_7); +lean_ctor_set_uint8(x_29, sizeof(void*)*3, x_5); +lean_ctor_set_uint8(x_29, sizeof(void*)*3 + 1, x_28); +lean_ctor_set_uint8(x_29, sizeof(void*)*3 + 2, x_6); +lean_ctor_set_uint8(x_29, sizeof(void*)*3 + 3, 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_14); +return x_30; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t 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_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2(lean_object* x_1, lean_object* x_2, 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, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_14; -x_14 = l_Lean_Syntax_getOptional_x3f(x_5); -if (lean_obj_tag(x_14) == 0) +lean_object* x_15; +x_15 = l_Lean_Syntax_getOptional_x3f(x_6); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_15; lean_object* x_16; -x_15 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_16 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__1(x_1, x_2, x_3, x_6, x_4, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_11); -lean_dec(x_7); -return x_16; +lean_object* x_16; lean_object* x_17; +x_16 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; +x_17 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_7, x_5, x_16, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_12); +lean_dec(x_8); +return x_17; } else { -lean_object* x_17; lean_object* x_18; -x_17 = lean_ctor_get(x_14, 0); -lean_inc(x_17); -lean_dec(x_14); -lean_inc(x_11); -lean_inc(x_7); -x_18 = l_Lean_Elab_elabDeclAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__2(x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_17); -if (lean_obj_tag(x_18) == 0) +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_15, 0); +lean_inc(x_18); +lean_dec(x_15); +lean_inc(x_12); +lean_inc(x_8); +x_19 = l_Lean_Elab_elabDeclAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__2(x_18, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_18); +if (lean_obj_tag(x_19) == 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_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_19, 0); lean_inc(x_20); -lean_dec(x_18); -x_21 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__1(x_1, x_2, x_3, x_6, x_4, x_19, x_7, x_8, x_9, x_10, x_11, x_12, x_20); -lean_dec(x_11); -lean_dec(x_7); -return x_21; +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_7, x_5, x_20, x_8, x_9, x_10, x_11, x_12, x_13, x_21); +lean_dec(x_12); +lean_dec(x_8); +return x_22; } else { -uint8_t x_22; -lean_dec(x_11); -lean_dec(x_7); +uint8_t x_23; +lean_dec(x_12); +lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); -x_22 = !lean_is_exclusive(x_18); -if (x_22 == 0) +x_23 = !lean_is_exclusive(x_19); +if (x_23 == 0) { -return x_18; +return x_19; } else { -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_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_19, 0); +x_25 = lean_ctor_get(x_19, 1); +lean_inc(x_25); 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; +lean_dec(x_19); +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; } } } @@ -4451,77 +4458,78 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___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_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___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_14; -x_14 = l_Lean_Syntax_getOptional_x3f(x_5); -if (lean_obj_tag(x_14) == 0) +lean_object* x_15; +x_15 = l_Lean_Syntax_getOptional_x3f(x_6); +if (lean_obj_tag(x_15) == 0) { -uint8_t x_15; lean_object* x_16; -x_15 = 0; -x_16 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2(x_1, x_2, x_6, x_3, x_4, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_16; +uint8_t x_16; lean_object* x_17; +x_16 = 0; +x_17 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2(x_1, x_2, x_3, x_7, x_4, x_5, x_16, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_17; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_17 = lean_ctor_get(x_14, 0); -lean_inc(x_17); -lean_dec(x_14); -lean_inc(x_17); -x_18 = l_Lean_Syntax_getKind(x_17); -x_19 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__3; -x_20 = lean_name_eq(x_18, x_19); -if (x_20 == 0) +lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_18 = lean_ctor_get(x_15, 0); +lean_inc(x_18); +lean_dec(x_15); +lean_inc(x_18); +x_19 = l_Lean_Syntax_getKind(x_18); +x_20 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__3; +x_21 = lean_name_eq(x_19, x_20); +if (x_21 == 0) { -lean_object* x_21; uint8_t x_22; -x_21 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__5; -x_22 = lean_name_eq(x_18, x_21); -lean_dec(x_18); -if (x_22 == 0) +lean_object* x_22; uint8_t x_23; +x_22 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__5; +x_23 = lean_name_eq(x_19, x_22); +lean_dec(x_19); +if (x_23 == 0) { -lean_object* x_23; lean_object* x_24; uint8_t x_25; -lean_dec(x_6); -x_23 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__7; -x_24 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__12(x_17, x_23, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_17); -x_25 = !lean_is_exclusive(x_24); -if (x_25 == 0) +lean_object* x_24; lean_object* x_25; uint8_t x_26; +lean_dec(x_7); +lean_dec(x_3); +x_24 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__7; +x_25 = l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__12(x_18, x_24, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_18); +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) { -return x_24; +return x_25; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_24, 0); -x_27 = lean_ctor_get(x_24, 1); +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_25, 0); +x_28 = lean_ctor_get(x_25, 1); +lean_inc(x_28); lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_24); -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_dec(x_25); +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_29; lean_object* x_30; -lean_dec(x_17); -x_29 = 1; -x_30 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2(x_1, x_2, x_6, x_3, x_4, x_29, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_30; +uint8_t x_30; lean_object* x_31; +lean_dec(x_18); +x_30 = 1; +x_31 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2(x_1, x_2, x_3, x_7, x_4, x_5, x_30, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_31; } } else { -uint8_t x_31; lean_object* x_32; +uint8_t x_32; lean_object* x_33; +lean_dec(x_19); lean_dec(x_18); -lean_dec(x_17); -x_31 = 2; -x_32 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2(x_1, x_2, x_6, x_3, x_4, x_31, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_32; +x_32 = 2; +x_33 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2(x_1, x_2, x_3, x_7, x_4, x_5, x_32, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_33; } } } @@ -4603,7 +4611,7 @@ if (lean_obj_tag(x_22) == 0) { lean_object* x_24; lean_object* x_25; x_24 = lean_box(0); -x_25 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3(x_16, x_18, x_23, x_12, x_14, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_25 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3(x_16, x_18, x_1, x_23, x_12, x_14, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_14); lean_dec(x_12); lean_dec(x_18); @@ -4631,7 +4639,7 @@ x_30 = lean_ctor_get(x_28, 1); lean_inc(x_30); lean_dec(x_28); lean_ctor_set(x_22, 0, x_29); -x_31 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3(x_16, x_18, x_23, x_12, x_14, x_22, x_2, x_3, x_4, x_5, x_6, x_7, x_30); +x_31 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3(x_16, x_18, x_1, x_23, x_12, x_14, x_22, x_2, x_3, x_4, x_5, x_6, x_7, x_30); lean_dec(x_14); lean_dec(x_12); lean_dec(x_18); @@ -4648,6 +4656,7 @@ lean_dec(x_14); lean_dec(x_12); lean_dec(x_6); lean_dec(x_2); +lean_dec(x_1); x_32 = !lean_is_exclusive(x_28); if (x_32 == 0) { @@ -4688,7 +4697,7 @@ lean_inc(x_39); lean_dec(x_37); x_40 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_40, 0, x_38); -x_41 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3(x_16, x_18, x_23, x_12, x_14, x_40, x_2, x_3, x_4, x_5, x_6, x_7, x_39); +x_41 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3(x_16, x_18, x_1, x_23, x_12, x_14, x_40, x_2, x_3, x_4, x_5, x_6, x_7, x_39); lean_dec(x_14); lean_dec(x_12); lean_dec(x_18); @@ -4704,6 +4713,7 @@ lean_dec(x_14); lean_dec(x_12); lean_dec(x_6); lean_dec(x_2); +lean_dec(x_1); x_42 = lean_ctor_get(x_37, 0); lean_inc(x_42); x_43 = lean_ctor_get(x_37, 1); @@ -4751,7 +4761,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___priva _start: { lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = lean_ctor_get(x_1, 1); +x_10 = lean_ctor_get(x_1, 2); x_11 = lean_array_get_size(x_10); x_12 = lean_unsigned_to_nat(0u); x_13 = lean_nat_dec_eq(x_11, x_12); @@ -4796,7 +4806,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___priva _start: { uint8_t x_10; -x_10 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); +x_10 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); if (x_10 == 0) { lean_object* x_11; lean_object* x_12; @@ -4906,7 +4916,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___priva _start: { uint8_t x_9; -x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); if (x_9 == 0) { lean_object* x_10; lean_object* x_11; @@ -4940,237 +4950,146 @@ return x_17; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_object* x_7, lean_object* x_8) { _start: { -lean_object* x_9; uint8_t 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 = 0; -x_11 = l_Lean_Syntax_getPos_x3f(x_1, x_10); -x_12 = l_Lean_Syntax_getTailPos_x3f(x_1, x_10); -if (lean_obj_tag(x_11) == 0) +uint8_t x_9; lean_object* x_10; +x_9 = 0; +x_10 = l_Lean_Syntax_getRange_x3f(x_1, x_9); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_unsigned_to_nat(0u); -lean_inc(x_9); -x_14 = l_Lean_FileMap_toPosition(x_9, x_13); -lean_inc(x_14); -x_15 = l_Lean_FileMap_leanPosToLspPos(x_9, x_14); -if (lean_obj_tag(x_12) == 0) +lean_object* x_11; lean_object* x_12; +lean_dec(x_6); +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_8); +return x_12; +} +else { -uint8_t x_16; -lean_dec(x_9); -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) +uint8_t x_13; +x_13 = !lean_is_exclusive(x_10); +if (x_13 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_15, 1); -x_18 = lean_ctor_get(x_15, 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_10, 0); +x_15 = lean_ctor_get(x_6, 1); +lean_inc(x_15); +lean_dec(x_6); +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_inc(x_15); +x_17 = l_Lean_FileMap_toPosition(x_15, x_16); +lean_dec(x_16); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_dec(x_14); +lean_inc(x_15); +x_19 = l_Lean_FileMap_toPosition(x_15, x_18); lean_dec(x_18); lean_inc(x_17); -lean_inc(x_14); -x_19 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_19, 0, x_14); -lean_ctor_set(x_19, 1, x_17); -lean_ctor_set(x_19, 2, x_14); -lean_ctor_set(x_19, 3, x_17); -lean_ctor_set(x_15, 1, x_8); -lean_ctor_set(x_15, 0, x_19); -return x_15; -} -else +x_20 = l_Lean_FileMap_leanPosToLspPos(x_15, x_17); +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) { -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_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, 1); +x_23 = lean_ctor_get(x_20, 0); +lean_dec(x_23); +lean_inc(x_19); +x_24 = l_Lean_FileMap_leanPosToLspPos(x_15, x_19); lean_dec(x_15); -lean_inc(x_20); -lean_inc(x_14); -x_21 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_21, 0, x_14); -lean_ctor_set(x_21, 1, x_20); -lean_ctor_set(x_21, 2, x_14); -lean_ctor_set(x_21, 3, 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_8); -return x_22; -} +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_26, 0, x_17); +lean_ctor_set(x_26, 1, x_22); +lean_ctor_set(x_26, 2, x_19); +lean_ctor_set(x_26, 3, x_25); +lean_ctor_set(x_10, 0, x_26); +lean_ctor_set(x_20, 1, x_8); +lean_ctor_set(x_20, 0, x_10); +return x_20; } else { -uint8_t x_23; -x_23 = !lean_is_exclusive(x_15); -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 = lean_ctor_get(x_15, 1); -x_25 = lean_ctor_get(x_15, 0); -lean_dec(x_25); -x_26 = lean_ctor_get(x_12, 0); -lean_inc(x_26); -lean_dec(x_12); -lean_inc(x_9); -x_27 = l_Lean_FileMap_toPosition(x_9, x_26); -lean_dec(x_26); +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_27 = lean_ctor_get(x_20, 1); lean_inc(x_27); -x_28 = l_Lean_FileMap_leanPosToLspPos(x_9, x_27); -lean_dec(x_9); +lean_dec(x_20); +lean_inc(x_19); +x_28 = l_Lean_FileMap_leanPosToLspPos(x_15, x_19); +lean_dec(x_15); x_29 = lean_ctor_get(x_28, 1); lean_inc(x_29); lean_dec(x_28); x_30 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_30, 0, x_14); -lean_ctor_set(x_30, 1, x_24); -lean_ctor_set(x_30, 2, x_27); +lean_ctor_set(x_30, 0, x_17); +lean_ctor_set(x_30, 1, x_27); +lean_ctor_set(x_30, 2, x_19); lean_ctor_set(x_30, 3, x_29); -lean_ctor_set(x_15, 1, x_8); -lean_ctor_set(x_15, 0, x_30); -return x_15; +lean_ctor_set(x_10, 0, x_30); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_10); +lean_ctor_set(x_31, 1, x_8); +return x_31; +} } 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_15, 1); -lean_inc(x_31); -lean_dec(x_15); -x_32 = lean_ctor_get(x_12, 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; lean_object* x_44; lean_object* x_45; +x_32 = lean_ctor_get(x_10, 0); lean_inc(x_32); -lean_dec(x_12); -lean_inc(x_9); -x_33 = l_Lean_FileMap_toPosition(x_9, x_32); +lean_dec(x_10); +x_33 = lean_ctor_get(x_6, 1); +lean_inc(x_33); +lean_dec(x_6); +x_34 = lean_ctor_get(x_32, 0); +lean_inc(x_34); +lean_inc(x_33); +x_35 = l_Lean_FileMap_toPosition(x_33, x_34); +lean_dec(x_34); +x_36 = lean_ctor_get(x_32, 1); +lean_inc(x_36); lean_dec(x_32); lean_inc(x_33); -x_34 = l_Lean_FileMap_leanPosToLspPos(x_9, x_33); -lean_dec(x_9); -x_35 = lean_ctor_get(x_34, 1); +x_37 = l_Lean_FileMap_toPosition(x_33, x_36); +lean_dec(x_36); lean_inc(x_35); -lean_dec(x_34); -x_36 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_36, 0, x_14); -lean_ctor_set(x_36, 1, x_31); -lean_ctor_set(x_36, 2, x_33); -lean_ctor_set(x_36, 3, 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; -} -} -} -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_11, 0); -lean_inc(x_38); -lean_dec(x_11); -lean_inc(x_9); -x_39 = l_Lean_FileMap_toPosition(x_9, x_38); -lean_dec(x_38); -lean_inc(x_39); -x_40 = l_Lean_FileMap_leanPosToLspPos(x_9, x_39); -if (lean_obj_tag(x_12) == 0) -{ -uint8_t x_41; -lean_dec(x_9); -x_41 = !lean_is_exclusive(x_40); -if (x_41 == 0) -{ -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_40, 1); -x_43 = lean_ctor_get(x_40, 0); -lean_dec(x_43); -lean_inc(x_42); -lean_inc(x_39); -x_44 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_44, 0, x_39); -lean_ctor_set(x_44, 1, x_42); -lean_ctor_set(x_44, 2, x_39); -lean_ctor_set(x_44, 3, x_42); -lean_ctor_set(x_40, 1, x_8); -lean_ctor_set(x_40, 0, x_44); -return x_40; -} -else -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_40, 1); -lean_inc(x_45); -lean_dec(x_40); -lean_inc(x_45); +x_38 = l_Lean_FileMap_leanPosToLspPos(x_33, x_35); +x_39 = lean_ctor_get(x_38, 1); lean_inc(x_39); -x_46 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_46, 0, x_39); -lean_ctor_set(x_46, 1, x_45); -lean_ctor_set(x_46, 2, x_39); -lean_ctor_set(x_46, 3, 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_8); -return x_47; -} -} -else -{ -uint8_t x_48; -x_48 = !lean_is_exclusive(x_40); -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; -x_49 = lean_ctor_get(x_40, 1); -x_50 = lean_ctor_get(x_40, 0); -lean_dec(x_50); -x_51 = lean_ctor_get(x_12, 0); -lean_inc(x_51); -lean_dec(x_12); -lean_inc(x_9); -x_52 = l_Lean_FileMap_toPosition(x_9, x_51); -lean_dec(x_51); -lean_inc(x_52); -x_53 = l_Lean_FileMap_leanPosToLspPos(x_9, x_52); -lean_dec(x_9); -x_54 = lean_ctor_get(x_53, 1); -lean_inc(x_54); -lean_dec(x_53); -x_55 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_55, 0, x_39); -lean_ctor_set(x_55, 1, x_49); -lean_ctor_set(x_55, 2, x_52); -lean_ctor_set(x_55, 3, x_54); -lean_ctor_set(x_40, 1, x_8); -lean_ctor_set(x_40, 0, x_55); -return x_40; +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); } -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_40, 1); -lean_inc(x_56); -lean_dec(x_40); -x_57 = lean_ctor_get(x_12, 0); -lean_inc(x_57); -lean_dec(x_12); -lean_inc(x_9); -x_58 = l_Lean_FileMap_toPosition(x_9, x_57); -lean_dec(x_57); -lean_inc(x_58); -x_59 = l_Lean_FileMap_leanPosToLspPos(x_9, x_58); -lean_dec(x_9); -x_60 = lean_ctor_get(x_59, 1); -lean_inc(x_60); -lean_dec(x_59); -x_61 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_61, 0, x_39); -lean_ctor_set(x_61, 1, x_56); -lean_ctor_set(x_61, 2, x_58); -lean_ctor_set(x_61, 3, x_60); -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_8); -return x_62; +lean_inc(x_37); +x_41 = l_Lean_FileMap_leanPosToLspPos(x_33, x_37); +lean_dec(x_33); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +x_43 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_43, 0, x_35); +lean_ctor_set(x_43, 1, x_39); +lean_ctor_set(x_43, 2, x_37); +lean_ctor_set(x_43, 3, x_42); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +if (lean_is_scalar(x_40)) { + x_45 = lean_alloc_ctor(0, 2, 0); +} else { + x_45 = x_40; } +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_8); +return x_45; } } } @@ -5617,42 +5536,97 @@ return x_116; LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__18(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, 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; uint8_t x_15; +lean_object* x_11; lean_object* x_12; lean_inc(x_8); -x_11 = l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(x_2, 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_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -lean_inc(x_8); -x_14 = l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) +if (lean_obj_tag(x_12) == 0) { -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_ctor_set(x_14, 1, x_16); -lean_ctor_set(x_14, 0, x_12); -x_18 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20(x_1, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_17); +uint8_t x_13; lean_dec(x_8); +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 = lean_box(0); +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 = 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; } +} else { 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_ctor_get(x_14, 1); -lean_inc(x_20); +x_19 = lean_ctor_get(x_11, 1); lean_inc(x_19); -lean_dec(x_14); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_12); -lean_ctor_set(x_21, 1, x_19); -x_22 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20(x_1, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_20); +lean_dec(x_11); +x_20 = lean_ctor_get(x_12, 0); +lean_inc(x_20); +lean_dec(x_12); +lean_inc(x_8); +x_21 = l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_19); +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_20); lean_dec(x_8); -return x_22; +lean_dec(x_1); +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 = lean_box(0); +lean_ctor_set(x_21, 0, x_25); +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 = 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_26); +return x_28; +} +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +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); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_20); +lean_ctor_set(x_31, 1, x_30); +x_32 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20(x_1, x_31, x_4, x_5, x_6, x_7, x_8, x_9, x_29); +lean_dec(x_8); +return x_32; +} } } } @@ -5665,7 +5639,7 @@ x_13 = l_Lean_Syntax_getArg(x_1, x_12); x_14 = l_Lean_Syntax_getId(x_13); lean_inc(x_14); x_15 = l_Lean_Name_append(x_2, x_14); -x_16 = lean_ctor_get_uint8(x_3, sizeof(void*)*2); +x_16 = lean_ctor_get_uint8(x_3, sizeof(void*)*3); lean_inc(x_5); x_17 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5(x_16, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11); if (lean_obj_tag(x_17) == 0) @@ -5676,7 +5650,7 @@ 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_3, 0); +x_20 = lean_ctor_get(x_3, 1); lean_inc(x_20); lean_inc(x_5); lean_inc(x_18); @@ -5869,20 +5843,31 @@ return x_2; static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3() { _start: { -lean_object* x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +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___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; x_1 = lean_box(0); -x_2 = 0; +x_2 = lean_box(0); x_3 = 0; -x_4 = 2; -x_5 = l_Lean_Elab_elabAttrs___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__3___closed__1; -x_6 = lean_alloc_ctor(0, 2, 4); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -lean_ctor_set_uint8(x_6, sizeof(void*)*2, x_2); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 1, x_3); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 2, x_4); -lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 3, x_3); -return x_6; +x_4 = 0; +x_5 = 0; +x_6 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3; +x_7 = lean_alloc_ctor(0, 3, 4); +lean_ctor_set(x_7, 0, x_2); +lean_ctor_set(x_7, 1, x_1); +lean_ctor_set(x_7, 2, x_6); +lean_ctor_set_uint8(x_7, sizeof(void*)*3, x_3); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 1, x_4); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 2, x_5); +lean_ctor_set_uint8(x_7, sizeof(void*)*3 + 3, x_4); +return x_7; } } LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { @@ -5924,7 +5909,6 @@ lean_ctor_set(x_8, 5, x_26); lean_inc(x_8); lean_inc(x_4); x_27 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1(x_23, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_23); if (lean_obj_tag(x_27) == 0) { lean_object* x_28; lean_object* x_29; lean_object* x_30; @@ -6097,7 +6081,6 @@ lean_ctor_set_uint8(x_67, sizeof(void*)*12 + 1, x_65); lean_inc(x_67); lean_inc(x_4); x_68 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1(x_23, x_4, x_5, x_6, x_7, x_67, x_9, x_10); -lean_dec(x_23); if (lean_obj_tag(x_68) == 0) { lean_object* x_69; lean_object* x_70; lean_object* x_71; @@ -6241,7 +6224,7 @@ if (x_94 == 0) lean_object* x_95; lean_object* x_96; lean_object* x_97; x_95 = lean_ctor_get(x_93, 0); lean_dec(x_95); -x_96 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3; +x_96 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__4; x_97 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_97, 0, x_15); lean_ctor_set(x_97, 1, x_96); @@ -6256,7 +6239,7 @@ lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; x_98 = lean_ctor_get(x_93, 1); lean_inc(x_98); lean_dec(x_93); -x_99 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3; +x_99 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__4; x_100 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_100, 0, x_15); lean_ctor_set(x_100, 1, x_99); @@ -6283,7 +6266,7 @@ if (x_103 == 0) lean_object* x_104; lean_object* x_105; lean_object* x_106; x_104 = lean_ctor_get(x_102, 0); lean_dec(x_104); -x_105 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3; +x_105 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__4; x_106 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_106, 0, x_15); lean_ctor_set(x_106, 1, x_105); @@ -6298,7 +6281,7 @@ lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; x_107 = lean_ctor_get(x_102, 1); lean_inc(x_107); lean_dec(x_102); -x_108 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3; +x_108 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__4; x_109 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_109, 0, x_15); lean_ctor_set(x_109, 1, x_108); @@ -6576,61 +6559,61 @@ lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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, lean_object* x_14) { _start: { -uint8_t x_14; uint8_t x_15; lean_object* x_16; -x_14 = lean_unbox(x_4); -lean_dec(x_4); +uint8_t x_15; uint8_t x_16; lean_object* x_17; x_15 = lean_unbox(x_5); lean_dec(x_5); -x_16 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__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); +x_16 = lean_unbox(x_6); +lean_dec(x_6); +x_17 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__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_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; +return x_17; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { _start: { -uint8_t x_14; uint8_t x_15; lean_object* x_16; -x_14 = lean_unbox(x_4); -lean_dec(x_4); -x_15 = lean_unbox(x_6); -lean_dec(x_6); -x_16 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2(x_1, x_2, x_3, x_14, x_5, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_12); +uint8_t x_15; uint8_t x_16; lean_object* x_17; +x_15 = lean_unbox(x_5); +lean_dec(x_5); +x_16 = lean_unbox(x_7); +lean_dec(x_7); +x_17 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_15, x_6, x_16, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_13); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_5); +lean_dec(x_6); lean_dec(x_2); lean_dec(x_1); -return x_16; +return x_17; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { _start: { -uint8_t x_14; lean_object* x_15; -x_14 = lean_unbox(x_3); -lean_dec(x_3); -x_15 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3(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); +uint8_t x_15; lean_object* x_16; +x_15 = lean_unbox(x_4); +lean_dec(x_4); +x_16 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___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_13); +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_2); lean_dec(x_1); -return x_15; +return x_16; } } LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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) { @@ -6642,7 +6625,6 @@ lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_1); return x_9; } } @@ -6705,11 +6687,11 @@ lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___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_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); @@ -6812,7 +6794,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__1 _start: { lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = lean_ctor_get(x_1, 1); +x_10 = lean_ctor_get(x_1, 2); x_11 = lean_array_get_size(x_10); x_12 = lean_unsigned_to_nat(0u); x_13 = lean_nat_dec_eq(x_11, x_12); @@ -6857,7 +6839,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier___lambda__2 _start: { uint8_t x_10; -x_10 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); +x_10 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 3); if (x_10 == 0) { lean_object* x_11; lean_object* x_12; @@ -6967,7 +6949,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidFieldModifier(lean_object _start: { uint8_t x_9; -x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); if (x_9 == 0) { lean_object* x_10; lean_object* x_11; @@ -7066,7 +7048,7 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Stru lean_object* x_19; uint8_t x_20; lean_object* x_21; lean_inc(x_2); x_19 = l_Lean_Name_append(x_1, x_2); -x_20 = lean_ctor_get_uint8(x_3, sizeof(void*)*2); +x_20 = lean_ctor_get_uint8(x_3, sizeof(void*)*3); lean_inc(x_12); x_21 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5(x_20, x_19, x_12, x_13, x_14, x_15, x_16, x_17, x_18); if (lean_obj_tag(x_21) == 0) @@ -7077,7 +7059,7 @@ 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_3, 0); +x_24 = lean_ctor_get(x_3, 1); lean_inc(x_24); lean_inc(x_22); x_25 = l_Lean_addDocString_x27___at_Lean_Elab_Term_expandDeclId___spec__8(x_22, x_24, x_12, x_13, x_14, x_15, x_16, x_17, x_23); @@ -7831,33 +7813,24 @@ return x_3; static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7() { _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_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__8() { -_start: -{ lean_object* x_1; x_1 = lean_mk_string_unchecked("app", 3, 3); return x_1; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__9() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___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_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__2; x_3 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__3; -x_4 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__8; +x_4 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__10() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__9() { _start: { lean_object* x_1; @@ -7865,56 +7838,56 @@ x_1 = lean_mk_string_unchecked("autoParam", 9, 9); return x_1; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__10; +x_1 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__9; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__10; +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__9; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__13() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12; +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11; 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_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__13; +x_2 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12; 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_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__15() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14() { _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_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; -x_3 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7; +x_3 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3; x_4 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -8095,7 +8068,7 @@ lean_ctor_set(x_59, 1, x_63); lean_ctor_set(x_59, 0, x_58); x_64 = l_Lean_Syntax_getArgs(x_32); lean_dec(x_32); -x_65 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7; +x_65 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3; x_66 = l_Array_append___rarg(x_65, x_64); lean_dec(x_64); x_67 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; @@ -8129,10 +8102,10 @@ x_78 = lean_ctor_get(x_76, 0); lean_inc(x_78); lean_dec(x_76); x_79 = lean_environment_main_module(x_78); -x_80 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12; +x_80 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11; x_81 = l_Lean_addMacroScope(x_79, x_80, x_74); -x_82 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11; -x_83 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14; +x_82 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__10; +x_83 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__13; lean_inc(x_58); x_84 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_84, 0, x_58); @@ -8143,10 +8116,10 @@ x_85 = l_Lean_mkIdentFrom(x_52, x_54, x_57); lean_dec(x_52); lean_inc(x_58); x_86 = l_Lean_Syntax_node2(x_58, x_67, x_73, x_85); -x_87 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__9; +x_87 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__8; x_88 = l_Lean_Syntax_node2(x_58, x_87, x_84, x_86); lean_ctor_set(x_33, 0, x_88); -x_89 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__15; +x_89 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14; lean_ctor_set(x_30, 0, x_89); x_90 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5, x_30, x_7, x_8, x_9, x_10, x_11, x_12, x_77); lean_dec(x_12); @@ -8169,7 +8142,7 @@ lean_ctor_set(x_93, 0, x_58); lean_ctor_set(x_93, 1, x_92); x_94 = l_Lean_Syntax_getArgs(x_32); lean_dec(x_32); -x_95 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7; +x_95 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3; x_96 = l_Array_append___rarg(x_95, x_94); lean_dec(x_94); x_97 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; @@ -8203,10 +8176,10 @@ x_108 = lean_ctor_get(x_106, 0); lean_inc(x_108); lean_dec(x_106); x_109 = lean_environment_main_module(x_108); -x_110 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12; +x_110 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11; x_111 = l_Lean_addMacroScope(x_109, x_110, x_104); -x_112 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11; -x_113 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14; +x_112 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__10; +x_113 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__13; lean_inc(x_58); x_114 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_114, 0, x_58); @@ -8217,10 +8190,10 @@ x_115 = l_Lean_mkIdentFrom(x_52, x_54, x_57); lean_dec(x_52); lean_inc(x_58); x_116 = l_Lean_Syntax_node2(x_58, x_97, x_103, x_115); -x_117 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__9; +x_117 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__8; x_118 = l_Lean_Syntax_node2(x_58, x_117, x_114, x_116); lean_ctor_set(x_33, 0, x_118); -x_119 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__15; +x_119 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14; lean_ctor_set(x_30, 0, x_119); x_120 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5, x_30, x_7, x_8, x_9, x_10, x_11, x_12, x_107); lean_dec(x_12); @@ -8321,7 +8294,7 @@ lean_ctor_set(x_138, 0, x_133); lean_ctor_set(x_138, 1, x_137); x_139 = l_Lean_Syntax_getArgs(x_32); lean_dec(x_32); -x_140 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7; +x_140 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3; x_141 = l_Array_append___rarg(x_140, x_139); lean_dec(x_139); x_142 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; @@ -8355,10 +8328,10 @@ x_153 = lean_ctor_get(x_151, 0); lean_inc(x_153); lean_dec(x_151); x_154 = lean_environment_main_module(x_153); -x_155 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12; +x_155 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11; x_156 = l_Lean_addMacroScope(x_154, x_155, x_149); -x_157 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11; -x_158 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14; +x_157 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__10; +x_158 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__13; lean_inc(x_133); x_159 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_159, 0, x_133); @@ -8369,11 +8342,11 @@ x_160 = l_Lean_mkIdentFrom(x_127, x_129, x_132); lean_dec(x_127); lean_inc(x_133); x_161 = l_Lean_Syntax_node2(x_133, x_142, x_148, x_160); -x_162 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__9; +x_162 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__8; x_163 = l_Lean_Syntax_node2(x_133, x_162, x_159, x_161); x_164 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_164, 0, x_163); -x_165 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__15; +x_165 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14; lean_ctor_set(x_30, 1, x_164); lean_ctor_set(x_30, 0, x_165); x_166 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5, x_30, x_7, x_8, x_9, x_10, x_11, x_12, x_152); @@ -8571,7 +8544,7 @@ lean_ctor_set(x_204, 0, x_199); lean_ctor_set(x_204, 1, x_203); x_205 = l_Lean_Syntax_getArgs(x_172); lean_dec(x_172); -x_206 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7; +x_206 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3; x_207 = l_Array_append___rarg(x_206, x_205); lean_dec(x_205); x_208 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; @@ -8605,10 +8578,10 @@ x_219 = lean_ctor_get(x_217, 0); lean_inc(x_219); lean_dec(x_217); x_220 = lean_environment_main_module(x_219); -x_221 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12; +x_221 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11; x_222 = l_Lean_addMacroScope(x_220, x_221, x_215); -x_223 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11; -x_224 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14; +x_223 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__10; +x_224 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__13; lean_inc(x_199); x_225 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_225, 0, x_199); @@ -8619,7 +8592,7 @@ x_226 = l_Lean_mkIdentFrom(x_193, x_195, x_198); lean_dec(x_193); lean_inc(x_199); x_227 = l_Lean_Syntax_node2(x_199, x_208, x_214, x_226); -x_228 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__9; +x_228 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__8; x_229 = l_Lean_Syntax_node2(x_199, x_228, x_225, x_227); if (lean_is_scalar(x_191)) { x_230 = lean_alloc_ctor(1, 1, 0); @@ -8627,7 +8600,7 @@ if (lean_is_scalar(x_191)) { x_230 = x_191; } lean_ctor_set(x_230, 0, x_229); -x_231 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__15; +x_231 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14; x_232 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_232, 0, x_231); lean_ctor_set(x_232, 1, x_230); @@ -8799,7 +8772,6 @@ x_14 = l_Lean_Syntax_getArg(x_1, x_13); lean_inc(x_10); lean_inc(x_6); x_15 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1(x_14, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_14); if (lean_obj_tag(x_15) == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; @@ -10802,7 +10774,7 @@ lean_dec(x_2); return x_4; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__1() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__1() { _start: { lean_object* x_1; @@ -10810,17 +10782,17 @@ x_1 = lean_mk_string_unchecked("structureDiamondWarning", 23, 23); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__2() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____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_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__1; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__3() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__3() { _start: { lean_object* x_1; @@ -10828,13 +10800,13 @@ x_1 = lean_mk_string_unchecked("enable/disable warning messages for structure di return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__4() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____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_getDocStringText___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__14___closed__3; -x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__3; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__3; x_4 = lean_box(x_1); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_4); @@ -10843,7 +10815,7 @@ lean_ctor_set(x_5, 2, x_3); return x_5; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__5() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__5() { _start: { lean_object* x_1; @@ -10851,25 +10823,25 @@ x_1 = lean_mk_string_unchecked("Elab", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__6() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____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_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__1; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__5; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__5; x_3 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1; -x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__1; +x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984_(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_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__2; -x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__4; -x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__6; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__2; +x_3 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__4; +x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__6; 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; } @@ -12032,7 +12004,7 @@ x_24 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_24, 0, x_2); lean_ctor_set(x_24, 1, x_10); x_25 = lean_array_mk(x_24); -x_26 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12; +x_26 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11; x_27 = l_Lean_Meta_mkAppM(x_26, x_25, x_5, x_6, x_7, x_8, x_18); if (lean_obj_tag(x_27) == 0) { @@ -12140,7 +12112,7 @@ x_45 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_45, 0, x_2); lean_ctor_set(x_45, 1, x_10); x_46 = lean_array_mk(x_45); -x_47 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12; +x_47 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11; x_48 = l_Lean_Meta_mkAppM(x_47, x_46, x_5, x_6, x_7, x_8, x_37); if (lean_obj_tag(x_48) == 0) { @@ -12310,7 +12282,7 @@ x_76 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_76, 0, x_2); lean_ctor_set(x_76, 1, x_75); x_77 = lean_array_mk(x_76); -x_78 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__12; +x_78 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__11; x_79 = l_Lean_Meta_mkAppM(x_78, x_77, x_5, x_6, x_7, x_8, x_66); if (lean_obj_tag(x_79) == 0) { @@ -19065,7 +19037,7 @@ lean_inc(x_28); lean_ctor_set_tag(x_29, 2); lean_ctor_set(x_29, 1, x_33); lean_ctor_set(x_29, 0, x_28); -x_34 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7; +x_34 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3; x_35 = l_Array_append___rarg(x_34, x_21); lean_dec(x_21); x_36 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; @@ -19104,7 +19076,7 @@ lean_inc(x_28); x_48 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_48, 0, x_28); lean_ctor_set(x_48, 1, x_47); -x_49 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__7; +x_49 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3; x_50 = l_Array_append___rarg(x_49, x_21); lean_dec(x_21); x_51 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; @@ -28697,7 +28669,7 @@ lean_ctor_set(x_43, 0, x_42); lean_ctor_set(x_43, 1, x_8); lean_ctor_set(x_43, 2, x_21); x_44 = lean_ctor_get(x_9, 1); -x_45 = lean_ctor_get_uint8(x_44, sizeof(void*)*2 + 3); +x_45 = lean_ctor_get_uint8(x_44, sizeof(void*)*3 + 3); lean_inc(x_42); lean_ctor_set_tag(x_33, 1); lean_ctor_set(x_33, 1, x_10); @@ -28909,7 +28881,7 @@ lean_ctor_set(x_90, 0, x_89); lean_ctor_set(x_90, 1, x_8); lean_ctor_set(x_90, 2, x_21); x_91 = lean_ctor_get(x_9, 1); -x_92 = lean_ctor_get_uint8(x_91, sizeof(void*)*2 + 3); +x_92 = lean_ctor_get_uint8(x_91, sizeof(void*)*3 + 3); lean_inc(x_89); x_93 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_93, 0, x_89); @@ -30960,7 +30932,7 @@ lean_ctor_set(x_86, 0, x_84); lean_ctor_set(x_86, 1, x_83); x_87 = lean_ctor_get(x_5, 1); lean_inc(x_87); -x_88 = lean_ctor_get_uint8(x_87, sizeof(void*)*2 + 3); +x_88 = lean_ctor_get_uint8(x_87, sizeof(void*)*3 + 3); lean_inc(x_85); lean_inc(x_67); x_89 = lean_alloc_ctor(6, 3, 1); @@ -31171,7 +31143,7 @@ lean_object* x_112; lean_object* x_113; uint8_t x_114; lean_object* x_115; x_112 = lean_ctor_get(x_111, 1); lean_inc(x_112); lean_dec(x_111); -x_113 = lean_ctor_get(x_87, 1); +x_113 = lean_ctor_get(x_87, 2); lean_inc(x_113); lean_dec(x_87); x_114 = 0; @@ -31795,7 +31767,7 @@ lean_ctor_set(x_236, 0, x_234); lean_ctor_set(x_236, 1, x_232); x_237 = lean_ctor_get(x_5, 1); lean_inc(x_237); -x_238 = lean_ctor_get_uint8(x_237, sizeof(void*)*2 + 3); +x_238 = lean_ctor_get_uint8(x_237, sizeof(void*)*3 + 3); lean_inc(x_235); lean_inc(x_67); x_239 = lean_alloc_ctor(6, 3, 1); @@ -32008,7 +31980,7 @@ lean_object* x_262; lean_object* x_263; uint8_t x_264; lean_object* x_265; x_262 = lean_ctor_get(x_261, 1); lean_inc(x_262); lean_dec(x_261); -x_263 = lean_ctor_get(x_237, 1); +x_263 = lean_ctor_get(x_237, 2); lean_inc(x_263); lean_dec(x_237); x_264 = 0; @@ -32738,7 +32710,7 @@ static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_e _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__5; x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___closed__4; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; @@ -33815,7 +33787,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at_Le _start: { uint8_t x_5; -x_5 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 1); +x_5 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 1); if (x_5 == 0) { lean_object* x_6; lean_object* x_7; @@ -33849,6 +33821,122 @@ return x_13; } } } +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___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) { +_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; +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); +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 = lean_box(2); +x_17 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__6; +x_18 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +lean_ctor_set(x_18, 2, x_15); +lean_inc(x_9); +x_19 = l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_18); +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_9); +lean_dec(x_3); +lean_dec(x_1); +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 = lean_box(0); +lean_ctor_set(x_19, 0, x_23); +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 = 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; +} +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +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); +x_29 = l_Lean_Elab_getDeclarationSelectionRef(x_1); +lean_inc(x_9); +x_30 = l_Lean_Elab_getDeclarationRange_x3f___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(x_29, x_5, x_6, x_7, x_8, x_9, x_10, x_27); +lean_dec(x_29); +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +if (lean_obj_tag(x_31) == 0) +{ +uint8_t x_32; +lean_dec(x_28); +lean_dec(x_9); +lean_dec(x_3); +x_32 = !lean_is_exclusive(x_30); +if (x_32 == 0) +{ +lean_object* x_33; lean_object* x_34; +x_33 = lean_ctor_get(x_30, 0); +lean_dec(x_33); +x_34 = lean_box(0); +lean_ctor_set(x_30, 0, x_34); +return x_30; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_30, 1); +lean_inc(x_35); +lean_dec(x_30); +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 +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_38 = lean_ctor_get(x_30, 1); +lean_inc(x_38); +lean_dec(x_30); +x_39 = lean_ctor_get(x_31, 0); +lean_inc(x_39); +lean_dec(x_31); +x_40 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_40, 0, x_28); +lean_ctor_set(x_40, 1, x_39); +x_41 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20(x_3, x_40, x_5, x_6, x_7, x_8, x_9, x_10, x_38); +lean_dec(x_9); +return x_41; +} +} +} +} static lean_object* _init_l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___closed__1() { _start: { @@ -33869,68 +33957,34 @@ x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___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_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___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_10; lean_object* x_11; uint8_t x_12; -lean_inc(x_2); -x_10 = l_Lean_Syntax_getKind(x_2); -x_11 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___closed__2; -x_12 = lean_name_eq(x_10, x_11); -lean_dec(x_10); -if (x_12 == 0) -{ -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_inc(x_7); -x_13 = l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -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_getDeclarationSelectionRef(x_2); -lean_inc(x_7); -x_17 = l_Lean_Elab_getDeclarationRange___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__19(x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_15); -lean_dec(x_16); -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 = lean_ctor_get(x_17, 1); -lean_ctor_set(x_17, 1, x_19); -lean_ctor_set(x_17, 0, x_14); -x_21 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20(x_1, x_17, x_3, x_4, x_5, x_6, x_7, x_8, x_20); -lean_dec(x_7); -return x_21; -} -else +lean_object* x_11; lean_object* x_12; uint8_t x_13; +lean_inc(x_3); +x_11 = l_Lean_Syntax_getKind(x_3); +x_12 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___closed__2; +x_13 = lean_name_eq(x_11, x_12); +lean_dec(x_11); +if (x_13 == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -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(0, 2, 0); -lean_ctor_set(x_24, 0, x_14); -lean_ctor_set(x_24, 1, x_22); -x_25 = l_Lean_addDeclarationRanges___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__20(x_1, x_24, x_3, x_4, x_5, x_6, x_7, x_8, x_23); -lean_dec(x_7); -return x_25; -} +lean_object* x_14; lean_object* x_15; +x_14 = lean_box(0); +x_15 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2___lambda__1(x_3, x_2, x_1, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_15; } else { -lean_object* x_26; lean_object* x_27; -lean_dec(x_7); +lean_object* x_16; lean_object* x_17; +lean_dec(x_8); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -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_9); -return x_27; +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_10); +return x_17; } } } @@ -34438,34 +34492,34 @@ return x_38; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__4(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, 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_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__4(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, 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) { _start: { -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_inc(x_16); -lean_inc(x_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_inc(x_17); +lean_inc(x_3); lean_inc(x_1); -x_19 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2(x_1, x_2, x_12, x_13, x_14, x_15, x_16, x_17, x_18); -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); -x_21 = lean_box(x_5); -x_22 = lean_box(x_9); +x_20 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2(x_1, x_2, x_3, x_13, x_14, x_15, x_16, x_17, x_18, x_19); +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = lean_box(x_6); +x_23 = lean_box(x_10); lean_inc(x_1); -x_23 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabStructure___lambda__3___boxed), 18, 11); -lean_closure_set(x_23, 0, x_2); -lean_closure_set(x_23, 1, x_3); -lean_closure_set(x_23, 2, x_1); -lean_closure_set(x_23, 3, x_4); -lean_closure_set(x_23, 4, x_21); -lean_closure_set(x_23, 5, x_6); -lean_closure_set(x_23, 6, x_7); -lean_closure_set(x_23, 7, x_8); -lean_closure_set(x_23, 8, x_22); -lean_closure_set(x_23, 9, x_10); -lean_closure_set(x_23, 10, x_11); -x_24 = l_Lean_Elab_Term_withDeclName___rarg(x_1, x_23, x_12, x_13, x_14, x_15, x_16, x_17, x_20); -return x_24; +x_24 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabStructure___lambda__3___boxed), 18, 11); +lean_closure_set(x_24, 0, x_3); +lean_closure_set(x_24, 1, x_4); +lean_closure_set(x_24, 2, x_1); +lean_closure_set(x_24, 3, x_5); +lean_closure_set(x_24, 4, x_22); +lean_closure_set(x_24, 5, x_7); +lean_closure_set(x_24, 6, x_8); +lean_closure_set(x_24, 7, x_9); +lean_closure_set(x_24, 8, x_23); +lean_closure_set(x_24, 9, x_11); +lean_closure_set(x_24, 10, x_12); +x_25 = l_Lean_Elab_Term_withDeclName___rarg(x_1, x_24, x_13, x_14, x_15, x_16, x_17, x_18, x_21); +return x_25; } } LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t 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) { @@ -34487,7 +34541,7 @@ lean_inc(x_18); x_21 = l_Lean_Elab_expandDeclId___at_Lean_Elab_Term_expandDeclId___spec__1(x_20, x_18, x_1, x_2, x_10, x_11, x_12, x_13, x_14, x_15, 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; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +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_22 = lean_ctor_get(x_21, 0); lean_inc(x_22); x_23 = lean_ctor_get(x_21, 1); @@ -34502,26 +34556,29 @@ lean_inc(x_26); lean_dec(x_22); x_27 = lean_alloc_closure((void*)(l_Lean_Name_beq___boxed), 2, 1); lean_closure_set(x_27, 0, x_24); -x_28 = lean_box(x_4); -x_29 = lean_box(x_7); -x_30 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabStructure___lambda__4___boxed), 18, 11); -lean_closure_set(x_30, 0, x_25); -lean_closure_set(x_30, 1, x_3); -lean_closure_set(x_30, 2, x_2); -lean_closure_set(x_30, 3, x_18); -lean_closure_set(x_30, 4, x_28); -lean_closure_set(x_30, 5, x_9); -lean_closure_set(x_30, 6, x_5); -lean_closure_set(x_30, 7, x_6); -lean_closure_set(x_30, 8, x_29); -lean_closure_set(x_30, 9, x_8); -lean_closure_set(x_30, 10, x_26); -x_31 = l_Lean_Elab_Term_withAutoBoundImplicitForbiddenPred___rarg(x_27, x_30, x_10, x_11, x_12, x_13, x_14, x_15, x_23); -return x_31; +x_28 = lean_ctor_get(x_2, 0); +lean_inc(x_28); +x_29 = lean_box(x_4); +x_30 = lean_box(x_7); +x_31 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabStructure___lambda__4___boxed), 19, 12); +lean_closure_set(x_31, 0, x_25); +lean_closure_set(x_31, 1, x_28); +lean_closure_set(x_31, 2, x_3); +lean_closure_set(x_31, 3, x_2); +lean_closure_set(x_31, 4, x_18); +lean_closure_set(x_31, 5, x_29); +lean_closure_set(x_31, 6, x_9); +lean_closure_set(x_31, 7, x_5); +lean_closure_set(x_31, 8, x_6); +lean_closure_set(x_31, 9, x_30); +lean_closure_set(x_31, 10, x_8); +lean_closure_set(x_31, 11, x_26); +x_32 = l_Lean_Elab_Term_withAutoBoundImplicitForbiddenPred___rarg(x_27, x_31, x_10, x_11, x_12, x_13, x_14, x_15, x_23); +return x_32; } else { -uint8_t x_32; +uint8_t x_33; lean_dec(x_18); lean_dec(x_15); lean_dec(x_14); @@ -34535,23 +34592,23 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); -x_32 = !lean_is_exclusive(x_21); -if (x_32 == 0) +x_33 = !lean_is_exclusive(x_21); +if (x_33 == 0) { return x_21; } else { -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_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_21, 0); +x_35 = lean_ctor_get(x_21, 1); +lean_inc(x_35); lean_inc(x_34); -lean_inc(x_33); lean_dec(x_21); -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; +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; } } } @@ -34560,7 +34617,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__6(lean_obje _start: { lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = lean_ctor_get(x_1, 1); +x_11 = lean_ctor_get(x_1, 2); lean_inc(x_11); lean_dec(x_1); x_12 = 1; @@ -35158,17 +35215,31 @@ lean_dec(x_1); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___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_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___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: { -lean_object* x_10; -x_10 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_object* x_12; +x_12 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___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_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -return x_10; +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___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) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabStructure___spec__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_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_11; } } LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabStructure___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) { @@ -35280,15 +35351,16 @@ 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]; _start: { -uint8_t x_19; uint8_t x_20; lean_object* x_21; -x_19 = lean_unbox(x_5); -lean_dec(x_5); -x_20 = lean_unbox(x_9); -lean_dec(x_9); -x_21 = l_Lean_Elab_Command_elabStructure___lambda__4(x_1, x_2, x_3, x_4, x_19, 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; +uint8_t x_20; uint8_t x_21; lean_object* x_22; +x_20 = lean_unbox(x_6); +lean_dec(x_6); +x_21 = lean_unbox(x_10); +lean_dec(x_10); +x_22 = l_Lean_Elab_Command_elabStructure___lambda__4(x_1, x_2, x_3, x_4, x_5, x_20, x_7, x_8, x_9, x_21, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19); +return x_22; } } LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___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) { @@ -35326,7 +35398,7 @@ lean_dec(x_8); return x_15; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__1() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -35336,27 +35408,27 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__2() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__1; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__1; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__3() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__2; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__2; x_2 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__1___lambda__3___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__4() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__4() { _start: { lean_object* x_1; @@ -35364,17 +35436,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__5() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__3; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__4; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__3; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__6() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__6() { _start: { lean_object* x_1; @@ -35382,37 +35454,37 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__7() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__5; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__6; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__5; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__8() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__7; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__7; x_2 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___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_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__9() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__8; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__5; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__8; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__10() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__10() { _start: { lean_object* x_1; @@ -35420,17 +35492,17 @@ x_1 = lean_mk_string_unchecked("Structure", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__11() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__9; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__10; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__9; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__10; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__12() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__12() { _start: { lean_object* x_1; @@ -35438,33 +35510,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__13() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__11; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__12; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__11; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__14() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__13; -x_2 = lean_unsigned_to_nat(14022u); +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__13; +x_2 = lean_unsigned_to_nat(14017u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017_(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_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__1; x_3 = 0; -x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__14; +x_4 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__14; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -35765,6 +35837,8 @@ l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__2 = _i lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__2); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__3); +l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__4 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__4(); +lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___closed__4); l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__1 = _init_l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__1(); lean_mark_persistent(l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__1); l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__2 = _init_l_Lean_Elab_Command_checkValidFieldModifier___lambda__1___closed__2(); @@ -35821,8 +35895,6 @@ l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Comman lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__13); l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14(); lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__14); -l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__15 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__15(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__15); l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__1 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__1(); lean_mark_persistent(l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__1); l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__2 = _init_l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__4___closed__2(); @@ -35918,19 +35990,19 @@ l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed_ lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__2); l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__3 = _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__3(); lean_mark_persistent(l___private_Lean_Elab_Structure_0__Lean_Elab_Command_findFieldInfo_x3f___closed__3); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__1); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__2); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__3(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__3); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__4(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__4); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__5(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__5); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__6(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990____closed__6); -if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3990_(lean_io_mk_world()); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__1); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__2); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__3); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__4(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__4); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__5(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__5); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__6(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984____closed__6); +if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3984_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Elab_Command_structureDiamondWarning = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_Command_structureDiamondWarning); @@ -36201,35 +36273,35 @@ l_Lean_Elab_Command_elabStructure___closed__8 = _init_l_Lean_Elab_Command_elabSt lean_mark_persistent(l_Lean_Elab_Command_elabStructure___closed__8); l_Lean_Elab_Command_elabStructure___closed__9 = _init_l_Lean_Elab_Command_elabStructure___closed__9(); lean_mark_persistent(l_Lean_Elab_Command_elabStructure___closed__9); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__1); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__2); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__3(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__3); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__4(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__4); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__5(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__5); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__6(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__6); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__7 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__7(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__7); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__8 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__8(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__8); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__9 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__9(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__9); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__10 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__10(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__10); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__11 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__11(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__11); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__12 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__12(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__12); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__13 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__13(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__13); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__14 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__14(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022____closed__14); -if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14022_(lean_io_mk_world()); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__1); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__2); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__3 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__3); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__4 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__4(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__4); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__5 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__5(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__5); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__6 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__6(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__6); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__7 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__7(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__7); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__8 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__8(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__8); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__9 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__9(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__9); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__10 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__10(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__10); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__11 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__11(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__11); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__12 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__12(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__12); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__13 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__13(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__13); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__14 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__14(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017____closed__14); +if (builtin) {res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_14017_(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/Syntax.c b/stage0/stdlib/Lean/Elab/Syntax.c index dfd6f9fe28d6..c73b915deade 100644 --- a/stage0/stdlib/Lean/Elab/Syntax.c +++ b/stage0/stdlib/Lean/Elab/Syntax.c @@ -413,7 +413,6 @@ static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyn static lean_object* l_Lean_Elab_Command_checkRuleKind___closed__2; lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); lean_object* l_Lean_Syntax_node3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___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*); static lean_object* l_Lean_Elab_Command_elabSyntax___lambda__7___closed__3; static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__61; lean_object* l_Lean_Name_append(lean_object*, lean_object*); @@ -612,6 +611,7 @@ uint8_t lean_uint32_dec_eq(uint32_t, uint32_t); static lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__19; static lean_object* l_Lean_Elab_Term_toParserDescr_processNonReserved___closed__11; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_toParserDescr_processAlias___spec__6___lambda__1___closed__11; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___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* l_Lean_Name_mkStr2(lean_object*, lean_object*); lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Command_runLinters___spec__11(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_checkLeftRec___spec__7___closed__4; @@ -633,6 +633,7 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_mkName lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_toParserDescr_processSeq___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_Term_toParserDescr_process___closed__7; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___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_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__66; static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__43; static lean_object* l_Lean_Elab_Command_elabSyntax___lambda__4___closed__15; @@ -660,7 +661,6 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclareSyntaxCat_d lean_object* l_Array_mkArray1___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_resolveSyntaxKind___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Term_elabParserName___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_Array_mapIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___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_Lean_throwError___at_Lean_Elab_Command_expandNoKindMacroRulesAux___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__12; static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__44; @@ -12040,7 +12040,7 @@ return x_84; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___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) { _start: { lean_object* x_16; uint8_t x_17; @@ -12406,7 +12406,7 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_20 = l_Array_mapIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___spec__1(x_11, x_11, x_18, x_12, lean_box(0), x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17); +x_20 = l_Array_mapFinIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___spec__1(x_11, x_11, x_18, x_12, lean_box(0), x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17); lean_dec(x_11); if (lean_obj_tag(x_20) == 0) { @@ -12822,11 +12822,11 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___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_mapFinIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___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: { lean_object* x_16; -x_16 = l_Array_mapIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___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 = l_Array_mapFinIdxM_map___at_Lean_Elab_Term_toParserDescr_processSeq___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); lean_dec(x_7); lean_dec(x_2); lean_dec(x_1); diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVExpr.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVExpr.c index 1f75fc0e3efa..9509f3241d0d 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVExpr.c +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVExpr.c @@ -13,307 +13,313 @@ #ifdef __cplusplus extern "C" { #endif -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__10; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__2; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31(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_ReifiedBVExpr_of_unaryReflection___closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__6; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__20; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___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_ReifiedBVExpr_of_binaryReflection___closed__13; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__1; lean_object* l_Lean_mkNatLit(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__24; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__3(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__4; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__1; lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_M_lookup(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_ReifiedBVExpr_of___lambda__2___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___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_ReifiedBVExpr_of_go___closed__51; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__60; lean_object* l_Lean_Meta_getNatValue_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19(lean_object*, 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_ReifiedBVExpr_getNatOrBvValue_x3f___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_ReifiedBVExpr_of___lambda__26___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__45; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__34; LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___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_ReifiedBVExpr_of___lambda__22___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___lambda__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_ReifiedBVExpr_of___closed__14; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__18; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, 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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__8; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__1; lean_object* l_Lean_mkAppB(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__13; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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_ReifiedBVExpr_getNatOrBvValue_x3f___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__27; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__4; uint8_t l_Lean_Expr_isApp(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__10; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__58; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__40; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__22; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__1(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12(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_ReifiedBVExpr_of_binaryReflection___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29(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_ReifiedBVExpr_of___closed__12; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__7; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__10; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__17; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__19; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__8; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__3(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__48; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24(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_ReifiedBVExpr_of_go___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstLikeReflection(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_ReifiedBVExpr_of___closed__32; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__21(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__38; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13(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_ReifiedBVExpr_of_go___lambda__2___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__50; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__33; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__26; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection(lean_object*, 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_ReifiedBVExpr_of_go___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection(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_ReifiedBVExpr_of_go___closed__20; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__14; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6(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_ReifiedBVExpr_of_goBvLit___closed__5; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__17; lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__4; lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__31; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__19; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10(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_ReifiedBVExpr_of_go___closed__53; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__8; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__44; lean_object* l_Lean_mkApp4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__9; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___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_ReifiedBVExpr_of_go___lambda__15(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__17(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25(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_ReifiedBVExpr_of_binaryReflection___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__57; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__7; lean_object* l_Lean_Level_ofNat(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__8; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__46; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29(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_ReifiedBVExpr_of_go___lambda__2___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___lambda__2(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_ReifiedBVExpr_mkEvalExpr___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__9; uint8_t l_Lean_Expr_hasMVar(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11(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_ReifiedBVExpr_of___closed__47; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16(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_ReifiedBVExpr_of_go___closed__39; lean_object* l_Lean_mkApp6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16(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_ReifiedBVExpr_of___lambda__25___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___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_ReifiedBVExpr_of_go___lambda__16___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14(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_ReifiedBVExpr_of_go___lambda__4___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__30; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection___boxed(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_ReifiedBVExpr_of_go___closed__56; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection___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_ReifiedBVExpr_of_go___lambda__16___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30(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_ReifiedBVExpr_of___closed__36; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__33; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__14; lean_object* lean_st_ref_take(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25(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_ReifiedBVExpr_of_go___lambda__22___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f(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_ReifiedBVExpr_of___lambda__22(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_ReifiedBVExpr_of___closed__43; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__39; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__7; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28(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_ReifiedBVExpr_mkEvalExpr___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_ReifiedBVExpr_of___closed__23; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12(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_ReifiedBVExpr_of___lambda__25___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__21(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__2; lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_M_atomsAssignment(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4(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_ReifiedBVExpr_of_go___lambda__22___closed__9; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___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_ReifiedBVExpr_of_go___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__15; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__31(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_ReifiedBVExpr_of_binaryReflection___closed__23; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__31; lean_object* l_Lean_Meta_getBitVecValue_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__5; lean_object* l_Lean_Expr_appArg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___lambda__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_ReifiedBVExpr_of_binaryReflection___closed__21; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__7; lean_object* lean_st_ref_get(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__25; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___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_ReifiedBVExpr_of___lambda__24(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_ReifiedBVExpr_of_go___closed__26; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___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_ReifiedBVExpr_of_go___lambda__25___closed__2; lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__7; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__31___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_ReifiedBVExpr_of___closed__9; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___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_ReifiedBVExpr_of___lambda__20(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22(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_ReifiedBVExpr_of_go___closed__54; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__55; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___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_ReifiedBVExpr_of___lambda__14___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__37; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__19; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__30; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__8; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30(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*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__38; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__22; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__3; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__8; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom(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_ReifiedBVExpr_of_binaryReflection___closed__15; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__10; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8(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_ReifiedBVExpr_of_go___closed__8; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14(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_ReifiedBVExpr_of_go___closed__41; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__25; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__11; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__7; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___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*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__32; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___lambda__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_ReifiedBVExpr_of___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*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__49; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__50; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___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*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__20; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__21; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___lambda__2(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_ReifiedBVExpr_of___closed__29; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2(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_ReifiedBVExpr_of_go___closed__10; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27(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_ReifiedBVExpr_of_go___lambda__2___closed__6; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__1; 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_ReifiedBVExpr_of___lambda__12___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28(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_ReifiedBVExpr_of_go___closed__28; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__3; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__5; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__4; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13(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_ReifiedBVExpr_of_binaryReflection___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__41; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11(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_ReifiedBVExpr_of_go___lambda__25___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__9; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__17(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31___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_ReifiedBVExpr_of_unaryReflection___closed__10; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__42; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__18(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__29; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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*, lean_object*); lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26(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_ReifiedBVExpr_of_go___closed__23; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__28; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__16; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__2; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__32(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_ReifiedBVExpr_of___closed__35; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__27; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__15; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__37; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__11; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__5; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__25; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__12; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__12; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___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*); uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__13; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__9; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__24; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__11; lean_object* lean_nat_mul(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10(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_ReifiedBVExpr_of___closed__22; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; lean_object* l_Lean_Meta_instantiateMVarsIfMVarApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__52; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__7; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__44; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstReflection(lean_object*, 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_ReifiedBVExpr_of_go___closed__49; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstReflection(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_ReifiedBVExpr_of_go___lambda__19___closed__8; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__1(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__43; lean_object* l_Lean_instantiateMVarsCore(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19(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_ReifiedBVExpr_of_go___closed__35; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection(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_ReifiedBVExpr_of___lambda__11___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__9; +LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__9; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__21; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__18; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__24; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__1; LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__46; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__47; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__10; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(lean_object*, lean_object*, lean_object*, 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_ReifiedBVExpr_of___lambda__27(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_ReifiedBVExpr_of_go___lambda__29___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(lean_object*, lean_object*, 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_ReifiedBVExpr_of_unaryCongrProof(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_ReifiedBVExpr_of___closed__34; -LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___spec__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_ReifiedBVExpr_of___lambda__26(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_ReifiedBVExpr_of_shiftReflection___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_ReifiedBVExpr_of___lambda__4___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__8; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__16; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6(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_ReifiedBVExpr_of___lambda__9___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___lambda__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_ReifiedBVExpr_of_go___closed__45; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__42; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__16; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__36; lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__15(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__20(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__2; lean_object* l_Lean_mkApp5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__51; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__18(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__18; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__48; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__5; -LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___spec__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_ReifiedBVExpr_of___lambda__27___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__4; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__59; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__11; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__10; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8(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_ReifiedBVExpr_of___closed__40; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__17; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryCongrProof(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_ReifiedBVExpr_of_go___lambda__2___closed__4; lean_object* l_Lean_Meta_whnfR(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__1; +LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1() { _start: @@ -1016,7 +1022,7 @@ lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___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_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___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: { uint8_t x_8; @@ -1123,7 +1129,7 @@ return x_35; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___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; @@ -1322,7 +1328,7 @@ return x_44; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(lean_object* x_1, lean_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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom(lean_object* x_1, 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; @@ -1353,7 +1359,7 @@ lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___spec__1(x_12, x_2, x_3, x_4, x_5, x_6, x_13); +x_14 = l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___spec__1(x_12, x_2, x_3, x_4, x_5, x_6, x_13); x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); x_16 = lean_ctor_get(x_14, 1); @@ -1391,7 +1397,7 @@ return x_27; else { lean_object* x_28; -x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___lambda__1(x_1, x_22, x_2, x_3, x_4, x_5, x_6, x_16); +x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___lambda__1(x_1, x_22, x_2, x_3, x_4, x_5, x_6, x_16); lean_dec(x_22); return x_28; } @@ -1456,11 +1462,11 @@ return x_36; } } } -LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___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_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___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: { lean_object* x_8; -x_8 = l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___spec__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); @@ -1469,11 +1475,11 @@ lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___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_ReifiedBVExpr_of_ofAtom___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___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; } @@ -1558,7 +1564,7 @@ lean_object* x_10; lean_object* x_11; x_10 = lean_ctor_get(x_8, 1); lean_inc(x_10); lean_dec(x_8); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); if (lean_obj_tag(x_11) == 0) { uint8_t x_12; @@ -2092,122 +2098,7 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(lean_object* x_1, 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_2); -lean_inc(x_1); -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(x_1, 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) == 0) -{ -lean_object* x_10; lean_object* x_11; -x_10 = lean_ctor_get(x_8, 1); -lean_inc(x_10); -lean_dec(x_8); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_11; -} -else -{ -uint8_t x_12; -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_12 = !lean_is_exclusive(x_8); -if (x_12 == 0) -{ -lean_object* x_13; uint8_t x_14; -x_13 = lean_ctor_get(x_8, 0); -lean_dec(x_13); -x_14 = !lean_is_exclusive(x_9); -if (x_14 == 0) -{ -return x_8; -} -else -{ -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_9, 0); -lean_inc(x_15); -lean_dec(x_9); -x_16 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_16, 0, x_15); -lean_ctor_set(x_8, 0, x_16); -return x_8; -} -} -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_8, 1); -lean_inc(x_17); -lean_dec(x_8); -x_18 = lean_ctor_get(x_9, 0); -lean_inc(x_18); -if (lean_is_exclusive(x_9)) { - lean_ctor_release(x_9, 0); - x_19 = x_9; -} else { - lean_dec_ref(x_9); - x_19 = lean_box(0); -} -if (lean_is_scalar(x_19)) { - x_20 = lean_alloc_ctor(1, 1, 0); -} else { - x_20 = x_19; -} -lean_ctor_set(x_20, 0, 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_17); -return x_21; -} -} -} -else -{ -uint8_t x_22; -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_22 = !lean_is_exclusive(x_8); -if (x_22 == 0) -{ -return x_8; -} -else -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_8, 0); -x_24 = lean_ctor_get(x_8, 1); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_8); -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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__1(lean_object* x_1) { _start: { lean_object* x_2; @@ -2216,7 +2107,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1() { _start: { lean_object* x_1; @@ -2224,7 +2115,7 @@ x_1 = lean_mk_string_unchecked("BVUnOp", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__2() { _start: { lean_object* x_1; @@ -2232,20 +2123,20 @@ x_1 = lean_mk_string_unchecked("rotateRight", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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; lean_object* x_6; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__2; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__2; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4() { _start: { lean_object* x_1; @@ -2253,7 +2144,7 @@ x_1 = lean_mk_string_unchecked("Reflect", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__5() { _start: { lean_object* x_1; @@ -2261,40 +2152,40 @@ x_1 = lean_mk_string_unchecked("rotateRight_congr", 17, 17); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___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_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__5; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___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_ReifiedBVExpr_of___lambda__2___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__7() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__1), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_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) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__7; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__3; -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__6; -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(x_1, x_3, x_2, x_10, x_11, x_12, x_4, x_5, x_6, x_7, x_8, x_9); -return x_13; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__7; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__3; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__6; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(x_2, x_1, x_9, x_10, x_11, x_3, x_4, x_5, x_6, x_7, x_8); +return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__3(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__3(lean_object* x_1) { _start: { lean_object* x_2; @@ -2303,7 +2194,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__1() { _start: { lean_object* x_1; @@ -2311,20 +2202,20 @@ x_1 = lean_mk_string_unchecked("rotateLeft", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__1; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__3() { _start: { lean_object* x_1; @@ -2332,40 +2223,40 @@ x_1 = lean_mk_string_unchecked("rotateLeft_congr", 16, 16); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___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_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__3; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___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_ReifiedBVExpr_of___lambda__4___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__3), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__3), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__5; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__2; -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__4; -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(x_1, x_3, x_2, x_10, x_11, x_12, x_4, x_5, x_6, x_7, x_8, x_9); -return x_13; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__5; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__2; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__4; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(x_2, x_1, x_9, x_10, x_11, 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_ReifiedBVExpr_of___lambda__5___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__1() { _start: { lean_object* x_1; @@ -2373,21 +2264,21 @@ x_1 = lean_mk_string_unchecked("extract_congr", 13, 13); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___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_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___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_ReifiedBVExpr_of___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, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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, lean_object* x_13) { _start: { lean_object* x_14; lean_object* x_15; @@ -2403,7 +2294,7 @@ 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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__2; +x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__2; x_19 = l_Lean_Expr_const___override(x_18, x_2); x_20 = l_Lean_mkApp6(x_19, x_3, x_4, x_5, x_6, x_7, x_17); lean_ctor_set(x_15, 0, x_20); @@ -2417,7 +2308,7 @@ x_22 = lean_ctor_get(x_15, 1); lean_inc(x_22); lean_inc(x_21); lean_dec(x_15); -x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__2; +x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__2; x_24 = l_Lean_Expr_const___override(x_23, x_2); x_25 = l_Lean_mkApp6(x_24, x_3, x_4, x_5, x_6, x_7, x_21); x_26 = lean_alloc_ctor(0, 2, 0); @@ -2456,7 +2347,7 @@ return x_30; } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__1() { _start: { lean_object* x_1; @@ -2464,7 +2355,7 @@ x_1 = lean_mk_string_unchecked("extract", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___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; @@ -2472,484 +2363,440 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___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_ReifiedBVExpr_of___lambda__6___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___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_ReifiedBVExpr_of___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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_11; -lean_inc(x_9); +lean_object* x_10; 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_inc(x_5); +x_10 = l_Lean_Meta_getNatValue_x3f(x_1, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_12; -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -if (lean_obj_tag(x_12) == 0) +lean_object* x_11; +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +if (lean_obj_tag(x_11) == 0) { -lean_object* x_13; lean_object* x_14; +uint8_t x_12; +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_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_5, x_6, x_7, 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) -{ -return x_14; -} -else -{ -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_17); -lean_inc(x_16); -lean_dec(x_14); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_16); -lean_ctor_set(x_18, 1, x_17); -return x_18; -} -} -else -{ -uint8_t x_19; -x_19 = !lean_is_exclusive(x_14); -if (x_19 == 0) +lean_dec(x_1); +x_12 = !lean_is_exclusive(x_10); +if (x_12 == 0) { -return x_14; +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_10, 0); +lean_dec(x_13); +x_14 = lean_box(0); +lean_ctor_set(x_10, 0, x_14); +return x_10; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_14, 0); -x_21 = lean_ctor_get(x_14, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_14); -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_10, 1); +lean_inc(x_15); +lean_dec(x_10); +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_15); +return x_17; } } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_11, 1); -lean_inc(x_23); +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_10, 1); +lean_inc(x_18); +lean_dec(x_10); +x_19 = lean_ctor_get(x_11, 0); +lean_inc(x_19); lean_dec(x_11); -x_24 = lean_ctor_get(x_12, 0); -lean_inc(x_24); -lean_dec(x_12); -lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_25 = l_Lean_Meta_getNatValue_x3f(x_3, x_6, x_7, x_8, x_9, x_23); -if (lean_obj_tag(x_25) == 0) +lean_inc(x_5); +x_20 = l_Lean_Meta_getNatValue_x3f(x_2, x_5, x_6, x_7, x_8, x_18); +if (lean_obj_tag(x_20) == 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_21; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +if (lean_obj_tag(x_21) == 0) { -lean_object* x_27; lean_object* x_28; -lean_dec(x_24); +uint8_t x_22; +lean_dec(x_19); +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_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); -lean_dec(x_25); -x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_5, x_6, x_7, x_8, x_9, x_27); -if (lean_obj_tag(x_28) == 0) -{ -uint8_t x_29; -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) +lean_dec(x_1); +x_22 = !lean_is_exclusive(x_20); +if (x_22 == 0) { -return x_28; +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_20, 0); +lean_dec(x_23); +x_24 = lean_box(0); +lean_ctor_set(x_20, 0, x_24); +return x_20; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_28, 0); -x_31 = lean_ctor_get(x_28, 1); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_28); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -return x_32; +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_20, 1); +lean_inc(x_25); +lean_dec(x_20); +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_33; -x_33 = !lean_is_exclusive(x_28); -if (x_33 == 0) +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_20, 1); +lean_inc(x_28); +lean_dec(x_20); +x_29 = lean_ctor_get(x_21, 0); +lean_inc(x_29); +lean_dec(x_21); +lean_inc(x_3); +x_30 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_3, x_4, x_5, x_6, x_7, x_8, x_28); +if (lean_obj_tag(x_30) == 0) { -return x_28; -} -else -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_28, 0); -x_35 = lean_ctor_get(x_28, 1); -lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_28); -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; lean_object* x_39; -lean_dec(x_1); -x_37 = lean_ctor_get(x_25, 1); -lean_inc(x_37); -lean_dec(x_25); -x_38 = lean_ctor_get(x_26, 0); -lean_inc(x_38); -lean_dec(x_26); -lean_inc(x_4); -x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_4, x_5, x_6, x_7, x_8, x_9, x_37); -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_31; +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +if (lean_obj_tag(x_31) == 0) { -uint8_t x_41; -lean_dec(x_38); -lean_dec(x_24); -lean_dec(x_4); +uint8_t x_32; +lean_dec(x_29); +lean_dec(x_19); lean_dec(x_3); lean_dec(x_2); -x_41 = !lean_is_exclusive(x_39); -if (x_41 == 0) +lean_dec(x_1); +x_32 = !lean_is_exclusive(x_30); +if (x_32 == 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; +lean_object* x_33; lean_object* x_34; +x_33 = lean_ctor_get(x_30, 0); +lean_dec(x_33); +x_34 = lean_box(0); +lean_ctor_set(x_30, 0, x_34); +return x_30; } 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; +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_30, 1); +lean_inc(x_35); +lean_dec(x_30); +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 { -uint8_t x_47; -x_47 = !lean_is_exclusive(x_40); -if (x_47 == 0) +uint8_t x_38; +x_38 = !lean_is_exclusive(x_31); +if (x_38 == 0) { -uint8_t x_48; -x_48 = !lean_is_exclusive(x_39); -if (x_48 == 0) +uint8_t x_39; +x_39 = !lean_is_exclusive(x_30); +if (x_39 == 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; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; -x_49 = lean_ctor_get(x_40, 0); -x_50 = lean_ctor_get(x_39, 0); -lean_dec(x_50); -x_51 = lean_ctor_get(x_49, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_49, 1); -lean_inc(x_52); -x_53 = lean_ctor_get(x_49, 3); -lean_inc(x_53); -lean_inc(x_38); -lean_inc(x_51); -x_54 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_54, 0, x_51); -lean_ctor_set(x_54, 1, x_24); -lean_ctor_set(x_54, 2, x_38); -lean_ctor_set(x_54, 3, x_52); -x_55 = lean_box(0); -lean_inc(x_51); -x_56 = l_Lean_mkNatLit(x_51); -x_57 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__3; -lean_inc(x_53); -lean_inc(x_3); +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; uint8_t x_52; +x_40 = lean_ctor_get(x_31, 0); +x_41 = lean_ctor_get(x_30, 0); +lean_dec(x_41); +x_42 = lean_ctor_get(x_40, 0); +lean_inc(x_42); +x_43 = lean_ctor_get(x_40, 1); +lean_inc(x_43); +x_44 = lean_ctor_get(x_40, 3); +lean_inc(x_44); +lean_inc(x_29); +lean_inc(x_42); +x_45 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_45, 0, x_42); +lean_ctor_set(x_45, 1, x_19); +lean_ctor_set(x_45, 2, x_29); +lean_ctor_set(x_45, 3, x_43); +x_46 = lean_box(0); +lean_inc(x_42); +x_47 = l_Lean_mkNatLit(x_42); +x_48 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__3; +lean_inc(x_44); lean_inc(x_2); -lean_inc(x_56); -x_58 = l_Lean_mkApp4(x_57, x_56, x_2, x_3, x_53); -x_59 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_59, 0, x_51); -lean_closure_set(x_59, 1, x_53); -lean_inc(x_49); -x_60 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5), 13, 6); -lean_closure_set(x_60, 0, x_49); -lean_closure_set(x_60, 1, x_55); -lean_closure_set(x_60, 2, x_2); -lean_closure_set(x_60, 3, x_3); -lean_closure_set(x_60, 4, x_56); -lean_closure_set(x_60, 5, x_4); -x_61 = !lean_is_exclusive(x_49); -if (x_61 == 0) -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_62 = lean_ctor_get(x_49, 3); -lean_dec(x_62); -x_63 = lean_ctor_get(x_49, 2); -lean_dec(x_63); -x_64 = lean_ctor_get(x_49, 1); -lean_dec(x_64); -x_65 = lean_ctor_get(x_49, 0); -lean_dec(x_65); -x_66 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_66, 0, x_59); -lean_closure_set(x_66, 1, x_60); -lean_ctor_set(x_49, 3, x_58); -lean_ctor_set(x_49, 2, x_66); -lean_ctor_set(x_49, 1, x_54); -lean_ctor_set(x_49, 0, x_38); -return x_39; +lean_inc(x_1); +lean_inc(x_47); +x_49 = l_Lean_mkApp4(x_48, x_47, x_1, x_2, x_44); +x_50 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_50, 0, x_42); +lean_closure_set(x_50, 1, x_44); +lean_inc(x_40); +x_51 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5), 13, 6); +lean_closure_set(x_51, 0, x_40); +lean_closure_set(x_51, 1, x_46); +lean_closure_set(x_51, 2, x_1); +lean_closure_set(x_51, 3, x_2); +lean_closure_set(x_51, 4, x_47); +lean_closure_set(x_51, 5, x_3); +x_52 = !lean_is_exclusive(x_40); +if (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_40, 3); +lean_dec(x_53); +x_54 = lean_ctor_get(x_40, 2); +lean_dec(x_54); +x_55 = lean_ctor_get(x_40, 1); +lean_dec(x_55); +x_56 = lean_ctor_get(x_40, 0); +lean_dec(x_56); +x_57 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_57, 0, x_50); +lean_closure_set(x_57, 1, x_51); +lean_ctor_set(x_40, 3, x_49); +lean_ctor_set(x_40, 2, x_57); +lean_ctor_set(x_40, 1, x_45); +lean_ctor_set(x_40, 0, x_29); +return x_30; } else { -lean_object* x_67; lean_object* x_68; -lean_dec(x_49); -x_67 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_67, 0, x_59); -lean_closure_set(x_67, 1, x_60); -x_68 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_68, 0, x_38); -lean_ctor_set(x_68, 1, x_54); -lean_ctor_set(x_68, 2, x_67); -lean_ctor_set(x_68, 3, x_58); -lean_ctor_set(x_40, 0, x_68); -return x_39; +lean_object* x_58; lean_object* x_59; +lean_dec(x_40); +x_58 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_58, 0, x_50); +lean_closure_set(x_58, 1, x_51); +x_59 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_59, 0, x_29); +lean_ctor_set(x_59, 1, x_45); +lean_ctor_set(x_59, 2, x_58); +lean_ctor_set(x_59, 3, x_49); +lean_ctor_set(x_31, 0, x_59); +return x_30; } } 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; 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_69 = lean_ctor_get(x_40, 0); -x_70 = lean_ctor_get(x_39, 1); -lean_inc(x_70); -lean_dec(x_39); -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, 3); -lean_inc(x_73); -lean_inc(x_38); -lean_inc(x_71); -x_74 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_74, 0, x_71); -lean_ctor_set(x_74, 1, x_24); -lean_ctor_set(x_74, 2, x_38); -lean_ctor_set(x_74, 3, x_72); -x_75 = lean_box(0); -lean_inc(x_71); -x_76 = l_Lean_mkNatLit(x_71); -x_77 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__3; -lean_inc(x_73); -lean_inc(x_3); +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; +x_60 = lean_ctor_get(x_31, 0); +x_61 = lean_ctor_get(x_30, 1); +lean_inc(x_61); +lean_dec(x_30); +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, 3); +lean_inc(x_64); +lean_inc(x_29); +lean_inc(x_62); +x_65 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_65, 0, x_62); +lean_ctor_set(x_65, 1, x_19); +lean_ctor_set(x_65, 2, x_29); +lean_ctor_set(x_65, 3, x_63); +x_66 = lean_box(0); +lean_inc(x_62); +x_67 = l_Lean_mkNatLit(x_62); +x_68 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__3; +lean_inc(x_64); lean_inc(x_2); -lean_inc(x_76); -x_78 = l_Lean_mkApp4(x_77, x_76, x_2, x_3, x_73); -x_79 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_79, 0, x_71); -lean_closure_set(x_79, 1, x_73); -lean_inc(x_69); -x_80 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5), 13, 6); -lean_closure_set(x_80, 0, x_69); -lean_closure_set(x_80, 1, x_75); -lean_closure_set(x_80, 2, x_2); -lean_closure_set(x_80, 3, x_3); -lean_closure_set(x_80, 4, x_76); -lean_closure_set(x_80, 5, x_4); -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); - x_81 = x_69; +lean_inc(x_1); +lean_inc(x_67); +x_69 = l_Lean_mkApp4(x_68, x_67, x_1, x_2, x_64); +x_70 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_70, 0, x_62); +lean_closure_set(x_70, 1, x_64); +lean_inc(x_60); +x_71 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5), 13, 6); +lean_closure_set(x_71, 0, x_60); +lean_closure_set(x_71, 1, x_66); +lean_closure_set(x_71, 2, x_1); +lean_closure_set(x_71, 3, x_2); +lean_closure_set(x_71, 4, x_67); +lean_closure_set(x_71, 5, x_3); +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); + x_72 = x_60; } else { - lean_dec_ref(x_69); - x_81 = lean_box(0); + lean_dec_ref(x_60); + x_72 = lean_box(0); } -x_82 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_82, 0, x_79); -lean_closure_set(x_82, 1, x_80); -if (lean_is_scalar(x_81)) { - x_83 = lean_alloc_ctor(0, 4, 0); +x_73 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_73, 0, x_70); +lean_closure_set(x_73, 1, x_71); +if (lean_is_scalar(x_72)) { + x_74 = lean_alloc_ctor(0, 4, 0); } else { - x_83 = x_81; + x_74 = x_72; } -lean_ctor_set(x_83, 0, x_38); -lean_ctor_set(x_83, 1, x_74); -lean_ctor_set(x_83, 2, x_82); -lean_ctor_set(x_83, 3, x_78); -lean_ctor_set(x_40, 0, x_83); -x_84 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_84, 0, x_40); -lean_ctor_set(x_84, 1, x_70); -return x_84; +lean_ctor_set(x_74, 0, x_29); +lean_ctor_set(x_74, 1, x_65); +lean_ctor_set(x_74, 2, x_73); +lean_ctor_set(x_74, 3, x_69); +lean_ctor_set(x_31, 0, x_74); +x_75 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_75, 0, x_31); +lean_ctor_set(x_75, 1, x_61); +return x_75; } } else { -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; -x_85 = lean_ctor_get(x_40, 0); -lean_inc(x_85); -lean_dec(x_40); -x_86 = lean_ctor_get(x_39, 1); -lean_inc(x_86); -if (lean_is_exclusive(x_39)) { - lean_ctor_release(x_39, 0); - lean_ctor_release(x_39, 1); - x_87 = x_39; +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; +x_76 = lean_ctor_get(x_31, 0); +lean_inc(x_76); +lean_dec(x_31); +x_77 = lean_ctor_get(x_30, 1); +lean_inc(x_77); +if (lean_is_exclusive(x_30)) { + lean_ctor_release(x_30, 0); + lean_ctor_release(x_30, 1); + x_78 = x_30; } else { - lean_dec_ref(x_39); - x_87 = lean_box(0); + lean_dec_ref(x_30); + x_78 = lean_box(0); } -x_88 = lean_ctor_get(x_85, 0); -lean_inc(x_88); -x_89 = lean_ctor_get(x_85, 1); -lean_inc(x_89); -x_90 = lean_ctor_get(x_85, 3); -lean_inc(x_90); -lean_inc(x_38); -lean_inc(x_88); -x_91 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_91, 0, x_88); -lean_ctor_set(x_91, 1, x_24); -lean_ctor_set(x_91, 2, x_38); -lean_ctor_set(x_91, 3, x_89); -x_92 = lean_box(0); -lean_inc(x_88); -x_93 = l_Lean_mkNatLit(x_88); -x_94 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__3; -lean_inc(x_90); -lean_inc(x_3); +x_79 = lean_ctor_get(x_76, 0); +lean_inc(x_79); +x_80 = lean_ctor_get(x_76, 1); +lean_inc(x_80); +x_81 = lean_ctor_get(x_76, 3); +lean_inc(x_81); +lean_inc(x_29); +lean_inc(x_79); +x_82 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_82, 0, x_79); +lean_ctor_set(x_82, 1, x_19); +lean_ctor_set(x_82, 2, x_29); +lean_ctor_set(x_82, 3, x_80); +x_83 = lean_box(0); +lean_inc(x_79); +x_84 = l_Lean_mkNatLit(x_79); +x_85 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__3; +lean_inc(x_81); lean_inc(x_2); -lean_inc(x_93); -x_95 = l_Lean_mkApp4(x_94, x_93, x_2, x_3, x_90); -x_96 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_96, 0, x_88); -lean_closure_set(x_96, 1, x_90); -lean_inc(x_85); -x_97 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5), 13, 6); -lean_closure_set(x_97, 0, x_85); -lean_closure_set(x_97, 1, x_92); -lean_closure_set(x_97, 2, x_2); -lean_closure_set(x_97, 3, x_3); -lean_closure_set(x_97, 4, x_93); -lean_closure_set(x_97, 5, x_4); -if (lean_is_exclusive(x_85)) { - lean_ctor_release(x_85, 0); - lean_ctor_release(x_85, 1); - lean_ctor_release(x_85, 2); - lean_ctor_release(x_85, 3); - x_98 = x_85; +lean_inc(x_1); +lean_inc(x_84); +x_86 = l_Lean_mkApp4(x_85, x_84, x_1, x_2, x_81); +x_87 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_87, 0, x_79); +lean_closure_set(x_87, 1, x_81); +lean_inc(x_76); +x_88 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5), 13, 6); +lean_closure_set(x_88, 0, x_76); +lean_closure_set(x_88, 1, x_83); +lean_closure_set(x_88, 2, x_1); +lean_closure_set(x_88, 3, x_2); +lean_closure_set(x_88, 4, x_84); +lean_closure_set(x_88, 5, x_3); +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); + x_89 = x_76; } else { - lean_dec_ref(x_85); - x_98 = lean_box(0); -} -x_99 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_99, 0, x_96); -lean_closure_set(x_99, 1, x_97); -if (lean_is_scalar(x_98)) { - x_100 = lean_alloc_ctor(0, 4, 0); + lean_dec_ref(x_76); + x_89 = lean_box(0); +} +x_90 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_90, 0, x_87); +lean_closure_set(x_90, 1, x_88); +if (lean_is_scalar(x_89)) { + x_91 = lean_alloc_ctor(0, 4, 0); } else { - x_100 = x_98; -} -lean_ctor_set(x_100, 0, x_38); -lean_ctor_set(x_100, 1, x_91); -lean_ctor_set(x_100, 2, x_99); -lean_ctor_set(x_100, 3, x_95); -x_101 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_101, 0, x_100); -if (lean_is_scalar(x_87)) { - x_102 = lean_alloc_ctor(0, 2, 0); + x_91 = x_89; +} +lean_ctor_set(x_91, 0, x_29); +lean_ctor_set(x_91, 1, x_82); +lean_ctor_set(x_91, 2, x_90); +lean_ctor_set(x_91, 3, x_86); +x_92 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_92, 0, x_91); +if (lean_is_scalar(x_78)) { + x_93 = lean_alloc_ctor(0, 2, 0); } else { - x_102 = x_87; + x_93 = x_78; } -lean_ctor_set(x_102, 0, x_101); -lean_ctor_set(x_102, 1, x_86); -return x_102; +lean_ctor_set(x_93, 0, x_92); +lean_ctor_set(x_93, 1, x_77); +return x_93; } } } else { -uint8_t x_103; -lean_dec(x_38); -lean_dec(x_24); -lean_dec(x_4); +uint8_t x_94; +lean_dec(x_29); +lean_dec(x_19); lean_dec(x_3); lean_dec(x_2); -x_103 = !lean_is_exclusive(x_39); -if (x_103 == 0) +lean_dec(x_1); +x_94 = !lean_is_exclusive(x_30); +if (x_94 == 0) { -return x_39; +return x_30; } else { -lean_object* x_104; lean_object* x_105; lean_object* x_106; -x_104 = lean_ctor_get(x_39, 0); -x_105 = lean_ctor_get(x_39, 1); -lean_inc(x_105); -lean_inc(x_104); -lean_dec(x_39); -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_95; lean_object* x_96; lean_object* x_97; +x_95 = lean_ctor_get(x_30, 0); +x_96 = lean_ctor_get(x_30, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_30); +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 { -uint8_t x_107; -lean_dec(x_24); -lean_dec(x_9); +uint8_t x_98; +lean_dec(x_19); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -2958,31 +2805,30 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_107 = !lean_is_exclusive(x_25); -if (x_107 == 0) +x_98 = !lean_is_exclusive(x_20); +if (x_98 == 0) { -return x_25; +return x_20; } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_108 = lean_ctor_get(x_25, 0); -x_109 = lean_ctor_get(x_25, 1); -lean_inc(x_109); -lean_inc(x_108); -lean_dec(x_25); -x_110 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_110, 0, x_108); -lean_ctor_set(x_110, 1, x_109); -return x_110; +lean_object* x_99; lean_object* x_100; lean_object* x_101; +x_99 = lean_ctor_get(x_20, 0); +x_100 = lean_ctor_get(x_20, 1); +lean_inc(x_100); +lean_inc(x_99); +lean_dec(x_20); +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; } } } } else { -uint8_t x_111; -lean_dec(x_9); +uint8_t x_102; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -2991,28 +2837,28 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_111 = !lean_is_exclusive(x_11); -if (x_111 == 0) +x_102 = !lean_is_exclusive(x_10); +if (x_102 == 0) { -return x_11; +return x_10; } else { -lean_object* x_112; lean_object* x_113; lean_object* x_114; -x_112 = lean_ctor_get(x_11, 0); -x_113 = lean_ctor_get(x_11, 1); -lean_inc(x_113); -lean_inc(x_112); -lean_dec(x_11); -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; +lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_103 = lean_ctor_get(x_10, 0); +x_104 = lean_ctor_get(x_10, 1); +lean_inc(x_104); +lean_inc(x_103); +lean_dec(x_10); +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; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__1() { _start: { lean_object* x_1; @@ -3020,21 +2866,21 @@ x_1 = lean_mk_string_unchecked("replicate_congr", 15, 15); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___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_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___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_ReifiedBVExpr_of___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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) { _start: { lean_object* x_13; lean_object* x_14; @@ -3050,7 +2896,7 @@ 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 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__2; +x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__2; x_18 = l_Lean_Expr_const___override(x_17, x_2); x_19 = l_Lean_mkApp5(x_18, x_3, x_4, x_5, x_6, x_16); lean_ctor_set(x_14, 0, x_19); @@ -3064,7 +2910,7 @@ x_21 = lean_ctor_get(x_14, 1); lean_inc(x_21); lean_inc(x_20); lean_dec(x_14); -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__2; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__2; x_23 = l_Lean_Expr_const___override(x_22, x_2); x_24 = l_Lean_mkApp5(x_23, x_3, x_4, x_5, x_6, x_20); x_25 = lean_alloc_ctor(0, 2, 0); @@ -3102,7 +2948,7 @@ return x_29; } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__1() { _start: { lean_object* x_1; @@ -3110,7 +2956,7 @@ x_1 = lean_mk_string_unchecked("replicate", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___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; @@ -3118,460 +2964,413 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___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_ReifiedBVExpr_of___lambda__8___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___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_ReifiedBVExpr_of___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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) { _start: { -lean_object* x_10; -lean_inc(x_8); +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_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_10) == 0) +lean_inc(x_2); +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_2, x_3, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_9) == 0) { -lean_object* x_11; -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -if (lean_obj_tag(x_11) == 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_12; -lean_dec(x_8); +uint8_t x_11; 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_is_exclusive(x_10); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_10, 0); -lean_dec(x_13); -x_14 = lean_box(0); -lean_ctor_set(x_10, 0, x_14); -return x_10; -} -else +lean_dec(x_2); +x_11 = !lean_is_exclusive(x_9); +if (x_11 == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_10, 1); -lean_inc(x_15); -lean_dec(x_10); -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_15); -return x_17; -} +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_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_10, 1); -lean_inc(x_18); +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; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_9, 1); +lean_inc(x_17); +lean_dec(x_9); +x_18 = lean_ctor_get(x_10, 0); +lean_inc(x_18); lean_dec(x_10); -x_19 = lean_ctor_get(x_11, 0); -lean_inc(x_19); -lean_dec(x_11); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -x_20 = l_Lean_Meta_getNatValue_x3f(x_2, x_5, x_6, x_7, x_8, x_18); +x_19 = l_Lean_Meta_getNatValue_x3f(x_1, x_4, x_5, x_6, x_7, x_17); +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) { -lean_object* x_21; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -if (lean_obj_tag(x_21) == 0) +uint8_t x_21; +lean_dec(x_18); +lean_dec(x_2); +x_21 = !lean_is_exclusive(x_19); +if (x_21 == 0) { lean_object* x_22; lean_object* x_23; -lean_dec(x_19); -lean_dec(x_3); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_4, x_5, x_6, x_7, x_8, x_22); -if (lean_obj_tag(x_23) == 0) -{ -uint8_t x_24; -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) -{ -return x_23; +x_22 = lean_ctor_get(x_19, 0); +lean_dec(x_22); +x_23 = lean_box(0); +lean_ctor_set(x_19, 0, x_23); +return x_19; } 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_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 = 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; } } else { -uint8_t x_28; -x_28 = !lean_is_exclusive(x_23); -if (x_28 == 0) +uint8_t x_27; +x_27 = !lean_is_exclusive(x_19); +if (x_27 == 0) { -return x_23; -} -else +lean_object* x_28; uint8_t x_29; +x_28 = lean_ctor_get(x_19, 0); +lean_dec(x_28); +x_29 = !lean_is_exclusive(x_20); +if (x_29 == 0) { -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_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_30 = lean_ctor_get(x_20, 0); +x_31 = lean_ctor_get(x_18, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_18, 1); +lean_inc(x_32); +x_33 = lean_ctor_get(x_18, 3); +lean_inc(x_33); lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_23); -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_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -x_32 = !lean_is_exclusive(x_20); -if (x_32 == 0) -{ -lean_object* x_33; uint8_t x_34; -x_33 = lean_ctor_get(x_20, 0); -lean_dec(x_33); -x_34 = !lean_is_exclusive(x_21); -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; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_35 = lean_ctor_get(x_21, 0); -x_36 = lean_ctor_get(x_19, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_19, 1); +lean_inc(x_31); +x_34 = lean_alloc_ctor(7, 3, 0); +lean_ctor_set(x_34, 0, x_31); +lean_ctor_set(x_34, 1, x_30); +lean_ctor_set(x_34, 2, x_32); +x_35 = lean_box(0); +lean_inc(x_31); +x_36 = l_Lean_mkNatLit(x_31); +lean_inc(x_30); +x_37 = l_Lean_mkNatLit(x_30); +x_38 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__3; +lean_inc(x_33); lean_inc(x_37); -x_38 = lean_ctor_get(x_19, 3); -lean_inc(x_38); -lean_inc(x_35); -lean_inc(x_36); -x_39 = lean_alloc_ctor(7, 3, 0); -lean_ctor_set(x_39, 0, x_36); -lean_ctor_set(x_39, 1, x_35); -lean_ctor_set(x_39, 2, x_37); -x_40 = lean_box(0); -lean_inc(x_36); -x_41 = l_Lean_mkNatLit(x_36); -lean_inc(x_35); -x_42 = l_Lean_mkNatLit(x_35); -x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__3; -lean_inc(x_38); -lean_inc(x_42); -lean_inc(x_41); -x_44 = l_Lean_mkApp3(x_43, x_41, x_42, x_38); lean_inc(x_36); -x_45 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_45, 0, x_36); -lean_closure_set(x_45, 1, x_38); -lean_inc(x_19); -x_46 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7), 12, 5); -lean_closure_set(x_46, 0, x_19); -lean_closure_set(x_46, 1, x_40); -lean_closure_set(x_46, 2, x_42); -lean_closure_set(x_46, 3, x_41); -lean_closure_set(x_46, 4, x_3); -x_47 = !lean_is_exclusive(x_19); -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; -x_48 = lean_ctor_get(x_19, 3); -lean_dec(x_48); -x_49 = lean_ctor_get(x_19, 2); -lean_dec(x_49); -x_50 = lean_ctor_get(x_19, 1); -lean_dec(x_50); -x_51 = lean_ctor_get(x_19, 0); -lean_dec(x_51); -x_52 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_52, 0, x_45); -lean_closure_set(x_52, 1, x_46); -x_53 = lean_nat_mul(x_36, x_35); -lean_dec(x_35); -lean_dec(x_36); -lean_ctor_set(x_19, 3, x_44); -lean_ctor_set(x_19, 2, x_52); -lean_ctor_set(x_19, 1, x_39); -lean_ctor_set(x_19, 0, x_53); -lean_ctor_set(x_21, 0, x_19); -return x_20; +x_39 = l_Lean_mkApp3(x_38, x_36, x_37, x_33); +lean_inc(x_31); +x_40 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_40, 0, x_31); +lean_closure_set(x_40, 1, x_33); +lean_inc(x_18); +x_41 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7), 12, 5); +lean_closure_set(x_41, 0, x_18); +lean_closure_set(x_41, 1, x_35); +lean_closure_set(x_41, 2, x_37); +lean_closure_set(x_41, 3, x_36); +lean_closure_set(x_41, 4, x_2); +x_42 = !lean_is_exclusive(x_18); +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; +x_43 = lean_ctor_get(x_18, 3); +lean_dec(x_43); +x_44 = lean_ctor_get(x_18, 2); +lean_dec(x_44); +x_45 = lean_ctor_get(x_18, 1); +lean_dec(x_45); +x_46 = lean_ctor_get(x_18, 0); +lean_dec(x_46); +x_47 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_47, 0, x_40); +lean_closure_set(x_47, 1, x_41); +x_48 = lean_nat_mul(x_31, x_30); +lean_dec(x_30); +lean_dec(x_31); +lean_ctor_set(x_18, 3, x_39); +lean_ctor_set(x_18, 2, x_47); +lean_ctor_set(x_18, 1, x_34); +lean_ctor_set(x_18, 0, x_48); +lean_ctor_set(x_20, 0, x_18); +return x_19; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; -lean_dec(x_19); -x_54 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_54, 0, x_45); -lean_closure_set(x_54, 1, x_46); -x_55 = lean_nat_mul(x_36, x_35); -lean_dec(x_35); -lean_dec(x_36); -x_56 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_56, 0, x_55); -lean_ctor_set(x_56, 1, x_39); -lean_ctor_set(x_56, 2, x_54); -lean_ctor_set(x_56, 3, x_44); -lean_ctor_set(x_21, 0, x_56); -return x_20; +lean_object* x_49; lean_object* x_50; lean_object* x_51; +lean_dec(x_18); +x_49 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_49, 0, x_40); +lean_closure_set(x_49, 1, x_41); +x_50 = lean_nat_mul(x_31, x_30); +lean_dec(x_30); +lean_dec(x_31); +x_51 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_34); +lean_ctor_set(x_51, 2, x_49); +lean_ctor_set(x_51, 3, x_39); +lean_ctor_set(x_20, 0, x_51); +return x_19; } } 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; 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_57 = lean_ctor_get(x_21, 0); -lean_inc(x_57); -lean_dec(x_21); -x_58 = lean_ctor_get(x_19, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_19, 1); +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; +x_52 = lean_ctor_get(x_20, 0); +lean_inc(x_52); +lean_dec(x_20); +x_53 = lean_ctor_get(x_18, 0); +lean_inc(x_53); +x_54 = lean_ctor_get(x_18, 1); +lean_inc(x_54); +x_55 = lean_ctor_get(x_18, 3); +lean_inc(x_55); +lean_inc(x_52); +lean_inc(x_53); +x_56 = lean_alloc_ctor(7, 3, 0); +lean_ctor_set(x_56, 0, x_53); +lean_ctor_set(x_56, 1, x_52); +lean_ctor_set(x_56, 2, x_54); +x_57 = lean_box(0); +lean_inc(x_53); +x_58 = l_Lean_mkNatLit(x_53); +lean_inc(x_52); +x_59 = l_Lean_mkNatLit(x_52); +x_60 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__3; +lean_inc(x_55); lean_inc(x_59); -x_60 = lean_ctor_get(x_19, 3); -lean_inc(x_60); -lean_inc(x_57); -lean_inc(x_58); -x_61 = lean_alloc_ctor(7, 3, 0); -lean_ctor_set(x_61, 0, x_58); -lean_ctor_set(x_61, 1, x_57); -lean_ctor_set(x_61, 2, x_59); -x_62 = lean_box(0); lean_inc(x_58); -x_63 = l_Lean_mkNatLit(x_58); -lean_inc(x_57); -x_64 = l_Lean_mkNatLit(x_57); -x_65 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__3; -lean_inc(x_60); -lean_inc(x_64); -lean_inc(x_63); -x_66 = l_Lean_mkApp3(x_65, x_63, x_64, x_60); -lean_inc(x_58); -x_67 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_67, 0, x_58); -lean_closure_set(x_67, 1, x_60); -lean_inc(x_19); -x_68 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7), 12, 5); -lean_closure_set(x_68, 0, x_19); -lean_closure_set(x_68, 1, x_62); -lean_closure_set(x_68, 2, x_64); -lean_closure_set(x_68, 3, x_63); -lean_closure_set(x_68, 4, x_3); -if (lean_is_exclusive(x_19)) { - lean_ctor_release(x_19, 0); - lean_ctor_release(x_19, 1); - lean_ctor_release(x_19, 2); - lean_ctor_release(x_19, 3); - x_69 = x_19; +x_61 = l_Lean_mkApp3(x_60, x_58, x_59, x_55); +lean_inc(x_53); +x_62 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_62, 0, x_53); +lean_closure_set(x_62, 1, x_55); +lean_inc(x_18); +x_63 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7), 12, 5); +lean_closure_set(x_63, 0, x_18); +lean_closure_set(x_63, 1, x_57); +lean_closure_set(x_63, 2, x_59); +lean_closure_set(x_63, 3, x_58); +lean_closure_set(x_63, 4, x_2); +if (lean_is_exclusive(x_18)) { + lean_ctor_release(x_18, 0); + lean_ctor_release(x_18, 1); + lean_ctor_release(x_18, 2); + lean_ctor_release(x_18, 3); + x_64 = x_18; } else { - lean_dec_ref(x_19); - x_69 = lean_box(0); + lean_dec_ref(x_18); + x_64 = lean_box(0); } -x_70 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_70, 0, x_67); -lean_closure_set(x_70, 1, x_68); -x_71 = lean_nat_mul(x_58, x_57); -lean_dec(x_57); -lean_dec(x_58); -if (lean_is_scalar(x_69)) { - x_72 = lean_alloc_ctor(0, 4, 0); +x_65 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_65, 0, x_62); +lean_closure_set(x_65, 1, x_63); +x_66 = lean_nat_mul(x_53, x_52); +lean_dec(x_52); +lean_dec(x_53); +if (lean_is_scalar(x_64)) { + x_67 = lean_alloc_ctor(0, 4, 0); } else { - x_72 = x_69; -} -lean_ctor_set(x_72, 0, x_71); -lean_ctor_set(x_72, 1, x_61); -lean_ctor_set(x_72, 2, x_70); -lean_ctor_set(x_72, 3, x_66); -x_73 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_73, 0, x_72); -lean_ctor_set(x_20, 0, x_73); -return x_20; + x_67 = x_64; +} +lean_ctor_set(x_67, 0, x_66); +lean_ctor_set(x_67, 1, x_56); +lean_ctor_set(x_67, 2, x_65); +lean_ctor_set(x_67, 3, x_61); +x_68 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_68, 0, x_67); +lean_ctor_set(x_19, 0, x_68); +return x_19; } } 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; 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; -x_74 = lean_ctor_get(x_20, 1); -lean_inc(x_74); -lean_dec(x_20); -x_75 = lean_ctor_get(x_21, 0); -lean_inc(x_75); -if (lean_is_exclusive(x_21)) { - lean_ctor_release(x_21, 0); - x_76 = x_21; +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; +x_69 = lean_ctor_get(x_19, 1); +lean_inc(x_69); +lean_dec(x_19); +x_70 = lean_ctor_get(x_20, 0); +lean_inc(x_70); +if (lean_is_exclusive(x_20)) { + lean_ctor_release(x_20, 0); + x_71 = x_20; } else { - lean_dec_ref(x_21); - x_76 = lean_box(0); + lean_dec_ref(x_20); + x_71 = lean_box(0); } -x_77 = lean_ctor_get(x_19, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_19, 1); +x_72 = lean_ctor_get(x_18, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_18, 1); +lean_inc(x_73); +x_74 = lean_ctor_get(x_18, 3); +lean_inc(x_74); +lean_inc(x_70); +lean_inc(x_72); +x_75 = lean_alloc_ctor(7, 3, 0); +lean_ctor_set(x_75, 0, x_72); +lean_ctor_set(x_75, 1, x_70); +lean_ctor_set(x_75, 2, x_73); +x_76 = lean_box(0); +lean_inc(x_72); +x_77 = l_Lean_mkNatLit(x_72); +lean_inc(x_70); +x_78 = l_Lean_mkNatLit(x_70); +x_79 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__3; +lean_inc(x_74); lean_inc(x_78); -x_79 = lean_ctor_get(x_19, 3); -lean_inc(x_79); -lean_inc(x_75); lean_inc(x_77); -x_80 = lean_alloc_ctor(7, 3, 0); -lean_ctor_set(x_80, 0, x_77); -lean_ctor_set(x_80, 1, x_75); -lean_ctor_set(x_80, 2, x_78); -x_81 = lean_box(0); -lean_inc(x_77); -x_82 = l_Lean_mkNatLit(x_77); -lean_inc(x_75); -x_83 = l_Lean_mkNatLit(x_75); -x_84 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__3; -lean_inc(x_79); -lean_inc(x_83); -lean_inc(x_82); -x_85 = l_Lean_mkApp3(x_84, x_82, x_83, x_79); -lean_inc(x_77); -x_86 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_86, 0, x_77); -lean_closure_set(x_86, 1, x_79); -lean_inc(x_19); -x_87 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7), 12, 5); -lean_closure_set(x_87, 0, x_19); -lean_closure_set(x_87, 1, x_81); -lean_closure_set(x_87, 2, x_83); -lean_closure_set(x_87, 3, x_82); -lean_closure_set(x_87, 4, x_3); -if (lean_is_exclusive(x_19)) { - lean_ctor_release(x_19, 0); - lean_ctor_release(x_19, 1); - lean_ctor_release(x_19, 2); - lean_ctor_release(x_19, 3); - x_88 = x_19; +x_80 = l_Lean_mkApp3(x_79, x_77, x_78, x_74); +lean_inc(x_72); +x_81 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_81, 0, x_72); +lean_closure_set(x_81, 1, x_74); +lean_inc(x_18); +x_82 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7), 12, 5); +lean_closure_set(x_82, 0, x_18); +lean_closure_set(x_82, 1, x_76); +lean_closure_set(x_82, 2, x_78); +lean_closure_set(x_82, 3, x_77); +lean_closure_set(x_82, 4, x_2); +if (lean_is_exclusive(x_18)) { + lean_ctor_release(x_18, 0); + lean_ctor_release(x_18, 1); + lean_ctor_release(x_18, 2); + lean_ctor_release(x_18, 3); + x_83 = x_18; } else { - lean_dec_ref(x_19); - x_88 = lean_box(0); -} -x_89 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_89, 0, x_86); -lean_closure_set(x_89, 1, x_87); -x_90 = lean_nat_mul(x_77, x_75); -lean_dec(x_75); -lean_dec(x_77); -if (lean_is_scalar(x_88)) { - x_91 = lean_alloc_ctor(0, 4, 0); + lean_dec_ref(x_18); + x_83 = lean_box(0); +} +x_84 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_84, 0, x_81); +lean_closure_set(x_84, 1, x_82); +x_85 = lean_nat_mul(x_72, x_70); +lean_dec(x_70); +lean_dec(x_72); +if (lean_is_scalar(x_83)) { + x_86 = lean_alloc_ctor(0, 4, 0); } else { - x_91 = x_88; -} -lean_ctor_set(x_91, 0, x_90); -lean_ctor_set(x_91, 1, x_80); -lean_ctor_set(x_91, 2, x_89); -lean_ctor_set(x_91, 3, x_85); -if (lean_is_scalar(x_76)) { - x_92 = lean_alloc_ctor(1, 1, 0); + x_86 = x_83; +} +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_75); +lean_ctor_set(x_86, 2, x_84); +lean_ctor_set(x_86, 3, x_80); +if (lean_is_scalar(x_71)) { + x_87 = lean_alloc_ctor(1, 1, 0); } else { - x_92 = x_76; + x_87 = x_71; } -lean_ctor_set(x_92, 0, x_91); -x_93 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_93, 0, x_92); -lean_ctor_set(x_93, 1, x_74); -return x_93; +lean_ctor_set(x_87, 0, x_86); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_87); +lean_ctor_set(x_88, 1, x_69); +return x_88; } } } else { -uint8_t x_94; -lean_dec(x_19); -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_94 = !lean_is_exclusive(x_20); -if (x_94 == 0) +uint8_t x_89; +lean_dec(x_18); +lean_dec(x_2); +x_89 = !lean_is_exclusive(x_19); +if (x_89 == 0) { -return x_20; +return x_19; } else { -lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_95 = lean_ctor_get(x_20, 0); -x_96 = lean_ctor_get(x_20, 1); -lean_inc(x_96); -lean_inc(x_95); -lean_dec(x_20); -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; +lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_90 = lean_ctor_get(x_19, 0); +x_91 = lean_ctor_get(x_19, 1); +lean_inc(x_91); +lean_inc(x_90); +lean_dec(x_19); +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_98; -lean_dec(x_8); +uint8_t x_93; 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_98 = !lean_is_exclusive(x_10); -if (x_98 == 0) +lean_dec(x_2); +x_93 = !lean_is_exclusive(x_9); +if (x_93 == 0) { -return x_10; +return x_9; } else { -lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_99 = lean_ctor_get(x_10, 0); -x_100 = lean_ctor_get(x_10, 1); -lean_inc(x_100); -lean_inc(x_99); -lean_dec(x_10); -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_94; lean_object* x_95; lean_object* x_96; +x_94 = lean_ctor_get(x_9, 0); +x_95 = lean_ctor_get(x_9, 1); +lean_inc(x_95); +lean_inc(x_94); +lean_dec(x_9); +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; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__1() { _start: { lean_object* x_1; @@ -3579,21 +3378,21 @@ x_1 = lean_mk_string_unchecked("append_congr", 12, 12); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___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_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___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_ReifiedBVExpr_of___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_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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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_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; @@ -3642,7 +3441,7 @@ if (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_25, 0); -x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__2; +x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__2; x_29 = l_Lean_Expr_const___override(x_28, x_5); x_30 = l_Lean_mkApp8(x_29, x_6, x_7, x_8, x_10, x_9, x_27, x_19, x_23); lean_ctor_set(x_25, 0, x_30); @@ -3656,7 +3455,7 @@ x_32 = lean_ctor_get(x_25, 1); lean_inc(x_32); lean_inc(x_31); lean_dec(x_25); -x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__2; +x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__2; x_34 = l_Lean_Expr_const___override(x_33, x_5); x_35 = l_Lean_mkApp8(x_34, x_6, x_7, x_8, x_10, x_9, x_31, x_19, x_23); x_36 = lean_alloc_ctor(0, 2, 0); @@ -3740,7 +3539,7 @@ return x_44; } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__1() { _start: { lean_object* x_1; @@ -3748,7 +3547,7 @@ x_1 = lean_mk_string_unchecked("append", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___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; @@ -3756,22 +3555,22 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___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_ReifiedBVExpr_of___lambda__10___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___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_ReifiedBVExpr_of___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, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; @@ -3781,7 +3580,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_1); -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_1, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(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; @@ -3830,7 +3629,7 @@ x_18 = lean_ctor_get(x_10, 0); lean_inc(x_18); lean_dec(x_10); lean_inc(x_2); -x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_2, x_3, x_4, x_5, x_6, x_7, x_17); +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_2, x_3, x_4, x_5, x_6, x_7, x_17); if (lean_obj_tag(x_19) == 0) { lean_object* x_20; @@ -3903,7 +3702,7 @@ lean_inc(x_34); x_39 = l_Lean_mkNatLit(x_34); x_40 = lean_ctor_get(x_30, 3); lean_inc(x_40); -x_41 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__3; +x_41 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__3; lean_inc(x_40); lean_inc(x_33); lean_inc(x_39); @@ -3915,7 +3714,7 @@ lean_closure_set(x_43, 0, x_31); lean_closure_set(x_43, 1, x_33); lean_inc(x_34); lean_inc(x_18); -x_44 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9), 16, 9); +x_44 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9), 16, 9); lean_closure_set(x_44, 0, x_18); lean_closure_set(x_44, 1, x_30); lean_closure_set(x_44, 2, x_34); @@ -3999,7 +3798,7 @@ lean_inc(x_59); x_64 = l_Lean_mkNatLit(x_59); x_65 = lean_ctor_get(x_55, 3); lean_inc(x_65); -x_66 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__3; +x_66 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__3; lean_inc(x_65); lean_inc(x_58); lean_inc(x_64); @@ -4011,7 +3810,7 @@ lean_closure_set(x_68, 0, x_56); lean_closure_set(x_68, 1, x_58); lean_inc(x_59); lean_inc(x_18); -x_69 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9), 16, 9); +x_69 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9), 16, 9); lean_closure_set(x_69, 0, x_18); lean_closure_set(x_69, 1, x_55); lean_closure_set(x_69, 2, x_59); @@ -4091,7 +3890,7 @@ lean_inc(x_81); x_86 = l_Lean_mkNatLit(x_81); x_87 = lean_ctor_get(x_76, 3); lean_inc(x_87); -x_88 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__3; +x_88 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__3; lean_inc(x_87); lean_inc(x_80); lean_inc(x_86); @@ -4103,7 +3902,7 @@ lean_closure_set(x_90, 0, x_78); lean_closure_set(x_90, 1, x_80); lean_inc(x_81); lean_inc(x_18); -x_91 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9), 16, 9); +x_91 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9), 16, 9); lean_closure_set(x_91, 0, x_18); lean_closure_set(x_91, 1, x_76); lean_closure_set(x_91, 2, x_81); @@ -4209,7 +4008,7 @@ return x_105; } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__1() { _start: { lean_object* x_1; @@ -4217,21 +4016,21 @@ x_1 = lean_mk_string_unchecked("signExtend_congr", 16, 16); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___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_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___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_ReifiedBVExpr_of___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, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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, 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; @@ -4247,7 +4046,7 @@ 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 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__2; +x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__2; x_18 = l_Lean_Expr_const___override(x_17, x_2); x_19 = l_Lean_mkApp5(x_18, x_3, x_4, x_5, x_6, x_16); lean_ctor_set(x_14, 0, x_19); @@ -4261,7 +4060,7 @@ x_21 = lean_ctor_get(x_14, 1); lean_inc(x_21); lean_inc(x_20); lean_dec(x_14); -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__2; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__2; x_23 = l_Lean_Expr_const___override(x_22, x_2); x_24 = l_Lean_mkApp5(x_23, x_3, x_4, x_5, x_6, x_20); x_25 = lean_alloc_ctor(0, 2, 0); @@ -4299,7 +4098,7 @@ return x_29; } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__1() { _start: { lean_object* x_1; @@ -4307,7 +4106,7 @@ x_1 = lean_mk_string_unchecked("signExtend", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___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; @@ -4315,394 +4114,371 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___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_ReifiedBVExpr_of___lambda__12___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___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_ReifiedBVExpr_of___lambda__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_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__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_object* x_7, lean_object* x_8) { _start: { -lean_object* x_10; -lean_inc(x_8); +lean_object* x_9; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_10 = l_Lean_Meta_getNatValue_x3f(x_2, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_10) == 0) +lean_inc(x_4); +x_9 = l_Lean_Meta_getNatValue_x3f(x_1, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_9) == 0) { -lean_object* x_11; -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -if (lean_obj_tag(x_11) == 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_object* x_12; lean_object* x_13; +uint8_t x_11; +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_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_4, x_5, x_6, x_7, x_8, x_12); -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_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_dec(x_1); +x_11 = !lean_is_exclusive(x_9); +if (x_11 == 0) { -return x_13; +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_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; -} +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_22; lean_object* x_23; lean_object* x_24; -lean_dec(x_1); -x_22 = lean_ctor_get(x_10, 1); -lean_inc(x_22); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_9, 1); +lean_inc(x_17); +lean_dec(x_9); +x_18 = lean_ctor_get(x_10, 0); +lean_inc(x_18); lean_dec(x_10); -x_23 = lean_ctor_get(x_11, 0); -lean_inc(x_23); -lean_dec(x_11); -lean_inc(x_3); -x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_3, x_4, x_5, x_6, x_7, x_8, x_22); -if (lean_obj_tag(x_24) == 0) +lean_inc(x_2); +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_2, x_3, x_4, x_5, x_6, x_7, x_17); +if (lean_obj_tag(x_19) == 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_20; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +if (lean_obj_tag(x_20) == 0) { -uint8_t x_26; -lean_dec(x_23); -lean_dec(x_3); +uint8_t x_21; +lean_dec(x_18); lean_dec(x_2); -x_26 = !lean_is_exclusive(x_24); -if (x_26 == 0) +lean_dec(x_1); +x_21 = !lean_is_exclusive(x_19); +if (x_21 == 0) { -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_24, 0); -lean_dec(x_27); -x_28 = lean_box(0); -lean_ctor_set(x_24, 0, x_28); -return x_24; +lean_object* x_22; lean_object* x_23; +x_22 = lean_ctor_get(x_19, 0); +lean_dec(x_22); +x_23 = lean_box(0); +lean_ctor_set(x_19, 0, x_23); +return x_19; } 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_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; +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 = 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; } } else { -uint8_t x_32; -x_32 = !lean_is_exclusive(x_25); -if (x_32 == 0) +uint8_t x_27; +x_27 = !lean_is_exclusive(x_20); +if (x_27 == 0) { -uint8_t x_33; -x_33 = !lean_is_exclusive(x_24); -if (x_33 == 0) +uint8_t x_28; +x_28 = !lean_is_exclusive(x_19); +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; 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_34 = lean_ctor_get(x_25, 0); -x_35 = lean_ctor_get(x_24, 0); -lean_dec(x_35); -x_36 = lean_ctor_get(x_34, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_34, 1); -lean_inc(x_37); -x_38 = lean_ctor_get(x_34, 3); -lean_inc(x_38); -lean_inc(x_23); -lean_inc(x_36); -x_39 = lean_alloc_ctor(8, 3, 0); -lean_ctor_set(x_39, 0, x_36); -lean_ctor_set(x_39, 1, x_23); -lean_ctor_set(x_39, 2, x_37); -x_40 = lean_box(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; uint8_t x_41; +x_29 = lean_ctor_get(x_20, 0); +x_30 = lean_ctor_get(x_19, 0); +lean_dec(x_30); +x_31 = lean_ctor_get(x_29, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_29, 1); +lean_inc(x_32); +x_33 = lean_ctor_get(x_29, 3); +lean_inc(x_33); +lean_inc(x_18); +lean_inc(x_31); +x_34 = lean_alloc_ctor(8, 3, 0); +lean_ctor_set(x_34, 0, x_31); +lean_ctor_set(x_34, 1, x_18); +lean_ctor_set(x_34, 2, x_32); +x_35 = lean_box(0); +lean_inc(x_31); +x_36 = l_Lean_mkNatLit(x_31); +x_37 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__3; +lean_inc(x_33); +lean_inc(x_1); lean_inc(x_36); -x_41 = l_Lean_mkNatLit(x_36); -x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__3; -lean_inc(x_38); -lean_inc(x_2); -lean_inc(x_41); -x_43 = l_Lean_mkApp3(x_42, x_41, x_2, x_38); -x_44 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_44, 0, x_36); -lean_closure_set(x_44, 1, x_38); -lean_inc(x_34); -x_45 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11), 12, 5); -lean_closure_set(x_45, 0, x_34); -lean_closure_set(x_45, 1, x_40); -lean_closure_set(x_45, 2, x_2); -lean_closure_set(x_45, 3, x_41); -lean_closure_set(x_45, 4, x_3); -x_46 = !lean_is_exclusive(x_34); -if (x_46 == 0) -{ -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_47 = lean_ctor_get(x_34, 3); -lean_dec(x_47); -x_48 = lean_ctor_get(x_34, 2); -lean_dec(x_48); -x_49 = lean_ctor_get(x_34, 1); -lean_dec(x_49); -x_50 = lean_ctor_get(x_34, 0); -lean_dec(x_50); -x_51 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_51, 0, x_44); -lean_closure_set(x_51, 1, x_45); -lean_ctor_set(x_34, 3, x_43); -lean_ctor_set(x_34, 2, x_51); -lean_ctor_set(x_34, 1, x_39); -lean_ctor_set(x_34, 0, x_23); -return x_24; +x_38 = l_Lean_mkApp3(x_37, x_36, x_1, x_33); +x_39 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_39, 0, x_31); +lean_closure_set(x_39, 1, x_33); +lean_inc(x_29); +x_40 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11), 12, 5); +lean_closure_set(x_40, 0, x_29); +lean_closure_set(x_40, 1, x_35); +lean_closure_set(x_40, 2, x_1); +lean_closure_set(x_40, 3, x_36); +lean_closure_set(x_40, 4, x_2); +x_41 = !lean_is_exclusive(x_29); +if (x_41 == 0) +{ +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_29, 3); +lean_dec(x_42); +x_43 = lean_ctor_get(x_29, 2); +lean_dec(x_43); +x_44 = lean_ctor_get(x_29, 1); +lean_dec(x_44); +x_45 = lean_ctor_get(x_29, 0); +lean_dec(x_45); +x_46 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_46, 0, x_39); +lean_closure_set(x_46, 1, x_40); +lean_ctor_set(x_29, 3, x_38); +lean_ctor_set(x_29, 2, x_46); +lean_ctor_set(x_29, 1, x_34); +lean_ctor_set(x_29, 0, x_18); +return x_19; } else { -lean_object* x_52; lean_object* x_53; -lean_dec(x_34); -x_52 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_52, 0, x_44); -lean_closure_set(x_52, 1, x_45); -x_53 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_53, 0, x_23); -lean_ctor_set(x_53, 1, x_39); -lean_ctor_set(x_53, 2, x_52); -lean_ctor_set(x_53, 3, x_43); -lean_ctor_set(x_25, 0, x_53); -return x_24; +lean_object* x_47; lean_object* x_48; +lean_dec(x_29); +x_47 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_47, 0, x_39); +lean_closure_set(x_47, 1, x_40); +x_48 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_48, 0, x_18); +lean_ctor_set(x_48, 1, x_34); +lean_ctor_set(x_48, 2, x_47); +lean_ctor_set(x_48, 3, x_38); +lean_ctor_set(x_20, 0, x_48); +return x_19; } } 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; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_54 = lean_ctor_get(x_25, 0); -x_55 = lean_ctor_get(x_24, 1); -lean_inc(x_55); -lean_dec(x_24); -x_56 = lean_ctor_get(x_54, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_54, 1); -lean_inc(x_57); -x_58 = lean_ctor_get(x_54, 3); -lean_inc(x_58); -lean_inc(x_23); -lean_inc(x_56); -x_59 = lean_alloc_ctor(8, 3, 0); -lean_ctor_set(x_59, 0, x_56); -lean_ctor_set(x_59, 1, x_23); -lean_ctor_set(x_59, 2, x_57); -x_60 = lean_box(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; 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_49 = lean_ctor_get(x_20, 0); +x_50 = lean_ctor_get(x_19, 1); +lean_inc(x_50); +lean_dec(x_19); +x_51 = lean_ctor_get(x_49, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_49, 1); +lean_inc(x_52); +x_53 = lean_ctor_get(x_49, 3); +lean_inc(x_53); +lean_inc(x_18); +lean_inc(x_51); +x_54 = lean_alloc_ctor(8, 3, 0); +lean_ctor_set(x_54, 0, x_51); +lean_ctor_set(x_54, 1, x_18); +lean_ctor_set(x_54, 2, x_52); +x_55 = lean_box(0); +lean_inc(x_51); +x_56 = l_Lean_mkNatLit(x_51); +x_57 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__3; +lean_inc(x_53); +lean_inc(x_1); lean_inc(x_56); -x_61 = l_Lean_mkNatLit(x_56); -x_62 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__3; -lean_inc(x_58); -lean_inc(x_2); -lean_inc(x_61); -x_63 = l_Lean_mkApp3(x_62, x_61, x_2, x_58); -x_64 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_64, 0, x_56); -lean_closure_set(x_64, 1, x_58); -lean_inc(x_54); -x_65 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11), 12, 5); -lean_closure_set(x_65, 0, x_54); -lean_closure_set(x_65, 1, x_60); -lean_closure_set(x_65, 2, x_2); -lean_closure_set(x_65, 3, x_61); -lean_closure_set(x_65, 4, x_3); -if (lean_is_exclusive(x_54)) { - lean_ctor_release(x_54, 0); - lean_ctor_release(x_54, 1); - lean_ctor_release(x_54, 2); - lean_ctor_release(x_54, 3); - x_66 = x_54; +x_58 = l_Lean_mkApp3(x_57, x_56, x_1, x_53); +x_59 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_59, 0, x_51); +lean_closure_set(x_59, 1, x_53); +lean_inc(x_49); +x_60 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11), 12, 5); +lean_closure_set(x_60, 0, x_49); +lean_closure_set(x_60, 1, x_55); +lean_closure_set(x_60, 2, x_1); +lean_closure_set(x_60, 3, x_56); +lean_closure_set(x_60, 4, x_2); +if (lean_is_exclusive(x_49)) { + lean_ctor_release(x_49, 0); + lean_ctor_release(x_49, 1); + lean_ctor_release(x_49, 2); + lean_ctor_release(x_49, 3); + x_61 = x_49; } else { - lean_dec_ref(x_54); - x_66 = lean_box(0); -} -x_67 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_67, 0, x_64); -lean_closure_set(x_67, 1, x_65); -if (lean_is_scalar(x_66)) { - x_68 = lean_alloc_ctor(0, 4, 0); + lean_dec_ref(x_49); + x_61 = lean_box(0); +} +x_62 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_62, 0, x_59); +lean_closure_set(x_62, 1, x_60); +if (lean_is_scalar(x_61)) { + x_63 = lean_alloc_ctor(0, 4, 0); } else { - x_68 = x_66; + x_63 = x_61; } -lean_ctor_set(x_68, 0, x_23); -lean_ctor_set(x_68, 1, x_59); -lean_ctor_set(x_68, 2, x_67); -lean_ctor_set(x_68, 3, x_63); -lean_ctor_set(x_25, 0, x_68); -x_69 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_69, 0, x_25); -lean_ctor_set(x_69, 1, x_55); -return x_69; +lean_ctor_set(x_63, 0, x_18); +lean_ctor_set(x_63, 1, x_54); +lean_ctor_set(x_63, 2, x_62); +lean_ctor_set(x_63, 3, x_58); +lean_ctor_set(x_20, 0, x_63); +x_64 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_64, 0, x_20); +lean_ctor_set(x_64, 1, x_50); +return x_64; } } 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_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_70 = lean_ctor_get(x_25, 0); -lean_inc(x_70); -lean_dec(x_25); -x_71 = lean_ctor_get(x_24, 1); -lean_inc(x_71); -if (lean_is_exclusive(x_24)) { - lean_ctor_release(x_24, 0); - lean_ctor_release(x_24, 1); - x_72 = x_24; +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; +x_65 = lean_ctor_get(x_20, 0); +lean_inc(x_65); +lean_dec(x_20); +x_66 = lean_ctor_get(x_19, 1); +lean_inc(x_66); +if (lean_is_exclusive(x_19)) { + lean_ctor_release(x_19, 0); + lean_ctor_release(x_19, 1); + x_67 = x_19; } else { - lean_dec_ref(x_24); - x_72 = lean_box(0); + lean_dec_ref(x_19); + x_67 = lean_box(0); } -x_73 = lean_ctor_get(x_70, 0); -lean_inc(x_73); -x_74 = lean_ctor_get(x_70, 1); -lean_inc(x_74); -x_75 = lean_ctor_get(x_70, 3); -lean_inc(x_75); -lean_inc(x_23); -lean_inc(x_73); -x_76 = lean_alloc_ctor(8, 3, 0); -lean_ctor_set(x_76, 0, x_73); -lean_ctor_set(x_76, 1, x_23); -lean_ctor_set(x_76, 2, x_74); -x_77 = lean_box(0); -lean_inc(x_73); -x_78 = l_Lean_mkNatLit(x_73); -x_79 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__3; -lean_inc(x_75); -lean_inc(x_2); -lean_inc(x_78); -x_80 = l_Lean_mkApp3(x_79, x_78, x_2, x_75); -x_81 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_81, 0, x_73); -lean_closure_set(x_81, 1, x_75); +x_68 = lean_ctor_get(x_65, 0); +lean_inc(x_68); +x_69 = lean_ctor_get(x_65, 1); +lean_inc(x_69); +x_70 = lean_ctor_get(x_65, 3); +lean_inc(x_70); +lean_inc(x_18); +lean_inc(x_68); +x_71 = lean_alloc_ctor(8, 3, 0); +lean_ctor_set(x_71, 0, x_68); +lean_ctor_set(x_71, 1, x_18); +lean_ctor_set(x_71, 2, x_69); +x_72 = lean_box(0); +lean_inc(x_68); +x_73 = l_Lean_mkNatLit(x_68); +x_74 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__3; lean_inc(x_70); -x_82 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11), 12, 5); -lean_closure_set(x_82, 0, x_70); -lean_closure_set(x_82, 1, x_77); -lean_closure_set(x_82, 2, x_2); -lean_closure_set(x_82, 3, x_78); -lean_closure_set(x_82, 4, x_3); -if (lean_is_exclusive(x_70)) { - lean_ctor_release(x_70, 0); - lean_ctor_release(x_70, 1); - lean_ctor_release(x_70, 2); - lean_ctor_release(x_70, 3); - x_83 = x_70; +lean_inc(x_1); +lean_inc(x_73); +x_75 = l_Lean_mkApp3(x_74, x_73, x_1, x_70); +x_76 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_76, 0, x_68); +lean_closure_set(x_76, 1, x_70); +lean_inc(x_65); +x_77 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11), 12, 5); +lean_closure_set(x_77, 0, x_65); +lean_closure_set(x_77, 1, x_72); +lean_closure_set(x_77, 2, x_1); +lean_closure_set(x_77, 3, x_73); +lean_closure_set(x_77, 4, x_2); +if (lean_is_exclusive(x_65)) { + lean_ctor_release(x_65, 0); + lean_ctor_release(x_65, 1); + lean_ctor_release(x_65, 2); + lean_ctor_release(x_65, 3); + x_78 = x_65; } else { - lean_dec_ref(x_70); - x_83 = lean_box(0); + lean_dec_ref(x_65); + x_78 = lean_box(0); } -x_84 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_84, 0, x_81); -lean_closure_set(x_84, 1, x_82); -if (lean_is_scalar(x_83)) { - x_85 = lean_alloc_ctor(0, 4, 0); +x_79 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_79, 0, x_76); +lean_closure_set(x_79, 1, x_77); +if (lean_is_scalar(x_78)) { + x_80 = lean_alloc_ctor(0, 4, 0); } else { - x_85 = x_83; -} -lean_ctor_set(x_85, 0, x_23); -lean_ctor_set(x_85, 1, x_76); -lean_ctor_set(x_85, 2, x_84); -lean_ctor_set(x_85, 3, x_80); -x_86 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_86, 0, x_85); -if (lean_is_scalar(x_72)) { - x_87 = lean_alloc_ctor(0, 2, 0); + x_80 = x_78; +} +lean_ctor_set(x_80, 0, x_18); +lean_ctor_set(x_80, 1, x_71); +lean_ctor_set(x_80, 2, x_79); +lean_ctor_set(x_80, 3, x_75); +x_81 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_81, 0, x_80); +if (lean_is_scalar(x_67)) { + x_82 = lean_alloc_ctor(0, 2, 0); } else { - x_87 = x_72; + x_82 = x_67; } -lean_ctor_set(x_87, 0, x_86); -lean_ctor_set(x_87, 1, x_71); -return x_87; +lean_ctor_set(x_82, 0, x_81); +lean_ctor_set(x_82, 1, x_66); +return x_82; } } } else { -uint8_t x_88; -lean_dec(x_23); -lean_dec(x_3); +uint8_t x_83; +lean_dec(x_18); lean_dec(x_2); -x_88 = !lean_is_exclusive(x_24); -if (x_88 == 0) +lean_dec(x_1); +x_83 = !lean_is_exclusive(x_19); +if (x_83 == 0) { -return x_24; +return x_19; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_89 = lean_ctor_get(x_24, 0); -x_90 = lean_ctor_get(x_24, 1); -lean_inc(x_90); -lean_inc(x_89); -lean_dec(x_24); -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_84; lean_object* x_85; lean_object* x_86; +x_84 = lean_ctor_get(x_19, 0); +x_85 = lean_ctor_get(x_19, 1); +lean_inc(x_85); +lean_inc(x_84); +lean_dec(x_19); +x_86 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_86, 0, x_84); +lean_ctor_set(x_86, 1, x_85); +return x_86; } } } } else { -uint8_t x_92; -lean_dec(x_8); +uint8_t x_87; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -4710,28 +4486,28 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_92 = !lean_is_exclusive(x_10); -if (x_92 == 0) +x_87 = !lean_is_exclusive(x_9); +if (x_87 == 0) { -return x_10; +return x_9; } else { -lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_93 = lean_ctor_get(x_10, 0); -x_94 = lean_ctor_get(x_10, 1); -lean_inc(x_94); -lean_inc(x_93); -lean_dec(x_10); -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_88; lean_object* x_89; lean_object* x_90; +x_88 = lean_ctor_get(x_9, 0); +x_89 = lean_ctor_get(x_9, 1); +lean_inc(x_89); +lean_inc(x_88); +lean_dec(x_9); +x_90 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_90, 0, x_88); +lean_ctor_set(x_90, 1, x_89); +return x_90; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__1() { _start: { lean_object* x_1; @@ -4739,21 +4515,21 @@ x_1 = lean_mk_string_unchecked("zeroExtend_congr", 16, 16); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___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_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___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_ReifiedBVExpr_of___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_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; @@ -4769,7 +4545,7 @@ 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 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__2; +x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__2; x_18 = l_Lean_Expr_const___override(x_17, x_2); x_19 = l_Lean_mkApp5(x_18, x_3, x_4, x_5, x_6, x_16); lean_ctor_set(x_14, 0, x_19); @@ -4783,7 +4559,7 @@ x_21 = lean_ctor_get(x_14, 1); lean_inc(x_21); lean_inc(x_20); lean_dec(x_14); -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__2; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__2; x_23 = l_Lean_Expr_const___override(x_22, x_2); x_24 = l_Lean_mkApp5(x_23, x_3, x_4, x_5, x_6, x_20); x_25 = lean_alloc_ctor(0, 2, 0); @@ -4821,7 +4597,7 @@ return x_29; } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__1() { _start: { lean_object* x_1; @@ -4829,7 +4605,7 @@ x_1 = lean_mk_string_unchecked("zeroExtend", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___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; @@ -4837,394 +4613,371 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___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_ReifiedBVExpr_of___lambda__14___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___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_ReifiedBVExpr_of___lambda__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, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__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, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_10; -lean_inc(x_8); +lean_object* x_9; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_10 = l_Lean_Meta_getNatValue_x3f(x_2, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_10) == 0) +lean_inc(x_4); +x_9 = l_Lean_Meta_getNatValue_x3f(x_1, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_9) == 0) { -lean_object* x_11; -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -if (lean_obj_tag(x_11) == 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_object* x_12; lean_object* x_13; +uint8_t x_11; +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_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_4, x_5, x_6, x_7, x_8, x_12); -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_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_dec(x_1); +x_11 = !lean_is_exclusive(x_9); +if (x_11 == 0) { -return x_13; +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_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; -} +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_22; lean_object* x_23; lean_object* x_24; -lean_dec(x_1); -x_22 = lean_ctor_get(x_10, 1); -lean_inc(x_22); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_9, 1); +lean_inc(x_17); +lean_dec(x_9); +x_18 = lean_ctor_get(x_10, 0); +lean_inc(x_18); lean_dec(x_10); -x_23 = lean_ctor_get(x_11, 0); -lean_inc(x_23); -lean_dec(x_11); -lean_inc(x_3); -x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_3, x_4, x_5, x_6, x_7, x_8, x_22); -if (lean_obj_tag(x_24) == 0) +lean_inc(x_2); +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_2, x_3, x_4, x_5, x_6, x_7, x_17); +if (lean_obj_tag(x_19) == 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_20; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +if (lean_obj_tag(x_20) == 0) { -uint8_t x_26; -lean_dec(x_23); -lean_dec(x_3); +uint8_t x_21; +lean_dec(x_18); lean_dec(x_2); -x_26 = !lean_is_exclusive(x_24); -if (x_26 == 0) +lean_dec(x_1); +x_21 = !lean_is_exclusive(x_19); +if (x_21 == 0) { -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_24, 0); -lean_dec(x_27); -x_28 = lean_box(0); -lean_ctor_set(x_24, 0, x_28); -return x_24; +lean_object* x_22; lean_object* x_23; +x_22 = lean_ctor_get(x_19, 0); +lean_dec(x_22); +x_23 = lean_box(0); +lean_ctor_set(x_19, 0, x_23); +return x_19; } 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_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; +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 = 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; } } else { -uint8_t x_32; -x_32 = !lean_is_exclusive(x_25); -if (x_32 == 0) +uint8_t x_27; +x_27 = !lean_is_exclusive(x_20); +if (x_27 == 0) { -uint8_t x_33; -x_33 = !lean_is_exclusive(x_24); -if (x_33 == 0) +uint8_t x_28; +x_28 = !lean_is_exclusive(x_19); +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; 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_34 = lean_ctor_get(x_25, 0); -x_35 = lean_ctor_get(x_24, 0); -lean_dec(x_35); -x_36 = lean_ctor_get(x_34, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_34, 1); -lean_inc(x_37); -x_38 = lean_ctor_get(x_34, 3); -lean_inc(x_38); -lean_inc(x_23); -lean_inc(x_36); -x_39 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_39, 0, x_36); -lean_ctor_set(x_39, 1, x_23); -lean_ctor_set(x_39, 2, x_37); -x_40 = lean_box(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; uint8_t x_41; +x_29 = lean_ctor_get(x_20, 0); +x_30 = lean_ctor_get(x_19, 0); +lean_dec(x_30); +x_31 = lean_ctor_get(x_29, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_29, 1); +lean_inc(x_32); +x_33 = lean_ctor_get(x_29, 3); +lean_inc(x_33); +lean_inc(x_18); +lean_inc(x_31); +x_34 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_34, 0, x_31); +lean_ctor_set(x_34, 1, x_18); +lean_ctor_set(x_34, 2, x_32); +x_35 = lean_box(0); +lean_inc(x_31); +x_36 = l_Lean_mkNatLit(x_31); +x_37 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__3; +lean_inc(x_33); +lean_inc(x_1); lean_inc(x_36); -x_41 = l_Lean_mkNatLit(x_36); -x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__3; -lean_inc(x_38); -lean_inc(x_2); -lean_inc(x_41); -x_43 = l_Lean_mkApp3(x_42, x_41, x_2, x_38); -x_44 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_44, 0, x_36); -lean_closure_set(x_44, 1, x_38); -lean_inc(x_34); -x_45 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13), 12, 5); -lean_closure_set(x_45, 0, x_34); -lean_closure_set(x_45, 1, x_40); -lean_closure_set(x_45, 2, x_2); -lean_closure_set(x_45, 3, x_41); -lean_closure_set(x_45, 4, x_3); -x_46 = !lean_is_exclusive(x_34); -if (x_46 == 0) -{ -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_47 = lean_ctor_get(x_34, 3); -lean_dec(x_47); -x_48 = lean_ctor_get(x_34, 2); -lean_dec(x_48); -x_49 = lean_ctor_get(x_34, 1); -lean_dec(x_49); -x_50 = lean_ctor_get(x_34, 0); -lean_dec(x_50); -x_51 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_51, 0, x_44); -lean_closure_set(x_51, 1, x_45); -lean_ctor_set(x_34, 3, x_43); -lean_ctor_set(x_34, 2, x_51); -lean_ctor_set(x_34, 1, x_39); -lean_ctor_set(x_34, 0, x_23); -return x_24; +x_38 = l_Lean_mkApp3(x_37, x_36, x_1, x_33); +x_39 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_39, 0, x_31); +lean_closure_set(x_39, 1, x_33); +lean_inc(x_29); +x_40 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13), 12, 5); +lean_closure_set(x_40, 0, x_29); +lean_closure_set(x_40, 1, x_35); +lean_closure_set(x_40, 2, x_1); +lean_closure_set(x_40, 3, x_36); +lean_closure_set(x_40, 4, x_2); +x_41 = !lean_is_exclusive(x_29); +if (x_41 == 0) +{ +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_29, 3); +lean_dec(x_42); +x_43 = lean_ctor_get(x_29, 2); +lean_dec(x_43); +x_44 = lean_ctor_get(x_29, 1); +lean_dec(x_44); +x_45 = lean_ctor_get(x_29, 0); +lean_dec(x_45); +x_46 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_46, 0, x_39); +lean_closure_set(x_46, 1, x_40); +lean_ctor_set(x_29, 3, x_38); +lean_ctor_set(x_29, 2, x_46); +lean_ctor_set(x_29, 1, x_34); +lean_ctor_set(x_29, 0, x_18); +return x_19; } else { -lean_object* x_52; lean_object* x_53; -lean_dec(x_34); -x_52 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_52, 0, x_44); -lean_closure_set(x_52, 1, x_45); -x_53 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_53, 0, x_23); -lean_ctor_set(x_53, 1, x_39); -lean_ctor_set(x_53, 2, x_52); -lean_ctor_set(x_53, 3, x_43); -lean_ctor_set(x_25, 0, x_53); -return x_24; +lean_object* x_47; lean_object* x_48; +lean_dec(x_29); +x_47 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_47, 0, x_39); +lean_closure_set(x_47, 1, x_40); +x_48 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_48, 0, x_18); +lean_ctor_set(x_48, 1, x_34); +lean_ctor_set(x_48, 2, x_47); +lean_ctor_set(x_48, 3, x_38); +lean_ctor_set(x_20, 0, x_48); +return x_19; } } 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; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_54 = lean_ctor_get(x_25, 0); -x_55 = lean_ctor_get(x_24, 1); -lean_inc(x_55); -lean_dec(x_24); -x_56 = lean_ctor_get(x_54, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_54, 1); -lean_inc(x_57); -x_58 = lean_ctor_get(x_54, 3); -lean_inc(x_58); -lean_inc(x_23); -lean_inc(x_56); -x_59 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_59, 0, x_56); -lean_ctor_set(x_59, 1, x_23); -lean_ctor_set(x_59, 2, x_57); -x_60 = lean_box(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; 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_49 = lean_ctor_get(x_20, 0); +x_50 = lean_ctor_get(x_19, 1); +lean_inc(x_50); +lean_dec(x_19); +x_51 = lean_ctor_get(x_49, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_49, 1); +lean_inc(x_52); +x_53 = lean_ctor_get(x_49, 3); +lean_inc(x_53); +lean_inc(x_18); +lean_inc(x_51); +x_54 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_54, 0, x_51); +lean_ctor_set(x_54, 1, x_18); +lean_ctor_set(x_54, 2, x_52); +x_55 = lean_box(0); +lean_inc(x_51); +x_56 = l_Lean_mkNatLit(x_51); +x_57 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__3; +lean_inc(x_53); +lean_inc(x_1); lean_inc(x_56); -x_61 = l_Lean_mkNatLit(x_56); -x_62 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__3; -lean_inc(x_58); -lean_inc(x_2); -lean_inc(x_61); -x_63 = l_Lean_mkApp3(x_62, x_61, x_2, x_58); -x_64 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_64, 0, x_56); -lean_closure_set(x_64, 1, x_58); -lean_inc(x_54); -x_65 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13), 12, 5); -lean_closure_set(x_65, 0, x_54); -lean_closure_set(x_65, 1, x_60); -lean_closure_set(x_65, 2, x_2); -lean_closure_set(x_65, 3, x_61); -lean_closure_set(x_65, 4, x_3); -if (lean_is_exclusive(x_54)) { - lean_ctor_release(x_54, 0); - lean_ctor_release(x_54, 1); - lean_ctor_release(x_54, 2); - lean_ctor_release(x_54, 3); - x_66 = x_54; +x_58 = l_Lean_mkApp3(x_57, x_56, x_1, x_53); +x_59 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_59, 0, x_51); +lean_closure_set(x_59, 1, x_53); +lean_inc(x_49); +x_60 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13), 12, 5); +lean_closure_set(x_60, 0, x_49); +lean_closure_set(x_60, 1, x_55); +lean_closure_set(x_60, 2, x_1); +lean_closure_set(x_60, 3, x_56); +lean_closure_set(x_60, 4, x_2); +if (lean_is_exclusive(x_49)) { + lean_ctor_release(x_49, 0); + lean_ctor_release(x_49, 1); + lean_ctor_release(x_49, 2); + lean_ctor_release(x_49, 3); + x_61 = x_49; } else { - lean_dec_ref(x_54); - x_66 = lean_box(0); -} -x_67 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_67, 0, x_64); -lean_closure_set(x_67, 1, x_65); -if (lean_is_scalar(x_66)) { - x_68 = lean_alloc_ctor(0, 4, 0); + lean_dec_ref(x_49); + x_61 = lean_box(0); +} +x_62 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_62, 0, x_59); +lean_closure_set(x_62, 1, x_60); +if (lean_is_scalar(x_61)) { + x_63 = lean_alloc_ctor(0, 4, 0); } else { - x_68 = x_66; + x_63 = x_61; } -lean_ctor_set(x_68, 0, x_23); -lean_ctor_set(x_68, 1, x_59); -lean_ctor_set(x_68, 2, x_67); -lean_ctor_set(x_68, 3, x_63); -lean_ctor_set(x_25, 0, x_68); -x_69 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_69, 0, x_25); -lean_ctor_set(x_69, 1, x_55); -return x_69; +lean_ctor_set(x_63, 0, x_18); +lean_ctor_set(x_63, 1, x_54); +lean_ctor_set(x_63, 2, x_62); +lean_ctor_set(x_63, 3, x_58); +lean_ctor_set(x_20, 0, x_63); +x_64 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_64, 0, x_20); +lean_ctor_set(x_64, 1, x_50); +return x_64; } } 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_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_70 = lean_ctor_get(x_25, 0); -lean_inc(x_70); -lean_dec(x_25); -x_71 = lean_ctor_get(x_24, 1); -lean_inc(x_71); -if (lean_is_exclusive(x_24)) { - lean_ctor_release(x_24, 0); - lean_ctor_release(x_24, 1); - x_72 = x_24; +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; +x_65 = lean_ctor_get(x_20, 0); +lean_inc(x_65); +lean_dec(x_20); +x_66 = lean_ctor_get(x_19, 1); +lean_inc(x_66); +if (lean_is_exclusive(x_19)) { + lean_ctor_release(x_19, 0); + lean_ctor_release(x_19, 1); + x_67 = x_19; } else { - lean_dec_ref(x_24); - x_72 = lean_box(0); + lean_dec_ref(x_19); + x_67 = lean_box(0); } -x_73 = lean_ctor_get(x_70, 0); -lean_inc(x_73); -x_74 = lean_ctor_get(x_70, 1); -lean_inc(x_74); -x_75 = lean_ctor_get(x_70, 3); -lean_inc(x_75); -lean_inc(x_23); -lean_inc(x_73); -x_76 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_76, 0, x_73); -lean_ctor_set(x_76, 1, x_23); -lean_ctor_set(x_76, 2, x_74); -x_77 = lean_box(0); -lean_inc(x_73); -x_78 = l_Lean_mkNatLit(x_73); -x_79 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__3; -lean_inc(x_75); -lean_inc(x_2); -lean_inc(x_78); -x_80 = l_Lean_mkApp3(x_79, x_78, x_2, x_75); -x_81 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_81, 0, x_73); -lean_closure_set(x_81, 1, x_75); +x_68 = lean_ctor_get(x_65, 0); +lean_inc(x_68); +x_69 = lean_ctor_get(x_65, 1); +lean_inc(x_69); +x_70 = lean_ctor_get(x_65, 3); +lean_inc(x_70); +lean_inc(x_18); +lean_inc(x_68); +x_71 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_71, 0, x_68); +lean_ctor_set(x_71, 1, x_18); +lean_ctor_set(x_71, 2, x_69); +x_72 = lean_box(0); +lean_inc(x_68); +x_73 = l_Lean_mkNatLit(x_68); +x_74 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__3; lean_inc(x_70); -x_82 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13), 12, 5); -lean_closure_set(x_82, 0, x_70); -lean_closure_set(x_82, 1, x_77); -lean_closure_set(x_82, 2, x_2); -lean_closure_set(x_82, 3, x_78); -lean_closure_set(x_82, 4, x_3); -if (lean_is_exclusive(x_70)) { - lean_ctor_release(x_70, 0); - lean_ctor_release(x_70, 1); - lean_ctor_release(x_70, 2); - lean_ctor_release(x_70, 3); - x_83 = x_70; +lean_inc(x_1); +lean_inc(x_73); +x_75 = l_Lean_mkApp3(x_74, x_73, x_1, x_70); +x_76 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_76, 0, x_68); +lean_closure_set(x_76, 1, x_70); +lean_inc(x_65); +x_77 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13), 12, 5); +lean_closure_set(x_77, 0, x_65); +lean_closure_set(x_77, 1, x_72); +lean_closure_set(x_77, 2, x_1); +lean_closure_set(x_77, 3, x_73); +lean_closure_set(x_77, 4, x_2); +if (lean_is_exclusive(x_65)) { + lean_ctor_release(x_65, 0); + lean_ctor_release(x_65, 1); + lean_ctor_release(x_65, 2); + lean_ctor_release(x_65, 3); + x_78 = x_65; } else { - lean_dec_ref(x_70); - x_83 = lean_box(0); + lean_dec_ref(x_65); + x_78 = lean_box(0); } -x_84 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_84, 0, x_81); -lean_closure_set(x_84, 1, x_82); -if (lean_is_scalar(x_83)) { - x_85 = lean_alloc_ctor(0, 4, 0); +x_79 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_79, 0, x_76); +lean_closure_set(x_79, 1, x_77); +if (lean_is_scalar(x_78)) { + x_80 = lean_alloc_ctor(0, 4, 0); } else { - x_85 = x_83; -} -lean_ctor_set(x_85, 0, x_23); -lean_ctor_set(x_85, 1, x_76); -lean_ctor_set(x_85, 2, x_84); -lean_ctor_set(x_85, 3, x_80); -x_86 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_86, 0, x_85); -if (lean_is_scalar(x_72)) { - x_87 = lean_alloc_ctor(0, 2, 0); + x_80 = x_78; +} +lean_ctor_set(x_80, 0, x_18); +lean_ctor_set(x_80, 1, x_71); +lean_ctor_set(x_80, 2, x_79); +lean_ctor_set(x_80, 3, x_75); +x_81 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_81, 0, x_80); +if (lean_is_scalar(x_67)) { + x_82 = lean_alloc_ctor(0, 2, 0); } else { - x_87 = x_72; + x_82 = x_67; } -lean_ctor_set(x_87, 0, x_86); -lean_ctor_set(x_87, 1, x_71); -return x_87; +lean_ctor_set(x_82, 0, x_81); +lean_ctor_set(x_82, 1, x_66); +return x_82; } } } else { -uint8_t x_88; -lean_dec(x_23); -lean_dec(x_3); +uint8_t x_83; +lean_dec(x_18); lean_dec(x_2); -x_88 = !lean_is_exclusive(x_24); -if (x_88 == 0) +lean_dec(x_1); +x_83 = !lean_is_exclusive(x_19); +if (x_83 == 0) { -return x_24; +return x_19; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_89 = lean_ctor_get(x_24, 0); -x_90 = lean_ctor_get(x_24, 1); -lean_inc(x_90); -lean_inc(x_89); -lean_dec(x_24); -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_84; lean_object* x_85; lean_object* x_86; +x_84 = lean_ctor_get(x_19, 0); +x_85 = lean_ctor_get(x_19, 1); +lean_inc(x_85); +lean_inc(x_84); +lean_dec(x_19); +x_86 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_86, 0, x_84); +lean_ctor_set(x_86, 1, x_85); +return x_86; } } } } else { -uint8_t x_92; -lean_dec(x_8); +uint8_t x_87; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -5232,28 +4985,28 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_92 = !lean_is_exclusive(x_10); -if (x_92 == 0) +x_87 = !lean_is_exclusive(x_9); +if (x_87 == 0) { -return x_10; +return x_9; } else { -lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_93 = lean_ctor_get(x_10, 0); -x_94 = lean_ctor_get(x_10, 1); -lean_inc(x_94); -lean_inc(x_93); -lean_dec(x_10); -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_88; lean_object* x_89; lean_object* x_90; +x_88 = lean_ctor_get(x_9, 0); +x_89 = lean_ctor_get(x_9, 1); +lean_inc(x_89); +lean_inc(x_88); +lean_dec(x_9); +x_90 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_90, 0, x_88); +lean_ctor_set(x_90, 1, x_89); +return x_90; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__15(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__15(lean_object* x_1) { _start: { lean_object* x_2; @@ -5262,7 +5015,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__1() { _start: { lean_object* x_1; @@ -5270,20 +5023,20 @@ x_1 = lean_mk_string_unchecked("arithShiftRightConst", 20, 20); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__1; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__3() { _start: { lean_object* x_1; @@ -5291,144 +5044,121 @@ x_1 = lean_mk_string_unchecked("arithShiftRight_congr", 21, 21); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__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; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__3; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___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_ReifiedBVExpr_of___lambda__16___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__15), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__15), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___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, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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_10; -lean_inc(x_8); +lean_object* x_9; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_10 = l_Lean_Meta_getNatValue_x3f(x_3, x_5, x_6, x_7, x_8, x_9); +lean_inc(x_4); +x_9 = l_Lean_Meta_getNatValue_x3f(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) { -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_11; +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_11 = !lean_is_exclusive(x_9); +if (x_11 == 0) { lean_object* x_12; lean_object* x_13; -lean_dec(x_2); -x_12 = lean_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_4, x_5, x_6, x_7, x_8, x_12); -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_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) -{ -return 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_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; -} +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_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -lean_dec(x_1); -x_22 = lean_ctor_get(x_10, 1); -lean_inc(x_22); +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_9, 1); +lean_inc(x_17); +lean_dec(x_9); +x_18 = lean_ctor_get(x_10, 0); +lean_inc(x_18); lean_dec(x_10); -x_23 = lean_ctor_get(x_11, 0); -lean_inc(x_23); -lean_dec(x_11); -x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__5; -x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__2; -x_26 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__4; -x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstLikeReflection(x_23, x_2, x_24, x_25, x_26, x_4, x_5, x_6, x_7, x_8, x_22); -return x_27; +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__5; +x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__2; +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__4; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstLikeReflection(x_18, x_1, x_19, x_20, x_21, x_3, x_4, x_5, x_6, x_7, x_17); +return x_22; } } else { -uint8_t x_28; -lean_dec(x_8); +uint8_t x_23; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_2); +lean_dec(x_3); lean_dec(x_1); -x_28 = !lean_is_exclusive(x_10); -if (x_28 == 0) +x_23 = !lean_is_exclusive(x_9); +if (x_23 == 0) { -return x_10; +return x_9; } 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; +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; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__17(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_ReifiedBVExpr_of_go___lambda__17(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; @@ -5440,7 +5170,7 @@ lean_ctor_set(x_5, 3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__18(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__18(lean_object* x_1) { _start: { lean_object* x_2; @@ -5449,7 +5179,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__1() { _start: { lean_object* x_1; @@ -5457,7 +5187,7 @@ x_1 = lean_mk_string_unchecked("shiftRight", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___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; @@ -5465,12 +5195,12 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__3() { _start: { lean_object* x_1; @@ -5478,29 +5208,29 @@ x_1 = lean_mk_string_unchecked("shiftRight_congr", 16, 16); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___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_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__3; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___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_ReifiedBVExpr_of___lambda__19___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__17), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__17), 4, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__6() { _start: { lean_object* x_1; @@ -5508,20 +5238,20 @@ x_1 = lean_mk_string_unchecked("shiftRightConst", 15, 15); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__6; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__6; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__8() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__8() { _start: { lean_object* x_1; @@ -5529,75 +5259,74 @@ x_1 = lean_mk_string_unchecked("shiftRightNat_congr", 19, 19); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__9() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___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; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__8; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__8; 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_ReifiedBVExpr_of___lambda__19___closed__10() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__10() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__18), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__18), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___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_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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_object* x_9) { _start: { -lean_object* x_11; -lean_inc(x_9); +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_2); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_inc(x_3); +lean_inc(x_1); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f(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; +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); if (lean_obj_tag(x_11) == 0) { -lean_object* x_12; -x_12 = lean_ctor_get(x_11, 0); +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_12 = lean_ctor_get(x_10, 1); lean_inc(x_12); -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; -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__5; -x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__2; -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__4; -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection(x_1, x_2, x_4, x_3, x_14, x_15, x_16, x_5, x_6, x_7, x_8, x_9, x_13); -return x_17; +lean_dec(x_10); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__5; +x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__2; +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__4; +x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection(x_1, x_3, x_2, x_13, x_14, x_15, x_4, x_5, x_6, x_7, x_8, x_12); +return x_16; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -lean_dec(x_12); -x_18 = lean_ctor_get(x_11, 1); -lean_inc(x_18); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_dec(x_11); -x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__10; -x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__7; -x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__9; -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstReflection(x_1, x_2, x_4, x_3, x_19, x_20, x_21, x_5, x_6, x_7, x_8, x_9, x_18); -return x_22; +x_17 = lean_ctor_get(x_10, 1); +lean_inc(x_17); +lean_dec(x_10); +x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__10; +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__7; +x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__9; +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstReflection(x_1, x_3, x_2, x_18, x_19, x_20, x_4, x_5, x_6, x_7, x_8, x_17); +return x_21; } } else { -uint8_t x_23; -lean_dec(x_9); +uint8_t x_22; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -5606,28 +5335,28 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_23 = !lean_is_exclusive(x_11); -if (x_23 == 0) +x_22 = !lean_is_exclusive(x_10); +if (x_22 == 0) { -return x_11; +return x_10; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_11, 0); -x_25 = lean_ctor_get(x_11, 1); -lean_inc(x_25); +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_10, 0); +x_24 = lean_ctor_get(x_10, 1); lean_inc(x_24); -lean_dec(x_11); -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_inc(x_23); +lean_dec(x_10); +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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__20(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_ReifiedBVExpr_of_go___lambda__20(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; @@ -5639,7 +5368,7 @@ lean_ctor_set(x_5, 3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__21(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__21(lean_object* x_1) { _start: { lean_object* x_2; @@ -5648,7 +5377,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__1() { _start: { lean_object* x_1; @@ -5656,7 +5385,7 @@ x_1 = lean_mk_string_unchecked("shiftLeft", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___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; @@ -5664,12 +5393,12 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__3() { _start: { lean_object* x_1; @@ -5677,29 +5406,29 @@ x_1 = lean_mk_string_unchecked("shiftLeft_congr", 15, 15); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___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_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__3; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___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_ReifiedBVExpr_of___lambda__22___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__20), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__20), 4, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__6() { _start: { lean_object* x_1; @@ -5707,20 +5436,20 @@ x_1 = lean_mk_string_unchecked("shiftLeftConst", 14, 14); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__6; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__6; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__8() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__8() { _start: { lean_object* x_1; @@ -5728,75 +5457,74 @@ x_1 = lean_mk_string_unchecked("shiftLeftNat_congr", 18, 18); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__9() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___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; lean_object* x_7; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__8; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__8; 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_ReifiedBVExpr_of___lambda__22___closed__10() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__10() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__21), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__21), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___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, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_11; -lean_inc(x_9); +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_2); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_inc(x_3); +lean_inc(x_1); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f(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; +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); if (lean_obj_tag(x_11) == 0) { -lean_object* x_12; -x_12 = lean_ctor_get(x_11, 0); +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_12 = lean_ctor_get(x_10, 1); lean_inc(x_12); -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; -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__5; -x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__2; -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__4; -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection(x_1, x_2, x_4, x_3, x_14, x_15, x_16, x_5, x_6, x_7, x_8, x_9, x_13); -return x_17; +lean_dec(x_10); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__5; +x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__2; +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__4; +x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection(x_1, x_3, x_2, x_13, x_14, x_15, x_4, x_5, x_6, x_7, x_8, x_12); +return x_16; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -lean_dec(x_12); -x_18 = lean_ctor_get(x_11, 1); -lean_inc(x_18); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_dec(x_11); -x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__10; -x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__7; -x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__9; -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstReflection(x_1, x_2, x_4, x_3, x_19, x_20, x_21, x_5, x_6, x_7, x_8, x_9, x_18); -return x_22; +x_17 = lean_ctor_get(x_10, 1); +lean_inc(x_17); +lean_dec(x_10); +x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__10; +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__7; +x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__9; +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstReflection(x_1, x_3, x_2, x_18, x_19, x_20, x_4, x_5, x_6, x_7, x_8, x_17); +return x_21; } } else { -uint8_t x_23; -lean_dec(x_9); +uint8_t x_22; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -5805,28 +5533,28 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_23 = !lean_is_exclusive(x_11); -if (x_23 == 0) +x_22 = !lean_is_exclusive(x_10); +if (x_22 == 0) { -return x_11; +return x_10; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_11, 0); -x_25 = lean_ctor_get(x_11, 1); -lean_inc(x_25); +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_10, 0); +x_24 = lean_ctor_get(x_10, 1); lean_inc(x_24); -lean_dec(x_11); -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_inc(x_23); +lean_dec(x_10); +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; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__1() { _start: { lean_object* x_1; @@ -5834,31 +5562,31 @@ x_1 = lean_mk_string_unchecked("not_congr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___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_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___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_ReifiedBVExpr_of___lambda__23(lean_object* x_1, lean_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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23(lean_object* x_1, 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; x_8 = lean_box(0); -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__2; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__2; x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection(x_1, x_8, x_9, x_2, x_3, x_4, x_5, x_6, x_7); return x_10; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__1() { _start: { lean_object* x_1; @@ -5866,31 +5594,31 @@ x_1 = lean_mk_string_unchecked("umod_congr", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___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_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___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_ReifiedBVExpr_of___lambda__24(lean_object* x_1, lean_object* x_2, lean_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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24(lean_object* x_1, lean_object* x_2, 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; lean_object* x_11; x_9 = 6; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__2; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__2; x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); return x_11; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__1() { _start: { lean_object* x_1; @@ -5898,31 +5626,31 @@ x_1 = lean_mk_string_unchecked("udiv_congr", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___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_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___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_ReifiedBVExpr_of___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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) { _start: { uint8_t x_9; lean_object* x_10; lean_object* x_11; x_9 = 5; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__2; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__2; x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); return x_11; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__1() { _start: { lean_object* x_1; @@ -5930,31 +5658,31 @@ x_1 = lean_mk_string_unchecked("mul_congr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___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_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___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_ReifiedBVExpr_of___lambda__26(lean_object* x_1, lean_object* x_2, lean_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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26(lean_object* x_1, lean_object* x_2, 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; lean_object* x_11; x_9 = 4; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__2; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__2; x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); return x_11; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__1() { _start: { lean_object* x_1; @@ -5962,31 +5690,31 @@ x_1 = lean_mk_string_unchecked("add_congr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___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_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___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_ReifiedBVExpr_of___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) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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: { uint8_t x_9; lean_object* x_10; lean_object* x_11; x_9 = 3; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__2; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__2; x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); return x_11; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__1() { _start: { lean_object* x_1; @@ -5994,31 +5722,31 @@ x_1 = lean_mk_string_unchecked("xor_congr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___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_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___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_ReifiedBVExpr_of___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, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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, lean_object* x_7, lean_object* x_8) { _start: { uint8_t x_9; lean_object* x_10; lean_object* x_11; x_9 = 2; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__2; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__2; x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); return x_11; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__1() { _start: { lean_object* x_1; @@ -6026,31 +5754,31 @@ x_1 = lean_mk_string_unchecked("or_congr", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___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_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___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_ReifiedBVExpr_of___lambda__29(lean_object* x_1, lean_object* x_2, lean_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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29(lean_object* x_1, lean_object* x_2, 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; lean_object* x_11; x_9 = 1; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__2; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__2; x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); return x_11; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__1() { _start: { lean_object* x_1; @@ -6058,31 +5786,31 @@ x_1 = lean_mk_string_unchecked("and_congr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___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_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___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_ReifiedBVExpr_of___lambda__30(lean_object* x_1, lean_object* x_2, lean_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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30(lean_object* x_1, lean_object* x_2, 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; lean_object* x_11; x_9 = 0; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__2; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__2; x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__31(lean_object* x_1, lean_object* x_2, lean_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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31(lean_object* x_1, lean_object* x_2, 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; @@ -6090,137 +5818,201 @@ x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit(x_1, x_3, x_ return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___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) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__1() { _start: { -lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_3, x_4, x_5, x_6, x_7, x_8); -return x_9; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___boxed), 8, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___boxed), 8, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6), 9, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___boxed), 8, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10), 8, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12), 8, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14), 8, 0); +return x_1; +} } +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___boxed), 8, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19), 9, 0); +return x_1; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__1() { +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__10() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22), 9, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__11() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23), 7, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23), 7, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__12() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__13() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__14() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__15() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__16() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__8() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__17() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__9() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__18() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__10() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___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_ReifiedBVExpr_of___closed__11() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__20() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___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_ReifiedBVExpr_of___closed__12() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__21() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___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_ReifiedBVExpr_of___closed__13() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__22() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___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_ReifiedBVExpr_of___closed__14() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__23() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___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_ReifiedBVExpr_of___closed__15() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__24() { _start: { lean_object* x_1; @@ -6228,17 +6020,17 @@ x_1 = lean_mk_string_unchecked("sshiftRight", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__16() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__25() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__15; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__24; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__17() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__26() { _start: { lean_object* x_1; @@ -6246,7 +6038,7 @@ x_1 = lean_mk_string_unchecked("Complement", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__18() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__27() { _start: { lean_object* x_1; @@ -6254,17 +6046,17 @@ x_1 = lean_mk_string_unchecked("complement", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__19() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__28() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__17; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__18; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__26; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__27; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__20() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__29() { _start: { lean_object* x_1; @@ -6272,17 +6064,17 @@ x_1 = lean_mk_string_unchecked("extractLsb'", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__21() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__30() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkBVRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__20; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__29; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__22() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__31() { _start: { lean_object* x_1; @@ -6290,7 +6082,7 @@ x_1 = lean_mk_string_unchecked("HAppend", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__23() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__32() { _start: { lean_object* x_1; @@ -6298,17 +6090,17 @@ x_1 = lean_mk_string_unchecked("hAppend", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__24() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__33() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__22; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__23; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__31; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__32; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__25() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__34() { _start: { lean_object* x_1; @@ -6316,7 +6108,7 @@ x_1 = lean_mk_string_unchecked("HShiftRight", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__26() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__35() { _start: { lean_object* x_1; @@ -6324,17 +6116,17 @@ x_1 = lean_mk_string_unchecked("hShiftRight", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__27() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__36() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__25; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__26; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__34; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__35; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__28() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__37() { _start: { lean_object* x_1; @@ -6342,7 +6134,7 @@ x_1 = lean_mk_string_unchecked("HShiftLeft", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__29() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__38() { _start: { lean_object* x_1; @@ -6350,17 +6142,17 @@ x_1 = lean_mk_string_unchecked("hShiftLeft", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__30() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__39() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__28; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__29; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__37; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__38; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__31() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__40() { _start: { lean_object* x_1; @@ -6368,7 +6160,7 @@ x_1 = lean_mk_string_unchecked("HMod", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__32() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__41() { _start: { lean_object* x_1; @@ -6376,17 +6168,17 @@ x_1 = lean_mk_string_unchecked("hMod", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__33() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__42() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__31; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__32; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__40; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__41; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__34() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__43() { _start: { lean_object* x_1; @@ -6394,7 +6186,7 @@ x_1 = lean_mk_string_unchecked("HDiv", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__35() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__44() { _start: { lean_object* x_1; @@ -6402,17 +6194,17 @@ x_1 = lean_mk_string_unchecked("hDiv", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__36() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__45() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__34; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__35; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__43; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__44; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__37() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__46() { _start: { lean_object* x_1; @@ -6420,7 +6212,7 @@ x_1 = lean_mk_string_unchecked("HMul", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__38() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__47() { _start: { lean_object* x_1; @@ -6428,17 +6220,17 @@ x_1 = lean_mk_string_unchecked("hMul", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__39() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__48() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__37; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__38; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__46; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__47; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__40() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__49() { _start: { lean_object* x_1; @@ -6446,7 +6238,7 @@ x_1 = lean_mk_string_unchecked("HAdd", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__41() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__50() { _start: { lean_object* x_1; @@ -6454,17 +6246,17 @@ x_1 = lean_mk_string_unchecked("hAdd", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__42() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__51() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__40; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__41; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__49; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__50; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__43() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__52() { _start: { lean_object* x_1; @@ -6472,7 +6264,7 @@ x_1 = lean_mk_string_unchecked("HXor", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__44() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__53() { _start: { lean_object* x_1; @@ -6480,17 +6272,17 @@ x_1 = lean_mk_string_unchecked("hXor", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__45() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__54() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__43; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__44; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__52; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__53; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__46() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__55() { _start: { lean_object* x_1; @@ -6498,7 +6290,7 @@ x_1 = lean_mk_string_unchecked("HOr", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__47() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__56() { _start: { lean_object* x_1; @@ -6506,17 +6298,17 @@ x_1 = lean_mk_string_unchecked("hOr", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__48() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__57() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__46; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__47; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__55; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__56; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__49() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__58() { _start: { lean_object* x_1; @@ -6524,7 +6316,7 @@ x_1 = lean_mk_string_unchecked("HAnd", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__50() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__59() { _start: { lean_object* x_1; @@ -6532,20 +6324,20 @@ x_1 = lean_mk_string_unchecked("hAnd", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__51() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__60() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__49; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__50; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__58; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__59; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(lean_object* x_1, lean_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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_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) { _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; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +lean_object* x_8; lean_object* x_9; 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; uint8_t x_31; lean_inc(x_1); x_8 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_1, x_3, x_4, x_5, x_6, x_7); x_9 = lean_ctor_get(x_8, 0); @@ -6553,383 +6345,390 @@ lean_inc(x_9); x_10 = lean_ctor_get(x_8, 1); lean_inc(x_10); lean_dec(x_8); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__1; -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__2; -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__3; -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__4; -x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__5; -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__6; -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__7; -x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__8; -x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__9; -x_20 = l_Lean_Expr_cleanupAnnotations(x_9); -x_21 = l_Lean_Expr_isApp(x_20); -if (x_21 == 0) +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__1; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__2; +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__3; +x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__4; +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__5; +x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__6; +x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__7; +x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__8; +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__9; +x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__10; +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__11; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__12; +x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__13; +x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__14; +x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__15; +x_26 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__16; +x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__17; +x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__18; +x_29 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___closed__1; +x_30 = l_Lean_Expr_cleanupAnnotations(x_9); +x_31 = l_Lean_Expr_isApp(x_30); +if (x_31 == 0) { -lean_object* x_22; -lean_dec(x_20); -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_22; +lean_object* x_32; lean_object* x_33; +lean_dec(x_30); +lean_dec(x_1); +x_32 = lean_box(0); +x_33 = lean_apply_7(x_29, x_32, x_2, x_3, x_4, x_5, x_6, x_10); +return x_33; } else { -lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_23 = l_Lean_Expr_appArg(x_20, lean_box(0)); -x_24 = l_Lean_Expr_appFnCleanup(x_20, lean_box(0)); -x_25 = l_Lean_Expr_isApp(x_24); -if (x_25 == 0) +lean_object* x_34; lean_object* x_35; uint8_t x_36; +x_34 = l_Lean_Expr_appArg(x_30, lean_box(0)); +x_35 = l_Lean_Expr_appFnCleanup(x_30, lean_box(0)); +x_36 = l_Lean_Expr_isApp(x_35); +if (x_36 == 0) { -lean_object* x_26; -lean_dec(x_24); -lean_dec(x_23); -x_26 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_26; +lean_object* x_37; lean_object* x_38; +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_1); +x_37 = lean_box(0); +x_38 = lean_apply_7(x_29, x_37, x_2, x_3, x_4, x_5, x_6, x_10); +return x_38; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; -x_27 = l_Lean_Expr_appArg(x_24, lean_box(0)); -x_28 = l_Lean_Expr_appFnCleanup(x_24, lean_box(0)); -x_29 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__5; -x_30 = l_Lean_Expr_isConstOf(x_28, x_29); -if (x_30 == 0) +lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; +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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__5; +x_42 = l_Lean_Expr_isConstOf(x_40, x_41); +if (x_42 == 0) { -uint8_t x_31; -x_31 = l_Lean_Expr_isApp(x_28); -if (x_31 == 0) +uint8_t x_43; +lean_dec(x_1); +x_43 = l_Lean_Expr_isApp(x_40); +if (x_43 == 0) { -lean_object* x_32; -lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_23); -x_32 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_32; +lean_object* x_44; lean_object* x_45; +lean_dec(x_40); +lean_dec(x_39); +lean_dec(x_34); +x_44 = lean_box(0); +x_45 = lean_apply_7(x_29, x_44, x_2, x_3, x_4, x_5, x_6, x_10); +return x_45; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; -x_33 = l_Lean_Expr_appArg(x_28, lean_box(0)); -x_34 = l_Lean_Expr_appFnCleanup(x_28, lean_box(0)); -x_35 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__10; -x_36 = l_Lean_Expr_isConstOf(x_34, x_35); -if (x_36 == 0) +lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; +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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__19; +x_49 = l_Lean_Expr_isConstOf(x_47, x_48); +if (x_49 == 0) { -lean_object* x_37; uint8_t x_38; -x_37 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__11; -x_38 = l_Lean_Expr_isConstOf(x_34, x_37); -if (x_38 == 0) +lean_object* x_50; uint8_t x_51; +x_50 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__20; +x_51 = l_Lean_Expr_isConstOf(x_47, x_50); +if (x_51 == 0) { -lean_object* x_39; uint8_t x_40; -x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__12; -x_40 = l_Lean_Expr_isConstOf(x_34, x_39); -if (x_40 == 0) +lean_object* x_52; uint8_t x_53; +x_52 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__21; +x_53 = l_Lean_Expr_isConstOf(x_47, x_52); +if (x_53 == 0) { -lean_object* x_41; uint8_t x_42; -x_41 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__13; -x_42 = l_Lean_Expr_isConstOf(x_34, x_41); -if (x_42 == 0) +lean_object* x_54; uint8_t x_55; +x_54 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__22; +x_55 = l_Lean_Expr_isConstOf(x_47, x_54); +if (x_55 == 0) { -lean_object* x_43; uint8_t x_44; -x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__14; -x_44 = l_Lean_Expr_isConstOf(x_34, x_43); -if (x_44 == 0) +lean_object* x_56; uint8_t x_57; +x_56 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__23; +x_57 = l_Lean_Expr_isConstOf(x_47, x_56); +if (x_57 == 0) { -lean_object* x_45; uint8_t x_46; -x_45 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__16; -x_46 = l_Lean_Expr_isConstOf(x_34, x_45); -if (x_46 == 0) +lean_object* x_58; uint8_t x_59; +x_58 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__25; +x_59 = l_Lean_Expr_isConstOf(x_47, x_58); +if (x_59 == 0) { -lean_object* x_47; uint8_t x_48; -x_47 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__19; -x_48 = l_Lean_Expr_isConstOf(x_34, x_47); -if (x_48 == 0) +lean_object* x_60; uint8_t x_61; +x_60 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__28; +x_61 = l_Lean_Expr_isConstOf(x_47, x_60); +if (x_61 == 0) { -uint8_t x_49; -x_49 = l_Lean_Expr_isApp(x_34); -if (x_49 == 0) +uint8_t x_62; +x_62 = l_Lean_Expr_isApp(x_47); +if (x_62 == 0) { -lean_object* x_50; +lean_object* x_63; lean_object* x_64; +lean_dec(x_47); +lean_dec(x_46); +lean_dec(x_39); lean_dec(x_34); -lean_dec(x_33); -lean_dec(x_27); -lean_dec(x_23); -x_50 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_50; +x_63 = lean_box(0); +x_64 = lean_apply_7(x_29, x_63, x_2, x_3, x_4, x_5, x_6, x_10); +return x_64; } else { -lean_object* x_51; lean_object* x_52; uint8_t x_53; -x_51 = l_Lean_Expr_appFnCleanup(x_34, lean_box(0)); -x_52 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__21; -x_53 = l_Lean_Expr_isConstOf(x_51, x_52); -if (x_53 == 0) +lean_object* x_65; lean_object* x_66; uint8_t x_67; +x_65 = l_Lean_Expr_appFnCleanup(x_47, lean_box(0)); +x_66 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__30; +x_67 = l_Lean_Expr_isConstOf(x_65, x_66); +if (x_67 == 0) { -uint8_t x_54; -lean_dec(x_33); -x_54 = l_Lean_Expr_isApp(x_51); -if (x_54 == 0) +uint8_t x_68; +lean_dec(x_46); +x_68 = l_Lean_Expr_isApp(x_65); +if (x_68 == 0) { -lean_object* x_55; -lean_dec(x_51); -lean_dec(x_27); -lean_dec(x_23); -x_55 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_55; +lean_object* x_69; lean_object* x_70; +lean_dec(x_65); +lean_dec(x_39); +lean_dec(x_34); +x_69 = lean_box(0); +x_70 = lean_apply_7(x_29, x_69, x_2, x_3, x_4, x_5, x_6, x_10); +return x_70; } else { -lean_object* x_56; lean_object* x_57; uint8_t x_58; -x_56 = l_Lean_Expr_appArg(x_51, lean_box(0)); -x_57 = l_Lean_Expr_appFnCleanup(x_51, lean_box(0)); -x_58 = l_Lean_Expr_isApp(x_57); -if (x_58 == 0) +lean_object* x_71; lean_object* x_72; uint8_t x_73; +x_71 = l_Lean_Expr_appArg(x_65, lean_box(0)); +x_72 = l_Lean_Expr_appFnCleanup(x_65, lean_box(0)); +x_73 = l_Lean_Expr_isApp(x_72); +if (x_73 == 0) { -lean_object* x_59; -lean_dec(x_57); -lean_dec(x_56); -lean_dec(x_27); -lean_dec(x_23); -x_59 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_59; +lean_object* x_74; lean_object* x_75; +lean_dec(x_72); +lean_dec(x_71); +lean_dec(x_39); +lean_dec(x_34); +x_74 = lean_box(0); +x_75 = lean_apply_7(x_29, x_74, x_2, x_3, x_4, x_5, x_6, x_10); +return x_75; } else { -lean_object* x_60; lean_object* x_61; uint8_t x_62; -x_60 = l_Lean_Expr_appFnCleanup(x_57, lean_box(0)); -x_61 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__24; -x_62 = l_Lean_Expr_isConstOf(x_60, x_61); -if (x_62 == 0) +lean_object* x_76; lean_object* x_77; uint8_t x_78; +x_76 = l_Lean_Expr_appFnCleanup(x_72, lean_box(0)); +x_77 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__33; +x_78 = l_Lean_Expr_isConstOf(x_76, x_77); +if (x_78 == 0) +{ +lean_object* x_79; uint8_t x_80; +x_79 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__36; +x_80 = l_Lean_Expr_isConstOf(x_76, x_79); +if (x_80 == 0) +{ +lean_object* x_81; uint8_t x_82; +x_81 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__39; +x_82 = l_Lean_Expr_isConstOf(x_76, x_81); +if (x_82 == 0) { -lean_object* x_63; uint8_t x_64; -x_63 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__27; -x_64 = l_Lean_Expr_isConstOf(x_60, x_63); -if (x_64 == 0) +lean_object* x_83; uint8_t x_84; +lean_dec(x_71); +x_83 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__42; +x_84 = l_Lean_Expr_isConstOf(x_76, x_83); +if (x_84 == 0) { -lean_object* x_65; uint8_t x_66; -x_65 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__30; -x_66 = l_Lean_Expr_isConstOf(x_60, x_65); -if (x_66 == 0) +lean_object* x_85; uint8_t x_86; +x_85 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__45; +x_86 = l_Lean_Expr_isConstOf(x_76, x_85); +if (x_86 == 0) { -lean_object* x_67; uint8_t x_68; -lean_dec(x_56); -x_67 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__33; -x_68 = l_Lean_Expr_isConstOf(x_60, x_67); -if (x_68 == 0) +lean_object* x_87; uint8_t x_88; +x_87 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__48; +x_88 = l_Lean_Expr_isConstOf(x_76, x_87); +if (x_88 == 0) { -lean_object* x_69; uint8_t x_70; -x_69 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__36; -x_70 = l_Lean_Expr_isConstOf(x_60, x_69); -if (x_70 == 0) -{ -lean_object* x_71; uint8_t x_72; -x_71 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__39; -x_72 = l_Lean_Expr_isConstOf(x_60, x_71); -if (x_72 == 0) -{ -lean_object* x_73; uint8_t x_74; -x_73 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__42; -x_74 = l_Lean_Expr_isConstOf(x_60, x_73); -if (x_74 == 0) -{ -lean_object* x_75; uint8_t x_76; -x_75 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__45; -x_76 = l_Lean_Expr_isConstOf(x_60, x_75); -if (x_76 == 0) -{ -lean_object* x_77; uint8_t x_78; -x_77 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__48; -x_78 = l_Lean_Expr_isConstOf(x_60, x_77); -if (x_78 == 0) +lean_object* x_89; uint8_t x_90; +x_89 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__51; +x_90 = l_Lean_Expr_isConstOf(x_76, x_89); +if (x_90 == 0) { -lean_object* x_79; uint8_t x_80; -x_79 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__51; -x_80 = l_Lean_Expr_isConstOf(x_60, x_79); -lean_dec(x_60); -if (x_80 == 0) +lean_object* x_91; uint8_t x_92; +x_91 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__54; +x_92 = l_Lean_Expr_isConstOf(x_76, x_91); +if (x_92 == 0) { -lean_object* x_81; -lean_dec(x_27); -lean_dec(x_23); -x_81 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_81; +lean_object* x_93; uint8_t x_94; +x_93 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__57; +x_94 = l_Lean_Expr_isConstOf(x_76, x_93); +if (x_94 == 0) +{ +lean_object* x_95; uint8_t x_96; +x_95 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__60; +x_96 = l_Lean_Expr_isConstOf(x_76, x_95); +lean_dec(x_76); +if (x_96 == 0) +{ +lean_object* x_97; lean_object* x_98; +lean_dec(x_39); +lean_dec(x_34); +x_97 = lean_box(0); +x_98 = lean_apply_7(x_29, x_97, x_2, x_3, x_4, x_5, x_6, x_10); +return x_98; } else { -lean_object* x_82; -lean_dec(x_1); -x_82 = lean_apply_8(x_19, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_82; +lean_object* x_99; +x_99 = lean_apply_8(x_28, x_39, x_34, x_2, x_3, x_4, x_5, x_6, x_10); +return x_99; } } else { -lean_object* x_83; -lean_dec(x_60); -lean_dec(x_1); -x_83 = lean_apply_8(x_18, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_83; +lean_object* x_100; +lean_dec(x_76); +x_100 = lean_apply_8(x_27, x_39, x_34, x_2, x_3, x_4, x_5, x_6, x_10); +return x_100; } } else { -lean_object* x_84; -lean_dec(x_60); -lean_dec(x_1); -x_84 = lean_apply_8(x_17, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_84; +lean_object* x_101; +lean_dec(x_76); +x_101 = lean_apply_8(x_26, x_39, x_34, x_2, x_3, x_4, x_5, x_6, x_10); +return x_101; } } else { -lean_object* x_85; -lean_dec(x_60); -lean_dec(x_1); -x_85 = lean_apply_8(x_16, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_85; +lean_object* x_102; +lean_dec(x_76); +x_102 = lean_apply_8(x_25, x_39, x_34, x_2, x_3, x_4, x_5, x_6, x_10); +return x_102; } } else { -lean_object* x_86; -lean_dec(x_60); -lean_dec(x_1); -x_86 = lean_apply_8(x_15, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_86; +lean_object* x_103; +lean_dec(x_76); +x_103 = lean_apply_8(x_24, x_39, x_34, x_2, x_3, x_4, x_5, x_6, x_10); +return x_103; } } else { -lean_object* x_87; -lean_dec(x_60); -lean_dec(x_1); -x_87 = lean_apply_8(x_14, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_87; +lean_object* x_104; +lean_dec(x_76); +x_104 = lean_apply_8(x_23, x_39, x_34, x_2, x_3, x_4, x_5, x_6, x_10); +return x_104; } } else { -lean_object* x_88; -lean_dec(x_60); -lean_dec(x_1); -x_88 = lean_apply_8(x_13, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_88; +lean_object* x_105; +lean_dec(x_76); +x_105 = lean_apply_8(x_22, x_39, x_34, x_2, x_3, x_4, x_5, x_6, x_10); +return x_105; } } else { -lean_object* x_89; -lean_dec(x_60); -x_89 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22(x_1, x_56, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_89; +lean_object* x_106; +lean_dec(x_76); +x_106 = lean_apply_9(x_20, x_71, x_39, x_34, x_2, x_3, x_4, x_5, x_6, x_10); +return x_106; } } else { -lean_object* x_90; -lean_dec(x_60); -x_90 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19(x_1, x_56, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_90; +lean_object* x_107; +lean_dec(x_76); +x_107 = lean_apply_9(x_19, x_71, x_39, x_34, x_2, x_3, x_4, x_5, x_6, x_10); +return x_107; } } else { -lean_object* x_91; -lean_dec(x_60); -lean_dec(x_56); -lean_dec(x_1); -x_91 = lean_apply_8(x_11, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_91; +lean_object* x_108; +lean_dec(x_76); +lean_dec(x_71); +x_108 = lean_apply_8(x_15, x_39, x_34, x_2, x_3, x_4, x_5, x_6, x_10); +return x_108; } } } } else { -lean_object* x_92; -lean_dec(x_51); -x_92 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6(x_1, x_33, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_92; +lean_object* x_109; +lean_dec(x_65); +x_109 = lean_apply_9(x_13, x_46, x_39, x_34, x_2, x_3, x_4, x_5, x_6, x_10); +return x_109; } } } else { -lean_object* x_93; -lean_dec(x_34); -lean_dec(x_33); -lean_dec(x_27); -lean_dec(x_1); -x_93 = lean_apply_7(x_12, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_93; +lean_object* x_110; +lean_dec(x_47); +lean_dec(x_46); +lean_dec(x_39); +x_110 = lean_apply_7(x_21, x_34, x_2, x_3, x_4, x_5, x_6, x_10); +return x_110; } } else { -lean_object* x_94; -lean_dec(x_34); -lean_dec(x_33); -x_94 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16(x_1, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -lean_dec(x_23); -return x_94; +lean_object* x_111; +lean_dec(x_47); +lean_dec(x_46); +x_111 = lean_apply_8(x_18, x_39, x_34, x_2, x_3, x_4, x_5, x_6, x_10); +return x_111; } } else { -lean_object* x_95; -lean_dec(x_34); -lean_dec(x_33); -x_95 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14(x_1, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_95; +lean_object* x_112; +lean_dec(x_47); +lean_dec(x_46); +x_112 = lean_apply_8(x_17, x_39, x_34, x_2, x_3, x_4, x_5, x_6, x_10); +return x_112; } } else { -lean_object* x_96; -lean_dec(x_34); -lean_dec(x_33); -x_96 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12(x_1, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_96; +lean_object* x_113; +lean_dec(x_47); +lean_dec(x_46); +x_113 = lean_apply_8(x_16, x_39, x_34, x_2, x_3, x_4, x_5, x_6, x_10); +return x_113; } } else { -lean_object* x_97; -lean_dec(x_34); -lean_dec(x_33); -x_97 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8(x_1, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -lean_dec(x_27); -return x_97; +lean_object* x_114; +lean_dec(x_47); +lean_dec(x_46); +x_114 = lean_apply_8(x_14, x_39, x_34, x_2, x_3, x_4, x_5, x_6, x_10); +return x_114; } } else { -lean_object* x_98; -lean_dec(x_34); -lean_dec(x_33); -x_98 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4(x_1, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -lean_dec(x_23); -return x_98; +lean_object* x_115; +lean_dec(x_47); +lean_dec(x_46); +x_115 = lean_apply_8(x_12, x_39, x_34, x_2, x_3, x_4, x_5, x_6, x_10); +return x_115; } } else { -lean_object* x_99; -lean_dec(x_34); -lean_dec(x_33); -x_99 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2(x_1, x_27, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -lean_dec(x_23); -return x_99; +lean_object* x_116; +lean_dec(x_47); +lean_dec(x_46); +x_116 = lean_apply_8(x_11, x_39, x_34, x_2, x_3, x_4, x_5, x_6, x_10); +return x_116; } } } else { -lean_object* x_100; -lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_23); -x_100 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_100; +lean_object* x_117; +lean_dec(x_40); +lean_dec(x_39); +lean_dec(x_34); +x_117 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +return x_117; } } } @@ -7201,7 +7000,7 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_1); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_1, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_1, x_5, x_6, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_11) == 0) { lean_object* x_12; @@ -7251,7 +7050,7 @@ x_20 = lean_ctor_get(x_12, 0); lean_inc(x_20); lean_dec(x_12); lean_inc(x_2); -x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_2, x_5, x_6, x_7, x_8, x_9, x_19); +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_2, x_5, x_6, x_7, x_8, x_9, x_19); if (lean_obj_tag(x_21) == 0) { lean_object* x_22; @@ -7520,6 +7319,121 @@ return x_70; } } } +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(lean_object* x_1, 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_2); +lean_inc(x_1); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go(x_1, 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) == 0) +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); +lean_dec(x_8); +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +return x_11; +} +else +{ +uint8_t x_12; +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_12 = !lean_is_exclusive(x_8); +if (x_12 == 0) +{ +lean_object* x_13; uint8_t x_14; +x_13 = lean_ctor_get(x_8, 0); +lean_dec(x_13); +x_14 = !lean_is_exclusive(x_9); +if (x_14 == 0) +{ +return x_8; +} +else +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_9, 0); +lean_inc(x_15); +lean_dec(x_9); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_8, 0, x_16); +return x_8; +} +} +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_8, 1); +lean_inc(x_17); +lean_dec(x_8); +x_18 = lean_ctor_get(x_9, 0); +lean_inc(x_18); +if (lean_is_exclusive(x_9)) { + lean_ctor_release(x_9, 0); + x_19 = x_9; +} else { + lean_dec_ref(x_9); + x_19 = lean_box(0); +} +if (lean_is_scalar(x_19)) { + x_20 = lean_alloc_ctor(1, 1, 0); +} else { + x_20 = x_19; +} +lean_ctor_set(x_20, 0, 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_17); +return x_21; +} +} +} +else +{ +uint8_t x_22; +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_22 = !lean_is_exclusive(x_8); +if (x_22 == 0) +{ +return x_8; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_8, 0); +x_24 = lean_ctor_get(x_8, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_8); +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; +} +} +} +} static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__1() { _start: { @@ -7566,7 +7480,7 @@ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_obj x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_unaryReflection___closed__4; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -7587,7 +7501,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ { 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_ReifiedBVExpr_of___lambda__22___closed__7; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__7; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } @@ -7597,7 +7511,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ { 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_ReifiedBVExpr_of___lambda__19___closed__7; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__7; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } @@ -7607,7 +7521,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ { 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_ReifiedBVExpr_of___lambda__4___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__2; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } @@ -7617,7 +7531,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ { 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_ReifiedBVExpr_of___lambda__2___closed__3; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__3; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } @@ -7627,7 +7541,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ { 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_ReifiedBVExpr_of___lambda__16___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__2; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } @@ -7637,7 +7551,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_u { lean_object* x_10; lean_inc(x_1); -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_1, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_1, x_4, x_5, x_6, x_7, x_8, x_9); if (lean_obj_tag(x_10) == 0) { lean_object* x_11; @@ -8392,7 +8306,7 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_1); -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(x_1, x_7, x_8, x_9, x_10, x_11, x_12); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_1, x_7, x_8, x_9, x_10, x_11, x_12); if (lean_obj_tag(x_13) == 0) { lean_object* x_14; @@ -8444,7 +8358,7 @@ x_22 = lean_ctor_get(x_14, 0); lean_inc(x_22); lean_dec(x_14); lean_inc(x_2); -x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(x_2, x_7, x_8, x_9, x_10, x_11, x_21); +x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_2, x_7, x_8, x_9, x_10, x_11, x_21); if (lean_obj_tag(x_23) == 0) { lean_object* x_24; @@ -8765,80 +8679,30 @@ return x_104; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___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; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, 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_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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_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_ReifiedBVExpr_of_shiftReflection(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, 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_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_14 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_2, 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_Lean_Expr_cleanupAnnotations(x_15); +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_13 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_1, 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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f___closed__1; +x_17 = l_Lean_Expr_cleanupAnnotations(x_14); 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_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); +lean_dec(x_2); x_19 = lean_box(0); -x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___lambda__2(x_1, x_19, x_8, x_9, x_10, x_11, x_12, x_16); +x_20 = lean_apply_7(x_16, x_19, x_7, x_8, x_9, x_10, x_11, x_15); return x_20; } else @@ -8851,115 +8715,91 @@ lean_dec(x_21); if (x_23 == 0) { lean_object* x_24; lean_object* x_25; -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_24 = lean_box(0); -x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___lambda__2(x_1, x_24, x_8, x_9, x_10, x_11, x_12, x_16); +x_25 = lean_apply_7(x_16, x_24, x_7, x_8, x_9, x_10, x_11, x_15); return x_25; } else { lean_object* x_26; lean_object* x_27; -lean_dec(x_1); x_26 = lean_box(0); -x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___lambda__1(x_4, x_3, x_5, x_6, x_7, x_26, x_8, x_9, x_10, x_11, x_12, x_16); +x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___lambda__1(x_3, x_2, x_4, x_5, x_6, x_26, x_7, x_8, x_9, x_10, x_11, x_15); return x_27; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstReflection(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_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_ReifiedBVExpr_of_shiftConstReflection(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, 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_14; -lean_inc(x_12); +lean_object* x_13; lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f(x_2, x_3, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_14) == 0) +lean_inc(x_7); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_getNatOrBvValue_x3f(x_1, x_2, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_15; -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -if (lean_obj_tag(x_15) == 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_16; lean_object* x_17; +uint8_t x_15; +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); -x_16 = lean_ctor_get(x_14, 1); -lean_inc(x_16); -lean_dec(x_14); -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_8, x_9, x_10, x_11, x_12, x_16); -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_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; -} -} -else -{ -uint8_t x_22; -x_22 = !lean_is_exclusive(x_17); -if (x_22 == 0) +lean_dec(x_3); +x_15 = !lean_is_exclusive(x_13); +if (x_15 == 0) { -return x_17; +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_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_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 { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -lean_dec(x_1); -x_26 = lean_ctor_get(x_14, 1); -lean_inc(x_26); +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_13, 1); +lean_inc(x_21); +lean_dec(x_13); +x_22 = lean_ctor_get(x_14, 0); +lean_inc(x_22); lean_dec(x_14); -x_27 = lean_ctor_get(x_15, 0); -lean_inc(x_27); -lean_dec(x_15); -x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstLikeReflection(x_27, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_26); -return x_28; +x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstLikeReflection(x_22, x_3, 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_29; -lean_dec(x_12); +uint8_t x_24; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -8968,24 +8808,24 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_1); -x_29 = !lean_is_exclusive(x_14); -if (x_29 == 0) +lean_dec(x_3); +x_24 = !lean_is_exclusive(x_13); +if (x_24 == 0) { -return x_14; +return x_13; } else { -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_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; } } } @@ -8995,7 +8835,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_s { lean_object* x_12; lean_inc(x_2); -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofOrAtom(x_2, x_6, x_7, x_8, x_9, x_10, x_11); +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_2, x_6, x_7, x_8, x_9, x_10, x_11); if (lean_obj_tag(x_12) == 0) { lean_object* x_13; @@ -9273,94 +9113,71 @@ return x_90; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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; -lean_inc(x_11); +lean_object* x_12; lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_13 = l_Lean_Meta_getNatValue_x3f(x_2, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_13) == 0) +lean_inc(x_7); +x_12 = l_Lean_Meta_getNatValue_x3f(x_1, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_12) == 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_13; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_15; lean_object* x_16; +uint8_t 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); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom(x_1, x_7, x_8, x_9, x_10, x_11, x_15); -if (lean_obj_tag(x_16) == 0) -{ -uint8_t x_17; -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) -{ -return x_16; -} -else -{ -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_21; -x_21 = !lean_is_exclusive(x_16); -if (x_21 == 0) +lean_dec(x_2); +x_14 = !lean_is_exclusive(x_12); +if (x_14 == 0) { -return x_16; +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); +return x_12; } 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; -} +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_25; lean_object* x_26; lean_object* x_27; -lean_dec(x_1); -x_25 = lean_ctor_get(x_13, 1); -lean_inc(x_25); +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_ctor_get(x_13, 0); +lean_inc(x_21); lean_dec(x_13); -x_26 = lean_ctor_get(x_14, 0); -lean_inc(x_26); -lean_dec(x_14); -x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstLikeReflection(x_26, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_25); -return x_27; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftConstLikeReflection(x_21, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_20); +return x_22; } } else { -uint8_t x_28; -lean_dec(x_11); +uint8_t x_23; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -9369,78 +9186,69 @@ 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_13); -if (x_28 == 0) +lean_dec(x_2); +x_23 = !lean_is_exclusive(x_12); +if (x_23 == 0) { -return x_13; +return x_12; } else { -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); -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_24; lean_object* x_25; lean_object* x_26; +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_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_ReifiedBVExpr_of___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_ReifiedBVExpr_of___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_3); -return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_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) { _start: { -lean_object* x_10; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_3); -return x_10; +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2(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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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) { _start: { -lean_object* x_10; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_2); -return x_10; +return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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) { _start: { -lean_object* x_10; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_3); -return x_10; +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8(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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__31(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16(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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___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) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___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) { _start: { lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__32(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__31(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_2); return x_9; } @@ -9464,22 +9272,21 @@ lean_dec(x_6); return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, 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_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_shiftReflection___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_2); -return x_9; +lean_object* x_12; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(lean_object* x_1, 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_13; -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_rotateReflection(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_2); -return x_13; +lean_object* x_8; +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +return x_8; } } lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_BVDecide_Reflect(uint8_t builtin, lean_object*); @@ -9551,264 +9358,282 @@ l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__5 = _ini lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__5); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__6(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goBvLit___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__2___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__4___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__5___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__6___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__7___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__8___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__9___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__10___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__11___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__12___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__13___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__14___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__16___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__8); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__9(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__9); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__10(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__19___closed__10); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__8); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__9(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__9); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__10(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__22___closed__10); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__23___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__24___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__25___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__26___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__27___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__28___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__29___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___lambda__30___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__8); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__9(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__9); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__10(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__10); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__11 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__11(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__11); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__12 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__12(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__12); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__13 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__13(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__13); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__14 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__14(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__14); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__15 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__15(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__15); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__16 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__16(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__16); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__17 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__17(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__17); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__18 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__18(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__18); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__19 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__19(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__19); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__20 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__20(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__20); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__21 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__21(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__21); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__22 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__22(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__22); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__23 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__23(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__23); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__24 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__24(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__24); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__25 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__25(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__25); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__26 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__26(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__26); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__27 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__27(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__27); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__28 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__28(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__28); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__29 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__29(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__29); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__30 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__30(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__30); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__31 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__31(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__31); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__32 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__32(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__32); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__33 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__33(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__33); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__34 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__34(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__34); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__35 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__35(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__35); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__36 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__36(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__36); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__37 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__37(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__37); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__38 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__38(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__38); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__39 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__39(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__39); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__40 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__40(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__40); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__41 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__41(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__41); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__42 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__42(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__42); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__43 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__43(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__43); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__44 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__44(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__44); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__45 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__45(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__45); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__46 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__46(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__46); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__47 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__47(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__47); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__48 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__48(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__48); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__49 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__49(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__49); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__50 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__50(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__50); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__51 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__51(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of___closed__51); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__2___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__4___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__5___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__6___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__7___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__8___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__9___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__10___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__11___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__12___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__13___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__14___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__16___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__9); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__10(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__19___closed__10); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__9); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__10(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__22___closed__10); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__23___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__24___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__25___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__26___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__27___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__28___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__29___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___lambda__30___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__9); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__10(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__10); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__11 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__11(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__11); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__12 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__12(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__12); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__13 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__13(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__13); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__14 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__14(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__14); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__15 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__15(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__15); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__16 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__16(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__16); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__17 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__17(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__17); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__18 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__18(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__18); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__19 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__19(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__19); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__20 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__20(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__20); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__21 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__21(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__21); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__22 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__22(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__22); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__23 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__23(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__23); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__24 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__24(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__24); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__25 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__25(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__25); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__26 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__26(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__26); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__27 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__27(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__27); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__28 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__28(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__28); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__29 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__29(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__29); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__30 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__30(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__30); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__31 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__31(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__31); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__32 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__32(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__32); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__33 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__33(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__33); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__34 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__34(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__34); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__35 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__35(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__35); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__36 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__36(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__36); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__37 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__37(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__37); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__38 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__38(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__38); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__39 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__39(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__39); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__40 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__40(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__40); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__41 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__41(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__41); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__42 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__42(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__42); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__43 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__43(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__43); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__44 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__44(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__44); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__45 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__45(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__45); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__46 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__46(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__46); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__47 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__47(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__47); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__48 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__48(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__48); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__49 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__49(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__49); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__50 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__50(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__50); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__51 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__51(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__51); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__52 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__52(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__52); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__53 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__53(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__53); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__54 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__54(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__54); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__55 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__55(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__55); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__56 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__56(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__56); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__57 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__57(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__57); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__58 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__58(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__58); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__59 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__59(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__59); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__60 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__60(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_go___closed__60); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__1); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_binaryReflection___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVLogical.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVLogical.c index 14b9500fffe9..aeaede831620 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVLogical.c +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVLogical.c @@ -13,132 +13,138 @@ #ifdef __cplusplus extern "C" { #endif +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__1(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_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__8; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goOrAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__5; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__6; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__9; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__9; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6(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_ReifiedBVLogical_mkTrans(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___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_ReifiedBVLogical_ofPred___closed__3; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__12; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__2; lean_object* l_Lean_mkAppB(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__11; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__1; uint8_t l_Lean_Expr_isApp(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__8; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__2; +lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__5; +LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); lean_object* l_Lean_mkApp4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__5; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__1; -LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__11; lean_object* l_Lean_Level_ofNat(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__9; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__6; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__5; lean_object* l_Lean_mkApp6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__6; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkTrans___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__9; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkTrans___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___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 lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__2; lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_M_atomsAssignment(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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_ReifiedBVLogical_of_go___closed__12; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; lean_object* l_Lean_Expr_appArg(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__1; lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__9; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__2; +LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___spec__1(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__7; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__2; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__10; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_boolAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5(lean_object*, lean_object*, lean_object*, 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*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5(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_ReifiedBVLogical_of___lambda__4___closed__2; -LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___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_ReifiedBVLogical_of___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__8; lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__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_ReifiedBVLogical_of___closed__8; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__6; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__8; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6(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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__3; -LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___spec__1(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__5; lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__7; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___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_ReifiedBVLogical_mkEvalExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___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_ReifiedBVLogical_of_goPred___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__13; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__6; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__7; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__8; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9(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*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__13; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__5; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkTrans___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__6; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__3; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__10; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__4; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__9; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__5; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__7; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__4; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__3; static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__1() { _start: { @@ -380,7 +386,7 @@ lean_dec(x_2); return x_8; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__1() { _start: { lean_object* x_1; @@ -388,7 +394,7 @@ x_1 = lean_mk_string_unchecked("BoolExpr", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__2() { _start: { lean_object* x_1; @@ -396,30 +402,30 @@ x_1 = lean_mk_string_unchecked("literal", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__2; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__2; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___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_ReifiedBVLogical_of_goPred___closed__3; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___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_ReifiedBVLogical_of_goPred___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__5() { _start: { lean_object* x_1; @@ -427,33 +433,103 @@ x_1 = lean_mk_string_unchecked("BVPred", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__5; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___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_ReifiedBVLogical_of_goPred___closed__6; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___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_ReifiedBVLogical_of_goPred(lean_object* x_1, lean_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_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred(lean_object* x_1, 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: +{ +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; +x_9 = lean_ctor_get(x_1, 0); +x_10 = lean_ctor_get(x_1, 2); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_9); +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__4; +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_14 = l_Lean_mkAppB(x_12, x_13, x_10); +lean_ctor_set(x_1, 2, x_14); +lean_ctor_set(x_1, 0, x_11); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, 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_7); +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; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_17 = lean_ctor_get(x_1, 0); +x_18 = lean_ctor_get(x_1, 1); +x_19 = lean_ctor_get(x_1, 2); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_1); +x_20 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_20, 0, x_17); +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__4; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_23 = l_Lean_mkAppB(x_21, x_22, x_19); +x_24 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_24, 0, x_20); +lean_ctor_set(x_24, 1, x_18); +lean_ctor_set(x_24, 2, x_23); +x_25 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_25, 0, 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_7); +return x_26; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___boxed(lean_object* x_1, 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_ReifiedBVPred_of(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred(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_ReifiedBVLogical_boolAtom(lean_object* x_1, 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_2); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_7); if (lean_obj_tag(x_8) == 0) { lean_object* x_9; @@ -462,6 +538,11 @@ lean_inc(x_9); if (lean_obj_tag(x_9) == 0) { uint8_t x_10; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); x_10 = !lean_is_exclusive(x_8); if (x_10 == 0) { @@ -487,1235 +568,1221 @@ return x_15; } else { -uint8_t x_16; -x_16 = !lean_is_exclusive(x_9); -if (x_16 == 0) -{ -uint8_t x_17; -x_17 = !lean_is_exclusive(x_8); -if (x_17 == 0) -{ -lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_18 = lean_ctor_get(x_9, 0); -x_19 = lean_ctor_get(x_8, 0); -lean_dec(x_19); -x_20 = !lean_is_exclusive(x_18); -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; -x_21 = lean_ctor_get(x_18, 0); -x_22 = lean_ctor_get(x_18, 2); -x_23 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_23, 0, x_21); -x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__4; -x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_26 = l_Lean_mkAppB(x_24, x_25, x_22); -lean_ctor_set(x_18, 2, x_26); -lean_ctor_set(x_18, 0, x_23); -return x_8; -} -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; -x_27 = lean_ctor_get(x_18, 0); -x_28 = lean_ctor_get(x_18, 1); -x_29 = lean_ctor_get(x_18, 2); -lean_inc(x_29); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_18); -x_30 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_30, 0, x_27); -x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__4; -x_32 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_33 = l_Lean_mkAppB(x_31, x_32, x_29); -x_34 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_34, 0, x_30); -lean_ctor_set(x_34, 1, x_28); -lean_ctor_set(x_34, 2, x_33); -lean_ctor_set(x_9, 0, x_34); -return x_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; 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_9, 0); -x_36 = lean_ctor_get(x_8, 1); -lean_inc(x_36); +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_8, 1); +lean_inc(x_16); lean_dec(x_8); -x_37 = lean_ctor_get(x_35, 0); -lean_inc(x_37); -x_38 = lean_ctor_get(x_35, 1); -lean_inc(x_38); -x_39 = lean_ctor_get(x_35, 2); -lean_inc(x_39); -if (lean_is_exclusive(x_35)) { - lean_ctor_release(x_35, 0); - lean_ctor_release(x_35, 1); - lean_ctor_release(x_35, 2); - x_40 = x_35; -} else { - lean_dec_ref(x_35); - x_40 = lean_box(0); -} -x_41 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_41, 0, x_37); -x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__4; -x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_44 = l_Lean_mkAppB(x_42, x_43, x_39); -if (lean_is_scalar(x_40)) { - x_45 = lean_alloc_ctor(0, 3, 0); -} else { - x_45 = x_40; -} -lean_ctor_set(x_45, 0, x_41); -lean_ctor_set(x_45, 1, x_38); -lean_ctor_set(x_45, 2, x_44); -lean_ctor_set(x_9, 0, x_45); -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_9); -lean_ctor_set(x_46, 1, x_36); -return x_46; -} -} -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; lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_47 = lean_ctor_get(x_9, 0); -lean_inc(x_47); +x_17 = lean_ctor_get(x_9, 0); +lean_inc(x_17); lean_dec(x_9); -x_48 = lean_ctor_get(x_8, 1); -lean_inc(x_48); -if (lean_is_exclusive(x_8)) { - lean_ctor_release(x_8, 0); - lean_ctor_release(x_8, 1); - x_49 = x_8; -} else { - lean_dec_ref(x_8); - x_49 = lean_box(0); -} -x_50 = lean_ctor_get(x_47, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_47, 1); -lean_inc(x_51); -x_52 = lean_ctor_get(x_47, 2); -lean_inc(x_52); -if (lean_is_exclusive(x_47)) { - lean_ctor_release(x_47, 0); - lean_ctor_release(x_47, 1); - lean_ctor_release(x_47, 2); - x_53 = x_47; -} else { - lean_dec_ref(x_47); - x_53 = lean_box(0); -} -x_54 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_54, 0, x_50); -x_55 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__4; -x_56 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_57 = l_Lean_mkAppB(x_55, x_56, x_52); -if (lean_is_scalar(x_53)) { - x_58 = lean_alloc_ctor(0, 3, 0); -} else { - x_58 = x_53; -} -lean_ctor_set(x_58, 0, x_54); -lean_ctor_set(x_58, 1, x_51); -lean_ctor_set(x_58, 2, x_57); -x_59 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_59, 0, x_58); -if (lean_is_scalar(x_49)) { - x_60 = lean_alloc_ctor(0, 2, 0); -} else { - x_60 = x_49; -} -lean_ctor_set(x_60, 0, x_59); -lean_ctor_set(x_60, 1, x_48); -return x_60; -} +x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred(x_17, x_2, x_3, x_4, x_5, x_6, x_16); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_18; } } else { -uint8_t x_61; -x_61 = !lean_is_exclusive(x_8); -if (x_61 == 0) +uint8_t x_19; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_19 = !lean_is_exclusive(x_8); +if (x_19 == 0) { return x_8; } else { -lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_62 = lean_ctor_get(x_8, 0); -x_63 = lean_ctor_get(x_8, 1); -lean_inc(x_63); -lean_inc(x_62); +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_8, 0); +x_21 = lean_ctor_get(x_8, 1); +lean_inc(x_21); +lean_inc(x_20); lean_dec(x_8); -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; +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_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(lean_object* x_1, 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_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_ReifiedBVLogical_mkEvalExpr(x_1, 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_ctor_get(x_15, 1); -lean_inc(x_17); -lean_dec(x_15); -x_18 = lean_ctor_get(x_2, 1); -lean_inc(x_18); -lean_dec(x_2); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); +lean_object* x_8; +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of(x_1, 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); -x_19 = lean_apply_6(x_18, x_9, x_10, x_11, x_12, x_13, x_17); -if (lean_obj_tag(x_19) == 0) +if (lean_obj_tag(x_9) == 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); -x_22 = lean_ctor_get(x_3, 1); -lean_inc(x_22); +uint8_t x_10; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); -x_23 = lean_apply_6(x_22, x_9, x_10, x_11, x_12, x_13, x_21); -if (lean_obj_tag(x_23) == 0) -{ -uint8_t x_24; -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) +lean_dec(x_2); +x_10 = !lean_is_exclusive(x_8); +if (x_10 == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_23, 0); -x_26 = l_Lean_Expr_const___override(x_4, x_5); -x_27 = l_Lean_mkApp6(x_26, x_6, x_7, x_8, x_16, x_20, x_25); -lean_ctor_set(x_23, 0, x_27); -return x_23; +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_8, 0); +lean_dec(x_11); +x_12 = lean_box(0); +lean_ctor_set(x_8, 0, x_12); +return x_8; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -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 = l_Lean_Expr_const___override(x_4, x_5); -x_31 = l_Lean_mkApp6(x_30, x_6, x_7, x_8, x_16, x_20, x_28); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_29); -return x_32; +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_8, 1); +lean_inc(x_13); +lean_dec(x_8); +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 { -uint8_t x_33; -lean_dec(x_20); -lean_dec(x_16); +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_8, 1); +lean_inc(x_16); lean_dec(x_8); -lean_dec(x_7); +x_17 = lean_ctor_get(x_9, 0); +lean_inc(x_17); +lean_dec(x_9); +x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred(x_17, x_2, x_3, x_4, x_5, x_6, x_16); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_33 = !lean_is_exclusive(x_23); -if (x_33 == 0) -{ -return x_23; -} -else -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_23, 0); -x_35 = lean_ctor_get(x_23, 1); -lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_23); -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_dec(x_3); +lean_dec(x_2); +return x_18; } } else { -uint8_t x_37; -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); +uint8_t x_19; lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_37 = !lean_is_exclusive(x_19); -if (x_37 == 0) +lean_dec(x_2); +x_19 = !lean_is_exclusive(x_8); +if (x_19 == 0) { -return x_19; +return x_8; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_19, 0); -x_39 = lean_ctor_get(x_19, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_19); -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_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_8, 0); +x_21 = lean_ctor_get(x_8, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_8); +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 lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__1() { +LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("gate", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__2() { +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_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___spec__1(lean_object* x_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; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__1; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___spec__1___rarg___boxed), 7, 0); +return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_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) { _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_ReifiedBVLogical_of_gateReflection___closed__2; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_3, x_4, x_5, x_6, x_7, x_8); +return x_9; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("Gate", 4, 4); +x_1 = lean_mk_string_unchecked("Reflect", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("and", 3, 3); +x_1 = lean_mk_string_unchecked("beq_congr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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; lean_object* x_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; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__5; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___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_ReifiedBVLogical_of_gateReflection___closed__7() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_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: +{ +uint8_t x_10; lean_object* x_11; lean_object* x_12; +x_10 = 2; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__3; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(x_1, x_2, x_10, x_11, x_4, x_5, x_6, x_7, x_8, x_9); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_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) { +_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_ReifiedBVLogical_of_go___lambda__4___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__3___boxed), 7, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__2() { +_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_ReifiedBVLogical_of_go___lambda__4___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_ReifiedBVLogical_of_gateReflection___closed__6; -x_3 = l_Lean_Expr_const___override(x_2, x_1); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___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_ReifiedBVLogical_of_gateReflection___closed__8() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +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_ReifiedBVLogical_of_go___lambda__4___closed__1; +x_15 = l_Lean_Expr_cleanupAnnotations(x_12); +x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__8; +x_17 = l_Lean_Expr_isConstOf(x_15, x_16); +if (x_17 == 0) +{ +uint8_t x_18; +lean_dec(x_4); +lean_dec(x_3); +x_18 = l_Lean_Expr_isApp(x_15); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_15); +lean_dec(x_1); +x_19 = lean_box(0); +x_20 = lean_apply_7(x_14, x_19, x_5, x_6, x_7, x_8, x_9, x_13); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = l_Lean_Expr_appFnCleanup(x_15, lean_box(0)); +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__3; +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_1); +x_24 = lean_box(0); +x_25 = lean_apply_7(x_14, x_24, x_5, x_6, x_7, x_8, x_9, x_13); +return x_25; +} +else +{ +lean_object* x_26; +x_26 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_5, x_6, x_7, x_8, x_9, x_13); +return x_26; +} +} +} +else +{ +lean_object* x_27; lean_object* x_28; +lean_dec(x_15); +lean_dec(x_1); +x_27 = lean_box(0); +x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2(x_3, x_4, x_27, x_5, x_6, x_7, x_8, x_9, x_13); +return x_28; +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("xor", 3, 3); +x_1 = lean_mk_string_unchecked("xor_congr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__9() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___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_1; 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_ReifiedBVLogical_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__8; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___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_ReifiedBVLogical_of_gateReflection___closed__10() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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) { _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_ReifiedBVLogical_of_gateReflection___closed__9; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; +uint8_t x_9; lean_object* x_10; lean_object* x_11; +x_9 = 1; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__2; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); +return x_11; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__11() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("beq", 3, 3); +x_1 = lean_mk_string_unchecked("and_congr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__12() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___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_1; 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_ReifiedBVLogical_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__11; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___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_ReifiedBVLogical_of_gateReflection___closed__13() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__12; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; +uint8_t x_9; lean_object* x_10; lean_object* x_11; +x_9 = 0; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__2; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); +return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(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) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__1() { _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_1); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of(x_1, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("not_congr", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__2() { +_start: { -lean_object* x_12; -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_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_object* x_7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___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_ReifiedBVLogical_of_go___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: +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_apply_6(x_11, x_5, x_6, x_7, x_8, x_9, x_10); 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_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_13 = !lean_is_exclusive(x_11); +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_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_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_12, 0); +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__2; +x_16 = l_Lean_Expr_const___override(x_15, x_2); +x_17 = l_Lean_mkApp3(x_16, x_3, x_4, x_14); +lean_ctor_set(x_12, 0, x_17); +return x_12; } 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_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_12, 0); +x_19 = lean_ctor_get(x_12, 1); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_12); +x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__2; +x_21 = l_Lean_Expr_const___override(x_20, x_2); +x_22 = l_Lean_mkApp3(x_21, x_3, x_4, x_18); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_19); +return x_23; } } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_11, 1); -lean_inc(x_19); -lean_dec(x_11); -x_20 = lean_ctor_get(x_12, 0); -lean_inc(x_20); -lean_dec(x_12); -lean_inc(x_2); -x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of(x_2, x_5, x_6, x_7, x_8, x_9, x_19); -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_20); +uint8_t x_24; lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_23 = !lean_is_exclusive(x_21); -if (x_23 == 0) +x_24 = !lean_is_exclusive(x_12); +if (x_24 == 0) { -lean_object* x_24; lean_object* x_25; -x_24 = lean_ctor_get(x_21, 0); -lean_dec(x_24); -x_25 = lean_box(0); -lean_ctor_set(x_21, 0, x_25); -return x_21; +return x_12; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_21, 1); +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_12, 0); +x_26 = lean_ctor_get(x_12, 1); lean_inc(x_26); -lean_dec(x_21); -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_26); -return x_28; +lean_inc(x_25); +lean_dec(x_12); +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_29; -x_29 = !lean_is_exclusive(x_21); -if (x_29 == 0) -{ -lean_object* x_30; uint8_t x_31; -x_30 = lean_ctor_get(x_21, 0); -lean_dec(x_30); -x_31 = !lean_is_exclusive(x_22); -if (x_31 == 0) +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__1() { +_start: { -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_32 = lean_ctor_get(x_22, 0); -x_33 = lean_ctor_get(x_20, 0); -lean_inc(x_33); -x_34 = lean_ctor_get(x_32, 0); -lean_inc(x_34); -x_35 = lean_alloc_ctor(3, 2, 1); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -lean_ctor_set_uint8(x_35, sizeof(void*)*2, x_3); -x_36 = lean_box(0); -x_37 = lean_ctor_get(x_20, 2); -lean_inc(x_37); -x_38 = lean_ctor_get(x_32, 2); -lean_inc(x_38); -lean_inc(x_37); -x_39 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); -lean_closure_set(x_39, 0, x_37); -lean_inc(x_38); -x_40 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___lambda__1), 14, 7); -lean_closure_set(x_40, 0, x_38); -lean_closure_set(x_40, 1, x_20); -lean_closure_set(x_40, 2, x_32); -lean_closure_set(x_40, 3, x_4); -lean_closure_set(x_40, 4, x_36); -lean_closure_set(x_40, 5, x_1); -lean_closure_set(x_40, 6, x_2); -x_41 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_41, 0, x_39); -lean_closure_set(x_41, 1, x_40); -switch (x_3) { -case 0: +lean_object* x_1; +x_1 = lean_mk_string_unchecked("not", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__2() { +_start: { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; -x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_44 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__7; -x_45 = l_Lean_mkApp4(x_42, x_43, x_44, x_37, x_38); -x_46 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_46, 0, x_35); -lean_ctor_set(x_46, 1, x_41); -lean_ctor_set(x_46, 2, x_45); -lean_ctor_set(x_22, 0, x_46); -return x_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; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__1; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; } -case 1: +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__3() { +_start: { -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_47 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; -x_48 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_49 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10; -x_50 = l_Lean_mkApp4(x_47, x_48, x_49, x_37, x_38); -x_51 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_51, 0, x_35); -lean_ctor_set(x_51, 1, x_41); -lean_ctor_set(x_51, 2, x_50); -lean_ctor_set(x_22, 0, x_51); -return x_21; +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_ReifiedBVLogical_of_go___lambda__8___closed__2; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; } -default: +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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) { +_start: { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_52 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; -x_53 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_54 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__13; -x_55 = l_Lean_mkApp4(x_52, x_53, x_54, x_37, x_38); -x_56 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_56, 0, x_35); -lean_ctor_set(x_56, 1, x_41); -lean_ctor_set(x_56, 2, x_55); -lean_ctor_set(x_22, 0, x_56); -return x_21; +lean_object* x_8; +lean_inc(x_1); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goOrAtom(x_1, 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) == 0) +{ +uint8_t x_10; +lean_dec(x_1); +x_10 = !lean_is_exclusive(x_8); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_8, 0); +lean_dec(x_11); +x_12 = lean_box(0); +lean_ctor_set(x_8, 0, x_12); +return x_8; } +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_8, 1); +lean_inc(x_13); +lean_dec(x_8); +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_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_57 = lean_ctor_get(x_22, 0); -lean_inc(x_57); -lean_dec(x_22); -x_58 = lean_ctor_get(x_20, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_57, 0); -lean_inc(x_59); -x_60 = lean_alloc_ctor(3, 2, 1); -lean_ctor_set(x_60, 0, x_58); -lean_ctor_set(x_60, 1, x_59); -lean_ctor_set_uint8(x_60, sizeof(void*)*2, x_3); -x_61 = lean_box(0); -x_62 = lean_ctor_get(x_20, 2); -lean_inc(x_62); -x_63 = lean_ctor_get(x_57, 2); -lean_inc(x_63); -lean_inc(x_62); -x_64 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); -lean_closure_set(x_64, 0, x_62); -lean_inc(x_63); -x_65 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___lambda__1), 14, 7); -lean_closure_set(x_65, 0, x_63); -lean_closure_set(x_65, 1, x_20); -lean_closure_set(x_65, 2, x_57); -lean_closure_set(x_65, 3, x_4); -lean_closure_set(x_65, 4, x_61); -lean_closure_set(x_65, 5, x_1); -lean_closure_set(x_65, 6, x_2); -x_66 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_66, 0, x_64); -lean_closure_set(x_66, 1, x_65); -switch (x_3) { -case 0: +uint8_t x_16; +x_16 = !lean_is_exclusive(x_9); +if (x_16 == 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; -x_67 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; -x_68 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_69 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__7; -x_70 = l_Lean_mkApp4(x_67, x_68, x_69, x_62, x_63); -x_71 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_71, 0, x_60); -lean_ctor_set(x_71, 1, x_66); -lean_ctor_set(x_71, 2, x_70); -x_72 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_72, 0, x_71); -lean_ctor_set(x_21, 0, x_72); -return x_21; -} -case 1: +uint8_t x_17; +x_17 = !lean_is_exclusive(x_8); +if (x_17 == 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 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; -x_74 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_75 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10; -x_76 = l_Lean_mkApp4(x_73, x_74, x_75, x_62, x_63); -x_77 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_77, 0, x_60); -lean_ctor_set(x_77, 1, x_66); -lean_ctor_set(x_77, 2, x_76); -x_78 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_78, 0, x_77); -lean_ctor_set(x_21, 0, x_78); -return x_21; -} -default: +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; uint8_t x_29; +x_18 = lean_ctor_get(x_9, 0); +x_19 = lean_ctor_get(x_8, 0); +lean_dec(x_19); +x_20 = lean_ctor_get(x_18, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_18, 2); +lean_inc(x_21); +x_22 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_22, 0, x_20); +x_23 = lean_box(0); +x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__3; +x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +lean_inc(x_21); +x_26 = l_Lean_mkAppB(x_24, x_25, x_21); +x_27 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); +lean_closure_set(x_27, 0, x_21); +lean_inc(x_18); +x_28 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7), 10, 3); +lean_closure_set(x_28, 0, x_18); +lean_closure_set(x_28, 1, x_23); +lean_closure_set(x_28, 2, x_1); +x_29 = !lean_is_exclusive(x_18); +if (x_29 == 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; -x_79 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; -x_80 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_81 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__13; -x_82 = l_Lean_mkApp4(x_79, x_80, x_81, x_62, x_63); -x_83 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_83, 0, x_60); -lean_ctor_set(x_83, 1, x_66); -lean_ctor_set(x_83, 2, x_82); -x_84 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_84, 0, x_83); -lean_ctor_set(x_21, 0, x_84); -return x_21; -} +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_30 = lean_ctor_get(x_18, 2); +lean_dec(x_30); +x_31 = lean_ctor_get(x_18, 1); +lean_dec(x_31); +x_32 = lean_ctor_get(x_18, 0); +lean_dec(x_32); +x_33 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_33, 0, x_27); +lean_closure_set(x_33, 1, x_28); +lean_ctor_set(x_18, 2, x_26); +lean_ctor_set(x_18, 1, x_33); +lean_ctor_set(x_18, 0, x_22); +return x_8; } +else +{ +lean_object* x_34; lean_object* x_35; +lean_dec(x_18); +x_34 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_34, 0, x_27); +lean_closure_set(x_34, 1, x_28); +x_35 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_35, 0, x_22); +lean_ctor_set(x_35, 1, x_34); +lean_ctor_set(x_35, 2, x_26); +lean_ctor_set(x_9, 0, x_35); +return x_8; } } else { -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_85 = lean_ctor_get(x_21, 1); -lean_inc(x_85); -lean_dec(x_21); -x_86 = lean_ctor_get(x_22, 0); -lean_inc(x_86); -if (lean_is_exclusive(x_22)) { - lean_ctor_release(x_22, 0); - x_87 = x_22; +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; +x_36 = lean_ctor_get(x_9, 0); +x_37 = lean_ctor_get(x_8, 1); +lean_inc(x_37); +lean_dec(x_8); +x_38 = lean_ctor_get(x_36, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_36, 2); +lean_inc(x_39); +x_40 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_40, 0, x_38); +x_41 = lean_box(0); +x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__3; +x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +lean_inc(x_39); +x_44 = l_Lean_mkAppB(x_42, x_43, x_39); +x_45 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); +lean_closure_set(x_45, 0, x_39); +lean_inc(x_36); +x_46 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7), 10, 3); +lean_closure_set(x_46, 0, x_36); +lean_closure_set(x_46, 1, x_41); +lean_closure_set(x_46, 2, x_1); +if (lean_is_exclusive(x_36)) { + lean_ctor_release(x_36, 0); + lean_ctor_release(x_36, 1); + lean_ctor_release(x_36, 2); + x_47 = x_36; } else { - lean_dec_ref(x_22); - x_87 = lean_box(0); + lean_dec_ref(x_36); + x_47 = lean_box(0); } -x_88 = lean_ctor_get(x_20, 0); -lean_inc(x_88); -x_89 = lean_ctor_get(x_86, 0); -lean_inc(x_89); -x_90 = lean_alloc_ctor(3, 2, 1); -lean_ctor_set(x_90, 0, x_88); -lean_ctor_set(x_90, 1, x_89); -lean_ctor_set_uint8(x_90, sizeof(void*)*2, x_3); -x_91 = lean_box(0); -x_92 = lean_ctor_get(x_20, 2); -lean_inc(x_92); -x_93 = lean_ctor_get(x_86, 2); -lean_inc(x_93); -lean_inc(x_92); -x_94 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); -lean_closure_set(x_94, 0, x_92); -lean_inc(x_93); -x_95 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___lambda__1), 14, 7); -lean_closure_set(x_95, 0, x_93); -lean_closure_set(x_95, 1, x_20); -lean_closure_set(x_95, 2, x_86); -lean_closure_set(x_95, 3, x_4); -lean_closure_set(x_95, 4, x_91); -lean_closure_set(x_95, 5, x_1); -lean_closure_set(x_95, 6, x_2); -x_96 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_96, 0, x_94); -lean_closure_set(x_96, 1, x_95); -switch (x_3) { -case 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; -x_97 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; -x_98 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_99 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__7; -x_100 = l_Lean_mkApp4(x_97, x_98, x_99, x_92, x_93); -x_101 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_101, 0, x_90); -lean_ctor_set(x_101, 1, x_96); -lean_ctor_set(x_101, 2, x_100); -if (lean_is_scalar(x_87)) { - x_102 = lean_alloc_ctor(1, 1, 0); +x_48 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_48, 0, x_45); +lean_closure_set(x_48, 1, x_46); +if (lean_is_scalar(x_47)) { + x_49 = lean_alloc_ctor(0, 3, 0); } else { - x_102 = x_87; + x_49 = x_47; } -lean_ctor_set(x_102, 0, x_101); -x_103 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_103, 0, x_102); -lean_ctor_set(x_103, 1, x_85); -return x_103; +lean_ctor_set(x_49, 0, x_40); +lean_ctor_set(x_49, 1, x_48); +lean_ctor_set(x_49, 2, x_44); +lean_ctor_set(x_9, 0, x_49); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_9); +lean_ctor_set(x_50, 1, x_37); +return x_50; } -case 1: +} +else { -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 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; -x_105 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_106 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10; -x_107 = l_Lean_mkApp4(x_104, x_105, x_106, x_92, x_93); -x_108 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_108, 0, x_90); -lean_ctor_set(x_108, 1, x_96); -lean_ctor_set(x_108, 2, x_107); -if (lean_is_scalar(x_87)) { - x_109 = lean_alloc_ctor(1, 1, 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; 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_51 = lean_ctor_get(x_9, 0); +lean_inc(x_51); +lean_dec(x_9); +x_52 = lean_ctor_get(x_8, 1); +lean_inc(x_52); +if (lean_is_exclusive(x_8)) { + lean_ctor_release(x_8, 0); + lean_ctor_release(x_8, 1); + x_53 = x_8; } else { - x_109 = x_87; -} -lean_ctor_set(x_109, 0, x_108); -x_110 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_110, 0, x_109); -lean_ctor_set(x_110, 1, x_85); -return x_110; + lean_dec_ref(x_8); + x_53 = lean_box(0); } -default: -{ -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_111 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; -x_112 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_113 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__13; -x_114 = l_Lean_mkApp4(x_111, x_112, x_113, x_92, x_93); -x_115 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_115, 0, x_90); -lean_ctor_set(x_115, 1, x_96); -lean_ctor_set(x_115, 2, x_114); -if (lean_is_scalar(x_87)) { - x_116 = lean_alloc_ctor(1, 1, 0); +x_54 = lean_ctor_get(x_51, 0); +lean_inc(x_54); +x_55 = lean_ctor_get(x_51, 2); +lean_inc(x_55); +x_56 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_56, 0, x_54); +x_57 = lean_box(0); +x_58 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__3; +x_59 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +lean_inc(x_55); +x_60 = l_Lean_mkAppB(x_58, x_59, x_55); +x_61 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); +lean_closure_set(x_61, 0, x_55); +lean_inc(x_51); +x_62 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7), 10, 3); +lean_closure_set(x_62, 0, x_51); +lean_closure_set(x_62, 1, x_57); +lean_closure_set(x_62, 2, x_1); +if (lean_is_exclusive(x_51)) { + lean_ctor_release(x_51, 0); + lean_ctor_release(x_51, 1); + lean_ctor_release(x_51, 2); + x_63 = x_51; } else { - x_116 = x_87; + lean_dec_ref(x_51); + x_63 = lean_box(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_85); -return x_117; +x_64 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_64, 0, x_61); +lean_closure_set(x_64, 1, x_62); +if (lean_is_scalar(x_63)) { + x_65 = lean_alloc_ctor(0, 3, 0); +} else { + x_65 = x_63; } +lean_ctor_set(x_65, 0, x_56); +lean_ctor_set(x_65, 1, x_64); +lean_ctor_set(x_65, 2, x_60); +x_66 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_66, 0, x_65); +if (lean_is_scalar(x_53)) { + x_67 = lean_alloc_ctor(0, 2, 0); +} else { + x_67 = x_53; } +lean_ctor_set(x_67, 0, x_66); +lean_ctor_set(x_67, 1, x_52); +return x_67; } } } else { -uint8_t x_118; -lean_dec(x_20); -lean_dec(x_4); -lean_dec(x_2); +uint8_t x_68; lean_dec(x_1); -x_118 = !lean_is_exclusive(x_21); -if (x_118 == 0) +x_68 = !lean_is_exclusive(x_8); +if (x_68 == 0) { -return x_21; +return x_8; } else { -lean_object* x_119; lean_object* x_120; lean_object* x_121; -x_119 = lean_ctor_get(x_21, 0); -x_120 = lean_ctor_get(x_21, 1); -lean_inc(x_120); -lean_inc(x_119); -lean_dec(x_21); -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_object* x_69; lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_8, 0); +x_70 = lean_ctor_get(x_8, 1); +lean_inc(x_70); +lean_inc(x_69); +lean_dec(x_8); +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_122; -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_122 = !lean_is_exclusive(x_11); -if (x_122 == 0) +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__1() { +_start: { -return x_11; +uint8_t x_1; lean_object* x_2; +x_1 = 0; +x_2 = lean_alloc_ctor(1, 0, 1); +lean_ctor_set_uint8(x_2, 0, x_1); +return x_2; } -else +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__2() { +_start: { -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_object* x_1; +x_1 = lean_mk_string_unchecked("const", 5, 5); +return x_1; } } +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___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_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___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) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__4() { _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_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__3; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; } } -LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___spec__1(lean_object* x_1) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__5() { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___spec__1___rarg___boxed), 7, 0); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("false", 5, 5); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___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) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__6() { _start: { -lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_3, x_4, x_5, x_6, x_7, x_8); -return x_9; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___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_ReifiedBVLogical_of___lambda__2___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__7() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Reflect", 7, 7); -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_ReifiedBVLogical_of_go___lambda__9___closed__6; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__8() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("beq_congr", 9, 9); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__4; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__7; +x_4 = l_Lean_mkAppB(x_1, x_2, x_3); +return x_4; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___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; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__2; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__7; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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) { _start: { -uint8_t x_10; lean_object* x_11; lean_object* x_12; -x_10 = 2; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__3; -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(x_1, x_2, x_10, x_11, x_4, x_5, x_6, x_7, x_8, x_9); -return x_12; +lean_object* x_8; 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_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__9; +x_9 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___spec__1___rarg___boxed), 7, 1); +lean_closure_set(x_9, 0, x_8); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__1; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__8; +x_12 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_12, 0, x_10); +lean_ctor_set(x_12, 1, x_9); +lean_ctor_set(x_12, 2, x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, 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_7); +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___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) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__1() { _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; +uint8_t x_1; lean_object* x_2; +x_1 = 1; +x_2 = lean_alloc_ctor(1, 0, 1); +lean_ctor_set_uint8(x_2, 0, x_1); +return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__3___boxed), 7, 0); +x_1 = lean_mk_string_unchecked("true", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("BitVec", 6, 6); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___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_ReifiedBVLogical_of___lambda__4___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___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_ReifiedBVLogical_of___lambda__4___closed__2; -x_3 = l_Lean_Name_str___override(x_1, x_2); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___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_ReifiedBVLogical_of___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) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__5() { _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; -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_ReifiedBVLogical_of___lambda__4___closed__1; -x_15 = l_Lean_Expr_cleanupAnnotations(x_12); -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__8; -x_17 = l_Lean_Expr_isConstOf(x_15, x_16); -if (x_17 == 0) -{ -uint8_t x_18; -lean_dec(x_4); -lean_dec(x_3); -x_18 = l_Lean_Expr_isApp(x_15); -if (x_18 == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__4; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__4; +x_4 = l_Lean_mkAppB(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__6() { +_start: { -lean_object* x_19; lean_object* x_20; -lean_dec(x_15); -lean_dec(x_1); -x_19 = lean_box(0); -x_20 = lean_apply_7(x_14, x_19, x_5, x_6, x_7, x_8, x_9, x_13); -return x_20; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__4; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl(x_1); +return x_2; } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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, lean_object* x_7) { +_start: { -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = l_Lean_Expr_appFnCleanup(x_15, lean_box(0)); -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__3; -x_23 = l_Lean_Expr_isConstOf(x_21, x_22); -lean_dec(x_21); -if (x_23 == 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; +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__6; +x_9 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___spec__1___rarg___boxed), 7, 1); +lean_closure_set(x_9, 0, x_8); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__1; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__5; +x_12 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_12, 0, x_10); +lean_ctor_set(x_12, 1, x_9); +lean_ctor_set(x_12, 2, x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, 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_7); +return x_14; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__1() { +_start: { -lean_object* x_24; lean_object* x_25; -lean_dec(x_1); -x_24 = lean_box(0); -x_25 = lean_apply_7(x_14, x_24, x_5, x_6, x_7, x_8, x_9, x_13); -return x_25; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5), 8, 0); +return x_1; } -else +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__2() { +_start: { -lean_object* x_26; -x_26 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_5, x_6, x_7, x_8, x_9, x_13); -return x_26; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6), 8, 0); +return x_1; } } +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8), 7, 0); +return x_1; +} } -else +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__4() { +_start: { -lean_object* x_27; lean_object* x_28; -lean_dec(x_15); -lean_dec(x_1); -x_27 = lean_box(0); -x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2(x_3, x_4, x_27, x_5, x_6, x_7, x_8, x_9, x_13); -return x_28; -} +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___boxed), 7, 0); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__5() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("xor_congr", 9, 9); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___boxed), 7, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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_ReifiedBVLogical_mkEvalExpr___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__1; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___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_ReifiedBVLogical_of___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) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__7() { _start: { -uint8_t x_9; lean_object* x_10; lean_object* x_11; -x_9 = 1; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__2; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); -return x_11; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("xor", 3, 3); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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_ReifiedBVLogical_of_go___closed__9() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("and_congr", 9, 9); +x_1 = lean_mk_string_unchecked("and", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__1; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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_ReifiedBVLogical_of___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) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__11() { _start: { -uint8_t x_9; lean_object* x_10; lean_object* x_11; -x_9 = 0; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__2; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); -return x_11; +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_ReifiedBVLogical_of___lambda__7___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__12() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("not_congr", 9, 9); +x_1 = lean_mk_string_unchecked("beq", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__1; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__11; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__12; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_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) { _start: { -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_1, 1); -lean_inc(x_11); -lean_dec(x_1); -x_12 = lean_apply_6(x_11, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_12) == 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; uint8_t x_18; +lean_inc(x_1); +x_8 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_1, x_3, x_4, x_5, x_6, x_7); +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_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__1; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__2; +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__3; +x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__4; +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__5; +x_16 = l_Lean_Expr_cleanupAnnotations(x_9); +x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__6; +x_18 = l_Lean_Expr_isConstOf(x_16, x_17); +if (x_18 == 0) { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_12); -if (x_13 == 0) +lean_object* x_19; uint8_t x_20; +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__3; +x_20 = l_Lean_Expr_isConstOf(x_16, x_19); +if (x_20 == 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 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__2; -x_16 = l_Lean_Expr_const___override(x_15, x_2); -x_17 = l_Lean_mkApp3(x_16, x_3, x_4, x_14); -lean_ctor_set(x_12, 0, x_17); -return x_12; +uint8_t x_21; +x_21 = l_Lean_Expr_isApp(x_16); +if (x_21 == 0) +{ +lean_object* x_22; +lean_dec(x_16); +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +return x_22; } 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; -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 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__2; -x_21 = l_Lean_Expr_const___override(x_20, x_2); -x_22 = l_Lean_mkApp3(x_21, x_3, x_4, x_18); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_19); -return x_23; +lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_23 = l_Lean_Expr_appArg(x_16, lean_box(0)); +x_24 = l_Lean_Expr_appFnCleanup(x_16, lean_box(0)); +x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__6; +x_26 = l_Lean_Expr_isConstOf(x_24, x_25); +if (x_26 == 0) +{ +uint8_t x_27; +x_27 = l_Lean_Expr_isApp(x_24); +if (x_27 == 0) +{ +lean_object* x_28; +lean_dec(x_24); +lean_dec(x_23); +x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +return x_28; } +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_29 = l_Lean_Expr_appArg(x_24, lean_box(0)); +x_30 = l_Lean_Expr_appFnCleanup(x_24, lean_box(0)); +x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__8; +x_32 = l_Lean_Expr_isConstOf(x_30, x_31); +if (x_32 == 0) +{ +lean_object* x_33; uint8_t x_34; +x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__10; +x_34 = l_Lean_Expr_isConstOf(x_30, x_33); +if (x_34 == 0) +{ +uint8_t x_35; +x_35 = l_Lean_Expr_isApp(x_30); +if (x_35 == 0) +{ +lean_object* x_36; +lean_dec(x_30); +lean_dec(x_29); +lean_dec(x_23); +x_36 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +return x_36; } else { -uint8_t x_24; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_24 = !lean_is_exclusive(x_12); -if (x_24 == 0) +lean_object* x_37; uint8_t x_38; +x_37 = l_Lean_Expr_appFnCleanup(x_30, lean_box(0)); +x_38 = l_Lean_Expr_isApp(x_37); +if (x_38 == 0) { -return x_12; +lean_object* x_39; +lean_dec(x_37); +lean_dec(x_29); +lean_dec(x_23); +x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +return x_39; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_12, 0); -x_26 = lean_ctor_get(x_12, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_12); -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_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; +x_40 = l_Lean_Expr_appArg(x_37, lean_box(0)); +x_41 = l_Lean_Expr_appFnCleanup(x_37, lean_box(0)); +x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__13; +x_43 = l_Lean_Expr_isConstOf(x_41, x_42); +lean_dec(x_41); +if (x_43 == 0) +{ +lean_object* x_44; +lean_dec(x_40); +lean_dec(x_29); +lean_dec(x_23); +x_44 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +return x_44; +} +else +{ +lean_object* x_45; +x_45 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4(x_1, x_40, x_29, x_23, x_2, x_3, x_4, x_5, x_6, x_10); +return x_45; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("not", 3, 3); -return x_1; +lean_object* x_46; +lean_dec(x_30); +lean_dec(x_1); +x_46 = lean_apply_8(x_12, x_29, x_23, x_2, x_3, x_4, x_5, x_6, x_10); +return x_46; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__2() { -_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; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__1; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; +lean_object* x_47; +lean_dec(x_30); +lean_dec(x_1); +x_47 = lean_apply_8(x_11, x_29, x_23, x_2, x_3, x_4, x_5, x_6, x_10); +return x_47; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__3() { -_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_ReifiedBVLogical_of___lambda__8___closed__2; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; +lean_object* x_48; +lean_dec(x_24); +lean_dec(x_1); +x_48 = lean_apply_7(x_13, x_23, x_2, x_3, x_4, x_5, x_6, x_10); +return x_48; +} +} +} +else +{ +lean_object* x_49; lean_object* x_50; +lean_dec(x_16); +lean_dec(x_1); +x_49 = lean_box(0); +x_50 = lean_apply_7(x_15, x_49, x_2, x_3, x_4, x_5, x_6, x_10); +return x_50; +} +} +else +{ +lean_object* x_51; lean_object* x_52; +lean_dec(x_16); +lean_dec(x_1); +x_51 = lean_box(0); +x_52 = lean_apply_7(x_14, x_51, x_2, x_3, x_4, x_5, x_6, x_10); +return x_52; +} } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goOrAtom(lean_object* x_1, 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_2); lean_inc(x_1); -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go(x_1, x_2, x_3, x_4, x_5, x_6, x_7); if (lean_obj_tag(x_8) == 0) { lean_object* x_9; @@ -1723,701 +1790,785 @@ x_9 = lean_ctor_get(x_8, 0); lean_inc(x_9); if (lean_obj_tag(x_9) == 0) { -uint8_t x_10; -lean_dec(x_1); -x_10 = !lean_is_exclusive(x_8); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_8, 0); -lean_dec(x_11); -x_12 = lean_box(0); -lean_ctor_set(x_8, 0, x_12); -return x_8; -} -else -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_8, 1); -lean_inc(x_13); +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); lean_dec(x_8); -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; -} +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_boolAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +return x_11; } else { -uint8_t x_16; -x_16 = !lean_is_exclusive(x_9); -if (x_16 == 0) -{ -uint8_t x_17; -x_17 = !lean_is_exclusive(x_8); -if (x_17 == 0) +uint8_t x_12; +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_12 = !lean_is_exclusive(x_8); +if (x_12 == 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_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; -x_18 = lean_ctor_get(x_9, 0); -x_19 = lean_ctor_get(x_8, 0); -lean_dec(x_19); -x_20 = lean_ctor_get(x_18, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_18, 2); -lean_inc(x_21); -x_22 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_22, 0, x_20); -x_23 = lean_box(0); -x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__3; -x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -lean_inc(x_21); -x_26 = l_Lean_mkAppB(x_24, x_25, x_21); -x_27 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); -lean_closure_set(x_27, 0, x_21); -lean_inc(x_18); -x_28 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7), 10, 3); -lean_closure_set(x_28, 0, x_18); -lean_closure_set(x_28, 1, x_23); -lean_closure_set(x_28, 2, x_1); -x_29 = !lean_is_exclusive(x_18); -if (x_29 == 0) +lean_object* x_13; uint8_t x_14; +x_13 = lean_ctor_get(x_8, 0); +lean_dec(x_13); +x_14 = !lean_is_exclusive(x_9); +if (x_14 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_30 = lean_ctor_get(x_18, 2); -lean_dec(x_30); -x_31 = lean_ctor_get(x_18, 1); -lean_dec(x_31); -x_32 = lean_ctor_get(x_18, 0); -lean_dec(x_32); -x_33 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_33, 0, x_27); -lean_closure_set(x_33, 1, x_28); -lean_ctor_set(x_18, 2, x_26); -lean_ctor_set(x_18, 1, x_33); -lean_ctor_set(x_18, 0, x_22); return x_8; } else { -lean_object* x_34; lean_object* x_35; -lean_dec(x_18); -x_34 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_34, 0, x_27); -lean_closure_set(x_34, 1, x_28); -x_35 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_35, 0, x_22); -lean_ctor_set(x_35, 1, x_34); -lean_ctor_set(x_35, 2, x_26); -lean_ctor_set(x_9, 0, x_35); +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_9, 0); +lean_inc(x_15); +lean_dec(x_9); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_8, 0, x_16); return x_8; } } 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; lean_object* x_49; lean_object* x_50; -x_36 = lean_ctor_get(x_9, 0); -x_37 = lean_ctor_get(x_8, 1); -lean_inc(x_37); +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_8, 1); +lean_inc(x_17); lean_dec(x_8); -x_38 = lean_ctor_get(x_36, 0); -lean_inc(x_38); -x_39 = lean_ctor_get(x_36, 2); -lean_inc(x_39); -x_40 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_40, 0, x_38); -x_41 = lean_box(0); -x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__3; -x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -lean_inc(x_39); -x_44 = l_Lean_mkAppB(x_42, x_43, x_39); -x_45 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); -lean_closure_set(x_45, 0, x_39); -lean_inc(x_36); -x_46 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7), 10, 3); -lean_closure_set(x_46, 0, x_36); -lean_closure_set(x_46, 1, x_41); -lean_closure_set(x_46, 2, x_1); -if (lean_is_exclusive(x_36)) { - lean_ctor_release(x_36, 0); - lean_ctor_release(x_36, 1); - lean_ctor_release(x_36, 2); - x_47 = x_36; +x_18 = lean_ctor_get(x_9, 0); +lean_inc(x_18); +if (lean_is_exclusive(x_9)) { + lean_ctor_release(x_9, 0); + x_19 = x_9; } else { - lean_dec_ref(x_36); - x_47 = lean_box(0); + lean_dec_ref(x_9); + x_19 = lean_box(0); } -x_48 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_48, 0, x_45); -lean_closure_set(x_48, 1, x_46); -if (lean_is_scalar(x_47)) { - x_49 = lean_alloc_ctor(0, 3, 0); +if (lean_is_scalar(x_19)) { + x_20 = lean_alloc_ctor(1, 1, 0); } else { - x_49 = x_47; + x_20 = x_19; +} +lean_ctor_set(x_20, 0, 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_17); +return x_21; } -lean_ctor_set(x_49, 0, x_40); -lean_ctor_set(x_49, 1, x_48); -lean_ctor_set(x_49, 2, x_44); -lean_ctor_set(x_9, 0, x_49); -x_50 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_50, 0, x_9); -lean_ctor_set(x_50, 1, x_37); -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; 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_51 = lean_ctor_get(x_9, 0); -lean_inc(x_51); -lean_dec(x_9); -x_52 = lean_ctor_get(x_8, 1); -lean_inc(x_52); -if (lean_is_exclusive(x_8)) { - lean_ctor_release(x_8, 0); - lean_ctor_release(x_8, 1); - x_53 = x_8; -} else { - lean_dec_ref(x_8); - x_53 = lean_box(0); +uint8_t x_22; +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_22 = !lean_is_exclusive(x_8); +if (x_22 == 0) +{ +return x_8; } -x_54 = lean_ctor_get(x_51, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_51, 2); -lean_inc(x_55); -x_56 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_56, 0, x_54); -x_57 = lean_box(0); -x_58 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__3; -x_59 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -lean_inc(x_55); -x_60 = l_Lean_mkAppB(x_58, x_59, x_55); -x_61 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); -lean_closure_set(x_61, 0, x_55); -lean_inc(x_51); -x_62 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7), 10, 3); -lean_closure_set(x_62, 0, x_51); -lean_closure_set(x_62, 1, x_57); -lean_closure_set(x_62, 2, x_1); -if (lean_is_exclusive(x_51)) { - lean_ctor_release(x_51, 0); - lean_ctor_release(x_51, 1); - lean_ctor_release(x_51, 2); - x_63 = x_51; -} else { - lean_dec_ref(x_51); - x_63 = lean_box(0); +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_8, 0); +x_24 = lean_ctor_get(x_8, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_8); +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_64 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_64, 0, x_61); -lean_closure_set(x_64, 1, x_62); -if (lean_is_scalar(x_63)) { - x_65 = lean_alloc_ctor(0, 3, 0); -} else { - x_65 = x_63; } -lean_ctor_set(x_65, 0, x_56); -lean_ctor_set(x_65, 1, x_64); -lean_ctor_set(x_65, 2, x_60); -x_66 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_66, 0, x_65); -if (lean_is_scalar(x_53)) { - x_67 = lean_alloc_ctor(0, 2, 0); -} else { - x_67 = x_53; } -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_52); -return x_67; } +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___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; lean_object* x_18; lean_object* x_19; +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr(x_1, 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_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +x_18 = lean_ctor_get(x_2, 1); +lean_inc(x_18); +lean_dec(x_2); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_19 = lean_apply_6(x_18, x_9, x_10, x_11, x_12, x_13, x_17); +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); +x_22 = lean_ctor_get(x_3, 1); +lean_inc(x_22); +lean_dec(x_3); +x_23 = lean_apply_6(x_22, x_9, x_10, x_11, x_12, x_13, x_21); +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; +x_25 = lean_ctor_get(x_23, 0); +x_26 = l_Lean_Expr_const___override(x_4, x_5); +x_27 = l_Lean_mkApp6(x_26, x_6, x_7, x_8, x_16, x_20, x_25); +lean_ctor_set(x_23, 0, x_27); +return x_23; +} +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +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 = l_Lean_Expr_const___override(x_4, x_5); +x_31 = l_Lean_mkApp6(x_30, x_6, x_7, x_8, x_16, x_20, x_28); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_29); +return x_32; } } else { -uint8_t x_68; -lean_dec(x_1); -x_68 = !lean_is_exclusive(x_8); -if (x_68 == 0) +uint8_t x_33; +lean_dec(x_20); +lean_dec(x_16); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_33 = !lean_is_exclusive(x_23); +if (x_33 == 0) { -return x_8; +return x_23; } else { -lean_object* x_69; lean_object* x_70; lean_object* x_71; -x_69 = lean_ctor_get(x_8, 0); -x_70 = lean_ctor_get(x_8, 1); -lean_inc(x_70); -lean_inc(x_69); -lean_dec(x_8); -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_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_23, 0); +x_35 = lean_ctor_get(x_23, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_23); +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_37; +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_4); +lean_dec(x_3); +x_37 = !lean_is_exclusive(x_19); +if (x_37 == 0) +{ +return x_19; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__1() { -_start: +else { -uint8_t x_1; lean_object* x_2; -x_1 = 0; -x_2 = lean_alloc_ctor(1, 0, 1); -lean_ctor_set_uint8(x_2, 0, x_1); -return x_2; +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_19, 0); +x_39 = lean_ctor_get(x_19, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_19); +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; +} } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__2() { +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("const", 5, 5); +x_1 = lean_mk_string_unchecked("gate", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__2; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__1; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___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_ReifiedBVLogical_of___lambda__9___closed__3; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___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_ReifiedBVLogical_of___lambda__9___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__4() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("false", 5, 5); +x_1 = lean_mk_string_unchecked("Gate", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__5() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__5; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_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_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__9; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___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_ReifiedBVLogical_of___lambda__9___closed__6; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__5; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___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_ReifiedBVLogical_of___lambda__9___closed__4; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__7; -x_4 = l_Lean_mkAppB(x_1, x_2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___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) { -_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; -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__9; -x_9 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___spec__1___rarg___boxed), 7, 1); -lean_closure_set(x_9, 0, x_8); -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__1; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__8; -x_12 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_12, 0, x_10); -lean_ctor_set(x_12, 1, x_9); -lean_ctor_set(x_12, 2, x_11); -x_13 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_13, 0, 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_7); -return x_14; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__1() { -_start: -{ -uint8_t x_1; lean_object* x_2; -x_1 = 1; -x_2 = lean_alloc_ctor(1, 0, 1); -lean_ctor_set_uint8(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___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_ReifiedBVLogical_of___lambda__10___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__7() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__2; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_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_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__7; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___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_ReifiedBVLogical_of___lambda__10___closed__3; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___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_ReifiedBVLogical_of___lambda__10___closed__5() { -_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_ReifiedBVLogical_of___lambda__9___closed__4; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__4; -x_4 = l_Lean_mkAppB(x_1, x_2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__4; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___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, 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; -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__6; -x_9 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___spec__1___rarg___boxed), 7, 1); -lean_closure_set(x_9, 0, x_8); -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__1; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__5; -x_12 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_12, 0, x_10); -lean_ctor_set(x_12, 1, x_9); -lean_ctor_set(x_12, 2, x_11); -x_13 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_13, 0, 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_7); -return x_14; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5), 8, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6), 8, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8), 7, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___boxed), 7, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___boxed), 7, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___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_ReifiedBVLogical_of___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___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_ReifiedBVLogical_of___closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkRefl___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___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_ReifiedBVLogical_of___closed__9() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__9() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("BEq", 3, 3); -return x_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; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__12; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__10() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__9; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__11; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__9; +x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of(lean_object* x_1, lean_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_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(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) { _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; -lean_inc(x_1); -x_8 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_1, x_3, x_4, x_5, x_6, x_7); -x_9 = lean_ctor_get(x_8, 0); +lean_object* x_11; lean_inc(x_9); -x_10 = lean_ctor_get(x_8, 1); -lean_inc(x_10); -lean_dec(x_8); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__1; -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__2; -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__3; -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__4; -x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__5; -x_16 = l_Lean_Expr_cleanupAnnotations(x_9); -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__6; -x_18 = l_Lean_Expr_isConstOf(x_16, x_17); -if (x_18 == 0) +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_1); +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goOrAtom(x_1, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) { -lean_object* x_19; uint8_t x_20; -x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__3; -x_20 = l_Lean_Expr_isConstOf(x_16, x_19); -if (x_20 == 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_21; -x_21 = l_Lean_Expr_isApp(x_16); -if (x_21 == 0) +uint8_t 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_2); +lean_dec(x_1); +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 0) { -lean_object* x_22; -lean_dec(x_16); -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_22; +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; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; -x_23 = l_Lean_Expr_appArg(x_16, lean_box(0)); -x_24 = l_Lean_Expr_appFnCleanup(x_16, lean_box(0)); -x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__6; -x_26 = l_Lean_Expr_isConstOf(x_24, x_25); -if (x_26 == 0) +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; +} +} +else { -uint8_t x_27; -x_27 = l_Lean_Expr_isApp(x_24); -if (x_27 == 0) +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_11, 1); +lean_inc(x_19); +lean_dec(x_11); +x_20 = lean_ctor_get(x_12, 0); +lean_inc(x_20); +lean_dec(x_12); +lean_inc(x_2); +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goOrAtom(x_2, x_5, x_6, x_7, x_8, x_9, x_19); +if (lean_obj_tag(x_21) == 0) { -lean_object* x_28; +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_20); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +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); -lean_dec(x_23); -x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +x_25 = lean_box(0); +lean_ctor_set(x_21, 0, x_25); +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 = 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_26); return x_28; } +} else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_29 = l_Lean_Expr_appArg(x_24, lean_box(0)); -x_30 = l_Lean_Expr_appFnCleanup(x_24, lean_box(0)); -x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__7; -x_32 = l_Lean_Expr_isConstOf(x_30, x_31); -if (x_32 == 0) +uint8_t x_29; +x_29 = !lean_is_exclusive(x_21); +if (x_29 == 0) { -lean_object* x_33; uint8_t x_34; -x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__8; -x_34 = l_Lean_Expr_isConstOf(x_30, x_33); -if (x_34 == 0) +lean_object* x_30; uint8_t x_31; +x_30 = lean_ctor_get(x_21, 0); +lean_dec(x_30); +x_31 = !lean_is_exclusive(x_22); +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; +x_32 = lean_ctor_get(x_22, 0); +x_33 = lean_ctor_get(x_20, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_32, 0); +lean_inc(x_34); +x_35 = lean_alloc_ctor(3, 2, 1); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +lean_ctor_set_uint8(x_35, sizeof(void*)*2, x_3); +x_36 = lean_box(0); +x_37 = lean_ctor_get(x_20, 2); +lean_inc(x_37); +x_38 = lean_ctor_get(x_32, 2); +lean_inc(x_38); +lean_inc(x_37); +x_39 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); +lean_closure_set(x_39, 0, x_37); +lean_inc(x_38); +x_40 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___lambda__1), 14, 7); +lean_closure_set(x_40, 0, x_38); +lean_closure_set(x_40, 1, x_20); +lean_closure_set(x_40, 2, x_32); +lean_closure_set(x_40, 3, x_4); +lean_closure_set(x_40, 4, x_36); +lean_closure_set(x_40, 5, x_1); +lean_closure_set(x_40, 6, x_2); +x_41 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_41, 0, x_39); +lean_closure_set(x_41, 1, x_40); +switch (x_3) { +case 0: +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_44 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__6; +x_45 = l_Lean_mkApp4(x_42, x_43, x_44, x_37, x_38); +x_46 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_46, 0, x_35); +lean_ctor_set(x_46, 1, x_41); +lean_ctor_set(x_46, 2, x_45); +lean_ctor_set(x_22, 0, x_46); +return x_21; +} +case 1: +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_47 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +x_48 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_49 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__8; +x_50 = l_Lean_mkApp4(x_47, x_48, x_49, x_37, x_38); +x_51 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_51, 0, x_35); +lean_ctor_set(x_51, 1, x_41); +lean_ctor_set(x_51, 2, x_50); +lean_ctor_set(x_22, 0, x_51); +return x_21; +} +default: +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_52 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +x_53 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_54 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10; +x_55 = l_Lean_mkApp4(x_52, x_53, x_54, x_37, x_38); +x_56 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_56, 0, x_35); +lean_ctor_set(x_56, 1, x_41); +lean_ctor_set(x_56, 2, x_55); +lean_ctor_set(x_22, 0, x_56); +return x_21; +} +} +} +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; lean_object* x_66; +x_57 = lean_ctor_get(x_22, 0); +lean_inc(x_57); +lean_dec(x_22); +x_58 = lean_ctor_get(x_20, 0); +lean_inc(x_58); +x_59 = lean_ctor_get(x_57, 0); +lean_inc(x_59); +x_60 = lean_alloc_ctor(3, 2, 1); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_59); +lean_ctor_set_uint8(x_60, sizeof(void*)*2, x_3); +x_61 = lean_box(0); +x_62 = lean_ctor_get(x_20, 2); +lean_inc(x_62); +x_63 = lean_ctor_get(x_57, 2); +lean_inc(x_63); +lean_inc(x_62); +x_64 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); +lean_closure_set(x_64, 0, x_62); +lean_inc(x_63); +x_65 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___lambda__1), 14, 7); +lean_closure_set(x_65, 0, x_63); +lean_closure_set(x_65, 1, x_20); +lean_closure_set(x_65, 2, x_57); +lean_closure_set(x_65, 3, x_4); +lean_closure_set(x_65, 4, x_61); +lean_closure_set(x_65, 5, x_1); +lean_closure_set(x_65, 6, x_2); +x_66 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_66, 0, x_64); +lean_closure_set(x_66, 1, x_65); +switch (x_3) { +case 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; +x_67 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +x_68 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_69 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__6; +x_70 = l_Lean_mkApp4(x_67, x_68, x_69, x_62, x_63); +x_71 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_71, 0, x_60); +lean_ctor_set(x_71, 1, x_66); +lean_ctor_set(x_71, 2, x_70); +x_72 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_72, 0, x_71); +lean_ctor_set(x_21, 0, x_72); +return x_21; +} +case 1: { -uint8_t x_35; -x_35 = l_Lean_Expr_isApp(x_30); -if (x_35 == 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 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +x_74 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_75 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__8; +x_76 = l_Lean_mkApp4(x_73, x_74, x_75, x_62, x_63); +x_77 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_77, 0, x_60); +lean_ctor_set(x_77, 1, x_66); +lean_ctor_set(x_77, 2, x_76); +x_78 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_78, 0, x_77); +lean_ctor_set(x_21, 0, x_78); +return x_21; +} +default: { -lean_object* x_36; -lean_dec(x_30); -lean_dec(x_29); -lean_dec(x_23); -x_36 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_36; +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_79 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +x_80 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_81 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10; +x_82 = l_Lean_mkApp4(x_79, x_80, x_81, x_62, x_63); +x_83 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_83, 0, x_60); +lean_ctor_set(x_83, 1, x_66); +lean_ctor_set(x_83, 2, x_82); +x_84 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_84, 0, x_83); +lean_ctor_set(x_21, 0, x_84); +return x_21; +} +} +} } else { -lean_object* x_37; uint8_t x_38; -x_37 = l_Lean_Expr_appFnCleanup(x_30, lean_box(0)); -x_38 = l_Lean_Expr_isApp(x_37); -if (x_38 == 0) -{ -lean_object* x_39; -lean_dec(x_37); -lean_dec(x_29); -lean_dec(x_23); -x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_39; +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_85 = lean_ctor_get(x_21, 1); +lean_inc(x_85); +lean_dec(x_21); +x_86 = lean_ctor_get(x_22, 0); +lean_inc(x_86); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + x_87 = x_22; +} else { + lean_dec_ref(x_22); + x_87 = lean_box(0); } -else +x_88 = lean_ctor_get(x_20, 0); +lean_inc(x_88); +x_89 = lean_ctor_get(x_86, 0); +lean_inc(x_89); +x_90 = lean_alloc_ctor(3, 2, 1); +lean_ctor_set(x_90, 0, x_88); +lean_ctor_set(x_90, 1, x_89); +lean_ctor_set_uint8(x_90, sizeof(void*)*2, x_3); +x_91 = lean_box(0); +x_92 = lean_ctor_get(x_20, 2); +lean_inc(x_92); +x_93 = lean_ctor_get(x_86, 2); +lean_inc(x_93); +lean_inc(x_92); +x_94 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___boxed), 7, 1); +lean_closure_set(x_94, 0, x_92); +lean_inc(x_93); +x_95 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___lambda__1), 14, 7); +lean_closure_set(x_95, 0, x_93); +lean_closure_set(x_95, 1, x_20); +lean_closure_set(x_95, 2, x_86); +lean_closure_set(x_95, 3, x_4); +lean_closure_set(x_95, 4, x_91); +lean_closure_set(x_95, 5, x_1); +lean_closure_set(x_95, 6, x_2); +x_96 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_96, 0, x_94); +lean_closure_set(x_96, 1, x_95); +switch (x_3) { +case 0: { -lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; -x_40 = l_Lean_Expr_appArg(x_37, lean_box(0)); -x_41 = l_Lean_Expr_appFnCleanup(x_37, lean_box(0)); -x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__10; -x_43 = l_Lean_Expr_isConstOf(x_41, x_42); -lean_dec(x_41); -if (x_43 == 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; +x_97 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +x_98 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_99 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__6; +x_100 = l_Lean_mkApp4(x_97, x_98, x_99, x_92, x_93); +x_101 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_101, 0, x_90); +lean_ctor_set(x_101, 1, x_96); +lean_ctor_set(x_101, 2, x_100); +if (lean_is_scalar(x_87)) { + x_102 = lean_alloc_ctor(1, 1, 0); +} else { + x_102 = x_87; +} +lean_ctor_set(x_102, 0, x_101); +x_103 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_103, 0, x_102); +lean_ctor_set(x_103, 1, x_85); +return x_103; +} +case 1: { -lean_object* x_44; -lean_dec(x_40); -lean_dec(x_29); -lean_dec(x_23); -x_44 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred(x_1, x_2, x_3, x_4, x_5, x_6, x_10); -return x_44; +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 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +x_105 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_106 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__8; +x_107 = l_Lean_mkApp4(x_104, x_105, x_106, x_92, x_93); +x_108 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_108, 0, x_90); +lean_ctor_set(x_108, 1, x_96); +lean_ctor_set(x_108, 2, x_107); +if (lean_is_scalar(x_87)) { + x_109 = lean_alloc_ctor(1, 1, 0); +} else { + x_109 = x_87; } -else +lean_ctor_set(x_109, 0, x_108); +x_110 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_110, 0, x_109); +lean_ctor_set(x_110, 1, x_85); +return x_110; +} +default: { -lean_object* x_45; -x_45 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4(x_1, x_40, x_29, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_45; +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_111 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__3; +x_112 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7; +x_113 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10; +x_114 = l_Lean_mkApp4(x_111, x_112, x_113, x_92, x_93); +x_115 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_115, 0, x_90); +lean_ctor_set(x_115, 1, x_96); +lean_ctor_set(x_115, 2, x_114); +if (lean_is_scalar(x_87)) { + x_116 = lean_alloc_ctor(1, 1, 0); +} else { + x_116 = x_87; } +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_85); +return x_117; } } } -else -{ -lean_object* x_46; -lean_dec(x_30); -lean_dec(x_1); -x_46 = lean_apply_8(x_12, x_29, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_46; } } else { -lean_object* x_47; -lean_dec(x_30); +uint8_t x_118; +lean_dec(x_20); +lean_dec(x_4); +lean_dec(x_2); lean_dec(x_1); -x_47 = lean_apply_8(x_11, x_29, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_47; -} -} +x_118 = !lean_is_exclusive(x_21); +if (x_118 == 0) +{ +return x_21; } else { -lean_object* x_48; -lean_dec(x_24); -lean_dec(x_1); -x_48 = lean_apply_7(x_13, x_23, x_2, x_3, x_4, x_5, x_6, x_10); -return x_48; +lean_object* x_119; lean_object* x_120; lean_object* x_121; +x_119 = lean_ctor_get(x_21, 0); +x_120 = lean_ctor_get(x_21, 1); +lean_inc(x_120); +lean_inc(x_119); +lean_dec(x_21); +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; +} } } } else { -lean_object* x_49; lean_object* x_50; -lean_dec(x_16); +uint8_t x_122; +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_49 = lean_box(0); -x_50 = lean_apply_7(x_15, x_49, x_2, x_3, x_4, x_5, x_6, x_10); -return x_50; -} +x_122 = !lean_is_exclusive(x_11); +if (x_122 == 0) +{ +return x_11; } else { -lean_object* x_51; lean_object* x_52; -lean_dec(x_16); -lean_dec(x_1); -x_51 = lean_box(0); -x_52 = lean_apply_7(x_14, x_51, x_2, x_3, x_4, x_5, x_6, x_10); -return x_52; -} +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_ReifiedBVLogical_of_gateReflection___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, 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_3); -lean_dec(x_3); -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(x_1, x_2, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_12; } } -LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___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_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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) { _start: { lean_object* x_8; -x_8 = l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_ReaderT_pure___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___spec__1___rarg(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); @@ -2426,29 +2577,29 @@ lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_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) { _start: { lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_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: { lean_object* x_10; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_3); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_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) { _start: { lean_object* x_8; -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__3(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); @@ -2458,11 +2609,11 @@ lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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) { _start: { lean_object* x_8; -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9(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); @@ -2472,11 +2623,11 @@ lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___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) { _start: { lean_object* x_8; -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10(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); @@ -2486,6 +2637,24 @@ lean_dec(x_1); return x_8; } } +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, 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_3); +lean_dec(x_3); +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection(x_1, x_2, x_11, x_4, 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_ReifiedBVLogical_of(lean_object* x_1, 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_ReifiedBVLogical_of_goOrAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +return x_8; +} +} lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_BVDecide_ReifiedBVPred(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_BVDecide_ReifiedBVLogical(uint8_t builtin, lean_object* w) { @@ -2533,20 +2702,106 @@ l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__6 = _ lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__6); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__7(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkEvalExpr___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goPred___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_ofPred___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__2___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__4___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__5___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__6___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__7___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__8___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__9___closed__9); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___lambda__10___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__9); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__10(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__10); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__11 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__11(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__11); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__12 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__12(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__12); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__13 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__13(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_go___closed__13); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__1); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__2(); @@ -2567,92 +2822,6 @@ l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__9); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__10); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__11 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__11(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__11); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__12 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__12(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__12); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__13 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__13(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_gateReflection___closed__13); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__2___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__4___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__5___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__6___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__7___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__8___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__8); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__9(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__9___closed__9); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___lambda__10___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__8); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__9(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__9); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__10(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of___closed__10); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVPred.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVPred.c index 546ecc9e5684..145557895eb5 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVPred.c +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/ReifiedBVPred.c @@ -14,219 +14,93 @@ extern "C" { #endif lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3(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_ReifiedBVPred_of___lambda__8(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_ReifiedBVPred_of_binaryReflection___closed__12; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__8; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__6; lean_object* l_Lean_Meta_getNatValue_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__9; lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkApp7(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_ReifiedBVPred_of___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2; uint8_t l_Lean_Expr_isApp(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__8; lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___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_cleanupAnnotations(lean_object*); 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_ReifiedBVPred_of___lambda__6(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_ReifiedBVPred_of_binaryReflection___closed__13; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___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_ReifiedBVPred_of___lambda__9___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__8; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection(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_ReifiedBVPred_of___lambda__8___closed__5; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__3; lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___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_ReifiedBVPred_of___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__8; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__7; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__2; lean_object* l_Lean_Expr_appArg(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__7; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2(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_ReifiedBVPred_of___lambda__8___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_ReifiedBVPred_of___lambda__9___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__5; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_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*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom(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_ReifiedBVPred_of___lambda__9(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_ReifiedBVPred_of_binaryReflection___closed__9; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__5___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, 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*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_app___override(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_Name_mkStr2(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__2; uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2(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*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__11; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__3; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__14; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4(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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___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_ReifiedBVPred_of___lambda__7___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, 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_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__7; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___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_ReifiedBVPred_of_binaryReflection___closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__6; lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr(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_ReifiedBVPred_of_binaryReflection___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); -lean_inc(x_12); -lean_inc(x_11); -x_17 = lean_apply_6(x_1, 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; -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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr(x_2, x_3, 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 = lean_ctor_get(x_4, 2); -lean_inc(x_23); -lean_dec(x_4); -x_24 = lean_apply_6(x_23, x_11, x_12, x_13, x_14, x_15, x_22); -if (lean_obj_tag(x_24) == 0) -{ -uint8_t x_25; -x_25 = !lean_is_exclusive(x_24); -if (x_25 == 0) -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_24, 0); -x_27 = l_Lean_Expr_const___override(x_5, x_6); -x_28 = l_Lean_mkApp7(x_27, x_7, x_8, x_9, x_10, x_21, x_18, x_26); -lean_ctor_set(x_24, 0, x_28); -return x_24; -} -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_24, 0); -x_30 = lean_ctor_get(x_24, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_24); -x_31 = l_Lean_Expr_const___override(x_5, x_6); -x_32 = l_Lean_mkApp7(x_31, x_7, x_8, x_9, x_10, x_21, x_18, x_29); -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; -} -} -else -{ -uint8_t x_34; -lean_dec(x_21); -lean_dec(x_18); -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_34 = !lean_is_exclusive(x_24); -if (x_34 == 0) -{ -return x_24; -} -else -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_24, 0); -x_36 = lean_ctor_get(x_24, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_24); -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_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_38 = !lean_is_exclusive(x_17); -if (x_38 == 0) -{ -return x_17; -} -else -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_17, 0); -x_40 = lean_ctor_get(x_17, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_17); -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; -} -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1() { _start: { lean_object* x_1; @@ -234,7 +108,7 @@ x_1 = lean_mk_string_unchecked("Std", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2() { _start: { lean_object* x_1; @@ -242,7 +116,7 @@ x_1 = lean_mk_string_unchecked("Tactic", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3() { _start: { lean_object* x_1; @@ -250,1601 +124,1750 @@ x_1 = lean_mk_string_unchecked("BVDecide", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__4() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("BVPred", 6, 6); +x_1 = lean_mk_string_unchecked("Reflect", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("bin", 3, 3); +x_1 = lean_mk_string_unchecked("BitVec", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___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; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__5; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ofBool_congr", 12, 12); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___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_ReifiedBVPred_of_binaryReflection___closed__6; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_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; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___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_ReifiedBVPred_of_binaryReflection___closed__8() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___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_1; -x_1 = lean_mk_string_unchecked("BVBinPred", 9, 9); -return x_1; +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_1, 2); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_apply_6(x_11, 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; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_12, 0); +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__7; +x_16 = l_Lean_Expr_const___override(x_15, x_2); +x_17 = l_Lean_mkApp3(x_16, x_3, x_4, x_14); +lean_ctor_set(x_12, 0, x_17); +return x_12; +} +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; +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 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__7; +x_21 = l_Lean_Expr_const___override(x_20, x_2); +x_22 = l_Lean_mkApp3(x_21, x_3, x_4, x_18); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_19); +return x_23; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__9() { +else +{ +uint8_t x_24; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_24 = !lean_is_exclusive(x_12); +if (x_24 == 0) +{ +return x_12; +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_12, 0); +x_26 = lean_ctor_get(x_12, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_12); +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; +} +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("eq", 2, 2); +x_1 = lean_mk_string_unchecked("ofBool", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__8; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__9; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___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_ReifiedBVPred_of_binaryReflection___closed__11() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___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_ReifiedBVPred_of_binaryReflection___closed__12() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__4() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("ult", 3, 3); +x_1 = lean_mk_string_unchecked("BVPred", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("getLsbD", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__13() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___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; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__8; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__12; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__5; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__14() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___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_ReifiedBVPred_of_binaryReflection___closed__13; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___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_ReifiedBVPred_of_binaryReflection(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) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__8() { _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_1); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(x_1, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) +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_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__9() { +_start: { -lean_object* x_12; -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -if (lean_obj_tag(x_12) == 0) +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; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___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: { -uint8_t 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_2); -lean_dec(x_1); -x_13 = !lean_is_exclusive(x_11); -if (x_13 == 0) +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = lean_box(0); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__3; +lean_inc(x_1); +x_11 = l_Lean_Expr_app___override(x_10, x_1); +x_12 = lean_unsigned_to_nat(1u); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom(x_11, x_12, x_3, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(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 = lean_box(0); -lean_ctor_set(x_11, 0, x_15); -return x_11; +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_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; +x_15 = lean_ctor_get(x_13, 0); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +x_18 = lean_ctor_get(x_15, 3); +lean_inc(x_18); +x_19 = lean_unsigned_to_nat(0u); +lean_inc(x_16); +x_20 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_20, 0, x_16); +lean_ctor_set(x_20, 1, x_17); +lean_ctor_set(x_20, 2, x_19); +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__7; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__8; +x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__9; +lean_inc(x_18); +x_24 = l_Lean_mkApp3(x_21, x_22, x_18, x_23); +x_25 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_25, 0, x_16); +lean_closure_set(x_25, 1, x_18); +x_26 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1), 10, 3); +lean_closure_set(x_26, 0, x_15); +lean_closure_set(x_26, 1, x_9); +lean_closure_set(x_26, 2, x_1); +x_27 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_27, 0, x_25); +lean_closure_set(x_27, 1, x_26); +x_28 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_28, 0, x_20); +lean_ctor_set(x_28, 1, x_27); +lean_ctor_set(x_28, 2, x_24); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_13, 0, x_29); +return x_13; } 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_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; +x_30 = lean_ctor_get(x_13, 0); +x_31 = lean_ctor_get(x_13, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_13); +x_32 = lean_ctor_get(x_30, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_30, 1); +lean_inc(x_33); +x_34 = lean_ctor_get(x_30, 3); +lean_inc(x_34); +x_35 = lean_unsigned_to_nat(0u); +lean_inc(x_32); +x_36 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_36, 0, x_32); +lean_ctor_set(x_36, 1, x_33); +lean_ctor_set(x_36, 2, x_35); +x_37 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__7; +x_38 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__8; +x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__9; +lean_inc(x_34); +x_40 = l_Lean_mkApp3(x_37, x_38, x_34, x_39); +x_41 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_41, 0, x_32); +lean_closure_set(x_41, 1, x_34); +x_42 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1), 10, 3); +lean_closure_set(x_42, 0, x_30); +lean_closure_set(x_42, 1, x_9); +lean_closure_set(x_42, 2, x_1); +x_43 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_43, 0, x_41); +lean_closure_set(x_43, 1, x_42); +x_44 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_44, 0, x_36); +lean_ctor_set(x_44, 1, x_43); +lean_ctor_set(x_44, 2, x_40); +x_45 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_45, 0, 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_31); +return x_46; } } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_11, 1); -lean_inc(x_19); -lean_dec(x_11); -x_20 = lean_ctor_get(x_12, 0); -lean_inc(x_20); -lean_dec(x_12); -lean_inc(x_2); -x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(x_2, x_5, x_6, x_7, x_8, x_9, x_19); -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_20); -lean_dec(x_4); -lean_dec(x_2); +uint8_t x_47; lean_dec(x_1); -x_23 = !lean_is_exclusive(x_21); -if (x_23 == 0) +x_47 = !lean_is_exclusive(x_13); +if (x_47 == 0) { -lean_object* x_24; lean_object* x_25; -x_24 = lean_ctor_get(x_21, 0); -lean_dec(x_24); -x_25 = lean_box(0); -lean_ctor_set(x_21, 0, x_25); -return x_21; +return x_13; } 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 = 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_26); -return x_28; +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_ctor_get(x_13, 0); +x_49 = lean_ctor_get(x_13, 1); +lean_inc(x_49); +lean_inc(x_48); +lean_dec(x_13); +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 +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___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) { +_start: { -uint8_t x_29; -x_29 = !lean_is_exclusive(x_21); -if (x_29 == 0) +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_ReifiedBVPred_boolAtom___closed__1() { +_start: { -lean_object* x_30; uint8_t x_31; -x_30 = lean_ctor_get(x_21, 0); -lean_dec(x_30); -x_31 = !lean_is_exclusive(x_22); -if (x_31 == 0) +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__3___boxed), 7, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__2() { +_start: { -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; -x_32 = lean_ctor_get(x_22, 0); -x_33 = lean_ctor_get(x_20, 0); -lean_inc(x_33); -x_34 = lean_ctor_get(x_20, 1); -lean_inc(x_34); -x_35 = lean_ctor_get(x_20, 2); -lean_inc(x_35); -x_36 = lean_ctor_get(x_20, 3); -lean_inc(x_36); -lean_dec(x_20); -x_37 = lean_ctor_get(x_32, 0); -lean_inc(x_37); -x_38 = lean_nat_dec_eq(x_33, x_37); -if (x_38 == 0) +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_ReifiedBVPred_boolAtom___closed__3() { +_start: { -lean_object* x_39; -lean_dec(x_37); -lean_dec(x_36); -lean_dec(x_35); -lean_dec(x_34); -lean_dec(x_33); -lean_free_object(x_22); -lean_dec(x_32); -lean_dec(x_4); -lean_dec(x_2); +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_ReifiedBVPred_boolAtom___closed__2; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom(lean_object* x_1, 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 = lean_infer_type(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; uint8_t x_14; +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_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__1; +x_12 = l_Lean_Expr_cleanupAnnotations(x_9); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___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_1); -x_39 = lean_box(0); -lean_ctor_set(x_21, 0, x_39); -return x_21; +x_15 = lean_box(0); +x_16 = lean_apply_7(x_11, x_15, x_2, x_3, x_4, x_5, x_6, x_10); +return x_16; } 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; -x_40 = lean_ctor_get(x_32, 1); -lean_inc(x_40); -lean_inc(x_33); -x_41 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_41, 0, x_33); -lean_ctor_set(x_41, 1, x_34); -lean_ctor_set(x_41, 2, x_40); -lean_ctor_set_uint8(x_41, sizeof(void*)*3, x_3); -x_42 = lean_box(0); -lean_inc(x_33); -x_43 = l_Lean_mkNatLit(x_33); -x_44 = lean_ctor_get(x_32, 3); -lean_inc(x_44); -lean_inc(x_36); -x_45 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_45, 0, x_33); -lean_closure_set(x_45, 1, x_36); -lean_inc(x_43); -lean_inc(x_44); -x_46 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___lambda__1), 16, 9); -lean_closure_set(x_46, 0, x_35); -lean_closure_set(x_46, 1, x_37); -lean_closure_set(x_46, 2, x_44); -lean_closure_set(x_46, 3, x_32); -lean_closure_set(x_46, 4, x_4); -lean_closure_set(x_46, 5, x_42); -lean_closure_set(x_46, 6, x_43); -lean_closure_set(x_46, 7, x_1); -lean_closure_set(x_46, 8, x_2); -x_47 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_47, 0, x_45); -lean_closure_set(x_47, 1, x_46); -if (x_3 == 0) +lean_object* x_17; lean_object* x_18; +x_17 = lean_box(0); +x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2(x_1, x_17, x_2, x_3, x_4, x_5, x_6, x_10); +return x_18; +} +} +else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_48 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; -x_49 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__11; -x_50 = l_Lean_mkApp4(x_48, x_43, x_36, x_49, x_44); -x_51 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_51, 0, x_41); -lean_ctor_set(x_51, 1, x_47); -lean_ctor_set(x_51, 2, x_50); -lean_ctor_set(x_22, 0, x_51); -return x_21; +uint8_t 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_19 = !lean_is_exclusive(x_8); +if (x_19 == 0) +{ +return x_8; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_52 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; -x_53 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__14; -x_54 = l_Lean_mkApp4(x_52, x_43, x_36, x_53, x_44); -x_55 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_55, 0, x_41); -lean_ctor_set(x_55, 1, x_47); -lean_ctor_set(x_55, 2, x_54); -lean_ctor_set(x_22, 0, x_55); -return x_21; +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_8, 0); +x_21 = lean_ctor_get(x_8, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_8); +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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___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_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; -x_56 = lean_ctor_get(x_22, 0); -lean_inc(x_56); -lean_dec(x_22); -x_57 = lean_ctor_get(x_20, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_20, 1); -lean_inc(x_58); -x_59 = lean_ctor_get(x_20, 2); -lean_inc(x_59); -x_60 = lean_ctor_get(x_20, 3); -lean_inc(x_60); -lean_dec(x_20); -x_61 = lean_ctor_get(x_56, 0); -lean_inc(x_61); -x_62 = lean_nat_dec_eq(x_57, x_61); -if (x_62 == 0) +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2(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_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___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) { +_start: { -lean_object* 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_object* x_8; +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__3(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_63 = lean_box(0); -lean_ctor_set(x_21, 0, x_63); -return x_21; +return x_8; } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___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_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_56, 1); -lean_inc(x_64); -lean_inc(x_57); -x_65 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_65, 0, x_57); -lean_ctor_set(x_65, 1, x_58); -lean_ctor_set(x_65, 2, x_64); -lean_ctor_set_uint8(x_65, sizeof(void*)*3, x_3); -x_66 = lean_box(0); -lean_inc(x_57); -x_67 = l_Lean_mkNatLit(x_57); -x_68 = lean_ctor_get(x_56, 3); -lean_inc(x_68); -lean_inc(x_60); -x_69 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_69, 0, x_57); -lean_closure_set(x_69, 1, x_60); -lean_inc(x_67); -lean_inc(x_68); -x_70 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___lambda__1), 16, 9); -lean_closure_set(x_70, 0, x_59); -lean_closure_set(x_70, 1, x_61); -lean_closure_set(x_70, 2, x_68); -lean_closure_set(x_70, 3, x_56); -lean_closure_set(x_70, 4, x_4); -lean_closure_set(x_70, 5, x_66); -lean_closure_set(x_70, 6, x_67); -lean_closure_set(x_70, 7, x_1); -lean_closure_set(x_70, 8, x_2); -x_71 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_71, 0, x_69); -lean_closure_set(x_71, 1, x_70); -if (x_3 == 0) +lean_object* x_17; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +x_17 = lean_apply_6(x_1, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_72 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; -x_73 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__11; -x_74 = l_Lean_mkApp4(x_72, x_67, x_60, x_73, x_68); -x_75 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_75, 0, x_65); -lean_ctor_set(x_75, 1, x_71); -lean_ctor_set(x_75, 2, x_74); -x_76 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_76, 0, x_75); -lean_ctor_set(x_21, 0, x_76); -return x_21; +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_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_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr(x_2, x_3, 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 = lean_ctor_get(x_4, 2); +lean_inc(x_23); +lean_dec(x_4); +x_24 = lean_apply_6(x_23, x_11, x_12, x_13, x_14, x_15, x_22); +if (lean_obj_tag(x_24) == 0) +{ +uint8_t x_25; +x_25 = !lean_is_exclusive(x_24); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_24, 0); +x_27 = l_Lean_Expr_const___override(x_5, x_6); +x_28 = l_Lean_mkApp7(x_27, x_7, x_8, x_9, x_10, x_21, x_18, x_26); +lean_ctor_set(x_24, 0, x_28); +return x_24; } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_77 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; -x_78 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__14; -x_79 = l_Lean_mkApp4(x_77, x_67, x_60, x_78, x_68); -x_80 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_80, 0, x_65); -lean_ctor_set(x_80, 1, x_71); -lean_ctor_set(x_80, 2, x_79); -x_81 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_81, 0, x_80); -lean_ctor_set(x_21, 0, x_81); -return x_21; -} -} +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_24, 0); +x_30 = lean_ctor_get(x_24, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_24); +x_31 = l_Lean_Expr_const___override(x_5, x_6); +x_32 = l_Lean_mkApp7(x_31, x_7, x_8, x_9, x_10, x_21, x_18, x_29); +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; } } 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; uint8_t x_90; -x_82 = lean_ctor_get(x_21, 1); -lean_inc(x_82); +uint8_t x_34; lean_dec(x_21); -x_83 = lean_ctor_get(x_22, 0); -lean_inc(x_83); -if (lean_is_exclusive(x_22)) { - lean_ctor_release(x_22, 0); - x_84 = x_22; -} else { - lean_dec_ref(x_22); - x_84 = lean_box(0); +lean_dec(x_18); +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_34 = !lean_is_exclusive(x_24); +if (x_34 == 0) +{ +return x_24; } -x_85 = lean_ctor_get(x_20, 0); -lean_inc(x_85); -x_86 = lean_ctor_get(x_20, 1); -lean_inc(x_86); -x_87 = lean_ctor_get(x_20, 2); -lean_inc(x_87); -x_88 = lean_ctor_get(x_20, 3); -lean_inc(x_88); -lean_dec(x_20); -x_89 = lean_ctor_get(x_83, 0); -lean_inc(x_89); -x_90 = lean_nat_dec_eq(x_85, x_89); -if (x_90 == 0) +else { -lean_object* x_91; lean_object* x_92; -lean_dec(x_89); -lean_dec(x_88); -lean_dec(x_87); -lean_dec(x_86); -lean_dec(x_85); -lean_dec(x_84); -lean_dec(x_83); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -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_82); -return x_92; -} -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; -x_93 = lean_ctor_get(x_83, 1); -lean_inc(x_93); -lean_inc(x_85); -x_94 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_94, 0, x_85); -lean_ctor_set(x_94, 1, x_86); -lean_ctor_set(x_94, 2, x_93); -lean_ctor_set_uint8(x_94, sizeof(void*)*3, x_3); -x_95 = lean_box(0); -lean_inc(x_85); -x_96 = l_Lean_mkNatLit(x_85); -x_97 = lean_ctor_get(x_83, 3); -lean_inc(x_97); -lean_inc(x_88); -x_98 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_98, 0, x_85); -lean_closure_set(x_98, 1, x_88); -lean_inc(x_96); -lean_inc(x_97); -x_99 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___lambda__1), 16, 9); -lean_closure_set(x_99, 0, x_87); -lean_closure_set(x_99, 1, x_89); -lean_closure_set(x_99, 2, x_97); -lean_closure_set(x_99, 3, x_83); -lean_closure_set(x_99, 4, x_4); -lean_closure_set(x_99, 5, x_95); -lean_closure_set(x_99, 6, x_96); -lean_closure_set(x_99, 7, x_1); -lean_closure_set(x_99, 8, x_2); -x_100 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_100, 0, x_98); -lean_closure_set(x_100, 1, x_99); -if (x_3 == 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; -x_101 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; -x_102 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__11; -x_103 = l_Lean_mkApp4(x_101, x_96, x_88, x_102, x_97); -x_104 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_104, 0, x_94); -lean_ctor_set(x_104, 1, x_100); -lean_ctor_set(x_104, 2, x_103); -if (lean_is_scalar(x_84)) { - x_105 = lean_alloc_ctor(1, 1, 0); -} else { - x_105 = x_84; -} -lean_ctor_set(x_105, 0, x_104); -x_106 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_106, 0, x_105); -lean_ctor_set(x_106, 1, x_82); -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; -x_107 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; -x_108 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__14; -x_109 = l_Lean_mkApp4(x_107, x_96, x_88, x_108, x_97); -x_110 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_110, 0, x_94); -lean_ctor_set(x_110, 1, x_100); -lean_ctor_set(x_110, 2, x_109); -if (lean_is_scalar(x_84)) { - x_111 = lean_alloc_ctor(1, 1, 0); -} else { - x_111 = x_84; -} -lean_ctor_set(x_111, 0, x_110); -x_112 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_112, 0, x_111); -lean_ctor_set(x_112, 1, x_82); -return x_112; -} -} -} -} -} -else -{ -uint8_t x_113; -lean_dec(x_20); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_113 = !lean_is_exclusive(x_21); -if (x_113 == 0) -{ -return x_21; -} -else -{ -lean_object* x_114; lean_object* x_115; lean_object* x_116; -x_114 = lean_ctor_get(x_21, 0); -x_115 = lean_ctor_get(x_21, 1); -lean_inc(x_115); -lean_inc(x_114); -lean_dec(x_21); -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_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_24, 0); +x_36 = lean_ctor_get(x_24, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_24); +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_117; +uint8_t x_38; +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_117 = !lean_is_exclusive(x_11); -if (x_117 == 0) +x_38 = !lean_is_exclusive(x_17); +if (x_38 == 0) { -return x_11; +return x_17; } else { -lean_object* x_118; lean_object* x_119; lean_object* x_120; -x_118 = lean_ctor_get(x_11, 0); -x_119 = lean_ctor_get(x_11, 1); -lean_inc(x_119); -lean_inc(x_118); -lean_dec(x_11); -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_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_17, 0); +x_40 = lean_ctor_get(x_17, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_17); +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_ReifiedBVPred_of_binaryReflection___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, 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_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1() { _start: { -uint8_t x_11; lean_object* x_12; -x_11 = lean_unbox(x_3); -lean_dec(x_3); -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection(x_1, x_2, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_12; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("bin", 3, 3); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Reflect", 7, 7); -return x_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; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; +} } +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___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_ReifiedBVPred_of_binaryReflection___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_ReifiedBVPred_of___lambda__1___closed__2() { +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__4() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("BitVec", 6, 6); +x_1 = lean_mk_string_unchecked("BVBinPred", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__5() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("getLsbD_congr", 13, 13); +x_1 = lean_mk_string_unchecked("eq", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___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_ReifiedBVPred_of_binaryReflection___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___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; +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_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__5; +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_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___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) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7() { _start: { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_1, 2); -lean_inc(x_13); -lean_dec(x_1); -x_14 = lean_apply_6(x_13, x_7, x_8, x_9, x_10, x_11, x_12); -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_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__6; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__8() { +_start: { -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 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__4; -x_18 = l_Lean_Expr_const___override(x_17, x_2); -x_19 = l_Lean_mkApp5(x_18, x_3, x_4, x_5, x_6, x_16); -lean_ctor_set(x_14, 0, x_19); -return x_14; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ult", 3, 3); +return x_1; } -else +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__9() { +_start: { -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_14, 0); -x_21 = lean_ctor_get(x_14, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_14); -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__4; -x_23 = l_Lean_Expr_const___override(x_22, x_2); -x_24 = l_Lean_mkApp5(x_23, x_3, x_4, x_5, x_6, x_20); -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; +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_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__8; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; } } -else -{ -uint8_t x_26; -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_14); -if (x_26 == 0) -{ -return x_14; -} -else -{ -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_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 lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("getLsbD", 7, 7); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__1; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__3() { -_start: +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___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_ReifiedBVPred_of___lambda__2___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__9; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection(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) { _start: { -lean_object* x_9; +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_1); -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of(x_1, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_9) == 0) +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_1, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 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_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_11; +uint8_t 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_2); lean_dec(x_1); -x_11 = !lean_is_exclusive(x_9); -if (x_11 == 0) +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 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; +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; } 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; +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; } } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_9, 1); -lean_inc(x_17); -lean_dec(x_9); -x_18 = lean_ctor_get(x_10, 0); -lean_inc(x_18); -lean_dec(x_10); -x_19 = l_Lean_Meta_getNatValue_x3f(x_2, x_4, x_5, x_6, x_7, x_17); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; -x_20 = lean_ctor_get(x_19, 0); +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_11, 1); +lean_inc(x_19); +lean_dec(x_11); +x_20 = lean_ctor_get(x_12, 0); lean_inc(x_20); -if (lean_obj_tag(x_20) == 0) +lean_dec(x_12); +lean_inc(x_2); +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_goOrAtom(x_2, x_5, x_6, x_7, x_8, x_9, x_19); +if (lean_obj_tag(x_21) == 0) { -uint8_t x_21; -lean_dec(x_18); +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_20); +lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_21 = !lean_is_exclusive(x_19); -if (x_21 == 0) +x_23 = !lean_is_exclusive(x_21); +if (x_23 == 0) { -lean_object* x_22; lean_object* x_23; -x_22 = lean_ctor_get(x_19, 0); -lean_dec(x_22); -x_23 = lean_box(0); -lean_ctor_set(x_19, 0, x_23); -return x_19; +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_21, 0); +lean_dec(x_24); +x_25 = lean_box(0); +lean_ctor_set(x_21, 0, x_25); +return x_21; } 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 = 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_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 = 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_26); +return x_28; } } else { -uint8_t x_27; -x_27 = !lean_is_exclusive(x_19); -if (x_27 == 0) -{ -lean_object* x_28; uint8_t x_29; -x_28 = lean_ctor_get(x_19, 0); -lean_dec(x_28); -x_29 = !lean_is_exclusive(x_20); +uint8_t x_29; +x_29 = !lean_is_exclusive(x_21); 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; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_30 = lean_ctor_get(x_20, 0); -x_31 = lean_ctor_get(x_18, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_18, 1); -lean_inc(x_32); -x_33 = lean_ctor_get(x_18, 3); -lean_inc(x_33); -lean_inc(x_31); -x_34 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_34, 0, x_31); -lean_ctor_set(x_34, 1, x_32); -lean_ctor_set(x_34, 2, x_30); -x_35 = lean_box(0); -lean_inc(x_31); -x_36 = l_Lean_mkNatLit(x_31); -x_37 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__3; -lean_inc(x_2); +lean_object* x_30; uint8_t x_31; +x_30 = lean_ctor_get(x_21, 0); +lean_dec(x_30); +x_31 = !lean_is_exclusive(x_22); +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; uint8_t x_38; +x_32 = lean_ctor_get(x_22, 0); +x_33 = lean_ctor_get(x_20, 0); lean_inc(x_33); +x_34 = lean_ctor_get(x_20, 1); +lean_inc(x_34); +x_35 = lean_ctor_get(x_20, 2); +lean_inc(x_35); +x_36 = lean_ctor_get(x_20, 3); lean_inc(x_36); -x_38 = l_Lean_mkApp3(x_37, x_36, x_33, x_2); -x_39 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_39, 0, x_31); -lean_closure_set(x_39, 1, x_33); -x_40 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1), 12, 5); -lean_closure_set(x_40, 0, x_18); -lean_closure_set(x_40, 1, x_35); -lean_closure_set(x_40, 2, x_2); -lean_closure_set(x_40, 3, x_36); -lean_closure_set(x_40, 4, x_1); -x_41 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_41, 0, x_39); -lean_closure_set(x_41, 1, x_40); -x_42 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_42, 0, x_34); -lean_ctor_set(x_42, 1, x_41); -lean_ctor_set(x_42, 2, x_38); -lean_ctor_set(x_20, 0, x_42); -return x_19; +lean_dec(x_20); +x_37 = lean_ctor_get(x_32, 0); +lean_inc(x_37); +x_38 = lean_nat_dec_eq(x_33, x_37); +if (x_38 == 0) +{ +lean_object* x_39; +lean_dec(x_37); +lean_dec(x_36); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_free_object(x_22); +lean_dec(x_32); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_39 = lean_box(0); +lean_ctor_set(x_21, 0, x_39); +return x_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; 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_20, 0); -lean_inc(x_43); -lean_dec(x_20); -x_44 = lean_ctor_get(x_18, 0); -lean_inc(x_44); -x_45 = lean_ctor_get(x_18, 1); -lean_inc(x_45); -x_46 = lean_ctor_get(x_18, 3); -lean_inc(x_46); -lean_inc(x_44); -x_47 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_47, 0, x_44); -lean_ctor_set(x_47, 1, x_45); -lean_ctor_set(x_47, 2, x_43); -x_48 = lean_box(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; +x_40 = lean_ctor_get(x_32, 1); +lean_inc(x_40); +lean_inc(x_33); +x_41 = lean_alloc_ctor(0, 3, 1); +lean_ctor_set(x_41, 0, x_33); +lean_ctor_set(x_41, 1, x_34); +lean_ctor_set(x_41, 2, x_40); +lean_ctor_set_uint8(x_41, sizeof(void*)*3, x_3); +x_42 = lean_box(0); +lean_inc(x_33); +x_43 = l_Lean_mkNatLit(x_33); +x_44 = lean_ctor_get(x_32, 3); lean_inc(x_44); -x_49 = l_Lean_mkNatLit(x_44); -x_50 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__3; -lean_inc(x_2); -lean_inc(x_46); -lean_inc(x_49); -x_51 = l_Lean_mkApp3(x_50, x_49, x_46, x_2); -x_52 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_52, 0, x_44); -lean_closure_set(x_52, 1, x_46); -x_53 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1), 12, 5); -lean_closure_set(x_53, 0, x_18); -lean_closure_set(x_53, 1, x_48); -lean_closure_set(x_53, 2, x_2); -lean_closure_set(x_53, 3, x_49); -lean_closure_set(x_53, 4, x_1); -x_54 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_54, 0, x_52); -lean_closure_set(x_54, 1, x_53); +lean_inc(x_36); +x_45 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_45, 0, x_33); +lean_closure_set(x_45, 1, x_36); +lean_inc(x_43); +lean_inc(x_44); +x_46 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___lambda__1), 16, 9); +lean_closure_set(x_46, 0, x_35); +lean_closure_set(x_46, 1, x_37); +lean_closure_set(x_46, 2, x_44); +lean_closure_set(x_46, 3, x_32); +lean_closure_set(x_46, 4, x_4); +lean_closure_set(x_46, 5, x_42); +lean_closure_set(x_46, 6, x_43); +lean_closure_set(x_46, 7, x_1); +lean_closure_set(x_46, 8, x_2); +x_47 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_47, 0, x_45); +lean_closure_set(x_47, 1, x_46); +if (x_3 == 0) +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_48 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; +x_49 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; +x_50 = l_Lean_mkApp4(x_48, x_43, x_36, x_49, x_44); +x_51 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_51, 0, x_41); +lean_ctor_set(x_51, 1, x_47); +lean_ctor_set(x_51, 2, x_50); +lean_ctor_set(x_22, 0, x_51); +return x_21; +} +else +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_52 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; +x_53 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10; +x_54 = l_Lean_mkApp4(x_52, x_43, x_36, x_53, x_44); x_55 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_55, 0, x_47); -lean_ctor_set(x_55, 1, x_54); -lean_ctor_set(x_55, 2, x_51); -x_56 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_56, 0, x_55); -lean_ctor_set(x_19, 0, x_56); -return x_19; +lean_ctor_set(x_55, 0, x_41); +lean_ctor_set(x_55, 1, x_47); +lean_ctor_set(x_55, 2, x_54); +lean_ctor_set(x_22, 0, x_55); +return x_21; +} } } 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; 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_57 = lean_ctor_get(x_19, 1); +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; +x_56 = lean_ctor_get(x_22, 0); +lean_inc(x_56); +lean_dec(x_22); +x_57 = lean_ctor_get(x_20, 0); lean_inc(x_57); -lean_dec(x_19); -x_58 = lean_ctor_get(x_20, 0); +x_58 = lean_ctor_get(x_20, 1); lean_inc(x_58); -if (lean_is_exclusive(x_20)) { - lean_ctor_release(x_20, 0); - x_59 = x_20; -} else { - lean_dec_ref(x_20); - x_59 = lean_box(0); -} -x_60 = lean_ctor_get(x_18, 0); +x_59 = lean_ctor_get(x_20, 2); +lean_inc(x_59); +x_60 = lean_ctor_get(x_20, 3); lean_inc(x_60); -x_61 = lean_ctor_get(x_18, 1); +lean_dec(x_20); +x_61 = lean_ctor_get(x_56, 0); lean_inc(x_61); -x_62 = lean_ctor_get(x_18, 3); -lean_inc(x_62); -lean_inc(x_60); -x_63 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_63, 0, x_60); -lean_ctor_set(x_63, 1, x_61); -lean_ctor_set(x_63, 2, x_58); -x_64 = lean_box(0); -lean_inc(x_60); -x_65 = l_Lean_mkNatLit(x_60); -x_66 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__3; -lean_inc(x_2); -lean_inc(x_62); -lean_inc(x_65); -x_67 = l_Lean_mkApp3(x_66, x_65, x_62, x_2); -x_68 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_68, 0, x_60); -lean_closure_set(x_68, 1, x_62); -x_69 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1), 12, 5); -lean_closure_set(x_69, 0, x_18); -lean_closure_set(x_69, 1, x_64); -lean_closure_set(x_69, 2, x_2); -lean_closure_set(x_69, 3, x_65); -lean_closure_set(x_69, 4, x_1); -x_70 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_70, 0, x_68); -lean_closure_set(x_70, 1, x_69); -x_71 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_71, 0, x_63); -lean_ctor_set(x_71, 1, x_70); -lean_ctor_set(x_71, 2, x_67); -if (lean_is_scalar(x_59)) { - x_72 = lean_alloc_ctor(1, 1, 0); -} else { - x_72 = x_59; -} -lean_ctor_set(x_72, 0, x_71); -x_73 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_73, 0, x_72); -lean_ctor_set(x_73, 1, x_57); -return x_73; -} -} -} -else +x_62 = lean_nat_dec_eq(x_57, x_61); +if (x_62 == 0) { -uint8_t x_74; -lean_dec(x_18); +lean_object* 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_4); lean_dec(x_2); lean_dec(x_1); -x_74 = !lean_is_exclusive(x_19); -if (x_74 == 0) -{ -return x_19; -} -else -{ -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_19, 0); -x_76 = lean_ctor_get(x_19, 1); -lean_inc(x_76); -lean_inc(x_75); -lean_dec(x_19); -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_63 = lean_box(0); +lean_ctor_set(x_21, 0, x_63); +return x_21; } else { -uint8_t x_78; -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_78 = !lean_is_exclusive(x_9); -if (x_78 == 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; +x_64 = lean_ctor_get(x_56, 1); +lean_inc(x_64); +lean_inc(x_57); +x_65 = lean_alloc_ctor(0, 3, 1); +lean_ctor_set(x_65, 0, x_57); +lean_ctor_set(x_65, 1, x_58); +lean_ctor_set(x_65, 2, x_64); +lean_ctor_set_uint8(x_65, sizeof(void*)*3, x_3); +x_66 = lean_box(0); +lean_inc(x_57); +x_67 = l_Lean_mkNatLit(x_57); +x_68 = lean_ctor_get(x_56, 3); +lean_inc(x_68); +lean_inc(x_60); +x_69 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_69, 0, x_57); +lean_closure_set(x_69, 1, x_60); +lean_inc(x_67); +lean_inc(x_68); +x_70 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___lambda__1), 16, 9); +lean_closure_set(x_70, 0, x_59); +lean_closure_set(x_70, 1, x_61); +lean_closure_set(x_70, 2, x_68); +lean_closure_set(x_70, 3, x_56); +lean_closure_set(x_70, 4, x_4); +lean_closure_set(x_70, 5, x_66); +lean_closure_set(x_70, 6, x_67); +lean_closure_set(x_70, 7, x_1); +lean_closure_set(x_70, 8, x_2); +x_71 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_71, 0, x_69); +lean_closure_set(x_71, 1, x_70); +if (x_3 == 0) { -return x_9; +lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_72 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; +x_73 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; +x_74 = l_Lean_mkApp4(x_72, x_67, x_60, x_73, x_68); +x_75 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_75, 0, x_65); +lean_ctor_set(x_75, 1, x_71); +lean_ctor_set(x_75, 2, x_74); +x_76 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_21, 0, x_76); +return x_21; } else { -lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_79 = lean_ctor_get(x_9, 0); -x_80 = lean_ctor_get(x_9, 1); -lean_inc(x_80); -lean_inc(x_79); -lean_dec(x_9); -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_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_77 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; +x_78 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10; +x_79 = l_Lean_mkApp4(x_77, x_67, x_60, x_78, x_68); +x_80 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_80, 0, x_65); +lean_ctor_set(x_80, 1, x_71); +lean_ctor_set(x_80, 2, x_79); +x_81 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_21, 0, x_81); +return x_21; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("ult_congr", 9, 9); -return x_1; -} +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; +x_82 = lean_ctor_get(x_21, 1); +lean_inc(x_82); +lean_dec(x_21); +x_83 = lean_ctor_get(x_22, 0); +lean_inc(x_83); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + x_84 = x_22; +} else { + lean_dec_ref(x_22); + x_84 = lean_box(0); } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__2() { -_start: +x_85 = lean_ctor_get(x_20, 0); +lean_inc(x_85); +x_86 = lean_ctor_get(x_20, 1); +lean_inc(x_86); +x_87 = lean_ctor_get(x_20, 2); +lean_inc(x_87); +x_88 = lean_ctor_get(x_20, 3); +lean_inc(x_88); +lean_dec(x_20); +x_89 = lean_ctor_get(x_83, 0); +lean_inc(x_89); +x_90 = lean_nat_dec_eq(x_85, x_89); +if (x_90 == 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; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__1; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; -} +lean_object* x_91; lean_object* x_92; +lean_dec(x_89); +lean_dec(x_88); +lean_dec(x_87); +lean_dec(x_86); +lean_dec(x_85); +lean_dec(x_84); +lean_dec(x_83); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +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_82); +return x_92; } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___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) { -_start: +else { -uint8_t x_9; lean_object* x_10; lean_object* x_11; -x_9 = 1; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__2; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); -return x_11; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__1() { -_start: +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_93 = lean_ctor_get(x_83, 1); +lean_inc(x_93); +lean_inc(x_85); +x_94 = lean_alloc_ctor(0, 3, 1); +lean_ctor_set(x_94, 0, x_85); +lean_ctor_set(x_94, 1, x_86); +lean_ctor_set(x_94, 2, x_93); +lean_ctor_set_uint8(x_94, sizeof(void*)*3, x_3); +x_95 = lean_box(0); +lean_inc(x_85); +x_96 = l_Lean_mkNatLit(x_85); +x_97 = lean_ctor_get(x_83, 3); +lean_inc(x_97); +lean_inc(x_88); +x_98 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_98, 0, x_85); +lean_closure_set(x_98, 1, x_88); +lean_inc(x_96); +lean_inc(x_97); +x_99 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___lambda__1), 16, 9); +lean_closure_set(x_99, 0, x_87); +lean_closure_set(x_99, 1, x_89); +lean_closure_set(x_99, 2, x_97); +lean_closure_set(x_99, 3, x_83); +lean_closure_set(x_99, 4, x_4); +lean_closure_set(x_99, 5, x_95); +lean_closure_set(x_99, 6, x_96); +lean_closure_set(x_99, 7, x_1); +lean_closure_set(x_99, 8, x_2); +x_100 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_100, 0, x_98); +lean_closure_set(x_100, 1, x_99); +if (x_3 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("beq_congr", 9, 9); -return x_1; +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_101 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; +x_102 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__7; +x_103 = l_Lean_mkApp4(x_101, x_96, x_88, x_102, x_97); +x_104 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_104, 0, x_94); +lean_ctor_set(x_104, 1, x_100); +lean_ctor_set(x_104, 2, x_103); +if (lean_is_scalar(x_84)) { + x_105 = lean_alloc_ctor(1, 1, 0); +} else { + x_105 = x_84; } +lean_ctor_set(x_105, 0, x_104); +x_106 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_106, 0, x_105); +lean_ctor_set(x_106, 1, x_82); +return x_106; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__2() { -_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_ReifiedBVPred_of_binaryReflection___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__1; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; +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_107 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; +x_108 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10; +x_109 = l_Lean_mkApp4(x_107, x_96, x_88, x_108, x_97); +x_110 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_110, 0, x_94); +lean_ctor_set(x_110, 1, x_100); +lean_ctor_set(x_110, 2, x_109); +if (lean_is_scalar(x_84)) { + x_111 = lean_alloc_ctor(1, 1, 0); +} else { + x_111 = x_84; } +lean_ctor_set(x_111, 0, x_110); +x_112 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_112, 0, x_111); +lean_ctor_set(x_112, 1, x_82); +return x_112; } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___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; lean_object* x_11; lean_object* x_12; -x_10 = 0; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__2; -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection(x_1, x_2, x_10, x_11, x_4, x_5, x_6, x_7, x_8, x_9); -return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___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) { -_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_ReifiedBVPred_of___lambda__6___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__5___boxed), 7, 0); -return x_1; -} +uint8_t x_113; +lean_dec(x_20); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_113 = !lean_is_exclusive(x_21); +if (x_113 == 0) +{ +return x_21; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__2() { -_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_ReifiedBVPred_of___lambda__1___closed__2; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_114; lean_object* x_115; lean_object* x_116; +x_114 = lean_ctor_get(x_21, 0); +x_115 = lean_ctor_get(x_21, 1); +lean_inc(x_115); +lean_inc(x_114); +lean_dec(x_21); +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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___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_10; lean_object* x_11; uint8_t x_12; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__1; -x_11 = l_Lean_Expr_cleanupAnnotations(x_1); -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_3); -lean_dec(x_2); -x_13 = lean_box(0); -x_14 = lean_apply_7(x_10, x_13, x_4, 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_appFnCleanup(x_11, lean_box(0)); -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__2; -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; -lean_dec(x_3); +uint8_t x_117; +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_18 = lean_box(0); -x_19 = lean_apply_7(x_10, x_18, x_4, x_5, x_6, x_7, x_8, x_9); -return x_19; +lean_dec(x_1); +x_117 = !lean_is_exclusive(x_11); +if (x_117 == 0) +{ +return x_11; } else { -lean_object* x_20; lean_object* x_21; -x_20 = lean_box(0); -x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4(x_2, x_3, x_20, x_4, x_5, x_6, x_7, x_8, x_9); -return x_21; +lean_object* x_118; lean_object* x_119; lean_object* x_120; +x_118 = lean_ctor_get(x_11, 0); +x_119 = lean_ctor_get(x_11, 1); +lean_inc(x_119); +lean_inc(x_118); +lean_dec(x_11); +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_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, 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_3); +lean_dec(x_3); +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection(x_1, x_2, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_12; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("ofBool_congr", 12, 12); +x_1 = lean_mk_string_unchecked("getLsbD_congr", 13, 13); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___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_ReifiedBVPred_of_binaryReflection___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__1; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__1; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___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_ReifiedBVPred_of___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_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_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) { _start: { -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_1, 2); -lean_inc(x_11); +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_1, 2); +lean_inc(x_13); lean_dec(x_1); -x_12 = lean_apply_6(x_11, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_12) == 0) +x_14 = lean_apply_6(x_13, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_14) == 0) { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_12); -if (x_13 == 0) +uint8_t x_15; +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 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 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__2; -x_16 = l_Lean_Expr_const___override(x_15, x_2); -x_17 = l_Lean_mkApp3(x_16, x_3, x_4, x_14); -lean_ctor_set(x_12, 0, x_17); -return x_12; +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 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__2; +x_18 = l_Lean_Expr_const___override(x_17, x_2); +x_19 = l_Lean_mkApp5(x_18, x_3, x_4, x_5, x_6, x_16); +lean_ctor_set(x_14, 0, x_19); +return x_14; } 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; -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 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__2; -x_21 = l_Lean_Expr_const___override(x_20, x_2); -x_22 = l_Lean_mkApp3(x_21, x_3, x_4, x_18); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_19); -return x_23; +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_14, 0); +x_21 = lean_ctor_get(x_14, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_14); +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__2; +x_23 = l_Lean_Expr_const___override(x_22, x_2); +x_24 = l_Lean_mkApp5(x_23, x_3, x_4, x_5, x_6, x_20); +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 { -uint8_t x_24; +uint8_t x_26; +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_24 = !lean_is_exclusive(x_12); -if (x_24 == 0) +x_26 = !lean_is_exclusive(x_14); +if (x_26 == 0) { -return x_12; +return x_14; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_12, 0); -x_26 = lean_ctor_get(x_12, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_12); -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; -} -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("ofBool", 6, 6); -return x_1; +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_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 lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___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_ReifiedBVPred_of___lambda__8___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2___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_ReifiedBVPred_of___lambda__8___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__6; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__4() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_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) { _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_ReifiedBVPred_of___lambda__2___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_ReifiedBVPred_of___lambda__8___closed__5() { -_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_ReifiedBVExpr_of_goOrAtom(x_1, x_3, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_9) == 0) { -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_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_dec(x_5); +lean_dec(x_4); +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; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__6() { -_start: +else { -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; +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; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___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) { -_start: -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_9 = lean_box(0); -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__3; -lean_inc(x_1); -x_11 = l_Lean_Expr_app___override(x_10, x_1); -x_12 = lean_unsigned_to_nat(1u); -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom(x_11, x_12, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_13) == 0) -{ -uint8_t x_14; -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) +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_object* x_27; lean_object* x_28; lean_object* x_29; -x_15 = lean_ctor_get(x_13, 0); -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_9, 1); lean_inc(x_17); -x_18 = lean_ctor_get(x_15, 3); -lean_inc(x_18); -x_19 = lean_unsigned_to_nat(0u); -lean_inc(x_16); -x_20 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_20, 0, x_16); -lean_ctor_set(x_20, 1, x_17); -lean_ctor_set(x_20, 2, x_19); -x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__4; -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__5; -x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__6; +lean_dec(x_9); +x_18 = lean_ctor_get(x_10, 0); lean_inc(x_18); -x_24 = l_Lean_mkApp3(x_21, x_22, x_18, x_23); -x_25 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_25, 0, x_16); -lean_closure_set(x_25, 1, x_18); -x_26 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7), 10, 3); -lean_closure_set(x_26, 0, x_15); -lean_closure_set(x_26, 1, x_9); -lean_closure_set(x_26, 2, x_1); -x_27 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_27, 0, x_25); -lean_closure_set(x_27, 1, x_26); -x_28 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_28, 0, x_20); -lean_ctor_set(x_28, 1, x_27); -lean_ctor_set(x_28, 2, x_24); -x_29 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_13, 0, x_29); -return x_13; +lean_dec(x_10); +x_19 = l_Lean_Meta_getNatValue_x3f(x_2, x_4, x_5, x_6, x_7, x_17); +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_18); +lean_dec(x_2); +lean_dec(x_1); +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 = lean_box(0); +lean_ctor_set(x_19, 0, x_23); +return x_19; } 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; lean_object* x_45; lean_object* x_46; -x_30 = lean_ctor_get(x_13, 0); -x_31 = lean_ctor_get(x_13, 1); +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 = 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; +} +} +else +{ +uint8_t x_27; +x_27 = !lean_is_exclusive(x_19); +if (x_27 == 0) +{ +lean_object* x_28; uint8_t x_29; +x_28 = lean_ctor_get(x_19, 0); +lean_dec(x_28); +x_29 = !lean_is_exclusive(x_20); +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; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_30 = lean_ctor_get(x_20, 0); +x_31 = lean_ctor_get(x_18, 0); lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_13); -x_32 = lean_ctor_get(x_30, 0); +x_32 = lean_ctor_get(x_18, 1); lean_inc(x_32); -x_33 = lean_ctor_get(x_30, 1); +x_33 = lean_ctor_get(x_18, 3); lean_inc(x_33); -x_34 = lean_ctor_get(x_30, 3); -lean_inc(x_34); -x_35 = lean_unsigned_to_nat(0u); -lean_inc(x_32); -x_36 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_36, 0, x_32); -lean_ctor_set(x_36, 1, x_33); -lean_ctor_set(x_36, 2, x_35); -x_37 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__4; -x_38 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__5; -x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__6; -lean_inc(x_34); -x_40 = l_Lean_mkApp3(x_37, x_38, x_34, x_39); -x_41 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); -lean_closure_set(x_41, 0, x_32); -lean_closure_set(x_41, 1, x_34); -x_42 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7), 10, 3); -lean_closure_set(x_42, 0, x_30); -lean_closure_set(x_42, 1, x_9); -lean_closure_set(x_42, 2, x_1); -x_43 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); -lean_closure_set(x_43, 0, x_41); -lean_closure_set(x_43, 1, x_42); -x_44 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_44, 0, x_36); -lean_ctor_set(x_44, 1, x_43); -lean_ctor_set(x_44, 2, x_40); -x_45 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_45, 0, 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_31); -return x_46; +lean_inc(x_31); +x_34 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_34, 0, x_31); +lean_ctor_set(x_34, 1, x_32); +lean_ctor_set(x_34, 2, x_30); +x_35 = lean_box(0); +lean_inc(x_31); +x_36 = l_Lean_mkNatLit(x_31); +x_37 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2___closed__1; +lean_inc(x_2); +lean_inc(x_33); +lean_inc(x_36); +x_38 = l_Lean_mkApp3(x_37, x_36, x_33, x_2); +x_39 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_39, 0, x_31); +lean_closure_set(x_39, 1, x_33); +x_40 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1), 12, 5); +lean_closure_set(x_40, 0, x_18); +lean_closure_set(x_40, 1, x_35); +lean_closure_set(x_40, 2, x_2); +lean_closure_set(x_40, 3, x_36); +lean_closure_set(x_40, 4, x_1); +x_41 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_41, 0, x_39); +lean_closure_set(x_41, 1, x_40); +x_42 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_42, 0, x_34); +lean_ctor_set(x_42, 1, x_41); +lean_ctor_set(x_42, 2, x_38); +lean_ctor_set(x_20, 0, x_42); +return x_19; +} +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_20, 0); +lean_inc(x_43); +lean_dec(x_20); +x_44 = lean_ctor_get(x_18, 0); +lean_inc(x_44); +x_45 = lean_ctor_get(x_18, 1); +lean_inc(x_45); +x_46 = lean_ctor_get(x_18, 3); +lean_inc(x_46); +lean_inc(x_44); +x_47 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_47, 0, x_44); +lean_ctor_set(x_47, 1, x_45); +lean_ctor_set(x_47, 2, x_43); +x_48 = lean_box(0); +lean_inc(x_44); +x_49 = l_Lean_mkNatLit(x_44); +x_50 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2___closed__1; +lean_inc(x_2); +lean_inc(x_46); +lean_inc(x_49); +x_51 = l_Lean_mkApp3(x_50, x_49, x_46, x_2); +x_52 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_52, 0, x_44); +lean_closure_set(x_52, 1, x_46); +x_53 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1), 12, 5); +lean_closure_set(x_53, 0, x_18); +lean_closure_set(x_53, 1, x_48); +lean_closure_set(x_53, 2, x_2); +lean_closure_set(x_53, 3, x_49); +lean_closure_set(x_53, 4, x_1); +x_54 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_54, 0, x_52); +lean_closure_set(x_54, 1, x_53); +x_55 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_55, 0, x_47); +lean_ctor_set(x_55, 1, x_54); +lean_ctor_set(x_55, 2, x_51); +x_56 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_56, 0, x_55); +lean_ctor_set(x_19, 0, x_56); +return x_19; +} +} +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; 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_57 = lean_ctor_get(x_19, 1); +lean_inc(x_57); +lean_dec(x_19); +x_58 = lean_ctor_get(x_20, 0); +lean_inc(x_58); +if (lean_is_exclusive(x_20)) { + lean_ctor_release(x_20, 0); + x_59 = x_20; +} else { + lean_dec_ref(x_20); + x_59 = lean_box(0); +} +x_60 = lean_ctor_get(x_18, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_18, 1); +lean_inc(x_61); +x_62 = lean_ctor_get(x_18, 3); +lean_inc(x_62); +lean_inc(x_60); +x_63 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_63, 0, x_60); +lean_ctor_set(x_63, 1, x_61); +lean_ctor_set(x_63, 2, x_58); +x_64 = lean_box(0); +lean_inc(x_60); +x_65 = l_Lean_mkNatLit(x_60); +x_66 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2___closed__1; +lean_inc(x_2); +lean_inc(x_62); +lean_inc(x_65); +x_67 = l_Lean_mkApp3(x_66, x_65, x_62, x_2); +x_68 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkEvalExpr___boxed), 8, 2); +lean_closure_set(x_68, 0, x_60); +lean_closure_set(x_68, 1, x_62); +x_69 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1), 12, 5); +lean_closure_set(x_69, 0, x_18); +lean_closure_set(x_69, 1, x_64); +lean_closure_set(x_69, 2, x_2); +lean_closure_set(x_69, 3, x_65); +lean_closure_set(x_69, 4, x_1); +x_70 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_mkAtom___spec__1___rarg), 8, 2); +lean_closure_set(x_70, 0, x_68); +lean_closure_set(x_70, 1, x_69); +x_71 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_71, 0, x_63); +lean_ctor_set(x_71, 1, x_70); +lean_ctor_set(x_71, 2, x_67); +if (lean_is_scalar(x_59)) { + x_72 = lean_alloc_ctor(1, 1, 0); +} else { + x_72 = x_59; +} +lean_ctor_set(x_72, 0, x_71); +x_73 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_73, 0, x_72); +lean_ctor_set(x_73, 1, x_57); +return x_73; +} +} +} +else +{ +uint8_t x_74; +lean_dec(x_18); +lean_dec(x_2); +lean_dec(x_1); +x_74 = !lean_is_exclusive(x_19); +if (x_74 == 0) +{ +return x_19; +} +else +{ +lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_75 = lean_ctor_get(x_19, 0); +x_76 = lean_ctor_get(x_19, 1); +lean_inc(x_76); +lean_inc(x_75); +lean_dec(x_19); +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_47; +uint8_t x_78; +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_47 = !lean_is_exclusive(x_13); -if (x_47 == 0) +x_78 = !lean_is_exclusive(x_9); +if (x_78 == 0) { -return x_13; +return x_9; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_13, 0); -x_49 = lean_ctor_get(x_13, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_13); -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_79; lean_object* x_80; lean_object* x_81; +x_79 = lean_ctor_get(x_9, 0); +x_80 = lean_ctor_get(x_9, 1); +lean_inc(x_80); +lean_inc(x_79); +lean_dec(x_9); +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; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("Bool", 4, 4); +x_1 = lean_mk_string_unchecked("ult_congr", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___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_ReifiedBVPred_boolAtom___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___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_ReifiedBVPred_of_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) { +_start: +{ +uint8_t x_9; lean_object* x_10; lean_object* x_11; +x_9 = 1; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__2; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection(x_1, x_2, x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); +return x_11; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("beq_congr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___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_ReifiedBVPred_boolAtom___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___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_ReifiedBVPred_of_go___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; lean_object* x_11; lean_object* x_12; +x_10 = 0; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__2; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection(x_1, x_2, x_10, x_11, x_4, x_5, x_6, x_7, x_8, x_9); +return x_12; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__5___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_ReifiedBVPred_of___lambda__9___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___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_9; -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_1); -x_9 = lean_infer_type(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; uint8_t x_15; -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_ReifiedBVPred_of___lambda__6___closed__1; -x_13 = l_Lean_Expr_cleanupAnnotations(x_10); -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__2; -x_15 = l_Lean_Expr_isConstOf(x_13, x_14); -lean_dec(x_13); -if (x_15 == 0) +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__1; +x_11 = l_Lean_Expr_cleanupAnnotations(x_1); +x_12 = l_Lean_Expr_isApp(x_11); +if (x_12 == 0) { -lean_object* x_16; lean_object* x_17; -lean_dec(x_1); -x_16 = lean_box(0); -x_17 = lean_apply_7(x_12, x_16, x_3, x_4, x_5, x_6, x_7, x_11); -return x_17; +lean_object* x_13; lean_object* x_14; +lean_dec(x_11); +lean_dec(x_3); +lean_dec(x_2); +x_13 = lean_box(0); +x_14 = lean_apply_7(x_10, x_13, x_4, 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_appFnCleanup(x_11, lean_box(0)); +x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__5___closed__1; +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; +lean_dec(x_3); +lean_dec(x_2); x_18 = lean_box(0); -x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8(x_1, x_18, x_3, x_4, x_5, x_6, x_7, x_11); +x_19 = lean_apply_7(x_10, x_18, x_4, x_5, x_6, x_7, x_8, x_9); return x_19; } -} -else -{ -uint8_t x_20; -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_9); -if (x_20 == 0) -{ -return x_9; -} else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_9, 0); -x_22 = lean_ctor_get(x_9, 1); -lean_inc(x_22); -lean_inc(x_21); -lean_dec(x_9); -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_20; lean_object* x_21; +x_20 = lean_box(0); +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4(x_2, x_3, x_20, x_4, x_5, x_6, x_7, x_8, x_9); +return x_21; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3), 8, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__3() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6), 9, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__5), 9, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__1; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___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_ReifiedBVPred_of___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__12; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___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_ReifiedBVPred_of___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__6() { _start: { lean_object* x_1; @@ -1852,7 +1875,7 @@ x_1 = lean_mk_string_unchecked("BEq", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__7() { _start: { lean_object* x_1; @@ -1860,184 +1883,264 @@ x_1 = lean_mk_string_unchecked("beq", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__8() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__6; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__6; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__7; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of(lean_object* x_1, lean_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_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_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) { _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; uint8_t x_15; -lean_inc(x_1); +lean_object* x_8; lean_object* x_9; lean_object* x_10; 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_8 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_1, x_3, x_4, x_5, x_6, x_7); 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_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__1; -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__2; -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__3; -x_14 = l_Lean_Expr_cleanupAnnotations(x_9); -x_15 = l_Lean_Expr_isApp(x_14); -if (x_15 == 0) -{ -lean_object* x_16; lean_object* x_17; -lean_dec(x_14); -x_16 = lean_box(0); -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9(x_1, x_16, x_2, x_3, x_4, x_5, x_6, x_10); -return x_17; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__1; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__2; +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__3; +x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__1; +x_15 = l_Lean_Expr_cleanupAnnotations(x_9); +x_16 = l_Lean_Expr_isApp(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +lean_dec(x_15); +x_17 = lean_box(0); +x_18 = lean_apply_7(x_14, x_17, x_2, x_3, x_4, x_5, x_6, x_10); +return x_18; } 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_19; lean_object* x_20; uint8_t x_21; +x_19 = l_Lean_Expr_appArg(x_15, lean_box(0)); +x_20 = l_Lean_Expr_appFnCleanup(x_15, lean_box(0)); +x_21 = l_Lean_Expr_isApp(x_20); +if (x_21 == 0) { -lean_object* x_21; lean_object* x_22; +lean_object* x_22; lean_object* x_23; +lean_dec(x_20); lean_dec(x_19); -lean_dec(x_18); -x_21 = lean_box(0); -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9(x_1, x_21, x_2, x_3, x_4, x_5, x_6, x_10); -return x_22; +x_22 = lean_box(0); +x_23 = lean_apply_7(x_14, x_22, x_2, x_3, x_4, x_5, x_6, x_10); +return x_23; } else { -lean_object* x_23; lean_object* x_24; uint8_t x_25; -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_Expr_isApp(x_24); -if (x_25 == 0) +lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_24 = l_Lean_Expr_appArg(x_20, lean_box(0)); +x_25 = l_Lean_Expr_appFnCleanup(x_20, lean_box(0)); +x_26 = l_Lean_Expr_isApp(x_25); +if (x_26 == 0) { -lean_object* x_26; lean_object* x_27; +lean_object* x_27; lean_object* x_28; +lean_dec(x_25); lean_dec(x_24); -lean_dec(x_23); -lean_dec(x_18); -x_26 = lean_box(0); -x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9(x_1, x_26, x_2, x_3, x_4, x_5, x_6, x_10); -return x_27; +lean_dec(x_19); +x_27 = lean_box(0); +x_28 = lean_apply_7(x_14, x_27, x_2, x_3, x_4, x_5, x_6, x_10); +return x_28; } else { -lean_object* x_28; lean_object* x_29; uint8_t x_30; -x_28 = l_Lean_Expr_appFnCleanup(x_24, lean_box(0)); -x_29 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__4; -x_30 = l_Lean_Expr_isConstOf(x_28, x_29); -if (x_30 == 0) -{ -lean_object* x_31; uint8_t x_32; -x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__5; -x_32 = l_Lean_Expr_isConstOf(x_28, x_31); -if (x_32 == 0) +lean_object* x_29; lean_object* x_30; uint8_t x_31; +x_29 = l_Lean_Expr_appFnCleanup(x_25, lean_box(0)); +x_30 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__4; +x_31 = l_Lean_Expr_isConstOf(x_29, x_30); +if (x_31 == 0) { -uint8_t x_33; -x_33 = l_Lean_Expr_isApp(x_28); +lean_object* x_32; uint8_t x_33; +x_32 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__5; +x_33 = l_Lean_Expr_isConstOf(x_29, x_32); if (x_33 == 0) { -lean_object* x_34; lean_object* x_35; -lean_dec(x_28); -lean_dec(x_23); -lean_dec(x_18); -x_34 = lean_box(0); -x_35 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9(x_1, x_34, x_2, x_3, x_4, x_5, x_6, x_10); -return x_35; -} -else -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; -x_36 = l_Lean_Expr_appArg(x_28, lean_box(0)); -x_37 = l_Lean_Expr_appFnCleanup(x_28, lean_box(0)); -x_38 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__8; -x_39 = l_Lean_Expr_isConstOf(x_37, x_38); -lean_dec(x_37); -if (x_39 == 0) +uint8_t x_34; +x_34 = l_Lean_Expr_isApp(x_29); +if (x_34 == 0) { -lean_object* x_40; lean_object* x_41; -lean_dec(x_36); -lean_dec(x_23); -lean_dec(x_18); -x_40 = lean_box(0); -x_41 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9(x_1, x_40, x_2, x_3, x_4, x_5, x_6, x_10); -return x_41; +lean_object* x_35; lean_object* x_36; +lean_dec(x_29); +lean_dec(x_24); +lean_dec(x_19); +x_35 = lean_box(0); +x_36 = lean_apply_7(x_14, x_35, x_2, x_3, x_4, x_5, x_6, x_10); +return x_36; } else { -lean_object* x_42; -lean_dec(x_1); -x_42 = lean_apply_9(x_13, x_36, x_23, x_18, x_2, x_3, x_4, x_5, x_6, x_10); +lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_37 = l_Lean_Expr_appArg(x_29, lean_box(0)); +x_38 = l_Lean_Expr_appFnCleanup(x_29, lean_box(0)); +x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__8; +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_37); +lean_dec(x_24); +lean_dec(x_19); +x_41 = lean_box(0); +x_42 = lean_apply_7(x_14, x_41, x_2, x_3, x_4, x_5, x_6, x_10); return x_42; } -} -} else { lean_object* x_43; -lean_dec(x_28); -lean_dec(x_1); -x_43 = lean_apply_8(x_12, x_23, x_18, x_2, x_3, x_4, x_5, x_6, x_10); +x_43 = lean_apply_9(x_13, x_37, x_24, x_19, x_2, x_3, x_4, x_5, x_6, x_10); return x_43; } } +} else { lean_object* x_44; -lean_dec(x_28); -lean_dec(x_1); -x_44 = lean_apply_8(x_11, x_23, x_18, x_2, x_3, x_4, x_5, x_6, x_10); +lean_dec(x_29); +x_44 = lean_apply_8(x_12, x_24, x_19, x_2, x_3, x_4, x_5, x_6, x_10); return x_44; } } +else +{ +lean_object* x_45; +lean_dec(x_29); +x_45 = lean_apply_8(x_11, x_24, x_19, x_2, x_3, x_4, x_5, x_6, x_10); +return x_45; +} } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_3); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of(lean_object* x_1, 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_ReifiedBVPred_of___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, 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_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go(x_1, 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) == 0) +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); +lean_dec(x_8); +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +return x_11; +} +else +{ +uint8_t x_12; 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_12 = !lean_is_exclusive(x_8); +if (x_12 == 0) +{ +lean_object* x_13; uint8_t x_14; +x_13 = lean_ctor_get(x_8, 0); +lean_dec(x_13); +x_14 = !lean_is_exclusive(x_9); +if (x_14 == 0) +{ +return x_8; +} +else +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_9, 0); +lean_inc(x_15); +lean_dec(x_9); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_8, 0, x_16); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___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) { -_start: +else { -lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_2); -return x_9; +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_8, 1); +lean_inc(x_17); +lean_dec(x_8); +x_18 = lean_ctor_get(x_9, 0); +lean_inc(x_18); +if (lean_is_exclusive(x_9)) { + lean_ctor_release(x_9, 0); + x_19 = x_9; +} else { + lean_dec_ref(x_9); + x_19 = lean_box(0); +} +if (lean_is_scalar(x_19)) { + x_20 = lean_alloc_ctor(1, 1, 0); +} else { + x_20 = x_19; +} +lean_ctor_set(x_20, 0, 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_17); +return x_21; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___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) { -_start: +} +else { -lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +uint8_t x_22; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -return x_9; +lean_dec(x_1); +x_22 = !lean_is_exclusive(x_8); +if (x_22 == 0) +{ +return x_8; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_8, 0); +x_24 = lean_ctor_get(x_8, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_8); +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_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_BVDecide_ReifiedBVExpr(uint8_t builtin, lean_object*); @@ -2049,6 +2152,44 @@ _G_initialized = true; res = initialize_Lean_Elab_Tactic_BVDecide_Frontend_BVDecide_ReifiedBVExpr(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__1___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___lambda__2___closed__9); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_boolAtom___closed__3); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__1); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__2(); @@ -2069,76 +2210,38 @@ l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed_ lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__9); l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__10); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__11 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__11(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__11); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__12 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__12(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__12); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__13 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__13(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__13); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__14 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__14(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_binaryReflection___closed__14); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__1___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__2___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__3___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__4___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__6___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__7___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__8___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___lambda__9___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__2___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__3___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__4___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__5___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__5___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___lambda__5___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVPred_of_go___closed__8); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/SatAtBVLogical.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/SatAtBVLogical.c index 1c8757fb750f..387d7ba4acfe 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/SatAtBVLogical.c +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide/SatAtBVLogical.c @@ -16,6 +16,7 @@ extern "C" { lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_of___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_of___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* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goOrAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_of___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_of___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_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_mkTrans(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -50,7 +51,6 @@ static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_and___la lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_and___lambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_and(lean_object*, lean_object*); -lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_and___closed__7; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_and___lambda__1___closed__3; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_proveFalse___closed__2; @@ -73,10 +73,10 @@ lean_object* l_Lean_Meta_instantiateMVarsIfMVarApp(lean_object*, lean_object*, l static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_and___closed__5; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_and___closed__9; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_of___lambda__4___closed__1; +lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___spec__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_SatAtBVLogical_of(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_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_proveFalse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_of___lambda__1___closed__2; lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_of___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -189,7 +189,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_SatAtBVLogical_of_ { lean_object* x_10; lean_inc(x_1); -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of(x_1, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVLogical_of_goOrAtom(x_1, x_4, x_5, x_6, x_7, x_8, x_9); if (lean_obj_tag(x_10) == 0) { lean_object* x_11; @@ -546,7 +546,7 @@ lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_of_ofAtom___spec__1(x_12, x_2, x_3, x_4, x_5, x_6, x_13); +x_14 = l_Lean_instantiateMVars___at_Lean_Elab_Tactic_BVDecide_Frontend_ReifiedBVExpr_bitVecAtom___spec__1(x_12, x_2, x_3, x_4, x_5, x_6, x_13); x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); x_16 = lean_ctor_get(x_14, 1); diff --git a/stage0/stdlib/Lean/Elab/Tactic/BuiltinTactic.c b/stage0/stdlib/Lean/Elab/Tactic/BuiltinTactic.c index cabd58b36fb0..6a7e3ea33346 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/BuiltinTactic.c +++ b/stage0/stdlib/Lean/Elab/Tactic/BuiltinTactic.c @@ -95,7 +95,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___at_Lean_Elab_Tactic LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at_Lean_Elab_Tactic_evalSepTactics_goEven___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*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalIntroMatch__1___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalTraceState_declRange__1___closed__4; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___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_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___boxed(lean_object**); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalClear_declRange__1___closed__6; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_evalOpen___spec__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*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalAnyGoals_declRange__1___closed__5; @@ -929,10 +929,10 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSleep_declRange__1( static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalFail_declRange__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRunTac_declRange__1___closed__7; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalIntroMatch_declRange__1(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___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_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1(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*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalSepTactics(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromise___at_Lean_Elab_Tactic_evalSepTactics_goEven___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_EXPORT lean_object* l_Lean_Elab_Tactic_evalCase___lambda__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*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCase___lambda__2(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*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithAnnotateState__1___closed__9; LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Tactic_evalOpen___spec__38___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalLeft_declRange__1___closed__1; @@ -1189,7 +1189,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAllGoals___boxed(lean_object*, l LEAN_EXPORT lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___at_Lean_Elab_Tactic_evalSepTactics_goEven___spec__10___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_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRotateLeft__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCase___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_Lean_Elab_Tactic_evalCase___lambda__2___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCase(lean_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_Elab_Tactic_renameInaccessibles___spec__14(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___regBuiltin_Lean_Elab_Tactic_evalRefl_declRange__1(lean_object*); @@ -1352,7 +1352,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalOpen__1___closed__2; LEAN_EXPORT lean_object* l_Lean_resolveNamespace___at_Lean_Elab_Tactic_evalOpen___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*); static lean_object* l_Lean_Elab_Tactic_evalSubstVars___rarg___closed__1; lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___spec__6(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*, lean_object*, lean_object*, lean_object*); lean_object* lean_local_ctx_num_indices(lean_object*); static lean_object* l_Lean_Elab_Tactic_evalRunTac___closed__10; LEAN_EXPORT lean_object* l_Lean_Core_withRestoreOrSaveFull___at_Lean_Elab_Tactic_evalSepTactics_goEven___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1413,7 +1413,7 @@ lean_object* l_Lean_MVarId_replaceLocalDeclDefEq(lean_object*, lean_object*, lea static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalClear_declRange__1___closed__4; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_renameInaccessibles___spec__16(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_Elab_pushInfoLeaf___at_Lean_Elab_Tactic_evalOpen___spec__28___closed__2; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___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*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___spec__6___boxed(lean_object**); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalTacticSeqBracketed__1___closed__4; uint8_t lean_nat_dec_le(lean_object*, lean_object*); @@ -40600,14 +40600,15 @@ return x_40; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___spec__6(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_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___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, lean_object* x_9, 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: { -uint8_t x_17; -x_17 = lean_usize_dec_lt(x_6, x_5); -if (x_17 == 0) +uint8_t x_18; +x_18 = lean_usize_dec_lt(x_7, x_6); +if (x_18 == 0) { -lean_object* x_18; +lean_object* x_19; +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -40615,72 +40616,73 @@ lean_dec(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_2); lean_dec(x_1); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_7); -lean_ctor_set(x_18, 1, x_16); -return x_18; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_8); +lean_ctor_set(x_19, 1, x_17); +return x_19; } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_19 = lean_array_uget(x_4, x_6); -x_29 = lean_ctor_get(x_7, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_7, 1); +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_20 = lean_array_uget(x_5, x_7); +x_30 = lean_ctor_get(x_8, 0); lean_inc(x_30); -x_31 = lean_ctor_get(x_7, 2); +x_31 = lean_ctor_get(x_8, 1); lean_inc(x_31); -x_32 = lean_nat_dec_lt(x_30, x_31); -if (x_32 == 0) +x_32 = lean_ctor_get(x_8, 2); +lean_inc(x_32); +x_33 = lean_nat_dec_lt(x_31, x_32); +if (x_33 == 0) { -lean_object* x_33; +lean_object* x_34; +lean_dec(x_32); lean_dec(x_31); lean_dec(x_30); -lean_dec(x_29); -lean_dec(x_19); -x_33 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_33, 0, x_7); -x_20 = x_33; -x_21 = x_16; -goto block_28; +lean_dec(x_20); +x_34 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_34, 0, x_8); +x_21 = x_34; +x_22 = x_17; +goto block_29; } else { -uint8_t x_34; -x_34 = !lean_is_exclusive(x_7); -if (x_34 == 0) +uint8_t x_35; +x_35 = !lean_is_exclusive(x_8); +if (x_35 == 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_7, 2); -lean_dec(x_35); -x_36 = lean_ctor_get(x_7, 1); +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_8, 2); lean_dec(x_36); -x_37 = lean_ctor_get(x_7, 0); +x_37 = lean_ctor_get(x_8, 1); lean_dec(x_37); -x_38 = lean_array_fget(x_29, x_30); -x_39 = lean_unsigned_to_nat(1u); -x_40 = lean_nat_add(x_30, x_39); -lean_dec(x_30); -lean_ctor_set(x_7, 1, x_40); -x_41 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_41) == 0) +x_38 = lean_ctor_get(x_8, 0); +lean_dec(x_38); +x_39 = lean_array_fget(x_30, x_31); +x_40 = lean_unsigned_to_nat(1u); +x_41 = lean_nat_add(x_31, x_40); +lean_dec(x_31); +lean_ctor_set(x_8, 1, x_41); +x_42 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_20, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +if (lean_obj_tag(x_42) == 0) { -lean_object* x_42; lean_object* x_43; uint8_t x_44; -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_41, 1); +lean_object* x_43; lean_object* x_44; uint8_t x_45; +x_43 = lean_ctor_get(x_42, 0); lean_inc(x_43); -lean_dec(x_41); -x_44 = !lean_is_exclusive(x_42); -if (x_44 == 0) +x_44 = lean_ctor_get(x_42, 1); +lean_inc(x_44); +lean_dec(x_42); +x_45 = !lean_is_exclusive(x_43); +if (x_45 == 0) { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_42, 0); -x_46 = lean_ctor_get(x_42, 1); +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_43, 0); +x_47 = lean_ctor_get(x_43, 1); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -40688,43 +40690,65 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); -x_47 = l_Lean_Elab_Tactic_renameInaccessibles(x_45, x_38, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_43); -if (lean_obj_tag(x_47) == 0) +x_48 = l_Lean_Elab_Tactic_renameInaccessibles(x_46, x_39, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_44); +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; 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_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; uint8_t x_53; +x_49 = lean_ctor_get(x_48, 0); lean_inc(x_49); -lean_dec(x_47); -x_50 = lean_box(0); -lean_inc(x_48); -lean_ctor_set_tag(x_42, 1); -lean_ctor_set(x_42, 1, x_50); -lean_ctor_set(x_42, 0, x_48); -x_51 = l_Lean_Elab_Tactic_setGoals(x_42, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_49); -x_52 = lean_ctor_get(x_51, 1); -lean_inc(x_52); -lean_dec(x_51); -x_53 = lean_box(0); -x_54 = l_Lean_MVarId_setTag(x_48, x_53, x_12, x_13, x_14, x_15, x_52); -x_55 = lean_ctor_get(x_54, 1); -lean_inc(x_55); -lean_dec(x_54); -x_56 = lean_unsigned_to_nat(3u); -x_57 = l_Lean_Elab_Tactic_evalWithAnnotateState___closed__1; -lean_inc(x_1); -x_58 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1), 12, 3); -lean_closure_set(x_58, 0, x_56); -lean_closure_set(x_58, 1, x_57); -lean_closure_set(x_58, 2, x_1); +x_50 = lean_ctor_get(x_48, 1); +lean_inc(x_50); +lean_dec(x_48); +x_51 = lean_box(0); +lean_inc(x_49); +lean_ctor_set_tag(x_43, 1); +lean_ctor_set(x_43, 1, x_51); +lean_ctor_set(x_43, 0, x_49); +x_52 = l_Lean_Elab_Tactic_setGoals(x_43, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, 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; uint8_t x_58; +x_54 = lean_ctor_get(x_52, 1); +x_55 = lean_ctor_get(x_52, 0); +lean_dec(x_55); +x_56 = lean_box(0); +x_57 = l_Lean_MVarId_setTag(x_49, x_56, x_13, x_14, x_15, x_16, x_54); +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, 1); +x_60 = lean_ctor_get(x_57, 0); +lean_dec(x_60); +lean_inc(x_3); +lean_ctor_set_tag(x_57, 1); +lean_ctor_set(x_57, 1, x_51); +lean_ctor_set(x_57, 0, x_3); +lean_inc(x_2); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_57); +lean_ctor_set(x_52, 0, x_2); +x_61 = lean_array_mk(x_52); +x_62 = lean_box(2); +x_63 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_64 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_64, 0, x_62); +lean_ctor_set(x_64, 1, x_63); +lean_ctor_set(x_64, 2, x_61); +x_65 = lean_unsigned_to_nat(3u); +x_66 = l_Lean_Elab_Tactic_evalWithAnnotateState___closed__1; lean_inc(x_1); -x_59 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); -lean_closure_set(x_59, 0, x_1); -lean_closure_set(x_59, 1, x_58); -x_60 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_closeUsingOrAdmit), 10, 1); -lean_closure_set(x_60, 0, x_59); +x_67 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1), 12, 3); +lean_closure_set(x_67, 0, x_65); +lean_closure_set(x_67, 1, x_66); +lean_closure_set(x_67, 2, x_1); +x_68 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_68, 0, x_64); +lean_closure_set(x_68, 1, x_67); +x_69 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_closeUsingOrAdmit), 10, 1); +lean_closure_set(x_69, 0, x_68); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -40732,31 +40756,31 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); +lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -x_61 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_2, x_3, x_60, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_55); -if (lean_obj_tag(x_61) == 0) +x_70 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_3, x_4, x_69, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_59); +if (lean_obj_tag(x_70) == 0) { -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_62 = lean_ctor_get(x_61, 1); -lean_inc(x_62); -lean_dec(x_61); -x_63 = l_Lean_Elab_Tactic_setGoals(x_46, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_62); -x_64 = lean_ctor_get(x_63, 1); -lean_inc(x_64); -lean_dec(x_63); -x_65 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_65, 0, x_7); -x_20 = x_65; -x_21 = x_64; -goto block_28; +lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_71 = lean_ctor_get(x_70, 1); +lean_inc(x_71); +lean_dec(x_70); +x_72 = l_Lean_Elab_Tactic_setGoals(x_47, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_71); +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_21 = x_74; +x_22 = x_73; +goto block_29; } else { -uint8_t x_66; -lean_dec(x_46); -lean_dec(x_7); +uint8_t x_75; +lean_dec(x_47); +lean_dec(x_8); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -40764,36 +40788,96 @@ lean_dec(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_2); lean_dec(x_1); -x_66 = !lean_is_exclusive(x_61); -if (x_66 == 0) +x_75 = !lean_is_exclusive(x_70); +if (x_75 == 0) { -return x_61; +return x_70; } else { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_61, 0); -x_68 = lean_ctor_get(x_61, 1); -lean_inc(x_68); -lean_inc(x_67); -lean_dec(x_61); -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_76; lean_object* x_77; lean_object* x_78; +x_76 = lean_ctor_get(x_70, 0); +x_77 = lean_ctor_get(x_70, 1); +lean_inc(x_77); +lean_inc(x_76); +lean_dec(x_70); +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_70; -lean_free_object(x_42); -lean_dec(x_46); -lean_dec(x_7); +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; +x_79 = lean_ctor_get(x_57, 1); +lean_inc(x_79); +lean_dec(x_57); +lean_inc(x_3); +x_80 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_80, 0, x_3); +lean_ctor_set(x_80, 1, x_51); +lean_inc(x_2); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_80); +lean_ctor_set(x_52, 0, x_2); +x_81 = lean_array_mk(x_52); +x_82 = lean_box(2); +x_83 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_84 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_83); +lean_ctor_set(x_84, 2, x_81); +x_85 = lean_unsigned_to_nat(3u); +x_86 = l_Lean_Elab_Tactic_evalWithAnnotateState___closed__1; +lean_inc(x_1); +x_87 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1), 12, 3); +lean_closure_set(x_87, 0, x_85); +lean_closure_set(x_87, 1, x_86); +lean_closure_set(x_87, 2, x_1); +x_88 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_88, 0, x_84); +lean_closure_set(x_88, 1, x_87); +x_89 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_closeUsingOrAdmit), 10, 1); +lean_closure_set(x_89, 0, x_88); +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_4); +lean_inc(x_3); +x_90 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_3, x_4, x_89, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_79); +if (lean_obj_tag(x_90) == 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); +x_92 = l_Lean_Elab_Tactic_setGoals(x_47, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_91); +x_93 = lean_ctor_get(x_92, 1); +lean_inc(x_93); +lean_dec(x_92); +x_94 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_94, 0, x_8); +x_21 = x_94; +x_22 = x_93; +goto block_29; +} +else +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +lean_dec(x_47); +lean_dec(x_8); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -40801,38 +40885,197 @@ lean_dec(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_2); lean_dec(x_1); -x_70 = !lean_is_exclusive(x_47); -if (x_70 == 0) +x_95 = lean_ctor_get(x_90, 0); +lean_inc(x_95); +x_96 = lean_ctor_get(x_90, 1); +lean_inc(x_96); +if (lean_is_exclusive(x_90)) { + lean_ctor_release(x_90, 0); + lean_ctor_release(x_90, 1); + x_97 = x_90; +} else { + lean_dec_ref(x_90); + 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 { -return x_47; +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_99 = lean_ctor_get(x_52, 1); +lean_inc(x_99); +lean_dec(x_52); +x_100 = lean_box(0); +x_101 = l_Lean_MVarId_setTag(x_49, x_100, x_13, x_14, x_15, x_16, x_99); +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); +} +lean_inc(x_3); +if (lean_is_scalar(x_103)) { + x_104 = lean_alloc_ctor(1, 2, 0); +} else { + x_104 = x_103; + lean_ctor_set_tag(x_104, 1); +} +lean_ctor_set(x_104, 0, x_3); +lean_ctor_set(x_104, 1, x_51); +lean_inc(x_2); +x_105 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_105, 0, x_2); +lean_ctor_set(x_105, 1, x_104); +x_106 = lean_array_mk(x_105); +x_107 = lean_box(2); +x_108 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_109 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_109, 0, x_107); +lean_ctor_set(x_109, 1, x_108); +lean_ctor_set(x_109, 2, x_106); +x_110 = lean_unsigned_to_nat(3u); +x_111 = l_Lean_Elab_Tactic_evalWithAnnotateState___closed__1; +lean_inc(x_1); +x_112 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1), 12, 3); +lean_closure_set(x_112, 0, x_110); +lean_closure_set(x_112, 1, x_111); +lean_closure_set(x_112, 2, x_1); +x_113 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_113, 0, x_109); +lean_closure_set(x_113, 1, x_112); +x_114 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_closeUsingOrAdmit), 10, 1); +lean_closure_set(x_114, 0, x_113); +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_4); +lean_inc(x_3); +x_115 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_3, x_4, x_114, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_102); +if (lean_obj_tag(x_115) == 0) +{ +lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; +x_116 = lean_ctor_get(x_115, 1); +lean_inc(x_116); +lean_dec(x_115); +x_117 = l_Lean_Elab_Tactic_setGoals(x_47, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_116); +x_118 = lean_ctor_get(x_117, 1); +lean_inc(x_118); +lean_dec(x_117); +x_119 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_119, 0, x_8); +x_21 = x_119; +x_22 = x_118; +goto block_29; } else { -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_ctor_get(x_47, 0); -x_72 = lean_ctor_get(x_47, 1); -lean_inc(x_72); -lean_inc(x_71); +lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_dec(x_47); -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_dec(x_8); +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_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_120 = lean_ctor_get(x_115, 0); +lean_inc(x_120); +x_121 = lean_ctor_get(x_115, 1); +lean_inc(x_121); +if (lean_is_exclusive(x_115)) { + lean_ctor_release(x_115, 0); + lean_ctor_release(x_115, 1); + x_122 = x_115; +} else { + lean_dec_ref(x_115); + x_122 = lean_box(0); +} +if (lean_is_scalar(x_122)) { + x_123 = lean_alloc_ctor(1, 2, 0); +} else { + x_123 = x_122; +} +lean_ctor_set(x_123, 0, x_120); +lean_ctor_set(x_123, 1, x_121); +return x_123; } } } else { -lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_74 = lean_ctor_get(x_42, 0); -x_75 = lean_ctor_get(x_42, 1); -lean_inc(x_75); -lean_inc(x_74); -lean_dec(x_42); +uint8_t x_124; +lean_free_object(x_43); +lean_dec(x_47); +lean_dec(x_8); +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_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_124 = !lean_is_exclusive(x_48); +if (x_124 == 0) +{ +return x_48; +} +else +{ +lean_object* x_125; lean_object* x_126; lean_object* x_127; +x_125 = lean_ctor_get(x_48, 0); +x_126 = lean_ctor_get(x_48, 1); +lean_inc(x_126); +lean_inc(x_125); +lean_dec(x_48); +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; lean_object* x_130; +x_128 = lean_ctor_get(x_43, 0); +x_129 = lean_ctor_get(x_43, 1); +lean_inc(x_129); +lean_inc(x_128); +lean_dec(x_43); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -40840,43 +41083,81 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); -x_76 = l_Lean_Elab_Tactic_renameInaccessibles(x_74, x_38, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_43); -if (lean_obj_tag(x_76) == 0) +x_130 = l_Lean_Elab_Tactic_renameInaccessibles(x_128, x_39, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_44); +if (lean_obj_tag(x_130) == 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; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; -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 = lean_box(0); -lean_inc(x_77); -x_80 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_80, 0, x_77); -lean_ctor_set(x_80, 1, x_79); -x_81 = l_Lean_Elab_Tactic_setGoals(x_80, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_78); -x_82 = lean_ctor_get(x_81, 1); -lean_inc(x_82); -lean_dec(x_81); -x_83 = lean_box(0); -x_84 = l_Lean_MVarId_setTag(x_77, x_83, x_12, x_13, x_14, x_15, x_82); -x_85 = lean_ctor_get(x_84, 1); -lean_inc(x_85); -lean_dec(x_84); -x_86 = lean_unsigned_to_nat(3u); -x_87 = l_Lean_Elab_Tactic_evalWithAnnotateState___closed__1; -lean_inc(x_1); -x_88 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1), 12, 3); -lean_closure_set(x_88, 0, x_86); -lean_closure_set(x_88, 1, x_87); -lean_closure_set(x_88, 2, x_1); +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; +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); +x_133 = lean_box(0); +lean_inc(x_131); +x_134 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_134, 0, x_131); +lean_ctor_set(x_134, 1, x_133); +x_135 = l_Lean_Elab_Tactic_setGoals(x_134, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_132); +x_136 = lean_ctor_get(x_135, 1); +lean_inc(x_136); +if (lean_is_exclusive(x_135)) { + lean_ctor_release(x_135, 0); + lean_ctor_release(x_135, 1); + x_137 = x_135; +} else { + lean_dec_ref(x_135); + x_137 = lean_box(0); +} +x_138 = lean_box(0); +x_139 = l_Lean_MVarId_setTag(x_131, x_138, x_13, x_14, x_15, x_16, x_136); +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); +} +lean_inc(x_3); +if (lean_is_scalar(x_141)) { + x_142 = lean_alloc_ctor(1, 2, 0); +} else { + x_142 = x_141; + lean_ctor_set_tag(x_142, 1); +} +lean_ctor_set(x_142, 0, x_3); +lean_ctor_set(x_142, 1, x_133); +lean_inc(x_2); +if (lean_is_scalar(x_137)) { + x_143 = lean_alloc_ctor(1, 2, 0); +} else { + x_143 = x_137; + lean_ctor_set_tag(x_143, 1); +} +lean_ctor_set(x_143, 0, x_2); +lean_ctor_set(x_143, 1, x_142); +x_144 = lean_array_mk(x_143); +x_145 = lean_box(2); +x_146 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_147 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_147, 0, x_145); +lean_ctor_set(x_147, 1, x_146); +lean_ctor_set(x_147, 2, x_144); +x_148 = lean_unsigned_to_nat(3u); +x_149 = l_Lean_Elab_Tactic_evalWithAnnotateState___closed__1; lean_inc(x_1); -x_89 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); -lean_closure_set(x_89, 0, x_1); -lean_closure_set(x_89, 1, x_88); -x_90 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_closeUsingOrAdmit), 10, 1); -lean_closure_set(x_90, 0, x_89); +x_150 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1), 12, 3); +lean_closure_set(x_150, 0, x_148); +lean_closure_set(x_150, 1, x_149); +lean_closure_set(x_150, 2, x_1); +x_151 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_151, 0, x_147); +lean_closure_set(x_151, 1, x_150); +x_152 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_closeUsingOrAdmit), 10, 1); +lean_closure_set(x_152, 0, x_151); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -40884,31 +41165,31 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); +lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -x_91 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_2, x_3, x_90, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_85); -if (lean_obj_tag(x_91) == 0) +x_153 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_3, x_4, x_152, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_140); +if (lean_obj_tag(x_153) == 0) { -lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_92 = lean_ctor_get(x_91, 1); -lean_inc(x_92); -lean_dec(x_91); -x_93 = l_Lean_Elab_Tactic_setGoals(x_75, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_92); -x_94 = lean_ctor_get(x_93, 1); -lean_inc(x_94); -lean_dec(x_93); -x_95 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_95, 0, x_7); -x_20 = x_95; -x_21 = x_94; -goto block_28; +lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; +x_154 = lean_ctor_get(x_153, 1); +lean_inc(x_154); +lean_dec(x_153); +x_155 = l_Lean_Elab_Tactic_setGoals(x_129, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_154); +x_156 = lean_ctor_get(x_155, 1); +lean_inc(x_156); +lean_dec(x_155); +x_157 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_157, 0, x_8); +x_21 = x_157; +x_22 = x_156; +goto block_29; } else { -lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; -lean_dec(x_75); -lean_dec(x_7); +lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; +lean_dec(x_129); +lean_dec(x_8); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -40916,37 +41197,38 @@ lean_dec(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_2); lean_dec(x_1); -x_96 = lean_ctor_get(x_91, 0); -lean_inc(x_96); -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; +x_158 = lean_ctor_get(x_153, 0); +lean_inc(x_158); +x_159 = lean_ctor_get(x_153, 1); +lean_inc(x_159); +if (lean_is_exclusive(x_153)) { + lean_ctor_release(x_153, 0); + lean_ctor_release(x_153, 1); + x_160 = x_153; } else { - lean_dec_ref(x_91); - x_98 = lean_box(0); + lean_dec_ref(x_153); + x_160 = lean_box(0); } -if (lean_is_scalar(x_98)) { - x_99 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_160)) { + x_161 = lean_alloc_ctor(1, 2, 0); } else { - x_99 = x_98; + x_161 = x_160; } -lean_ctor_set(x_99, 0, x_96); -lean_ctor_set(x_99, 1, x_97); -return x_99; +lean_ctor_set(x_161, 0, x_158); +lean_ctor_set(x_161, 1, x_159); +return x_161; } } else { -lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -lean_dec(x_75); -lean_dec(x_7); +lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; +lean_dec(x_129); +lean_dec(x_8); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -40954,38 +41236,39 @@ lean_dec(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_2); lean_dec(x_1); -x_100 = lean_ctor_get(x_76, 0); -lean_inc(x_100); -x_101 = lean_ctor_get(x_76, 1); -lean_inc(x_101); -if (lean_is_exclusive(x_76)) { - lean_ctor_release(x_76, 0); - lean_ctor_release(x_76, 1); - x_102 = x_76; +x_162 = lean_ctor_get(x_130, 0); +lean_inc(x_162); +x_163 = lean_ctor_get(x_130, 1); +lean_inc(x_163); +if (lean_is_exclusive(x_130)) { + lean_ctor_release(x_130, 0); + lean_ctor_release(x_130, 1); + x_164 = x_130; } else { - lean_dec_ref(x_76); - x_102 = lean_box(0); + lean_dec_ref(x_130); + x_164 = lean_box(0); } -if (lean_is_scalar(x_102)) { - x_103 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_164)) { + x_165 = lean_alloc_ctor(1, 2, 0); } else { - x_103 = x_102; + x_165 = x_164; } -lean_ctor_set(x_103, 0, x_100); -lean_ctor_set(x_103, 1, x_101); -return x_103; +lean_ctor_set(x_165, 0, x_162); +lean_ctor_set(x_165, 1, x_163); +return x_165; } } } else { -uint8_t x_104; -lean_dec(x_7); -lean_dec(x_38); +uint8_t x_166; +lean_dec(x_8); +lean_dec(x_39); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -40993,63 +41276,64 @@ lean_dec(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_2); lean_dec(x_1); -x_104 = !lean_is_exclusive(x_41); -if (x_104 == 0) +x_166 = !lean_is_exclusive(x_42); +if (x_166 == 0) { -return x_41; +return x_42; } else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_105 = lean_ctor_get(x_41, 0); -x_106 = lean_ctor_get(x_41, 1); -lean_inc(x_106); -lean_inc(x_105); -lean_dec(x_41); -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_167; lean_object* x_168; lean_object* x_169; +x_167 = lean_ctor_get(x_42, 0); +x_168 = lean_ctor_get(x_42, 1); +lean_inc(x_168); +lean_inc(x_167); +lean_dec(x_42); +x_169 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_169, 0, x_167); +lean_ctor_set(x_169, 1, x_168); +return x_169; } } } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; -lean_dec(x_7); -x_108 = lean_array_fget(x_29, x_30); -x_109 = lean_unsigned_to_nat(1u); -x_110 = lean_nat_add(x_30, x_109); -lean_dec(x_30); -x_111 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_111, 0, x_29); -lean_ctor_set(x_111, 1, x_110); -lean_ctor_set(x_111, 2, x_31); -x_112 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_112) == 0) +lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; +lean_dec(x_8); +x_170 = lean_array_fget(x_30, x_31); +x_171 = lean_unsigned_to_nat(1u); +x_172 = lean_nat_add(x_31, x_171); +lean_dec(x_31); +x_173 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_173, 0, x_30); +lean_ctor_set(x_173, 1, x_172); +lean_ctor_set(x_173, 2, x_32); +x_174 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_20, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +if (lean_obj_tag(x_174) == 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; -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); -x_115 = lean_ctor_get(x_113, 0); -lean_inc(x_115); -x_116 = lean_ctor_get(x_113, 1); -lean_inc(x_116); -if (lean_is_exclusive(x_113)) { - lean_ctor_release(x_113, 0); - lean_ctor_release(x_113, 1); - x_117 = x_113; +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_174, 0); +lean_inc(x_175); +x_176 = lean_ctor_get(x_174, 1); +lean_inc(x_176); +lean_dec(x_174); +x_177 = lean_ctor_get(x_175, 0); +lean_inc(x_177); +x_178 = lean_ctor_get(x_175, 1); +lean_inc(x_178); +if (lean_is_exclusive(x_175)) { + lean_ctor_release(x_175, 0); + lean_ctor_release(x_175, 1); + x_179 = x_175; } else { - lean_dec_ref(x_113); - x_117 = lean_box(0); + lean_dec_ref(x_175); + x_179 = lean_box(0); } +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -41057,48 +41341,86 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); -x_118 = l_Lean_Elab_Tactic_renameInaccessibles(x_115, x_108, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_114); -if (lean_obj_tag(x_118) == 0) +x_180 = l_Lean_Elab_Tactic_renameInaccessibles(x_177, x_170, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_176); +if (lean_obj_tag(x_180) == 0) { -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; -x_119 = lean_ctor_get(x_118, 0); -lean_inc(x_119); -x_120 = lean_ctor_get(x_118, 1); -lean_inc(x_120); -lean_dec(x_118); -x_121 = lean_box(0); -lean_inc(x_119); -if (lean_is_scalar(x_117)) { - x_122 = lean_alloc_ctor(1, 2, 0); +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; +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_box(0); +lean_inc(x_181); +if (lean_is_scalar(x_179)) { + x_184 = lean_alloc_ctor(1, 2, 0); } else { - x_122 = x_117; - lean_ctor_set_tag(x_122, 1); + x_184 = x_179; + lean_ctor_set_tag(x_184, 1); } -lean_ctor_set(x_122, 0, x_119); -lean_ctor_set(x_122, 1, x_121); -x_123 = l_Lean_Elab_Tactic_setGoals(x_122, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_120); -x_124 = lean_ctor_get(x_123, 1); -lean_inc(x_124); -lean_dec(x_123); -x_125 = lean_box(0); -x_126 = l_Lean_MVarId_setTag(x_119, x_125, x_12, x_13, x_14, x_15, x_124); -x_127 = lean_ctor_get(x_126, 1); -lean_inc(x_127); -lean_dec(x_126); -x_128 = lean_unsigned_to_nat(3u); -x_129 = l_Lean_Elab_Tactic_evalWithAnnotateState___closed__1; -lean_inc(x_1); -x_130 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1), 12, 3); -lean_closure_set(x_130, 0, x_128); -lean_closure_set(x_130, 1, x_129); -lean_closure_set(x_130, 2, x_1); +lean_ctor_set(x_184, 0, x_181); +lean_ctor_set(x_184, 1, x_183); +x_185 = l_Lean_Elab_Tactic_setGoals(x_184, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_182); +x_186 = lean_ctor_get(x_185, 1); +lean_inc(x_186); +if (lean_is_exclusive(x_185)) { + lean_ctor_release(x_185, 0); + lean_ctor_release(x_185, 1); + x_187 = x_185; +} else { + lean_dec_ref(x_185); + x_187 = lean_box(0); +} +x_188 = lean_box(0); +x_189 = l_Lean_MVarId_setTag(x_181, x_188, x_13, x_14, x_15, x_16, x_186); +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); +} +lean_inc(x_3); +if (lean_is_scalar(x_191)) { + x_192 = lean_alloc_ctor(1, 2, 0); +} else { + x_192 = x_191; + lean_ctor_set_tag(x_192, 1); +} +lean_ctor_set(x_192, 0, x_3); +lean_ctor_set(x_192, 1, x_183); +lean_inc(x_2); +if (lean_is_scalar(x_187)) { + x_193 = lean_alloc_ctor(1, 2, 0); +} else { + x_193 = x_187; + lean_ctor_set_tag(x_193, 1); +} +lean_ctor_set(x_193, 0, x_2); +lean_ctor_set(x_193, 1, x_192); +x_194 = lean_array_mk(x_193); +x_195 = lean_box(2); +x_196 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_197 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_197, 0, x_195); +lean_ctor_set(x_197, 1, x_196); +lean_ctor_set(x_197, 2, x_194); +x_198 = lean_unsigned_to_nat(3u); +x_199 = l_Lean_Elab_Tactic_evalWithAnnotateState___closed__1; lean_inc(x_1); -x_131 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); -lean_closure_set(x_131, 0, x_1); -lean_closure_set(x_131, 1, x_130); -x_132 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_closeUsingOrAdmit), 10, 1); -lean_closure_set(x_132, 0, x_131); +x_200 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1), 12, 3); +lean_closure_set(x_200, 0, x_198); +lean_closure_set(x_200, 1, x_199); +lean_closure_set(x_200, 2, x_1); +x_201 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_201, 0, x_197); +lean_closure_set(x_201, 1, x_200); +x_202 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_closeUsingOrAdmit), 10, 1); +lean_closure_set(x_202, 0, x_201); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -41106,31 +41428,31 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); +lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -x_133 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_2, x_3, x_132, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_127); -if (lean_obj_tag(x_133) == 0) +x_203 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_3, x_4, x_202, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_190); +if (lean_obj_tag(x_203) == 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); -x_135 = l_Lean_Elab_Tactic_setGoals(x_116, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_134); -x_136 = lean_ctor_get(x_135, 1); -lean_inc(x_136); -lean_dec(x_135); -x_137 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_137, 0, x_111); -x_20 = x_137; -x_21 = x_136; -goto block_28; +lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; +x_204 = lean_ctor_get(x_203, 1); +lean_inc(x_204); +lean_dec(x_203); +x_205 = l_Lean_Elab_Tactic_setGoals(x_178, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_204); +x_206 = lean_ctor_get(x_205, 1); +lean_inc(x_206); +lean_dec(x_205); +x_207 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_207, 0, x_173); +x_21 = x_207; +x_22 = x_206; +goto block_29; } else { -lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; -lean_dec(x_116); -lean_dec(x_111); +lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; +lean_dec(x_178); +lean_dec(x_173); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -41138,38 +41460,39 @@ lean_dec(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_2); lean_dec(x_1); -x_138 = lean_ctor_get(x_133, 0); -lean_inc(x_138); -x_139 = lean_ctor_get(x_133, 1); -lean_inc(x_139); -if (lean_is_exclusive(x_133)) { - lean_ctor_release(x_133, 0); - lean_ctor_release(x_133, 1); - x_140 = x_133; +x_208 = lean_ctor_get(x_203, 0); +lean_inc(x_208); +x_209 = lean_ctor_get(x_203, 1); +lean_inc(x_209); +if (lean_is_exclusive(x_203)) { + lean_ctor_release(x_203, 0); + lean_ctor_release(x_203, 1); + x_210 = x_203; } else { - lean_dec_ref(x_133); - x_140 = lean_box(0); + lean_dec_ref(x_203); + x_210 = lean_box(0); } -if (lean_is_scalar(x_140)) { - x_141 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_210)) { + x_211 = lean_alloc_ctor(1, 2, 0); } else { - x_141 = x_140; + x_211 = x_210; } -lean_ctor_set(x_141, 0, x_138); -lean_ctor_set(x_141, 1, x_139); -return x_141; +lean_ctor_set(x_211, 0, x_208); +lean_ctor_set(x_211, 1, x_209); +return x_211; } } else { -lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; -lean_dec(x_117); -lean_dec(x_116); -lean_dec(x_111); +lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; +lean_dec(x_179); +lean_dec(x_178); +lean_dec(x_173); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -41177,37 +41500,38 @@ lean_dec(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_2); lean_dec(x_1); -x_142 = lean_ctor_get(x_118, 0); -lean_inc(x_142); -x_143 = lean_ctor_get(x_118, 1); -lean_inc(x_143); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - x_144 = x_118; +x_212 = lean_ctor_get(x_180, 0); +lean_inc(x_212); +x_213 = lean_ctor_get(x_180, 1); +lean_inc(x_213); +if (lean_is_exclusive(x_180)) { + lean_ctor_release(x_180, 0); + lean_ctor_release(x_180, 1); + x_214 = x_180; } else { - lean_dec_ref(x_118); - x_144 = lean_box(0); + lean_dec_ref(x_180); + x_214 = lean_box(0); } -if (lean_is_scalar(x_144)) { - x_145 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_214)) { + x_215 = lean_alloc_ctor(1, 2, 0); } else { - x_145 = x_144; + x_215 = x_214; } -lean_ctor_set(x_145, 0, x_142); -lean_ctor_set(x_145, 1, x_143); -return x_145; +lean_ctor_set(x_215, 0, x_212); +lean_ctor_set(x_215, 1, x_213); +return x_215; } } else { -lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; -lean_dec(x_111); -lean_dec(x_108); +lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; +lean_dec(x_173); +lean_dec(x_170); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -41215,38 +41539,39 @@ lean_dec(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_2); lean_dec(x_1); -x_146 = lean_ctor_get(x_112, 0); -lean_inc(x_146); -x_147 = lean_ctor_get(x_112, 1); -lean_inc(x_147); -if (lean_is_exclusive(x_112)) { - lean_ctor_release(x_112, 0); - lean_ctor_release(x_112, 1); - x_148 = x_112; +x_216 = lean_ctor_get(x_174, 0); +lean_inc(x_216); +x_217 = lean_ctor_get(x_174, 1); +lean_inc(x_217); +if (lean_is_exclusive(x_174)) { + lean_ctor_release(x_174, 0); + lean_ctor_release(x_174, 1); + x_218 = x_174; } else { - lean_dec_ref(x_112); - x_148 = lean_box(0); + lean_dec_ref(x_174); + x_218 = lean_box(0); } -if (lean_is_scalar(x_148)) { - x_149 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_218)) { + x_219 = lean_alloc_ctor(1, 2, 0); } else { - x_149 = x_148; + x_219 = x_218; } -lean_ctor_set(x_149, 0, x_146); -lean_ctor_set(x_149, 1, x_147); -return x_149; +lean_ctor_set(x_219, 0, x_216); +lean_ctor_set(x_219, 1, x_217); +return x_219; } } } -block_28: +block_29: { -if (lean_obj_tag(x_20) == 0) +if (lean_obj_tag(x_21) == 0) { -lean_object* x_22; lean_object* x_23; +lean_object* x_23; lean_object* x_24; +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -41254,29 +41579,29 @@ lean_dec(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_2); lean_dec(x_1); -x_22 = lean_ctor_get(x_20, 0); -lean_inc(x_22); -lean_dec(x_20); -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; +x_23 = lean_ctor_get(x_21, 0); +lean_inc(x_23); +lean_dec(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 { -lean_object* x_24; size_t x_25; size_t x_26; -x_24 = lean_ctor_get(x_20, 0); -lean_inc(x_24); -lean_dec(x_20); -x_25 = 1; -x_26 = lean_usize_add(x_6, x_25); -x_6 = x_26; -x_7 = x_24; -x_16 = x_21; +lean_object* x_25; size_t x_26; size_t x_27; +x_25 = lean_ctor_get(x_21, 0); +lean_inc(x_25); +lean_dec(x_21); +x_26 = 1; +x_27 = lean_usize_add(x_7, x_26); +x_7 = x_27; +x_8 = x_25; +x_17 = x_22; goto _start; } } @@ -41336,57 +41661,57 @@ return x_11; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCase___lambda__2(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_Lean_Elab_Tactic_evalCase___lambda__2(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_object* x_9, 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_17; -x_17 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___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); -if (lean_obj_tag(x_17) == 0) +lean_object* x_18; +x_18 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___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, x_17); +if (lean_obj_tag(x_18) == 0) { -uint8_t x_18; -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) +uint8_t x_19; +x_19 = !lean_is_exclusive(x_18); +if (x_19 == 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; +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; } 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; +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; } } else { -uint8_t x_24; -x_24 = !lean_is_exclusive(x_17); -if (x_24 == 0) +uint8_t x_25; +x_25 = !lean_is_exclusive(x_18); +if (x_25 == 0) { -return x_17; +return x_18; } else { -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_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_18, 0); +x_27 = lean_ctor_get(x_18, 1); +lean_inc(x_27); 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; +lean_dec(x_18); +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; } } } @@ -41452,61 +41777,63 @@ return x_13; } else { -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_14 = lean_unsigned_to_nat(1u); +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; +x_14 = lean_unsigned_to_nat(0u); x_15 = l_Lean_Syntax_getArg(x_1, x_14); -x_16 = l_Lean_Syntax_getArgs(x_15); -lean_dec(x_15); -x_17 = lean_array_get_size(x_16); -x_18 = lean_unsigned_to_nat(0u); -x_19 = lean_nat_dec_lt(x_18, x_17); -if (x_19 == 0) -{ -lean_object* x_50; +x_16 = lean_unsigned_to_nat(1u); +x_17 = l_Lean_Syntax_getArg(x_1, x_16); +x_18 = l_Lean_Syntax_getArgs(x_17); lean_dec(x_17); -lean_dec(x_16); -x_50 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__12; -x_20 = x_50; -goto block_49; +x_19 = lean_array_get_size(x_18); +x_20 = lean_nat_dec_lt(x_14, x_19); +if (x_20 == 0) +{ +lean_object* x_51; +lean_dec(x_19); +lean_dec(x_18); +x_51 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__12; +x_21 = x_51; +goto block_50; } else { -uint8_t x_51; -x_51 = lean_nat_dec_le(x_17, x_17); -if (x_51 == 0) +uint8_t x_52; +x_52 = lean_nat_dec_le(x_19, x_19); +if (x_52 == 0) { -lean_object* x_52; -lean_dec(x_17); -lean_dec(x_16); -x_52 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__12; -x_20 = x_52; -goto block_49; +lean_object* x_53; +lean_dec(x_19); +lean_dec(x_18); +x_53 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__12; +x_21 = x_53; +goto block_50; } else { -size_t x_53; size_t x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_53 = 0; -x_54 = lean_usize_of_nat(x_17); -lean_dec(x_17); -x_55 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__13; -x_56 = l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1(x_16, x_53, x_54, x_55); -lean_dec(x_16); -x_57 = lean_ctor_get(x_56, 1); -lean_inc(x_57); -lean_dec(x_56); -x_20 = x_57; -goto block_49; +size_t x_54; size_t x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_54 = 0; +x_55 = lean_usize_of_nat(x_19); +lean_dec(x_19); +x_56 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__13; +x_57 = l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1(x_18, x_54, x_55, x_56); +lean_dec(x_18); +x_58 = lean_ctor_get(x_57, 1); +lean_inc(x_58); +lean_dec(x_57); +x_21 = x_58; +goto block_50; } } -block_49: +block_50: { -lean_object* x_21; lean_object* x_22; -x_21 = l_Lean_Elab_Tactic_evalCase___closed__3; -x_22 = l_Array_sequenceMap___at_Lean_Elab_Tactic_evalCase___spec__1(x_20, x_21); -lean_dec(x_20); -if (lean_obj_tag(x_22) == 0) +lean_object* x_22; lean_object* x_23; +x_22 = l_Lean_Elab_Tactic_evalCase___closed__3; +x_23 = l_Array_sequenceMap___at_Lean_Elab_Tactic_evalCase___spec__1(x_21, x_22); +lean_dec(x_21); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_23; +lean_object* x_24; +lean_dec(x_15); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -41516,34 +41843,35 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_23 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); -return x_23; +x_24 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); +return x_24; } else { -lean_object* x_24; size_t x_25; size_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; uint8_t x_34; -x_24 = lean_ctor_get(x_22, 0); -lean_inc(x_24); -lean_dec(x_22); -x_25 = lean_array_size(x_24); -x_26 = 0; -lean_inc(x_24); -x_27 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalCase___spec__3(x_25, x_26, x_24); -x_28 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalCase___spec__4(x_25, x_26, x_24); -x_29 = lean_unsigned_to_nat(2u); -x_30 = l_Lean_Syntax_getArg(x_1, x_29); -x_31 = lean_unsigned_to_nat(3u); -x_32 = l_Lean_Syntax_getArg(x_1, x_31); -x_33 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_addCheckpoints___spec__1___closed__4; -lean_inc(x_32); -x_34 = l_Lean_Syntax_isOfKind(x_32, x_33); -if (x_34 == 0) +lean_object* x_25; size_t x_26; size_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; uint8_t x_35; +x_25 = lean_ctor_get(x_23, 0); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_array_size(x_25); +x_27 = 0; +lean_inc(x_25); +x_28 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalCase___spec__3(x_26, x_27, x_25); +x_29 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalCase___spec__4(x_26, x_27, x_25); +x_30 = lean_unsigned_to_nat(2u); +x_31 = l_Lean_Syntax_getArg(x_1, x_30); +x_32 = lean_unsigned_to_nat(3u); +x_33 = l_Lean_Syntax_getArg(x_1, x_32); +x_34 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_addCheckpoints___spec__1___closed__4; +lean_inc(x_33); +x_35 = l_Lean_Syntax_isOfKind(x_33, x_34); +if (x_35 == 0) { -lean_object* x_35; -lean_dec(x_32); -lean_dec(x_30); +lean_object* x_36; +lean_dec(x_33); +lean_dec(x_31); +lean_dec(x_29); lean_dec(x_28); -lean_dec(x_27); +lean_dec(x_15); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -41553,24 +41881,25 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_35 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); -return x_35; +x_36 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); +return x_36; } else { -lean_object* x_36; lean_object* x_37; uint8_t x_38; -x_36 = l_Lean_Syntax_getArg(x_32, x_18); -lean_dec(x_32); -x_37 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_addCheckpoints___spec__1___closed__6; -lean_inc(x_36); -x_38 = l_Lean_Syntax_isOfKind(x_36, x_37); -if (x_38 == 0) +lean_object* x_37; lean_object* x_38; uint8_t x_39; +x_37 = l_Lean_Syntax_getArg(x_33, x_14); +lean_dec(x_33); +x_38 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_addCheckpoints___spec__1___closed__6; +lean_inc(x_37); +x_39 = l_Lean_Syntax_isOfKind(x_37, x_38); +if (x_39 == 0) { -lean_object* x_39; -lean_dec(x_36); -lean_dec(x_30); +lean_object* x_40; +lean_dec(x_37); +lean_dec(x_31); +lean_dec(x_29); lean_dec(x_28); -lean_dec(x_27); +lean_dec(x_15); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -41580,30 +41909,31 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_39 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); -return x_39; +x_40 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); +return x_40; } else { -lean_object* x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; size_t x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_40 = lean_array_get_size(x_28); -x_41 = lean_nat_dec_lt(x_14, x_40); -lean_dec(x_40); -x_42 = lean_array_get_size(x_27); -x_43 = l_Array_toSubarray___rarg(x_27, x_18, x_42); -x_44 = lean_array_size(x_28); -x_45 = lean_box_usize(x_44); -x_46 = l_Lean_Elab_Tactic_evalCase___boxed__const__1; -x_47 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalCase___lambda__2___boxed), 16, 7); -lean_closure_set(x_47, 0, x_1); -lean_closure_set(x_47, 1, x_30); -lean_closure_set(x_47, 2, x_36); -lean_closure_set(x_47, 3, x_28); -lean_closure_set(x_47, 4, x_45); -lean_closure_set(x_47, 5, x_46); -lean_closure_set(x_47, 6, x_43); -x_48 = l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_evalTactic_eval___spec__3(x_41, x_47, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_48; +lean_object* x_41; uint8_t x_42; lean_object* x_43; lean_object* x_44; size_t x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_41 = lean_array_get_size(x_29); +x_42 = lean_nat_dec_lt(x_16, x_41); +lean_dec(x_41); +x_43 = lean_array_get_size(x_28); +x_44 = l_Array_toSubarray___rarg(x_28, x_14, x_43); +x_45 = lean_array_size(x_29); +x_46 = lean_box_usize(x_45); +x_47 = l_Lean_Elab_Tactic_evalCase___boxed__const__1; +x_48 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalCase___lambda__2___boxed), 17, 8); +lean_closure_set(x_48, 0, x_1); +lean_closure_set(x_48, 1, x_15); +lean_closure_set(x_48, 2, x_31); +lean_closure_set(x_48, 3, x_37); +lean_closure_set(x_48, 4, x_29); +lean_closure_set(x_48, 5, x_46); +lean_closure_set(x_48, 6, x_47); +lean_closure_set(x_48, 7, x_44); +x_49 = l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_evalTactic_eval___spec__3(x_42, x_48, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_49; } } } @@ -41653,30 +41983,64 @@ x_6 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalCase___spec__4(x_4, x_5, return x_6; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___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) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___spec__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]; _start: { -size_t x_17; size_t x_18; lean_object* x_19; -x_17 = lean_unbox_usize(x_5); -lean_dec(x_5); +size_t x_18; size_t x_19; lean_object* x_20; x_18 = lean_unbox_usize(x_6); lean_dec(x_6); -x_19 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___spec__6(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); -return x_19; +x_19 = lean_unbox_usize(x_7); +lean_dec(x_7); +x_20 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase___spec__6(x_1, x_2, x_3, x_4, x_5, x_18, x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +lean_dec(x_5); +return x_20; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCase___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_Lean_Elab_Tactic_evalCase___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: { -size_t x_17; size_t x_18; lean_object* x_19; -x_17 = lean_unbox_usize(x_5); -lean_dec(x_5); +size_t x_18; size_t x_19; lean_object* x_20; x_18 = lean_unbox_usize(x_6); lean_dec(x_6); -x_19 = l_Lean_Elab_Tactic_evalCase___lambda__2(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); -return x_19; +x_19 = lean_unbox_usize(x_7); +lean_dec(x_7); +x_20 = l_Lean_Elab_Tactic_evalCase___lambda__2(x_1, x_2, x_3, x_4, x_5, x_18, x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +lean_dec(x_5); +return x_20; } } static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalCase__1___closed__1() { @@ -41868,14 +42232,15 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___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_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1(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_object* x_9, 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: { -uint8_t x_17; -x_17 = lean_usize_dec_lt(x_6, x_5); -if (x_17 == 0) +uint8_t x_18; +x_18 = lean_usize_dec_lt(x_7, x_6); +if (x_18 == 0) { -lean_object* x_18; +lean_object* x_19; +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -41883,79 +42248,80 @@ lean_dec(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_2); lean_dec(x_1); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_7); -lean_ctor_set(x_18, 1, x_16); -return x_18; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_8); +lean_ctor_set(x_19, 1, x_17); +return x_19; } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_29; -x_19 = lean_array_uget(x_4, x_6); -x_29 = !lean_is_exclusive(x_7); -if (x_29 == 0) +lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_30; +x_20 = lean_array_uget(x_5, x_7); +x_30 = !lean_is_exclusive(x_8); +if (x_30 == 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_7, 0); -x_31 = lean_ctor_get(x_7, 1); -x_32 = lean_ctor_get(x_30, 0); -lean_inc(x_32); -x_33 = 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; uint8_t x_36; +x_31 = lean_ctor_get(x_8, 0); +x_32 = lean_ctor_get(x_8, 1); +x_33 = lean_ctor_get(x_31, 0); lean_inc(x_33); -x_34 = lean_ctor_get(x_30, 2); +x_34 = lean_ctor_get(x_31, 1); lean_inc(x_34); -x_35 = lean_nat_dec_lt(x_33, x_34); -if (x_35 == 0) +x_35 = lean_ctor_get(x_31, 2); +lean_inc(x_35); +x_36 = lean_nat_dec_lt(x_34, x_35); +if (x_36 == 0) { -lean_object* x_36; +lean_object* x_37; +lean_dec(x_35); lean_dec(x_34); lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_19); -x_36 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_36, 0, x_7); -x_20 = x_36; -x_21 = x_16; -goto block_28; +lean_dec(x_20); +x_37 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_37, 0, x_8); +x_21 = x_37; +x_22 = x_17; +goto block_29; } else { -uint8_t x_37; -lean_free_object(x_7); -x_37 = !lean_is_exclusive(x_30); -if (x_37 == 0) +uint8_t x_38; +lean_free_object(x_8); +x_38 = !lean_is_exclusive(x_31); +if (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; -x_38 = lean_ctor_get(x_30, 2); -lean_dec(x_38); -x_39 = lean_ctor_get(x_30, 1); +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_31, 2); lean_dec(x_39); -x_40 = lean_ctor_get(x_30, 0); +x_40 = lean_ctor_get(x_31, 1); lean_dec(x_40); -x_41 = lean_array_fget(x_32, x_33); -x_42 = lean_unsigned_to_nat(1u); -x_43 = lean_nat_add(x_33, x_42); -lean_dec(x_33); -lean_ctor_set(x_30, 1, x_43); -x_44 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_44) == 0) +x_41 = lean_ctor_get(x_31, 0); +lean_dec(x_41); +x_42 = lean_array_fget(x_33, x_34); +x_43 = lean_unsigned_to_nat(1u); +x_44 = lean_nat_add(x_34, x_43); +lean_dec(x_34); +lean_ctor_set(x_31, 1, x_44); +x_45 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_20, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +if (lean_obj_tag(x_45) == 0) { -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_object* x_46; lean_object* x_47; uint8_t x_48; +x_46 = lean_ctor_get(x_45, 0); lean_inc(x_46); -lean_dec(x_44); -x_47 = !lean_is_exclusive(x_45); -if (x_47 == 0) +x_47 = lean_ctor_get(x_45, 1); +lean_inc(x_47); +lean_dec(x_45); +x_48 = !lean_is_exclusive(x_46); +if (x_48 == 0) { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_45, 0); -x_49 = lean_ctor_get(x_45, 1); +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_46, 0); +x_50 = lean_ctor_get(x_46, 1); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -41963,37 +42329,60 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); -x_50 = l_Lean_Elab_Tactic_renameInaccessibles(x_48, x_41, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_46); -if (lean_obj_tag(x_50) == 0) +x_51 = l_Lean_Elab_Tactic_renameInaccessibles(x_49, x_42, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_47); +if (lean_obj_tag(x_51) == 0) { -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_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_51, 0); lean_inc(x_52); -lean_dec(x_50); -lean_inc(x_51); -x_53 = l_Lean_MVarId_getTag(x_51, x_12, x_13, x_14, x_15, x_52); -if (lean_obj_tag(x_53) == 0) +x_53 = lean_ctor_get(x_51, 1); +lean_inc(x_53); +lean_dec(x_51); +lean_inc(x_52); +x_54 = l_Lean_MVarId_getTag(x_52, x_13, x_14, x_15, x_16, x_53); +if (lean_obj_tag(x_54) == 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; -x_54 = lean_ctor_get(x_53, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_53, 1); +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); -lean_dec(x_53); -lean_inc(x_3); -lean_ctor_set_tag(x_45, 1); -lean_ctor_set(x_45, 1, x_3); -lean_ctor_set(x_45, 0, x_51); -x_56 = l_Lean_Elab_Tactic_setGoals(x_45, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_55); -x_57 = lean_ctor_get(x_56, 1); -lean_inc(x_57); -lean_dec(x_56); +x_56 = lean_ctor_get(x_54, 1); +lean_inc(x_56); +lean_dec(x_54); +lean_inc(x_4); +lean_ctor_set_tag(x_46, 1); +lean_ctor_set(x_46, 1, x_4); +lean_ctor_set(x_46, 0, x_52); +x_57 = l_Lean_Elab_Tactic_setGoals(x_46, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, 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; +x_59 = lean_ctor_get(x_57, 1); +x_60 = lean_ctor_get(x_57, 0); +lean_dec(x_60); +x_61 = lean_box(0); lean_inc(x_2); -x_58 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); -lean_closure_set(x_58, 0, x_2); +lean_ctor_set_tag(x_57, 1); +lean_ctor_set(x_57, 1, x_61); +lean_ctor_set(x_57, 0, x_2); +lean_inc(x_1); +x_62 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_62, 0, x_1); +lean_ctor_set(x_62, 1, x_57); +x_63 = lean_array_mk(x_62); +x_64 = lean_box(2); +x_65 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_66 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +lean_ctor_set(x_66, 2, x_63); +lean_inc(x_3); +x_67 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); +lean_closure_set(x_67, 0, x_3); +x_68 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_68, 0, x_66); +lean_closure_set(x_68, 1, x_67); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -42001,172 +42390,95 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); +lean_inc(x_3); lean_inc(x_2); -lean_inc(x_1); -x_59 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_1, x_2, x_58, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_57); -if (lean_obj_tag(x_59) == 0) -{ -lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_60 = lean_ctor_get(x_59, 1); -lean_inc(x_60); -lean_dec(x_59); -x_61 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_60); -x_62 = lean_ctor_get(x_61, 0); -lean_inc(x_62); -if (lean_obj_tag(x_62) == 0) -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -lean_dec(x_54); -x_63 = lean_ctor_get(x_61, 1); -lean_inc(x_63); -lean_dec(x_61); -x_64 = lean_box(0); -x_65 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_62, x_49, x_30, x_31, x_64, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_63); -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_20 = x_66; -x_21 = x_67; -goto block_28; -} -else -{ -lean_object* x_68; -x_68 = lean_ctor_get(x_62, 1); -lean_inc(x_68); -if (lean_obj_tag(x_68) == 0) +x_69 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_2, x_3, x_68, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_59); +if (lean_obj_tag(x_69) == 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; -x_69 = lean_ctor_get(x_61, 1); -lean_inc(x_69); -lean_dec(x_61); -x_70 = lean_ctor_get(x_62, 0); +lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_70 = lean_ctor_get(x_69, 1); lean_inc(x_70); -x_71 = l_Lean_MVarId_setTag(x_70, x_54, x_12, x_13, x_14, x_15, x_69); +lean_dec(x_69); +x_71 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_70); 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_object* x_77; +lean_dec(x_55); x_73 = lean_ctor_get(x_71, 1); lean_inc(x_73); lean_dec(x_71); -x_74 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_62, x_49, x_30, x_31, x_72, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_73); -lean_dec(x_72); -x_75 = lean_ctor_get(x_74, 0); -lean_inc(x_75); -x_76 = lean_ctor_get(x_74, 1); +x_74 = lean_box(0); +x_75 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_72, x_50, x_31, x_32, x_74, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_73); +x_76 = lean_ctor_get(x_75, 0); lean_inc(x_76); -lean_dec(x_74); -x_20 = x_75; -x_21 = x_76; -goto block_28; -} -else -{ -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -lean_dec(x_68); -lean_dec(x_54); -x_77 = lean_ctor_get(x_61, 1); +x_77 = lean_ctor_get(x_75, 1); lean_inc(x_77); -lean_dec(x_61); -x_78 = lean_box(0); -x_79 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_62, x_49, x_30, x_31, x_78, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, 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); -lean_dec(x_79); -x_20 = x_80; -x_21 = x_81; -goto block_28; -} -} +lean_dec(x_75); +x_21 = x_76; +x_22 = x_77; +goto block_29; } else { -uint8_t x_82; -lean_dec(x_54); -lean_dec(x_49); -lean_dec(x_30); -lean_dec(x_31); -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_3); -lean_dec(x_2); -lean_dec(x_1); -x_82 = !lean_is_exclusive(x_59); -if (x_82 == 0) -{ -return x_59; -} -else +lean_object* x_78; +x_78 = lean_ctor_get(x_72, 1); +lean_inc(x_78); +if (lean_obj_tag(x_78) == 0) { -lean_object* x_83; lean_object* x_84; lean_object* x_85; -x_83 = lean_ctor_get(x_59, 0); -x_84 = lean_ctor_get(x_59, 1); -lean_inc(x_84); +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_71, 1); +lean_inc(x_79); +lean_dec(x_71); +x_80 = lean_ctor_get(x_72, 0); +lean_inc(x_80); +x_81 = l_Lean_MVarId_setTag(x_80, x_55, x_13, x_14, x_15, x_16, x_79); +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_59); -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_51); -lean_free_object(x_45); -lean_dec(x_49); -lean_dec(x_30); -lean_dec(x_31); -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_3); -lean_dec(x_2); -lean_dec(x_1); -x_86 = !lean_is_exclusive(x_53); -if (x_86 == 0) -{ -return x_53; +lean_dec(x_81); +x_84 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_72, x_50, x_31, x_32, x_82, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_83); +lean_dec(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_21 = x_85; +x_22 = x_86; +goto block_29; } else { -lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_87 = lean_ctor_get(x_53, 0); -x_88 = lean_ctor_get(x_53, 1); -lean_inc(x_88); +lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; +lean_dec(x_78); +lean_dec(x_55); +x_87 = lean_ctor_get(x_71, 1); lean_inc(x_87); -lean_dec(x_53); -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_dec(x_71); +x_88 = lean_box(0); +x_89 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_72, x_50, x_31, x_32, x_88, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_87); +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_21 = x_90; +x_22 = x_91; +goto block_29; } } } else { -uint8_t x_90; -lean_free_object(x_45); -lean_dec(x_49); -lean_dec(x_30); +uint8_t x_92; +lean_dec(x_55); +lean_dec(x_50); lean_dec(x_31); +lean_dec(x_32); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -42174,76 +42486,59 @@ lean_dec(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_2); lean_dec(x_1); -x_90 = !lean_is_exclusive(x_50); -if (x_90 == 0) +x_92 = !lean_is_exclusive(x_69); +if (x_92 == 0) { -return x_50; +return x_69; } else { -lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_91 = lean_ctor_get(x_50, 0); -x_92 = lean_ctor_get(x_50, 1); -lean_inc(x_92); -lean_inc(x_91); -lean_dec(x_50); -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_93; lean_object* x_94; lean_object* x_95; +x_93 = lean_ctor_get(x_69, 0); +x_94 = lean_ctor_get(x_69, 1); +lean_inc(x_94); +lean_inc(x_93); +lean_dec(x_69); +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 { -lean_object* x_94; lean_object* x_95; lean_object* x_96; -x_94 = lean_ctor_get(x_45, 0); -x_95 = lean_ctor_get(x_45, 1); -lean_inc(x_95); -lean_inc(x_94); -lean_dec(x_45); -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_96 = l_Lean_Elab_Tactic_renameInaccessibles(x_94, x_41, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_46); -if (lean_obj_tag(x_96) == 0) -{ -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_inc(x_97); -x_99 = l_Lean_MVarId_getTag(x_97, x_12, x_13, x_14, x_15, x_98); -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; 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); -lean_dec(x_99); -lean_inc(x_3); -x_102 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_102, 0, x_97); -lean_ctor_set(x_102, 1, x_3); -x_103 = l_Lean_Elab_Tactic_setGoals(x_102, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_101); -x_104 = lean_ctor_get(x_103, 1); -lean_inc(x_104); -lean_dec(x_103); +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_96 = lean_ctor_get(x_57, 1); +lean_inc(x_96); +lean_dec(x_57); +x_97 = lean_box(0); lean_inc(x_2); -x_105 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); -lean_closure_set(x_105, 0, x_2); +x_98 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_98, 0, x_2); +lean_ctor_set(x_98, 1, x_97); +lean_inc(x_1); +x_99 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_99, 0, x_1); +lean_ctor_set(x_99, 1, x_98); +x_100 = lean_array_mk(x_99); +x_101 = lean_box(2); +x_102 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_103 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_103, 0, x_101); +lean_ctor_set(x_103, 1, x_102); +lean_ctor_set(x_103, 2, x_100); +lean_inc(x_3); +x_104 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); +lean_closure_set(x_104, 0, x_3); +x_105 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_105, 0, x_103); +lean_closure_set(x_105, 1, x_104); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -42251,36 +42546,35 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); +lean_inc(x_3); lean_inc(x_2); -lean_inc(x_1); -x_106 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_1, x_2, x_105, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_104); +x_106 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_2, x_3, x_105, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_96); 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, 1); lean_inc(x_107); lean_dec(x_106); -x_108 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_107); +x_108 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_107); x_109 = lean_ctor_get(x_108, 0); lean_inc(x_109); 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_dec(x_100); +lean_dec(x_55); x_110 = lean_ctor_get(x_108, 1); lean_inc(x_110); lean_dec(x_108); x_111 = lean_box(0); -x_112 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_109, x_95, x_30, x_31, x_111, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_110); +x_112 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_109, x_50, x_31, x_32, x_111, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_110); 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); -x_20 = x_113; -x_21 = x_114; -goto block_28; +x_21 = x_113; +x_22 = x_114; +goto block_29; } else { @@ -42295,51 +42589,52 @@ lean_inc(x_116); lean_dec(x_108); x_117 = lean_ctor_get(x_109, 0); lean_inc(x_117); -x_118 = l_Lean_MVarId_setTag(x_117, x_100, x_12, x_13, x_14, x_15, x_116); +x_118 = l_Lean_MVarId_setTag(x_117, x_55, x_13, x_14, x_15, x_16, x_116); x_119 = lean_ctor_get(x_118, 0); lean_inc(x_119); x_120 = lean_ctor_get(x_118, 1); lean_inc(x_120); lean_dec(x_118); -x_121 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_109, x_95, x_30, x_31, x_119, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_120); +x_121 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_109, x_50, x_31, x_32, x_119, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_120); lean_dec(x_119); x_122 = lean_ctor_get(x_121, 0); lean_inc(x_122); x_123 = lean_ctor_get(x_121, 1); lean_inc(x_123); lean_dec(x_121); -x_20 = x_122; -x_21 = x_123; -goto block_28; +x_21 = x_122; +x_22 = x_123; +goto block_29; } else { lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_dec(x_115); -lean_dec(x_100); +lean_dec(x_55); x_124 = lean_ctor_get(x_108, 1); lean_inc(x_124); lean_dec(x_108); x_125 = lean_box(0); -x_126 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_109, x_95, x_30, x_31, x_125, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_124); +x_126 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_109, x_50, x_31, x_32, x_125, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_124); x_127 = lean_ctor_get(x_126, 0); lean_inc(x_127); x_128 = lean_ctor_get(x_126, 1); lean_inc(x_128); lean_dec(x_126); -x_20 = x_127; -x_21 = x_128; -goto block_28; +x_21 = x_127; +x_22 = x_128; +goto block_29; } } } else { lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; -lean_dec(x_100); -lean_dec(x_95); -lean_dec(x_30); +lean_dec(x_55); +lean_dec(x_50); lean_dec(x_31); +lean_dec(x_32); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -42347,7 +42642,7 @@ lean_dec(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_2); lean_dec(x_1); @@ -42373,13 +42668,16 @@ 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_dec(x_97); -lean_dec(x_95); -lean_dec(x_30); +uint8_t x_133; +lean_dec(x_52); +lean_free_object(x_46); +lean_dec(x_50); lean_dec(x_31); +lean_dec(x_32); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -42387,38 +42685,324 @@ lean_dec(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_2); lean_dec(x_1); -x_133 = lean_ctor_get(x_99, 0); -lean_inc(x_133); -x_134 = lean_ctor_get(x_99, 1); +x_133 = !lean_is_exclusive(x_54); +if (x_133 == 0) +{ +return x_54; +} +else +{ +lean_object* x_134; lean_object* x_135; lean_object* x_136; +x_134 = lean_ctor_get(x_54, 0); +x_135 = lean_ctor_get(x_54, 1); +lean_inc(x_135); lean_inc(x_134); -if (lean_is_exclusive(x_99)) { - lean_ctor_release(x_99, 0); - lean_ctor_release(x_99, 1); - x_135 = x_99; +lean_dec(x_54); +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_137; +lean_free_object(x_46); +lean_dec(x_50); +lean_dec(x_31); +lean_dec(x_32); +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_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_137 = !lean_is_exclusive(x_51); +if (x_137 == 0) +{ +return x_51; +} +else +{ +lean_object* x_138; lean_object* x_139; lean_object* x_140; +x_138 = lean_ctor_get(x_51, 0); +x_139 = lean_ctor_get(x_51, 1); +lean_inc(x_139); +lean_inc(x_138); +lean_dec(x_51); +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_object* x_141; lean_object* x_142; lean_object* x_143; +x_141 = lean_ctor_get(x_46, 0); +x_142 = lean_ctor_get(x_46, 1); +lean_inc(x_142); +lean_inc(x_141); +lean_dec(x_46); +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); +x_143 = l_Lean_Elab_Tactic_renameInaccessibles(x_141, x_42, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_47); +if (lean_obj_tag(x_143) == 0) +{ +lean_object* x_144; lean_object* x_145; lean_object* x_146; +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); +lean_inc(x_144); +x_146 = l_Lean_MVarId_getTag(x_144, x_13, x_14, x_15, x_16, x_145); +if (lean_obj_tag(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; 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; +x_147 = lean_ctor_get(x_146, 0); +lean_inc(x_147); +x_148 = lean_ctor_get(x_146, 1); +lean_inc(x_148); +lean_dec(x_146); +lean_inc(x_4); +x_149 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_149, 0, x_144); +lean_ctor_set(x_149, 1, x_4); +x_150 = l_Lean_Elab_Tactic_setGoals(x_149, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_148); +x_151 = lean_ctor_get(x_150, 1); +lean_inc(x_151); +if (lean_is_exclusive(x_150)) { + lean_ctor_release(x_150, 0); + lean_ctor_release(x_150, 1); + x_152 = x_150; } else { - lean_dec_ref(x_99); - x_135 = lean_box(0); + lean_dec_ref(x_150); + x_152 = lean_box(0); +} +x_153 = lean_box(0); +lean_inc(x_2); +if (lean_is_scalar(x_152)) { + x_154 = lean_alloc_ctor(1, 2, 0); +} else { + x_154 = x_152; + lean_ctor_set_tag(x_154, 1); +} +lean_ctor_set(x_154, 0, x_2); +lean_ctor_set(x_154, 1, x_153); +lean_inc(x_1); +x_155 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_155, 0, x_1); +lean_ctor_set(x_155, 1, x_154); +x_156 = lean_array_mk(x_155); +x_157 = lean_box(2); +x_158 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_159 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_159, 0, x_157); +lean_ctor_set(x_159, 1, x_158); +lean_ctor_set(x_159, 2, x_156); +lean_inc(x_3); +x_160 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); +lean_closure_set(x_160, 0, x_3); +x_161 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_161, 0, x_159); +lean_closure_set(x_161, 1, x_160); +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_3); +lean_inc(x_2); +x_162 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_2, x_3, x_161, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_151); +if (lean_obj_tag(x_162) == 0) +{ +lean_object* x_163; lean_object* x_164; lean_object* x_165; +x_163 = lean_ctor_get(x_162, 1); +lean_inc(x_163); +lean_dec(x_162); +x_164 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_163); +x_165 = lean_ctor_get(x_164, 0); +lean_inc(x_165); +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_dec(x_147); +x_166 = lean_ctor_get(x_164, 1); +lean_inc(x_166); +lean_dec(x_164); +x_167 = lean_box(0); +x_168 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_165, x_142, x_31, x_32, x_167, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_166); +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_21 = x_169; +x_22 = x_170; +goto block_29; +} +else +{ +lean_object* x_171; +x_171 = lean_ctor_get(x_165, 1); +lean_inc(x_171); +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; +x_172 = lean_ctor_get(x_164, 1); +lean_inc(x_172); +lean_dec(x_164); +x_173 = lean_ctor_get(x_165, 0); +lean_inc(x_173); +x_174 = l_Lean_MVarId_setTag(x_173, x_147, x_13, x_14, x_15, x_16, 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); +lean_dec(x_174); +x_177 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_165, x_142, x_31, x_32, x_175, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_176); +lean_dec(x_175); +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_21 = x_178; +x_22 = x_179; +goto block_29; +} +else +{ +lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; +lean_dec(x_171); +lean_dec(x_147); +x_180 = lean_ctor_get(x_164, 1); +lean_inc(x_180); +lean_dec(x_164); +x_181 = lean_box(0); +x_182 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_165, x_142, x_31, x_32, x_181, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_180); +x_183 = lean_ctor_get(x_182, 0); +lean_inc(x_183); +x_184 = lean_ctor_get(x_182, 1); +lean_inc(x_184); +lean_dec(x_182); +x_21 = x_183; +x_22 = x_184; +goto block_29; +} +} +} +else +{ +lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; +lean_dec(x_147); +lean_dec(x_142); +lean_dec(x_31); +lean_dec(x_32); +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_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_185 = lean_ctor_get(x_162, 0); +lean_inc(x_185); +x_186 = lean_ctor_get(x_162, 1); +lean_inc(x_186); +if (lean_is_exclusive(x_162)) { + lean_ctor_release(x_162, 0); + lean_ctor_release(x_162, 1); + x_187 = x_162; +} else { + lean_dec_ref(x_162); + x_187 = lean_box(0); +} +if (lean_is_scalar(x_187)) { + x_188 = lean_alloc_ctor(1, 2, 0); +} else { + x_188 = x_187; +} +lean_ctor_set(x_188, 0, x_185); +lean_ctor_set(x_188, 1, x_186); +return x_188; +} +} +else +{ +lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; +lean_dec(x_144); +lean_dec(x_142); +lean_dec(x_31); +lean_dec(x_32); +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_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_189 = lean_ctor_get(x_146, 0); +lean_inc(x_189); +x_190 = lean_ctor_get(x_146, 1); +lean_inc(x_190); +if (lean_is_exclusive(x_146)) { + lean_ctor_release(x_146, 0); + lean_ctor_release(x_146, 1); + x_191 = x_146; +} else { + lean_dec_ref(x_146); + x_191 = lean_box(0); } -if (lean_is_scalar(x_135)) { - x_136 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_191)) { + x_192 = lean_alloc_ctor(1, 2, 0); } else { - x_136 = x_135; + x_192 = x_191; } -lean_ctor_set(x_136, 0, x_133); -lean_ctor_set(x_136, 1, x_134); -return x_136; +lean_ctor_set(x_192, 0, x_189); +lean_ctor_set(x_192, 1, x_190); +return x_192; } } else { -lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; -lean_dec(x_95); -lean_dec(x_30); +lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; +lean_dec(x_142); lean_dec(x_31); +lean_dec(x_32); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -42426,39 +43010,40 @@ lean_dec(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_2); lean_dec(x_1); -x_137 = lean_ctor_get(x_96, 0); -lean_inc(x_137); -x_138 = lean_ctor_get(x_96, 1); -lean_inc(x_138); -if (lean_is_exclusive(x_96)) { - lean_ctor_release(x_96, 0); - lean_ctor_release(x_96, 1); - x_139 = x_96; +x_193 = lean_ctor_get(x_143, 0); +lean_inc(x_193); +x_194 = lean_ctor_get(x_143, 1); +lean_inc(x_194); +if (lean_is_exclusive(x_143)) { + lean_ctor_release(x_143, 0); + lean_ctor_release(x_143, 1); + x_195 = x_143; } else { - lean_dec_ref(x_96); - x_139 = lean_box(0); + lean_dec_ref(x_143); + x_195 = lean_box(0); } -if (lean_is_scalar(x_139)) { - x_140 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_195)) { + x_196 = lean_alloc_ctor(1, 2, 0); } else { - x_140 = x_139; + x_196 = x_195; } -lean_ctor_set(x_140, 0, x_137); -lean_ctor_set(x_140, 1, x_138); -return x_140; +lean_ctor_set(x_196, 0, x_193); +lean_ctor_set(x_196, 1, x_194); +return x_196; } } } else { -uint8_t x_141; -lean_dec(x_30); -lean_dec(x_41); +uint8_t x_197; lean_dec(x_31); +lean_dec(x_42); +lean_dec(x_32); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -42466,63 +43051,64 @@ lean_dec(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_2); lean_dec(x_1); -x_141 = !lean_is_exclusive(x_44); -if (x_141 == 0) +x_197 = !lean_is_exclusive(x_45); +if (x_197 == 0) { -return x_44; +return x_45; } else { -lean_object* x_142; lean_object* x_143; lean_object* x_144; -x_142 = lean_ctor_get(x_44, 0); -x_143 = lean_ctor_get(x_44, 1); -lean_inc(x_143); -lean_inc(x_142); -lean_dec(x_44); -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; +lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_198 = lean_ctor_get(x_45, 0); +x_199 = lean_ctor_get(x_45, 1); +lean_inc(x_199); +lean_inc(x_198); +lean_dec(x_45); +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_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; -lean_dec(x_30); -x_145 = lean_array_fget(x_32, x_33); -x_146 = lean_unsigned_to_nat(1u); -x_147 = lean_nat_add(x_33, x_146); -lean_dec(x_33); -x_148 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_148, 0, x_32); -lean_ctor_set(x_148, 1, x_147); -lean_ctor_set(x_148, 2, x_34); -x_149 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_149) == 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; -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 = lean_ctor_get(x_150, 0); -lean_inc(x_152); -x_153 = lean_ctor_get(x_150, 1); -lean_inc(x_153); -if (lean_is_exclusive(x_150)) { - lean_ctor_release(x_150, 0); - lean_ctor_release(x_150, 1); - x_154 = x_150; +lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; +lean_dec(x_31); +x_201 = lean_array_fget(x_33, x_34); +x_202 = lean_unsigned_to_nat(1u); +x_203 = lean_nat_add(x_34, x_202); +lean_dec(x_34); +x_204 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_204, 0, x_33); +lean_ctor_set(x_204, 1, x_203); +lean_ctor_set(x_204, 2, x_35); +x_205 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_20, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +if (lean_obj_tag(x_205) == 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_205, 0); +lean_inc(x_206); +x_207 = lean_ctor_get(x_205, 1); +lean_inc(x_207); +lean_dec(x_205); +x_208 = lean_ctor_get(x_206, 0); +lean_inc(x_208); +x_209 = lean_ctor_get(x_206, 1); +lean_inc(x_209); +if (lean_is_exclusive(x_206)) { + lean_ctor_release(x_206, 0); + lean_ctor_release(x_206, 1); + x_210 = x_206; } else { - lean_dec_ref(x_150); - x_154 = lean_box(0); + lean_dec_ref(x_206); + x_210 = lean_box(0); } +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -42530,42 +43116,73 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); -x_155 = l_Lean_Elab_Tactic_renameInaccessibles(x_152, x_145, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_151); -if (lean_obj_tag(x_155) == 0) +x_211 = l_Lean_Elab_Tactic_renameInaccessibles(x_208, x_201, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_207); +if (lean_obj_tag(x_211) == 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); -x_157 = lean_ctor_get(x_155, 1); -lean_inc(x_157); -lean_dec(x_155); -lean_inc(x_156); -x_158 = l_Lean_MVarId_getTag(x_156, x_12, x_13, x_14, x_15, x_157); -if (lean_obj_tag(x_158) == 0) +lean_object* x_212; lean_object* x_213; lean_object* x_214; +x_212 = lean_ctor_get(x_211, 0); +lean_inc(x_212); +x_213 = lean_ctor_get(x_211, 1); +lean_inc(x_213); +lean_dec(x_211); +lean_inc(x_212); +x_214 = l_Lean_MVarId_getTag(x_212, x_13, x_14, x_15, x_16, x_213); +if (lean_obj_tag(x_214) == 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; -x_159 = lean_ctor_get(x_158, 0); -lean_inc(x_159); -x_160 = lean_ctor_get(x_158, 1); -lean_inc(x_160); -lean_dec(x_158); -lean_inc(x_3); -if (lean_is_scalar(x_154)) { - x_161 = lean_alloc_ctor(1, 2, 0); +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; +x_215 = lean_ctor_get(x_214, 0); +lean_inc(x_215); +x_216 = lean_ctor_get(x_214, 1); +lean_inc(x_216); +lean_dec(x_214); +lean_inc(x_4); +if (lean_is_scalar(x_210)) { + x_217 = lean_alloc_ctor(1, 2, 0); } else { - x_161 = x_154; - lean_ctor_set_tag(x_161, 1); + x_217 = x_210; + lean_ctor_set_tag(x_217, 1); } -lean_ctor_set(x_161, 0, x_156); -lean_ctor_set(x_161, 1, x_3); -x_162 = l_Lean_Elab_Tactic_setGoals(x_161, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_160); -x_163 = lean_ctor_get(x_162, 1); -lean_inc(x_163); -lean_dec(x_162); +lean_ctor_set(x_217, 0, x_212); +lean_ctor_set(x_217, 1, x_4); +x_218 = l_Lean_Elab_Tactic_setGoals(x_217, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_216); +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; +} else { + lean_dec_ref(x_218); + x_220 = lean_box(0); +} +x_221 = lean_box(0); lean_inc(x_2); -x_164 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); -lean_closure_set(x_164, 0, x_2); +if (lean_is_scalar(x_220)) { + x_222 = lean_alloc_ctor(1, 2, 0); +} else { + x_222 = x_220; + lean_ctor_set_tag(x_222, 1); +} +lean_ctor_set(x_222, 0, x_2); +lean_ctor_set(x_222, 1, x_221); +lean_inc(x_1); +x_223 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_223, 0, x_1); +lean_ctor_set(x_223, 1, x_222); +x_224 = lean_array_mk(x_223); +x_225 = lean_box(2); +x_226 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_227 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_227, 0, x_225); +lean_ctor_set(x_227, 1, x_226); +lean_ctor_set(x_227, 2, x_224); +lean_inc(x_3); +x_228 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); +lean_closure_set(x_228, 0, x_3); +x_229 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_229, 0, x_227); +lean_closure_set(x_229, 1, x_228); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -42573,95 +43190,95 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); +lean_inc(x_3); lean_inc(x_2); -lean_inc(x_1); -x_165 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_1, x_2, x_164, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_163); -if (lean_obj_tag(x_165) == 0) +x_230 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_2, x_3, x_229, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_219); +if (lean_obj_tag(x_230) == 0) { -lean_object* x_166; lean_object* x_167; lean_object* x_168; -x_166 = lean_ctor_get(x_165, 1); -lean_inc(x_166); -lean_dec(x_165); -x_167 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_166); -x_168 = lean_ctor_get(x_167, 0); -lean_inc(x_168); -if (lean_obj_tag(x_168) == 0) +lean_object* x_231; lean_object* x_232; lean_object* x_233; +x_231 = lean_ctor_get(x_230, 1); +lean_inc(x_231); +lean_dec(x_230); +x_232 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_231); +x_233 = lean_ctor_get(x_232, 0); +lean_inc(x_233); +if (lean_obj_tag(x_233) == 0) { -lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; -lean_dec(x_159); -x_169 = lean_ctor_get(x_167, 1); -lean_inc(x_169); -lean_dec(x_167); -x_170 = lean_box(0); -x_171 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_168, x_153, x_148, x_31, x_170, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, 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_20 = x_172; -x_21 = x_173; -goto block_28; +lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; +lean_dec(x_215); +x_234 = lean_ctor_get(x_232, 1); +lean_inc(x_234); +lean_dec(x_232); +x_235 = lean_box(0); +x_236 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_233, x_209, x_204, x_32, x_235, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_234); +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_21 = x_237; +x_22 = x_238; +goto block_29; } else { -lean_object* x_174; -x_174 = lean_ctor_get(x_168, 1); -lean_inc(x_174); -if (lean_obj_tag(x_174) == 0) +lean_object* x_239; +x_239 = lean_ctor_get(x_233, 1); +lean_inc(x_239); +if (lean_obj_tag(x_239) == 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; lean_object* x_182; -x_175 = lean_ctor_get(x_167, 1); -lean_inc(x_175); -lean_dec(x_167); -x_176 = lean_ctor_get(x_168, 0); -lean_inc(x_176); -x_177 = l_Lean_MVarId_setTag(x_176, x_159, x_12, x_13, x_14, x_15, x_175); -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_180 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_168, x_153, x_148, x_31, x_178, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_179); -lean_dec(x_178); -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_20 = x_181; -x_21 = x_182; -goto block_28; +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; +x_240 = lean_ctor_get(x_232, 1); +lean_inc(x_240); +lean_dec(x_232); +x_241 = lean_ctor_get(x_233, 0); +lean_inc(x_241); +x_242 = l_Lean_MVarId_setTag(x_241, x_215, x_13, x_14, x_15, x_16, 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); +lean_dec(x_242); +x_245 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_233, x_209, x_204, x_32, x_243, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_244); +lean_dec(x_243); +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_21 = x_246; +x_22 = x_247; +goto block_29; } else { -lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; -lean_dec(x_174); -lean_dec(x_159); -x_183 = lean_ctor_get(x_167, 1); -lean_inc(x_183); -lean_dec(x_167); -x_184 = lean_box(0); -x_185 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_168, x_153, x_148, x_31, x_184, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_183); -x_186 = lean_ctor_get(x_185, 0); -lean_inc(x_186); -x_187 = lean_ctor_get(x_185, 1); -lean_inc(x_187); -lean_dec(x_185); -x_20 = x_186; -x_21 = x_187; -goto block_28; +lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; +lean_dec(x_239); +lean_dec(x_215); +x_248 = lean_ctor_get(x_232, 1); +lean_inc(x_248); +lean_dec(x_232); +x_249 = lean_box(0); +x_250 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_233, x_209, x_204, x_32, x_249, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_248); +x_251 = lean_ctor_get(x_250, 0); +lean_inc(x_251); +x_252 = lean_ctor_get(x_250, 1); +lean_inc(x_252); +lean_dec(x_250); +x_21 = x_251; +x_22 = x_252; +goto block_29; } } } else { -lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; -lean_dec(x_159); -lean_dec(x_153); -lean_dec(x_148); -lean_dec(x_31); +lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; +lean_dec(x_215); +lean_dec(x_209); +lean_dec(x_204); +lean_dec(x_32); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -42669,40 +43286,41 @@ lean_dec(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_2); lean_dec(x_1); -x_188 = lean_ctor_get(x_165, 0); -lean_inc(x_188); -x_189 = lean_ctor_get(x_165, 1); -lean_inc(x_189); -if (lean_is_exclusive(x_165)) { - lean_ctor_release(x_165, 0); - lean_ctor_release(x_165, 1); - x_190 = x_165; +x_253 = lean_ctor_get(x_230, 0); +lean_inc(x_253); +x_254 = lean_ctor_get(x_230, 1); +lean_inc(x_254); +if (lean_is_exclusive(x_230)) { + lean_ctor_release(x_230, 0); + lean_ctor_release(x_230, 1); + x_255 = x_230; } else { - lean_dec_ref(x_165); - x_190 = lean_box(0); + lean_dec_ref(x_230); + x_255 = lean_box(0); } -if (lean_is_scalar(x_190)) { - x_191 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_255)) { + x_256 = lean_alloc_ctor(1, 2, 0); } else { - x_191 = x_190; + x_256 = x_255; } -lean_ctor_set(x_191, 0, x_188); -lean_ctor_set(x_191, 1, x_189); -return x_191; +lean_ctor_set(x_256, 0, x_253); +lean_ctor_set(x_256, 1, x_254); +return x_256; } } else { -lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; -lean_dec(x_156); -lean_dec(x_154); -lean_dec(x_153); -lean_dec(x_148); -lean_dec(x_31); +lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; +lean_dec(x_212); +lean_dec(x_210); +lean_dec(x_209); +lean_dec(x_204); +lean_dec(x_32); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -42710,39 +43328,40 @@ lean_dec(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_2); lean_dec(x_1); -x_192 = lean_ctor_get(x_158, 0); -lean_inc(x_192); -x_193 = lean_ctor_get(x_158, 1); -lean_inc(x_193); -if (lean_is_exclusive(x_158)) { - lean_ctor_release(x_158, 0); - lean_ctor_release(x_158, 1); - x_194 = x_158; +x_257 = lean_ctor_get(x_214, 0); +lean_inc(x_257); +x_258 = lean_ctor_get(x_214, 1); +lean_inc(x_258); +if (lean_is_exclusive(x_214)) { + lean_ctor_release(x_214, 0); + lean_ctor_release(x_214, 1); + x_259 = x_214; } else { - lean_dec_ref(x_158); - x_194 = lean_box(0); + lean_dec_ref(x_214); + x_259 = lean_box(0); } -if (lean_is_scalar(x_194)) { - x_195 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_259)) { + x_260 = lean_alloc_ctor(1, 2, 0); } else { - x_195 = x_194; + x_260 = x_259; } -lean_ctor_set(x_195, 0, x_192); -lean_ctor_set(x_195, 1, x_193); -return x_195; +lean_ctor_set(x_260, 0, x_257); +lean_ctor_set(x_260, 1, x_258); +return x_260; } } else { -lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; -lean_dec(x_154); -lean_dec(x_153); -lean_dec(x_148); -lean_dec(x_31); +lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; +lean_dec(x_210); +lean_dec(x_209); +lean_dec(x_204); +lean_dec(x_32); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -42750,38 +43369,39 @@ lean_dec(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_2); lean_dec(x_1); -x_196 = lean_ctor_get(x_155, 0); -lean_inc(x_196); -x_197 = lean_ctor_get(x_155, 1); -lean_inc(x_197); -if (lean_is_exclusive(x_155)) { - lean_ctor_release(x_155, 0); - lean_ctor_release(x_155, 1); - x_198 = x_155; +x_261 = lean_ctor_get(x_211, 0); +lean_inc(x_261); +x_262 = lean_ctor_get(x_211, 1); +lean_inc(x_262); +if (lean_is_exclusive(x_211)) { + lean_ctor_release(x_211, 0); + lean_ctor_release(x_211, 1); + x_263 = x_211; } else { - lean_dec_ref(x_155); - x_198 = lean_box(0); + lean_dec_ref(x_211); + x_263 = lean_box(0); } -if (lean_is_scalar(x_198)) { - x_199 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_263)) { + x_264 = lean_alloc_ctor(1, 2, 0); } else { - x_199 = x_198; + x_264 = x_263; } -lean_ctor_set(x_199, 0, x_196); -lean_ctor_set(x_199, 1, x_197); -return x_199; +lean_ctor_set(x_264, 0, x_261); +lean_ctor_set(x_264, 1, x_262); +return x_264; } } else { -lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; -lean_dec(x_148); -lean_dec(x_145); -lean_dec(x_31); +lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; +lean_dec(x_204); +lean_dec(x_201); +lean_dec(x_32); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -42789,110 +43409,111 @@ lean_dec(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_2); lean_dec(x_1); -x_200 = lean_ctor_get(x_149, 0); -lean_inc(x_200); -x_201 = lean_ctor_get(x_149, 1); -lean_inc(x_201); -if (lean_is_exclusive(x_149)) { - lean_ctor_release(x_149, 0); - lean_ctor_release(x_149, 1); - x_202 = x_149; +x_265 = lean_ctor_get(x_205, 0); +lean_inc(x_265); +x_266 = lean_ctor_get(x_205, 1); +lean_inc(x_266); +if (lean_is_exclusive(x_205)) { + lean_ctor_release(x_205, 0); + lean_ctor_release(x_205, 1); + x_267 = x_205; } else { - lean_dec_ref(x_149); - x_202 = lean_box(0); + lean_dec_ref(x_205); + x_267 = lean_box(0); } -if (lean_is_scalar(x_202)) { - x_203 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_267)) { + x_268 = lean_alloc_ctor(1, 2, 0); } else { - x_203 = x_202; + x_268 = x_267; } -lean_ctor_set(x_203, 0, x_200); -lean_ctor_set(x_203, 1, x_201); -return x_203; +lean_ctor_set(x_268, 0, x_265); +lean_ctor_set(x_268, 1, x_266); +return x_268; } } } } else { -lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; uint8_t x_209; -x_204 = lean_ctor_get(x_7, 0); -x_205 = lean_ctor_get(x_7, 1); -lean_inc(x_205); -lean_inc(x_204); -lean_dec(x_7); -x_206 = lean_ctor_get(x_204, 0); -lean_inc(x_206); -x_207 = lean_ctor_get(x_204, 1); -lean_inc(x_207); -x_208 = lean_ctor_get(x_204, 2); -lean_inc(x_208); -x_209 = lean_nat_dec_lt(x_207, x_208); -if (x_209 == 0) +lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; uint8_t x_274; +x_269 = lean_ctor_get(x_8, 0); +x_270 = lean_ctor_get(x_8, 1); +lean_inc(x_270); +lean_inc(x_269); +lean_dec(x_8); +x_271 = lean_ctor_get(x_269, 0); +lean_inc(x_271); +x_272 = lean_ctor_get(x_269, 1); +lean_inc(x_272); +x_273 = lean_ctor_get(x_269, 2); +lean_inc(x_273); +x_274 = lean_nat_dec_lt(x_272, x_273); +if (x_274 == 0) { -lean_object* x_210; lean_object* x_211; -lean_dec(x_208); -lean_dec(x_207); -lean_dec(x_206); -lean_dec(x_19); -x_210 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_210, 0, x_204); -lean_ctor_set(x_210, 1, x_205); -x_211 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_211, 0, x_210); -x_20 = x_211; -x_21 = x_16; -goto block_28; +lean_object* x_275; lean_object* x_276; +lean_dec(x_273); +lean_dec(x_272); +lean_dec(x_271); +lean_dec(x_20); +x_275 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_275, 0, x_269); +lean_ctor_set(x_275, 1, x_270); +x_276 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_276, 0, x_275); +x_21 = x_276; +x_22 = x_17; +goto block_29; } 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; -if (lean_is_exclusive(x_204)) { - lean_ctor_release(x_204, 0); - lean_ctor_release(x_204, 1); - lean_ctor_release(x_204, 2); - x_212 = x_204; +lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; +if (lean_is_exclusive(x_269)) { + lean_ctor_release(x_269, 0); + lean_ctor_release(x_269, 1); + lean_ctor_release(x_269, 2); + x_277 = x_269; } else { - lean_dec_ref(x_204); - x_212 = lean_box(0); + lean_dec_ref(x_269); + x_277 = lean_box(0); } -x_213 = lean_array_fget(x_206, x_207); -x_214 = lean_unsigned_to_nat(1u); -x_215 = lean_nat_add(x_207, x_214); -lean_dec(x_207); -if (lean_is_scalar(x_212)) { - x_216 = lean_alloc_ctor(0, 3, 0); +x_278 = lean_array_fget(x_271, x_272); +x_279 = lean_unsigned_to_nat(1u); +x_280 = lean_nat_add(x_272, x_279); +lean_dec(x_272); +if (lean_is_scalar(x_277)) { + x_281 = lean_alloc_ctor(0, 3, 0); } else { - x_216 = x_212; + x_281 = x_277; } -lean_ctor_set(x_216, 0, x_206); -lean_ctor_set(x_216, 1, x_215); -lean_ctor_set(x_216, 2, x_208); -x_217 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_217) == 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; -x_218 = lean_ctor_get(x_217, 0); -lean_inc(x_218); -x_219 = lean_ctor_get(x_217, 1); -lean_inc(x_219); -lean_dec(x_217); -x_220 = lean_ctor_get(x_218, 0); -lean_inc(x_220); -x_221 = lean_ctor_get(x_218, 1); -lean_inc(x_221); -if (lean_is_exclusive(x_218)) { - lean_ctor_release(x_218, 0); - lean_ctor_release(x_218, 1); - x_222 = x_218; +lean_ctor_set(x_281, 0, x_271); +lean_ctor_set(x_281, 1, x_280); +lean_ctor_set(x_281, 2, x_273); +x_282 = l___private_Lean_Elab_Tactic_BuiltinTactic_0__Lean_Elab_Tactic_getCaseGoals(x_20, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +if (lean_obj_tag(x_282) == 0) +{ +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_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 = lean_ctor_get(x_283, 0); +lean_inc(x_285); +x_286 = lean_ctor_get(x_283, 1); +lean_inc(x_286); +if (lean_is_exclusive(x_283)) { + lean_ctor_release(x_283, 0); + lean_ctor_release(x_283, 1); + x_287 = x_283; } else { - lean_dec_ref(x_218); - x_222 = lean_box(0); + lean_dec_ref(x_283); + x_287 = lean_box(0); } +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -42900,42 +43521,73 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); -x_223 = l_Lean_Elab_Tactic_renameInaccessibles(x_220, x_213, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_219); -if (lean_obj_tag(x_223) == 0) -{ -lean_object* x_224; lean_object* x_225; lean_object* x_226; -x_224 = lean_ctor_get(x_223, 0); -lean_inc(x_224); -x_225 = lean_ctor_get(x_223, 1); -lean_inc(x_225); -lean_dec(x_223); -lean_inc(x_224); -x_226 = l_Lean_MVarId_getTag(x_224, x_12, x_13, x_14, x_15, x_225); -if (lean_obj_tag(x_226) == 0) +x_288 = l_Lean_Elab_Tactic_renameInaccessibles(x_285, x_278, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_284); +if (lean_obj_tag(x_288) == 0) { -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; -x_227 = lean_ctor_get(x_226, 0); -lean_inc(x_227); -x_228 = lean_ctor_get(x_226, 1); -lean_inc(x_228); -lean_dec(x_226); -lean_inc(x_3); -if (lean_is_scalar(x_222)) { - x_229 = lean_alloc_ctor(1, 2, 0); +lean_object* x_289; lean_object* x_290; lean_object* x_291; +x_289 = lean_ctor_get(x_288, 0); +lean_inc(x_289); +x_290 = lean_ctor_get(x_288, 1); +lean_inc(x_290); +lean_dec(x_288); +lean_inc(x_289); +x_291 = l_Lean_MVarId_getTag(x_289, x_13, x_14, x_15, x_16, x_290); +if (lean_obj_tag(x_291) == 0) +{ +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; +x_292 = lean_ctor_get(x_291, 0); +lean_inc(x_292); +x_293 = lean_ctor_get(x_291, 1); +lean_inc(x_293); +lean_dec(x_291); +lean_inc(x_4); +if (lean_is_scalar(x_287)) { + x_294 = lean_alloc_ctor(1, 2, 0); +} else { + x_294 = x_287; + lean_ctor_set_tag(x_294, 1); +} +lean_ctor_set(x_294, 0, x_289); +lean_ctor_set(x_294, 1, x_4); +x_295 = l_Lean_Elab_Tactic_setGoals(x_294, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_293); +x_296 = lean_ctor_get(x_295, 1); +lean_inc(x_296); +if (lean_is_exclusive(x_295)) { + lean_ctor_release(x_295, 0); + lean_ctor_release(x_295, 1); + x_297 = x_295; +} else { + lean_dec_ref(x_295); + x_297 = lean_box(0); +} +x_298 = lean_box(0); +lean_inc(x_2); +if (lean_is_scalar(x_297)) { + x_299 = lean_alloc_ctor(1, 2, 0); } else { - x_229 = x_222; - lean_ctor_set_tag(x_229, 1); + x_299 = x_297; + lean_ctor_set_tag(x_299, 1); } -lean_ctor_set(x_229, 0, x_224); -lean_ctor_set(x_229, 1, x_3); -x_230 = l_Lean_Elab_Tactic_setGoals(x_229, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_228); -x_231 = lean_ctor_get(x_230, 1); -lean_inc(x_231); -lean_dec(x_230); -lean_inc(x_2); -x_232 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); -lean_closure_set(x_232, 0, x_2); +lean_ctor_set(x_299, 0, x_2); +lean_ctor_set(x_299, 1, x_298); +lean_inc(x_1); +x_300 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_300, 0, x_1); +lean_ctor_set(x_300, 1, x_299); +x_301 = lean_array_mk(x_300); +x_302 = lean_box(2); +x_303 = l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalWithAnnotateState___spec__1___lambda__1___closed__2; +x_304 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_304, 0, x_302); +lean_ctor_set(x_304, 1, x_303); +lean_ctor_set(x_304, 2, x_301); +lean_inc(x_3); +x_305 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); +lean_closure_set(x_305, 0, x_3); +x_306 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_306, 0, x_304); +lean_closure_set(x_306, 1, x_305); +lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -42943,95 +43595,95 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); +lean_inc(x_3); lean_inc(x_2); -lean_inc(x_1); -x_233 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_1, x_2, x_232, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_231); -if (lean_obj_tag(x_233) == 0) +x_307 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalCase___spec__5(x_2, x_3, x_306, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_296); +if (lean_obj_tag(x_307) == 0) { -lean_object* x_234; lean_object* x_235; lean_object* x_236; -x_234 = lean_ctor_get(x_233, 1); -lean_inc(x_234); -lean_dec(x_233); -x_235 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_234); -x_236 = lean_ctor_get(x_235, 0); -lean_inc(x_236); -if (lean_obj_tag(x_236) == 0) +lean_object* x_308; lean_object* x_309; lean_object* x_310; +x_308 = lean_ctor_get(x_307, 1); +lean_inc(x_308); +lean_dec(x_307); +x_309 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_308); +x_310 = lean_ctor_get(x_309, 0); +lean_inc(x_310); +if (lean_obj_tag(x_310) == 0) { -lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; -lean_dec(x_227); -x_237 = lean_ctor_get(x_235, 1); -lean_inc(x_237); -lean_dec(x_235); -x_238 = lean_box(0); -x_239 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_236, x_221, x_216, x_205, x_238, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_237); -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_20 = x_240; -x_21 = x_241; -goto block_28; +lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; +lean_dec(x_292); +x_311 = lean_ctor_get(x_309, 1); +lean_inc(x_311); +lean_dec(x_309); +x_312 = lean_box(0); +x_313 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_310, x_286, x_281, x_270, x_312, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_311); +x_314 = lean_ctor_get(x_313, 0); +lean_inc(x_314); +x_315 = lean_ctor_get(x_313, 1); +lean_inc(x_315); +lean_dec(x_313); +x_21 = x_314; +x_22 = x_315; +goto block_29; } else { -lean_object* x_242; -x_242 = lean_ctor_get(x_236, 1); -lean_inc(x_242); -if (lean_obj_tag(x_242) == 0) +lean_object* x_316; +x_316 = lean_ctor_get(x_310, 1); +lean_inc(x_316); +if (lean_obj_tag(x_316) == 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; lean_object* x_249; lean_object* x_250; -x_243 = lean_ctor_get(x_235, 1); -lean_inc(x_243); -lean_dec(x_235); -x_244 = lean_ctor_get(x_236, 0); -lean_inc(x_244); -x_245 = l_Lean_MVarId_setTag(x_244, x_227, x_12, x_13, x_14, x_15, x_243); -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_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_236, x_221, x_216, x_205, x_246, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_247); -lean_dec(x_246); -x_249 = lean_ctor_get(x_248, 0); -lean_inc(x_249); -x_250 = lean_ctor_get(x_248, 1); -lean_inc(x_250); -lean_dec(x_248); -x_20 = x_249; -x_21 = x_250; -goto block_28; +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; +x_317 = lean_ctor_get(x_309, 1); +lean_inc(x_317); +lean_dec(x_309); +x_318 = lean_ctor_get(x_310, 0); +lean_inc(x_318); +x_319 = l_Lean_MVarId_setTag(x_318, x_292, x_13, x_14, x_15, x_16, x_317); +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_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_310, x_286, x_281, x_270, x_320, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_321); +lean_dec(x_320); +x_323 = lean_ctor_get(x_322, 0); +lean_inc(x_323); +x_324 = lean_ctor_get(x_322, 1); +lean_inc(x_324); +lean_dec(x_322); +x_21 = x_323; +x_22 = x_324; +goto block_29; } else { -lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; -lean_dec(x_242); -lean_dec(x_227); -x_251 = lean_ctor_get(x_235, 1); -lean_inc(x_251); -lean_dec(x_235); -x_252 = lean_box(0); -x_253 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_236, x_221, x_216, x_205, x_252, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_251); -x_254 = lean_ctor_get(x_253, 0); -lean_inc(x_254); -x_255 = lean_ctor_get(x_253, 1); -lean_inc(x_255); -lean_dec(x_253); -x_20 = x_254; -x_21 = x_255; -goto block_28; +lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; +lean_dec(x_316); +lean_dec(x_292); +x_325 = lean_ctor_get(x_309, 1); +lean_inc(x_325); +lean_dec(x_309); +x_326 = lean_box(0); +x_327 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1___lambda__1(x_310, x_286, x_281, x_270, x_326, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_325); +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); +x_21 = x_328; +x_22 = x_329; +goto block_29; } } } else { -lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; -lean_dec(x_227); -lean_dec(x_221); -lean_dec(x_216); -lean_dec(x_205); +lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; +lean_dec(x_292); +lean_dec(x_286); +lean_dec(x_281); +lean_dec(x_270); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -43039,40 +43691,41 @@ lean_dec(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_2); lean_dec(x_1); -x_256 = lean_ctor_get(x_233, 0); -lean_inc(x_256); -x_257 = lean_ctor_get(x_233, 1); -lean_inc(x_257); -if (lean_is_exclusive(x_233)) { - lean_ctor_release(x_233, 0); - lean_ctor_release(x_233, 1); - x_258 = x_233; +x_330 = lean_ctor_get(x_307, 0); +lean_inc(x_330); +x_331 = lean_ctor_get(x_307, 1); +lean_inc(x_331); +if (lean_is_exclusive(x_307)) { + lean_ctor_release(x_307, 0); + lean_ctor_release(x_307, 1); + x_332 = x_307; } else { - lean_dec_ref(x_233); - x_258 = lean_box(0); + lean_dec_ref(x_307); + x_332 = lean_box(0); } -if (lean_is_scalar(x_258)) { - x_259 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_332)) { + x_333 = lean_alloc_ctor(1, 2, 0); } else { - x_259 = x_258; + x_333 = x_332; } -lean_ctor_set(x_259, 0, x_256); -lean_ctor_set(x_259, 1, x_257); -return x_259; +lean_ctor_set(x_333, 0, x_330); +lean_ctor_set(x_333, 1, x_331); +return x_333; } } else { -lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; -lean_dec(x_224); -lean_dec(x_222); -lean_dec(x_221); -lean_dec(x_216); -lean_dec(x_205); +lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; +lean_dec(x_289); +lean_dec(x_287); +lean_dec(x_286); +lean_dec(x_281); +lean_dec(x_270); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -43080,39 +43733,40 @@ lean_dec(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_2); lean_dec(x_1); -x_260 = lean_ctor_get(x_226, 0); -lean_inc(x_260); -x_261 = lean_ctor_get(x_226, 1); -lean_inc(x_261); -if (lean_is_exclusive(x_226)) { - lean_ctor_release(x_226, 0); - lean_ctor_release(x_226, 1); - x_262 = x_226; +x_334 = lean_ctor_get(x_291, 0); +lean_inc(x_334); +x_335 = lean_ctor_get(x_291, 1); +lean_inc(x_335); +if (lean_is_exclusive(x_291)) { + lean_ctor_release(x_291, 0); + lean_ctor_release(x_291, 1); + x_336 = x_291; } else { - lean_dec_ref(x_226); - x_262 = lean_box(0); + lean_dec_ref(x_291); + x_336 = lean_box(0); } -if (lean_is_scalar(x_262)) { - x_263 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_336)) { + x_337 = lean_alloc_ctor(1, 2, 0); } else { - x_263 = x_262; + x_337 = x_336; } -lean_ctor_set(x_263, 0, x_260); -lean_ctor_set(x_263, 1, x_261); -return x_263; +lean_ctor_set(x_337, 0, x_334); +lean_ctor_set(x_337, 1, x_335); +return x_337; } } else { -lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; -lean_dec(x_222); -lean_dec(x_221); -lean_dec(x_216); -lean_dec(x_205); +lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; +lean_dec(x_287); +lean_dec(x_286); +lean_dec(x_281); +lean_dec(x_270); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -43120,38 +43774,39 @@ lean_dec(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_2); lean_dec(x_1); -x_264 = lean_ctor_get(x_223, 0); -lean_inc(x_264); -x_265 = lean_ctor_get(x_223, 1); -lean_inc(x_265); -if (lean_is_exclusive(x_223)) { - lean_ctor_release(x_223, 0); - lean_ctor_release(x_223, 1); - x_266 = x_223; +x_338 = lean_ctor_get(x_288, 0); +lean_inc(x_338); +x_339 = lean_ctor_get(x_288, 1); +lean_inc(x_339); +if (lean_is_exclusive(x_288)) { + lean_ctor_release(x_288, 0); + lean_ctor_release(x_288, 1); + x_340 = x_288; } else { - lean_dec_ref(x_223); - x_266 = lean_box(0); + lean_dec_ref(x_288); + x_340 = lean_box(0); } -if (lean_is_scalar(x_266)) { - x_267 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_340)) { + x_341 = lean_alloc_ctor(1, 2, 0); } else { - x_267 = x_266; + x_341 = x_340; } -lean_ctor_set(x_267, 0, x_264); -lean_ctor_set(x_267, 1, x_265); -return x_267; +lean_ctor_set(x_341, 0, x_338); +lean_ctor_set(x_341, 1, x_339); +return x_341; } } else { -lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; -lean_dec(x_216); -lean_dec(x_213); -lean_dec(x_205); +lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; +lean_dec(x_281); +lean_dec(x_278); +lean_dec(x_270); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -43159,38 +43814,39 @@ lean_dec(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_2); lean_dec(x_1); -x_268 = lean_ctor_get(x_217, 0); -lean_inc(x_268); -x_269 = lean_ctor_get(x_217, 1); -lean_inc(x_269); -if (lean_is_exclusive(x_217)) { - lean_ctor_release(x_217, 0); - lean_ctor_release(x_217, 1); - x_270 = x_217; +x_342 = lean_ctor_get(x_282, 0); +lean_inc(x_342); +x_343 = lean_ctor_get(x_282, 1); +lean_inc(x_343); +if (lean_is_exclusive(x_282)) { + lean_ctor_release(x_282, 0); + lean_ctor_release(x_282, 1); + x_344 = x_282; } else { - lean_dec_ref(x_217); - x_270 = lean_box(0); + lean_dec_ref(x_282); + x_344 = lean_box(0); } -if (lean_is_scalar(x_270)) { - x_271 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_344)) { + x_345 = lean_alloc_ctor(1, 2, 0); } else { - x_271 = x_270; + x_345 = x_344; } -lean_ctor_set(x_271, 0, x_268); -lean_ctor_set(x_271, 1, x_269); -return x_271; +lean_ctor_set(x_345, 0, x_342); +lean_ctor_set(x_345, 1, x_343); +return x_345; } } } -block_28: +block_29: { -if (lean_obj_tag(x_20) == 0) +if (lean_obj_tag(x_21) == 0) { -lean_object* x_22; lean_object* x_23; +lean_object* x_23; lean_object* x_24; +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -43198,29 +43854,29 @@ lean_dec(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_2); lean_dec(x_1); -x_22 = lean_ctor_get(x_20, 0); -lean_inc(x_22); -lean_dec(x_20); -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; +x_23 = lean_ctor_get(x_21, 0); +lean_inc(x_23); +lean_dec(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 { -lean_object* x_24; size_t x_25; size_t x_26; -x_24 = lean_ctor_get(x_20, 0); -lean_inc(x_24); -lean_dec(x_20); -x_25 = 1; -x_26 = lean_usize_add(x_6, x_25); -x_6 = x_26; -x_7 = x_24; -x_16 = x_21; +lean_object* x_25; size_t x_26; size_t x_27; +x_25 = lean_ctor_get(x_21, 0); +lean_inc(x_25); +lean_dec(x_21); +x_26 = 1; +x_27 = lean_usize_add(x_7, x_26); +x_7 = x_27; +x_8 = x_25; +x_17 = x_22; goto _start; } } @@ -43271,61 +43927,63 @@ return x_13; } else { -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_14 = lean_unsigned_to_nat(1u); +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; +x_14 = lean_unsigned_to_nat(0u); x_15 = l_Lean_Syntax_getArg(x_1, x_14); -x_16 = l_Lean_Syntax_getArgs(x_15); -lean_dec(x_15); -x_17 = lean_array_get_size(x_16); -x_18 = lean_unsigned_to_nat(0u); -x_19 = lean_nat_dec_lt(x_18, x_17); -if (x_19 == 0) -{ -lean_object* x_57; +x_16 = lean_unsigned_to_nat(1u); +x_17 = l_Lean_Syntax_getArg(x_1, x_16); +x_18 = l_Lean_Syntax_getArgs(x_17); lean_dec(x_17); -lean_dec(x_16); -x_57 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__12; -x_20 = x_57; -goto block_56; +x_19 = lean_array_get_size(x_18); +x_20 = lean_nat_dec_lt(x_14, x_19); +if (x_20 == 0) +{ +lean_object* x_58; +lean_dec(x_19); +lean_dec(x_18); +x_58 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__12; +x_21 = x_58; +goto block_57; } else { -uint8_t x_58; -x_58 = lean_nat_dec_le(x_17, x_17); -if (x_58 == 0) +uint8_t x_59; +x_59 = lean_nat_dec_le(x_19, x_19); +if (x_59 == 0) { -lean_object* x_59; -lean_dec(x_17); -lean_dec(x_16); -x_59 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__12; -x_20 = x_59; -goto block_56; +lean_object* x_60; +lean_dec(x_19); +lean_dec(x_18); +x_60 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__12; +x_21 = x_60; +goto block_57; } else { -size_t x_60; size_t x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_60 = 0; -x_61 = lean_usize_of_nat(x_17); -lean_dec(x_17); -x_62 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__13; -x_63 = l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1(x_16, x_60, x_61, x_62); -lean_dec(x_16); -x_64 = lean_ctor_get(x_63, 1); -lean_inc(x_64); -lean_dec(x_63); -x_20 = x_64; -goto block_56; +size_t x_61; size_t x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_61 = 0; +x_62 = lean_usize_of_nat(x_19); +lean_dec(x_19); +x_63 = l_Lean_Elab_OpenDecl_elabOpenDecl___at_Lean_Elab_Tactic_evalOpen___spec__3___closed__13; +x_64 = l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1(x_18, x_61, x_62, x_63); +lean_dec(x_18); +x_65 = lean_ctor_get(x_64, 1); +lean_inc(x_65); +lean_dec(x_64); +x_21 = x_65; +goto block_57; } } -block_56: +block_57: { -lean_object* x_21; lean_object* x_22; -x_21 = l_Lean_Elab_Tactic_evalCase___closed__3; -x_22 = l_Array_sequenceMap___at_Lean_Elab_Tactic_evalCase___spec__1(x_20, x_21); -lean_dec(x_20); -if (lean_obj_tag(x_22) == 0) +lean_object* x_22; lean_object* x_23; +x_22 = l_Lean_Elab_Tactic_evalCase___closed__3; +x_23 = l_Array_sequenceMap___at_Lean_Elab_Tactic_evalCase___spec__1(x_21, x_22); +lean_dec(x_21); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_23; +lean_object* x_24; +lean_dec(x_15); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -43335,35 +43993,36 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_23 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); -return x_23; +x_24 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); +return x_24; } else { -lean_object* x_24; size_t x_25; size_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; uint8_t x_34; -x_24 = lean_ctor_get(x_22, 0); -lean_inc(x_24); -lean_dec(x_22); -x_25 = lean_array_size(x_24); -x_26 = 0; -lean_inc(x_24); -x_27 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalCase___spec__3(x_25, x_26, x_24); -x_28 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalCase___spec__4(x_25, x_26, x_24); -x_29 = lean_unsigned_to_nat(2u); -x_30 = l_Lean_Syntax_getArg(x_1, x_29); -x_31 = lean_unsigned_to_nat(3u); -x_32 = l_Lean_Syntax_getArg(x_1, x_31); -lean_dec(x_1); -x_33 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_addCheckpoints___spec__1___closed__4; -lean_inc(x_32); -x_34 = l_Lean_Syntax_isOfKind(x_32, x_33); -if (x_34 == 0) +lean_object* x_25; size_t x_26; size_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; uint8_t x_35; +x_25 = lean_ctor_get(x_23, 0); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_array_size(x_25); +x_27 = 0; +lean_inc(x_25); +x_28 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalCase___spec__3(x_26, x_27, x_25); +x_29 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalCase___spec__4(x_26, x_27, x_25); +x_30 = lean_unsigned_to_nat(2u); +x_31 = l_Lean_Syntax_getArg(x_1, x_30); +x_32 = lean_unsigned_to_nat(3u); +x_33 = l_Lean_Syntax_getArg(x_1, x_32); +lean_dec(x_1); +x_34 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_addCheckpoints___spec__1___closed__4; +lean_inc(x_33); +x_35 = l_Lean_Syntax_isOfKind(x_33, x_34); +if (x_35 == 0) { -lean_object* x_35; -lean_dec(x_32); -lean_dec(x_30); +lean_object* x_36; +lean_dec(x_33); +lean_dec(x_31); +lean_dec(x_29); lean_dec(x_28); -lean_dec(x_27); +lean_dec(x_15); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -43372,20 +44031,20 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_35 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); -return x_35; +x_36 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); +return x_36; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; size_t x_41; lean_object* x_42; -x_36 = lean_box(0); -x_37 = lean_array_get_size(x_27); -x_38 = l_Array_toSubarray___rarg(x_27, x_18, x_37); -x_39 = l_Lean_Elab_Tactic_addCheckpoints___lambda__1___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_array_size(x_28); +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; size_t x_42; lean_object* x_43; +x_37 = lean_box(0); +x_38 = lean_array_get_size(x_28); +x_39 = l_Array_toSubarray___rarg(x_28, x_14, x_38); +x_40 = l_Lean_Elab_Tactic_addCheckpoints___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_42 = lean_array_size(x_29); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); @@ -43394,28 +44053,28 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_42 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1(x_30, x_32, x_36, x_28, x_41, x_26, x_40, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_28); -if (lean_obj_tag(x_42) == 0) +x_43 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1(x_15, x_31, x_33, x_37, x_29, x_42, x_27, x_41, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_29); +if (lean_obj_tag(x_43) == 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 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); +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_44 = lean_ctor_get(x_43, 0); lean_inc(x_44); -lean_dec(x_42); x_45 = lean_ctor_get(x_43, 1); lean_inc(x_45); lean_dec(x_43); -x_46 = l_Lean_Elab_Tactic_getGoals___rarg(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_44); -x_47 = lean_ctor_get(x_46, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_46, 1); +x_46 = lean_ctor_get(x_44, 1); +lean_inc(x_46); +lean_dec(x_44); +x_47 = l_Lean_Elab_Tactic_getGoals___rarg(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_45); +x_48 = lean_ctor_get(x_47, 0); lean_inc(x_48); -lean_dec(x_46); -x_49 = lean_array_to_list(x_45); -x_50 = l_List_appendTR___rarg(x_49, x_47); -x_51 = l_Lean_Elab_Tactic_setGoals(x_50, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_48); +x_49 = lean_ctor_get(x_47, 1); +lean_inc(x_49); +lean_dec(x_47); +x_50 = lean_array_to_list(x_46); +x_51 = l_List_appendTR___rarg(x_50, x_48); +x_52 = l_Lean_Elab_Tactic_setGoals(x_51, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_49); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -43424,11 +44083,11 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -return x_51; +return x_52; } else { -uint8_t x_52; +uint8_t x_53; lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -43437,23 +44096,23 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_52 = !lean_is_exclusive(x_42); -if (x_52 == 0) +x_53 = !lean_is_exclusive(x_43); +if (x_53 == 0) { -return x_42; +return x_43; } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_53 = lean_ctor_get(x_42, 0); -x_54 = lean_ctor_get(x_42, 1); +lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_54 = lean_ctor_get(x_43, 0); +x_55 = lean_ctor_get(x_43, 1); +lean_inc(x_55); lean_inc(x_54); -lean_inc(x_53); -lean_dec(x_42); -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_dec(x_43); +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; } } } @@ -43479,17 +44138,34 @@ lean_dec(x_5); return x_15; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___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_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__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]; _start: { -size_t x_17; size_t x_18; lean_object* x_19; -x_17 = lean_unbox_usize(x_5); -lean_dec(x_5); +size_t x_18; size_t x_19; lean_object* x_20; x_18 = lean_unbox_usize(x_6); lean_dec(x_6); -x_19 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___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); -return x_19; +x_19 = lean_unbox_usize(x_7); +lean_dec(x_7); +x_20 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalCase_x27___spec__1(x_1, x_2, x_3, x_4, x_5, x_18, x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +lean_dec(x_5); +return x_20; } } static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalCase_x27__1___closed__1() { diff --git a/stage0/stdlib/Lean/Elab/Tactic/Conv/Pattern.c b/stage0/stdlib/Lean/Elab/Tactic/Conv/Pattern.c index cc0dadb28b5f..009ab12c4df6 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Conv/Pattern.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Conv/Pattern.c @@ -58,7 +58,6 @@ static lean_object* l___private_Lean_Elab_Tactic_Conv_Pattern_0__Lean_Elab_Tacti static lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__11___closed__3; uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__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* l_Lean_stringToMessageData(lean_object*); static lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__11___closed__6; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Conv_evalPattern___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -84,6 +83,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalPattern(lean_object*, lean_ static lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__9___closed__4; lean_object* l_Lean_Elab_Term_withoutErrToSorryImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_Conv_getLhs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__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* l_Array_forInUnsafe_loop___at_Lean_Meta_Simp_visitFn___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*); static lean_object* l_Array_qsort_sort___at_Lean_Elab_Tactic_Conv_evalPattern___spec__3___closed__1; lean_object* l_Lean_Meta_withNewMCtxDepth___at_Lean_Meta_matchesInstance___spec__1___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -91,7 +91,6 @@ lean_object* l_Lean_MessageData_ofFormat(lean_object*); lean_object* l_Lean_Elab_Tactic_Conv_getRhs(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_Conv_evalPattern___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_Conv_matchPattern_x3f_go_x3f___closed__1; -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2; lean_object* l_Lean_Elab_Tactic_withMainContext___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_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Conv_evalPattern___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static uint32_t l___private_Lean_Elab_Tactic_Conv_Pattern_0__Lean_Elab_Tactic_Conv_getContext___rarg___closed__1; @@ -118,7 +117,9 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalPattern_declRange__ LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Elab_Tactic_Conv_evalPattern___spec__9___boxed(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Conv_evalPattern___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_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___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_object*); lean_object* l_Lean_Expr_appFn_x21(lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalPattern_declRange__1___closed__2; static lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__9___closed__3; static lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__9___closed__1; @@ -139,7 +140,6 @@ static lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___closed__1; static lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__11___closed__8; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); uint8_t l___private_Lean_HeadIndex_0__Lean_beqHeadIndex____x40_Lean_HeadIndex___hyg_68_(lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___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* l_Lean_indentExpr(lean_object*); lean_object* l_Lean_Meta_isExprDefEqGuarded(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -147,6 +147,7 @@ static lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__11___closed__7 LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Conv_evalPattern___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_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_PatternMatchState_accept(lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1; LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Elab_Tactic_Conv_evalPattern___spec__3___boxed(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*); uint8_t l_Lean_Syntax_isNone(lean_object*); @@ -192,7 +193,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_matchPattern_x3f___lambda__1(le LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Conv_Pattern_0__Lean_Elab_Tactic_Conv_getContext___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Elab_Tactic_Conv_evalPattern___spec__3___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalPattern__1(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___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_object*); lean_object* l_Lean_Expr_mvarId_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___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_array_uset(lean_object*, size_t, lean_object*); @@ -2431,7 +2431,7 @@ return x_32; } } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1() { _start: { lean_object* x_1; @@ -2439,16 +2439,16 @@ x_1 = lean_mk_string_unchecked("positive integer expected", 25, 25); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1; +x_1 = l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___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, 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_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___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, 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; @@ -2489,7 +2489,7 @@ lean_dec(x_21); lean_dec(x_19); lean_dec(x_6); lean_dec(x_4); -x_28 = l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2; +x_28 = l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2; x_29 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Conv_evalPattern___spec__6(x_20, x_28, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); lean_dec(x_20); x_30 = !lean_is_exclusive(x_29); @@ -4647,7 +4647,7 @@ lean_dec(x_60); x_62 = lean_array_get_size(x_61); x_63 = lean_mk_empty_array_with_capacity(x_62); lean_inc(x_10); -x_64 = l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8(x_61, x_61, x_62, x_59, lean_box(0), x_63, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_47); +x_64 = l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8(x_61, x_61, x_62, x_59, lean_box(0), x_63, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_47); lean_dec(x_61); if (lean_obj_tag(x_64) == 0) { @@ -5049,11 +5049,11 @@ lean_dec(x_1); return x_12; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___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, 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_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___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, 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_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8(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 = l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8(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_12); lean_dec(x_11); @@ -5396,10 +5396,10 @@ l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Conv_evalPattern___spec lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Conv_evalPattern___spec__5___rarg___closed__1); l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Conv_evalPattern___spec__5___rarg___closed__2 = _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Conv_evalPattern___spec__5___rarg___closed__2(); lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Conv_evalPattern___spec__5___rarg___closed__2); -l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1); -l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2); +l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__1); +l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2 = _init_l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_Conv_evalPattern___spec__8___closed__2); l_Lean_Elab_Tactic_Conv_evalPattern___lambda__9___closed__1 = _init_l_Lean_Elab_Tactic_Conv_evalPattern___lambda__9___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_Conv_evalPattern___lambda__9___closed__1); l_Lean_Elab_Tactic_Conv_evalPattern___lambda__9___closed__2 = _init_l_Lean_Elab_Tactic_Conv_evalPattern___lambda__9___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Tactic/Ext.c b/stage0/stdlib/Lean/Elab/Tactic/Ext.c index 30b95bca24a0..544197862c57 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Ext.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Ext.c @@ -14,92 +14,89 @@ extern "C" { #endif LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_withExtHyps___spec__2(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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem_declRange__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__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_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___closed__6; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_evalPrio(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Elab_Tactic_Ext_evalExt___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_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_withExtN___spec__4___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkEqHEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_beqKey____x40_Lean_Meta_DiscrTreeTypes___hyg_101_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_tryIntros___spec__1___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__9(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_Elab_Tactic_Ext_evalExt___lambda__2___closed__1; lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_reprPrec(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt__1(lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__29; +LEAN_EXPORT lean_object* l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3199____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1(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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__12; uint8_t l_Lean_PersistentHashMap_contains___at_Lean_NameSSet_contains___spec__2(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__3; lean_object* l_Lean_MapDeclarationExtension_insert___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___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_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__30; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__27; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___lambda__1___closed__6; lean_object* lean_mk_empty_array_with_capacity(lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal_loop___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__10(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___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*); size_t lean_usize_shift_right(size_t, size_t); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__32; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__19; lean_object* l_Lean_addBuiltinDocString(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__18; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__5___closed__3; static lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__2___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem__1___closed__4; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__5(lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); 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_Elab_Tactic_Ext_realizeExtTheorem___lambda__5___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalApplyExtTheorem___rarg(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_Ext_evalApplyExtTheorem_docString__1(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__35; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__5(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__2; lean_object* l_Lean_throwError___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_declRangeExt; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____lambda__1(lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_RCases_rintro(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_Ext_realizeExtTheorem___lambda__2___closed__28; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__5___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_Ext_tryIntros___rarg___lambda__4(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__59; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ConstantInfo_type(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__25; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___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_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10(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_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__9___closed__1; +LEAN_EXPORT uint8_t l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3199_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_Ext_withExtHyps___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__3___closed__1; extern lean_object* l_Lean_maxRecDepthErrorMessage; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__7; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__27; uint8_t lean_usize_dec_le(size_t, size_t); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___closed__2; -LEAN_EXPORT uint64_t l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___rarg___closed__1; lean_object* l_Lean_ConstantInfo_levelParams(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__55; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalApplyExtTheorem___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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__2; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__21; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191_(lean_object*, lean_object*); lean_object* l_Lean_indentD(lean_object*); uint8_t l_Lean_Exception_isInterrupt(lean_object*); static lean_object* l_Lean_Linter_logLint___at_Lean_Elab_Tactic_Ext_evalExt___spec__3___closed__5; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__9___closed__2; +static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__4; uint64_t lean_uint64_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__3(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_mix_hash(uint64_t, uint64_t); @@ -107,92 +104,87 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___at_Lean_Elab_Tactic_E lean_object* l_Lean_mkIff(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__22; 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_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__7(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___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_FileMap_toPosition(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__17; +LEAN_EXPORT lean_object* l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__1; size_t lean_uint64_to_usize(uint64_t); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__6; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__23; lean_object* lean_array_fswap(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_logAt___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__2(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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___closed__1; uint8_t l_Lean_Expr_isAppOfArity(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__2; +LEAN_EXPORT uint64_t l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3289____spec__1(lean_object*, size_t, size_t, uint64_t); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_extCore___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_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__7; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__44; static lean_object* l_Lean_Elab_Tactic_Ext_evalExt___lambda__2___closed__4; static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__2___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem_declRange__1___closed__5; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___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* l_Lean_Elab_Term_elabTermEnsuringType(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Array_findIdx_x3f_loop___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___lambda__1___closed__4; lean_object* l_Lean_MessageData_ofList(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_extCore___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*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__13; lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__16; static lean_object* l_Lean_Elab_Tactic_Ext_instBEqExtTheorem___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_evalExt___lambda__2___closed__5; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__28; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___closed__4; size_t lean_usize_mul(size_t, size_t); lean_object* l_Lean_PersistentHashMap_insert___at_Lean_NameSSet_insert___spec__2(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_DiscrTree_instInhabited(lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__4; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__31; lean_object* lean_mk_array(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__21; uint8_t lean_usize_dec_eq(size_t, size_t); static lean_object* l_Lean_Elab_Tactic_Ext_extExt_config___closed__1; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__7___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_getExtTheorems___spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_Trie_foldValuesM___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__11; lean_object* l_Lean_Syntax_getArgs(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___rarg___boxed(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_Tactic_Ext_applyExtTheoremAt___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6(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* l_Lean_replaceRef(lean_object*, lean_object*); lean_object* l_Lean_MVarId_getType_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__4(lean_object*, 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___regBuiltin_Lean_Elab_Tactic_Ext_evalExt_declRange__1(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___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___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__5; 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_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_eraseCore(lean_object*, lean_object*); -lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___rarg___lambda__1___boxed(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_Ext_ExtTheorems_erase___spec__4___boxed(lean_object*, lean_object*, lean_object*, 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*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__17; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__2(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* lean_array_fset(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___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*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__8; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__3(size_t, lean_object*, 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_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__23; 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*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_tryIntros___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__12; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__22; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__13; +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__4; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___at_Lean_Elab_Tactic_Ext_extCore___spec__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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__19; lean_object* l_ReaderT_read___at_Lean_Macro_instMonadRefMacroM___spec__1(lean_object*, lean_object*); -static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__29; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__38; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorem; @@ -202,171 +194,167 @@ lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, 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_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__3(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6(lean_object*, size_t, size_t, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__2___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_foldlMAux___at_Lean_mkModuleData___spec__3___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Elab_Tactic_Ext_mkExtType___spec__1(lean_object*, size_t, size_t, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__4; lean_object* l_Lean_Syntax_node5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__20; uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__11; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__14; lean_object* l_Lean_stringToMessageData(lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Tactic_Ext_evalExt___spec__2(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__36; static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__2___closed__1; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__16; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__6(lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_MapDeclarationExtension_contains___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__13(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696_(lean_object*); lean_object* l_Lean_RBNode_findCore___at_Lean_Meta_mkGeneralizationForbiddenSet_visit___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__2(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__4; uint8_t lean_string_dec_eq(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem_declRange__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___rarg___closed__2; lean_object* l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__1; lean_object* l_Lean_Exception_toMessageData(lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__6; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__29; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__10; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___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_Ext_withExtHyps___rarg___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_repr___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__3___closed__7; lean_object* l_Lean_Expr_appArg_x21(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem_declRange__1___closed__3; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__3; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__56; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_tryIntros___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt_declRange__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___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_Ext_mkExtIffType___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_Elab_Tactic_Ext_withExt1___at_Lean_Elab_Tactic_Ext_extCore___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_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___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*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__21; lean_object* l_Lean_getStructureFields(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__4___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__16; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__14; uint8_t l_Lean_Expr_hasMVar(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase(lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__3; static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__1___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_logLint___at_Lean_Elab_Tactic_Ext_evalExt___spec__3___closed__1; +LEAN_EXPORT uint64_t l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3289_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___at_Lean_Elab_Tactic_Ext_withExtN___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_extCore(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static size_t l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__4___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__2; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___lambda__2(lean_object*, uint8_t, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__11; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__19; lean_object* l_Lean_Elab_Tactic_RCases_expandRIntroPats(lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10(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_Ext_mkExtIffType___lambda__2___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___closed__5; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__26; lean_object* l_Lean_FVarId_getBinderInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__34; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__10; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__15; static lean_object* l_Lean_Linter_logLint___at_Lean_Elab_Tactic_Ext_evalExt___spec__3___closed__3; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_Ext_evalExt___spec__1(size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___rarg(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___closed__1; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__8; -LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_getExtTheorems(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_logLint___at_Lean_Elab_Tactic_Ext_evalExt___spec__3___closed__6; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269____boxed(lean_object*, lean_object*); lean_object* l_Array_reverse___rarg(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__17; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__14; -static lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__1; lean_object* l_Lean_getConstInfo___at_Lean_Elab_Command_expandDeclId___spec__9(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*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__50; +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem_declRange__1(lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__8; +static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__3; 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_List_foldl___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____spec__3(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___closed__2; lean_object* l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__4; +static lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__3; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__4___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___closed__1; lean_object* l_Lean_Elab_expandMacroImpl_x3f(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorems___closed__1; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__15; uint8_t lean_expr_eqv(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__7; lean_object* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__28; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__4; lean_object* l_Lean_registerSimpleScopedEnvExtension___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__25; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___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_Ext_realizeExtIffTheorem___lambda__1___closed__31; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_bind___at_Lean_Macro_instMonadRefMacroM___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_to_int(lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__7; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__1; lean_object* l_Lean_MessageData_ofSyntax(lean_object*); lean_object* l_Lean_Syntax_node6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__24; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__15; lean_object* lean_nat_div(lean_object*, lean_object*); static lean_object* l_Lean_Linter_logLint___at_Lean_Elab_Tactic_Ext_evalExt___spec__3___closed__4; 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_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallMetaTelescopeReducingAux(lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_instHashableExtTheorem___closed__1; lean_object* l_Lean_Elab_Term_withoutErrToSorryImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___closed__5; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_withExtHyps___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_Elab_Tactic_Ext_realizeExtTheorem___lambda__4(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___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___closed__2; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__7; LEAN_EXPORT uint8_t l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___lambda__3(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__4(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1(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*); lean_object* l_Lean_Elab_Command_getRef(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Elab_Tactic_Ext_mkExtType___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__18; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__18; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__4___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_Ext_tryIntros___rarg___lambda__6___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__3___closed__8; -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__10; lean_object* l_Lean_Meta_withNewMCtxDepth___at_Lean_Meta_matchesInstance___spec__1___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__1; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__4; lean_object* l_Lean_MessageData_ofFormat(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___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_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkCIdentFrom(lean_object*, lean_object*, uint8_t); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__6; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__5; lean_object* l_Lean_Elab_getBetterRef(lean_object*, lean_object*); uint8_t l_Lean_Expr_isMVar(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt_declRange__1___closed__2; 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_Lean_Elab_Tactic_Ext_tryIntros___rarg___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_Ext_realizeExtIffTheorem___lambda__1___closed__33; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6(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_Tactic_Ext_realizeExtTheorem___lambda__2___closed__15; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__11; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_withExtN___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -375,120 +363,122 @@ lean_object* l_outOfBounds___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps(lean_object*); lean_object* l_Lean_Elab_Tactic_withMainContext___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_Elab_Tactic_Ext_applyExtTheoremAt___lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__13; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__63; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__60; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_liftTermElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__5(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__24; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__3; lean_object* lean_st_ref_get(lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_registerTagAttribute___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___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_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__12___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__6___closed__4; 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*); lean_object* l_Lean_liftCommandElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkAndN(lean_object*); +LEAN_EXPORT uint8_t l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3199____spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__3___closed__2; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__8; lean_object* l_Lean_Syntax_getOptional_x3f(lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); -static lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6___closed__1; -static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__2; +static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__13(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_to_list(lean_object*); lean_object* l_ReaderT_instApplicativeOfMonad___rarg(lean_object*); 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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__13; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_getExtTheorems___closed__1; -static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__5; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359____boxed(lean_object*); +static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__5; lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); lean_object* l_Lean_Syntax_node3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__4; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__9; lean_object* l_Lean_ScopedEnvExtension_modifyState___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__24; -static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___closed__4; static lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_evalExt___closed__1; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__12; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__57; uint8_t l_Lean_Meta_DiscrTree_Key_lt(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__15; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___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_Elab_Tactic_Ext_instReprExtTheorem___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__4___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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__2(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__21; +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__5___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__5(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__1___closed__1; -static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__1; lean_object* l_Lean_Elab_Command_getCurrMacroScope(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___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_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__13___closed__1; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__20; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___closed__8; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__13; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__10; static lean_object* l_Lean_Elab_Tactic_Ext_evalExt___lambda__2___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__13(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__12___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_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__8(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__4___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__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_Ext_realizeExtTheorem___lambda__2___closed__4; uint8_t lean_name_eq(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__26; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__54; -LEAN_EXPORT lean_object* l_repr___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____spec__1(lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__9; static lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__3___closed__1; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___closed__2; -static size_t l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__2; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__4; lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__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_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__2; 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_Elab_Tactic_Ext_instInhabitedExtTheorems; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__1___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___closed__1; -LEAN_EXPORT uint8_t l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269_(lean_object*, lean_object*); +static lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__6___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__3___closed__6; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__14; lean_object* l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArg(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_Lean_Elab_Tactic_Ext_evalExt(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_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__9; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__37; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__1; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__7; uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__5; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__6; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__17; +LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___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_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__5; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_tryIntros___spec__1___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_withExtN___spec__2___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Tactic_Ext_evalExt___spec__2___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_saveState___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__16; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___at_Lean_Elab_Tactic_Ext_extCore___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_Elab_Tactic_Ext_mkExtIffType___lambda__3___closed__4; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__23; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__5___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtType(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__13; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_extExt_config; lean_object* l_Lean_Expr_appFn_x21(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__2___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___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_Elab_Command_getScope___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_instHashableExtTheorem; @@ -496,46 +486,41 @@ lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesi lean_object* l_Lean_CollectFVars_main(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__1___lambda__1___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__46; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_withExt1___spec__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__18; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3199____boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__52; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__30; +LEAN_EXPORT lean_object* l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlM___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__6(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___at_Lean_Elab_Tactic_Ext_withExtN___spec__3(lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__6; -static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401_(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__53; lean_object* l_Lean_Meta_DiscrTree_mkPath(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_usize_to_nat(size_t); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___at_Lean_Elab_Tactic_Ext_withExtN___spec__3___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Meta_mkSimpCongrTheorem___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__1(lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofConstName(lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__47; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__6; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__8; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3(lean_object*, size_t, lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___lambda__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__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_Array_insertionSort_swapLoop___at_Lean_Elab_Tactic_Ext_getExtTheorems___spec__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__6___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_Ext_withExtN___at_Lean_Elab_Tactic_Ext_extCore___spec__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*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_instMonadControlTOfPure___rarg(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__2; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__11; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3289____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__10; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__33; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__2___closed__2; lean_object* l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -544,18 +529,18 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros(lean_object*); lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___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_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__1(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_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__4; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_getExtTheorems___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___closed__1; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__17; +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_evalExt___lambda__2___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__6(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_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_extCore___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_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__43; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt__1___closed__2; -LEAN_EXPORT uint8_t l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269____spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalExt___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_FileMap_leanPosToLspPos(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__34; @@ -564,66 +549,65 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem__1__ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__2(lean_object*, lean_object*); static lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___closed__4; static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___closed__3; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__9; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt_declRange__1___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__15; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3289____boxed(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__26; LEAN_EXPORT uint8_t l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__2(lean_object*, lean_object*, size_t, size_t, uint8_t); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_evalApplyExtTheorem___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__6; static lean_object* l_Lean_Elab_Tactic_Ext_getExtTheorems___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__7; lean_object* l_Lean_throwError___rarg(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Meta_DiscrTree_instInhabitedKey; +static lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__4; static lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__6___closed__1; static lean_object* l_Lean_Linter_logLint___at_Lean_Elab_Tactic_Ext_evalExt___spec__3___closed__2; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___closed__2; uint8_t l_Lean_Name_isAtomic(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__16; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__4___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___closed__2; lean_object* lean_string_length(lean_object*); -static lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__3; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__19; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___closed__6; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__19; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__9; +static lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem__1___closed__6; lean_object* l_Lean_TSyntax_getNat(lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_instReprExtTheorem; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___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_Elab_Tactic_Ext_realizeExtIffTheorem___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_List_forIn_loop___at_Lean_Elab_Tactic_Ext_withExtN___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__17; 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*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__21; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___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_Lean_Elab_Tactic_Ext_instInhabitedExtTheorem___closed__1; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); -static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__4; lean_object* lean_environment_main_module(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___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_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__20; LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Elab_Tactic_Ext_evalExt___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___regBuiltin_Lean_Elab_Tactic_Ext_evalExt_declRange__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___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_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_tryIntros___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__58; -static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__3; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_Ext_evalExt___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9(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_id___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___at_Lean_Elab_Tactic_Ext_extCore___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* l_Lean_Name_mkStr2(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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*); static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__3___closed__1; lean_object* l_Lean_indentExpr(lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3; lean_object* l_List_forM___at_Lean_Elab_Command_elabCommand___spec__8(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_mkEmptyEntries(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -631,67 +615,71 @@ lean_object* l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_reprKey LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__2(lean_object*, size_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_Lean_Elab_Tactic_Ext_withExtHyps___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node7(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_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__3; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__6; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__39; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__2; +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalApplyExtTheorem___boxed(lean_object*); lean_object* l_Lean_TagDeclarationExtension_tag(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__1___closed__2; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_withExtN___spec__4(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_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__7; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__5___closed__2; -LEAN_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__6(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__3; uint64_t l_Lean_Name_hash___override(lean_object*); +static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__1; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__1; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__7___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___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_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_Elab_Tactic_Ext_realizeExtTheorem___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt__1___closed__1; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__12; uint8_t l_Lean_Syntax_isNone(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__4___closed__2; lean_object* lean_panic_fn(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalApplyExtTheorem(lean_object*); LEAN_EXPORT lean_object* l_Array_insertionSort_traverse___at_Lean_Elab_Tactic_Ext_getExtTheorems___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___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_Ext_withExtHyps___rarg___lambda__4___boxed__const__1; -static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__3; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__2; lean_object* l_Lean_ResolveName_resolveGlobalName(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__24; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__8(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ScopedEnvExtension_getState___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__8(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); lean_object* l_Array_insertAt_x21___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_withLCtx___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_isStructure(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___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_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); lean_object* l_Lean_ScopedEnvExtension_addCore___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_evalExt___lambda__2___closed__6; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___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_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__2; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__4; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__3___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___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_Elab_Tactic_Ext_realizeExtIffTheorem___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_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___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_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__21; lean_object* l_Lean_PersistentHashMap_mkCollisionNode___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__12(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__2___closed__3; LEAN_EXPORT uint8_t l_Lean_Meta_DiscrTree_Trie_foldValuesM___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__1(lean_object*, uint8_t, lean_object*); -static lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__6___closed__3; -static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem__1___closed__3; extern lean_object* l_Lean_Elab_Tactic_RCases_linter_unusedRCasesPattern; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__49; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); lean_object* l_Array_ofSubarray___rarg(lean_object*); -static size_t l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__1; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__12; extern lean_object* l_Lean_Core_instMonadCoreM; lean_object* l_Lean_MVarId_apply(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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___closed__1; extern lean_object* l_Lean_protectedExt; extern lean_object* l_Lean_instInhabitedDeclarationRanges; @@ -700,10 +688,11 @@ lean_object* l_Array_back___rarg(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__4(lean_object*, lean_object*, size_t, size_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_reverse___rarg(lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalExt___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_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__14; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__14; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___at_Lean_Elab_Tactic_Ext_extCore___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_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__32; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__23; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_extCore___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -713,20 +702,18 @@ lean_object* lean_array_mk(lean_object*); lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalRepeat_x27___spec__1___rarg(lean_object*); static lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___closed__3; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_withExtN___spec__2(lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__2; lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__2___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__45; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___rarg___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_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__5; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__8(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_extExtension; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___rarg___lambda__2(lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); -static lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_extCore___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_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___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_Lean_Elab_Tactic_Ext_withExt1(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__3___closed__2; @@ -734,12 +721,15 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalApplyExtTheorem___rarg___lam LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalExt___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_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__27; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalExt___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_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121_(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt__1___closed__3; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___closed__3; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__19; lean_object* lean_array_uget(lean_object*, size_t); -LEAN_EXPORT uint64_t l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359____spec__1(lean_object*, size_t, size_t, uint64_t); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__25; size_t lean_array_size(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__3; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__5; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___at_Lean_Elab_Tactic_Ext_mkExtIffType___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_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_Ext_withExtHyps___spec__1(size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___closed__3; @@ -747,60 +737,65 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg(lean_ob LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__4___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___closed__1; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__12___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__29; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__6; size_t lean_usize_shift_left(size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___lambda__1___closed__2; lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__2___boxed(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt_declRange__1___closed__5; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__62; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___lambda__1___closed__3; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__12; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__8; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__22; +static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__4; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_withExt1___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__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_forIn_loop___at_Lean_Elab_Tactic_Ext_withExt1___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem_declRange__1___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__8; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__18; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_evalExt___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_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__41; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__40; lean_object* lean_array_get_size(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem__1___closed__5; -LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____spec__3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_mkExtType___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_instBEqExtTheorem; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__48; -LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__3___closed__3; lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_arrowDomainsN___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__6; 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_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__2; extern lean_object* l_Lean_Elab_unsupportedSyntaxExceptionId; +LEAN_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__6(lean_object*, lean_object*, uint8_t, 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_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__5(lean_object*, lean_object*, size_t, size_t, uint8_t); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkProjection(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___lambda__1___closed__1; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__5; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__7(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__51; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_intros(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_erase___at_Lean_Meta_addInstanceEntry___spec__18(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal_loop___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__10(lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__7; lean_object* l_Lean_PersistentHashMap_getCollisionNodeSize___rarg(lean_object*); uint8_t l_Lean_Exception_isRuntime(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_mkExtIffType___spec__1___lambda__1___closed__7; @@ -810,60 +805,66 @@ static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___cl static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__30; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem_declRange__1___closed__2; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__61; -LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__8; static lean_object* l_Lean_Elab_Tactic_Ext_extCore___closed__1; uint8_t l_Lean_Expr_isForall(lean_object*); lean_object* l_Lean_Meta_mkConstWithFreshMVarLevels(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getStructureFieldsFlattened(lean_object*, lean_object*, uint8_t); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__3; +LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___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_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__4; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__10; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_tryIntros___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_String_toSubstring_x27(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__1___lambda__1___closed__2; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__25; -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__13(lean_object*); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__18; +static size_t l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__3___closed__2; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__20; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExtN___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_withExt1___at_Lean_Elab_Tactic_Ext_withExtN___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_run___spec__1___rarg(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_Elab_Tactic_Ext_withExt1___at_Lean_Elab_Tactic_Ext_withExtN___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__13___closed__1; lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); 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_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__6; lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__8___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t l_Lean_Meta_DiscrTree_Key_hash(lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__6; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__26; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__5; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__22; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__20; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Ext_tryIntros___spec__1(lean_object*); +static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__1; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__20; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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_object* l_Lean_Meta_isProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__30; lean_object* l_Lean_addDecl(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_instMonad___rarg(lean_object*); extern lean_object* l_Lean_PersistentHashMap_empty___at_Lean_Meta_Match_instInhabitedMatchEqnsExtState___spec__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__7; -static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__11; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__16; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_applyExtTheoremAt___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_Std_Format_joinSep___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____spec__2(lean_object*, lean_object*); lean_object* l_Lean_Meta_withNewBinderInfos___at_Lean_Meta_withInstImplicitAsImplict___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__8___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1___closed__28; -static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__1; lean_object* l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt_declRange__1___closed__7; static lean_object* l_Lean_Elab_Tactic_Ext_mkExtIffType___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__12(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_Ext_ExtTheorems_erase___spec__3(lean_object*, lean_object*, size_t, size_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Array_isEmpty___rarg(lean_object*); +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__3; +static lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__7; +static lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__27; static lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___closed__3; lean_object* l_Lean_Elab_Term_withDeclName___rarg(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_Elab_Tactic_Ext_withExtHyps___spec__1(size_t x_1, size_t x_2, lean_object* x_3) { @@ -3565,242 +3566,151 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___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_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___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: { -lean_object* x_9; uint8_t 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 = 0; -x_11 = l_Lean_Syntax_getPos_x3f(x_1, x_10); -x_12 = l_Lean_Syntax_getTailPos_x3f(x_1, x_10); -if (lean_obj_tag(x_11) == 0) +uint8_t x_9; lean_object* x_10; +x_9 = 0; +x_10 = l_Lean_Syntax_getRange_x3f(x_1, x_9); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_unsigned_to_nat(0u); -lean_inc(x_9); -x_14 = l_Lean_FileMap_toPosition(x_9, x_13); -lean_inc(x_14); -x_15 = l_Lean_FileMap_leanPosToLspPos(x_9, x_14); -if (lean_obj_tag(x_12) == 0) +lean_object* x_11; lean_object* x_12; +lean_dec(x_6); +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_8); +return x_12; +} +else { -uint8_t x_16; -lean_dec(x_9); -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) +uint8_t x_13; +x_13 = !lean_is_exclusive(x_10); +if (x_13 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_15, 1); -x_18 = lean_ctor_get(x_15, 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_10, 0); +x_15 = lean_ctor_get(x_6, 1); +lean_inc(x_15); +lean_dec(x_6); +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_inc(x_15); +x_17 = l_Lean_FileMap_toPosition(x_15, x_16); +lean_dec(x_16); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_dec(x_14); +lean_inc(x_15); +x_19 = l_Lean_FileMap_toPosition(x_15, x_18); lean_dec(x_18); lean_inc(x_17); -lean_inc(x_14); -x_19 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_19, 0, x_14); -lean_ctor_set(x_19, 1, x_17); -lean_ctor_set(x_19, 2, x_14); -lean_ctor_set(x_19, 3, x_17); -lean_ctor_set(x_15, 1, x_8); -lean_ctor_set(x_15, 0, x_19); -return x_15; -} -else +x_20 = l_Lean_FileMap_leanPosToLspPos(x_15, x_17); +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) { -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_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, 1); +x_23 = lean_ctor_get(x_20, 0); +lean_dec(x_23); +lean_inc(x_19); +x_24 = l_Lean_FileMap_leanPosToLspPos(x_15, x_19); lean_dec(x_15); -lean_inc(x_20); -lean_inc(x_14); -x_21 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_21, 0, x_14); -lean_ctor_set(x_21, 1, x_20); -lean_ctor_set(x_21, 2, x_14); -lean_ctor_set(x_21, 3, 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_8); -return x_22; -} +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_26, 0, x_17); +lean_ctor_set(x_26, 1, x_22); +lean_ctor_set(x_26, 2, x_19); +lean_ctor_set(x_26, 3, x_25); +lean_ctor_set(x_10, 0, x_26); +lean_ctor_set(x_20, 1, x_8); +lean_ctor_set(x_20, 0, x_10); +return x_20; } else { -uint8_t x_23; -x_23 = !lean_is_exclusive(x_15); -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 = lean_ctor_get(x_15, 1); -x_25 = lean_ctor_get(x_15, 0); -lean_dec(x_25); -x_26 = lean_ctor_get(x_12, 0); -lean_inc(x_26); -lean_dec(x_12); -lean_inc(x_9); -x_27 = l_Lean_FileMap_toPosition(x_9, x_26); -lean_dec(x_26); +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_27 = lean_ctor_get(x_20, 1); lean_inc(x_27); -x_28 = l_Lean_FileMap_leanPosToLspPos(x_9, x_27); -lean_dec(x_9); +lean_dec(x_20); +lean_inc(x_19); +x_28 = l_Lean_FileMap_leanPosToLspPos(x_15, x_19); +lean_dec(x_15); x_29 = lean_ctor_get(x_28, 1); lean_inc(x_29); lean_dec(x_28); x_30 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_30, 0, x_14); -lean_ctor_set(x_30, 1, x_24); -lean_ctor_set(x_30, 2, x_27); +lean_ctor_set(x_30, 0, x_17); +lean_ctor_set(x_30, 1, x_27); +lean_ctor_set(x_30, 2, x_19); lean_ctor_set(x_30, 3, x_29); -lean_ctor_set(x_15, 1, x_8); -lean_ctor_set(x_15, 0, x_30); -return x_15; +lean_ctor_set(x_10, 0, x_30); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_10); +lean_ctor_set(x_31, 1, x_8); +return x_31; +} } 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_15, 1); -lean_inc(x_31); -lean_dec(x_15); -x_32 = lean_ctor_get(x_12, 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; lean_object* x_44; lean_object* x_45; +x_32 = lean_ctor_get(x_10, 0); lean_inc(x_32); -lean_dec(x_12); -lean_inc(x_9); -x_33 = l_Lean_FileMap_toPosition(x_9, x_32); +lean_dec(x_10); +x_33 = lean_ctor_get(x_6, 1); +lean_inc(x_33); +lean_dec(x_6); +x_34 = lean_ctor_get(x_32, 0); +lean_inc(x_34); +lean_inc(x_33); +x_35 = l_Lean_FileMap_toPosition(x_33, x_34); +lean_dec(x_34); +x_36 = lean_ctor_get(x_32, 1); +lean_inc(x_36); lean_dec(x_32); lean_inc(x_33); -x_34 = l_Lean_FileMap_leanPosToLspPos(x_9, x_33); -lean_dec(x_9); -x_35 = lean_ctor_get(x_34, 1); +x_37 = l_Lean_FileMap_toPosition(x_33, x_36); +lean_dec(x_36); lean_inc(x_35); -lean_dec(x_34); -x_36 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_36, 0, x_14); -lean_ctor_set(x_36, 1, x_31); -lean_ctor_set(x_36, 2, x_33); -lean_ctor_set(x_36, 3, 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; -} -} -} -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_11, 0); -lean_inc(x_38); -lean_dec(x_11); -lean_inc(x_9); -x_39 = l_Lean_FileMap_toPosition(x_9, x_38); -lean_dec(x_38); +x_38 = l_Lean_FileMap_leanPosToLspPos(x_33, x_35); +x_39 = lean_ctor_get(x_38, 1); lean_inc(x_39); -x_40 = l_Lean_FileMap_leanPosToLspPos(x_9, x_39); -if (lean_obj_tag(x_12) == 0) -{ -uint8_t x_41; -lean_dec(x_9); -x_41 = !lean_is_exclusive(x_40); -if (x_41 == 0) -{ -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_40, 1); -x_43 = lean_ctor_get(x_40, 0); -lean_dec(x_43); -lean_inc(x_42); -lean_inc(x_39); -x_44 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_44, 0, x_39); -lean_ctor_set(x_44, 1, x_42); -lean_ctor_set(x_44, 2, x_39); -lean_ctor_set(x_44, 3, x_42); -lean_ctor_set(x_40, 1, x_8); -lean_ctor_set(x_40, 0, x_44); -return x_40; -} -else -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_40, 1); -lean_inc(x_45); -lean_dec(x_40); -lean_inc(x_45); -lean_inc(x_39); -x_46 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_46, 0, x_39); -lean_ctor_set(x_46, 1, x_45); -lean_ctor_set(x_46, 2, x_39); -lean_ctor_set(x_46, 3, 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_8); -return x_47; -} -} -else -{ -uint8_t x_48; -x_48 = !lean_is_exclusive(x_40); -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; -x_49 = lean_ctor_get(x_40, 1); -x_50 = lean_ctor_get(x_40, 0); -lean_dec(x_50); -x_51 = lean_ctor_get(x_12, 0); -lean_inc(x_51); -lean_dec(x_12); -lean_inc(x_9); -x_52 = l_Lean_FileMap_toPosition(x_9, x_51); -lean_dec(x_51); -lean_inc(x_52); -x_53 = l_Lean_FileMap_leanPosToLspPos(x_9, x_52); -lean_dec(x_9); -x_54 = lean_ctor_get(x_53, 1); -lean_inc(x_54); -lean_dec(x_53); -x_55 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_55, 0, x_39); -lean_ctor_set(x_55, 1, x_49); -lean_ctor_set(x_55, 2, x_52); -lean_ctor_set(x_55, 3, x_54); -lean_ctor_set(x_40, 1, x_8); -lean_ctor_set(x_40, 0, x_55); -return x_40; +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); } -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_40, 1); -lean_inc(x_56); -lean_dec(x_40); -x_57 = lean_ctor_get(x_12, 0); -lean_inc(x_57); -lean_dec(x_12); -lean_inc(x_9); -x_58 = l_Lean_FileMap_toPosition(x_9, x_57); -lean_dec(x_57); -lean_inc(x_58); -x_59 = l_Lean_FileMap_leanPosToLspPos(x_9, x_58); -lean_dec(x_9); -x_60 = lean_ctor_get(x_59, 1); -lean_inc(x_60); -lean_dec(x_59); -x_61 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_61, 0, x_39); -lean_ctor_set(x_61, 1, x_56); -lean_ctor_set(x_61, 2, x_58); -lean_ctor_set(x_61, 3, x_60); -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_8); -return x_62; +lean_inc(x_37); +x_41 = l_Lean_FileMap_leanPosToLspPos(x_33, x_37); +lean_dec(x_33); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +x_43 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_43, 0, x_35); +lean_ctor_set(x_43, 1, x_39); +lean_ctor_set(x_43, 2, x_37); +lean_ctor_set(x_43, 3, x_42); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +if (lean_is_scalar(x_40)) { + x_45 = lean_alloc_ctor(0, 2, 0); +} else { + x_45 = x_40; } +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_8); +return x_45; } } } } -static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__1() { +static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__1() { _start: { lean_object* x_1; @@ -3808,7 +3718,7 @@ x_1 = l_Lean_declRangeExt; return x_1; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2() { +static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2() { _start: { lean_object* x_1; lean_object* x_2; @@ -3819,7 +3729,7 @@ lean_ctor_set(x_2, 1, x_1); return x_2; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__3() { +static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__3() { _start: { lean_object* x_1; lean_object* x_2; @@ -3830,7 +3740,7 @@ lean_ctor_set(x_2, 1, x_1); return x_2; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__4() { +static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__4() { _start: { lean_object* x_1; lean_object* x_2; @@ -3843,13 +3753,13 @@ lean_ctor_set(x_2, 3, x_1); return x_2; } } -static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5() { +static lean_object* _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__3; +x_1 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__3; x_2 = l_Lean_Elab_Tactic_Ext_mkExtType___closed__2; -x_3 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__4; +x_3 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__4; x_4 = lean_alloc_ctor(0, 7, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -3861,7 +3771,7 @@ lean_ctor_set(x_4, 6, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___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_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___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) { _start: { lean_object* x_10; uint8_t x_11; @@ -3876,7 +3786,7 @@ x_14 = lean_ctor_get(x_12, 0); lean_inc(x_14); lean_dec(x_12); x_15 = l_Lean_instInhabitedDeclarationRanges; -x_16 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__1; +x_16 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__1; lean_inc(x_1); x_17 = l_Lean_MapDeclarationExtension_contains___rarg(x_15, x_16, x_14, x_1); lean_dec(x_14); @@ -3898,7 +3808,7 @@ x_22 = lean_ctor_get(x_19, 0); x_23 = lean_ctor_get(x_19, 4); lean_dec(x_23); x_24 = l_Lean_MapDeclarationExtension_insert___rarg(x_16, x_22, x_1, x_2); -x_25 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; +x_25 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; lean_ctor_set(x_19, 4, x_25); lean_ctor_set(x_19, 0, x_24); x_26 = lean_st_ref_set(x_8, x_19, x_20); @@ -3917,7 +3827,7 @@ if (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_29, 1); lean_dec(x_32); -x_33 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +x_33 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; lean_ctor_set(x_29, 1, x_33); x_34 = lean_st_ref_set(x_6, x_29, x_30); x_35 = !lean_is_exclusive(x_34); @@ -3955,7 +3865,7 @@ lean_inc(x_43); lean_inc(x_42); lean_inc(x_41); lean_dec(x_29); -x_45 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +x_45 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; x_46 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_46, 0, x_41); lean_ctor_set(x_46, 1, x_45); @@ -4001,7 +3911,7 @@ lean_inc(x_53); lean_inc(x_52); lean_dec(x_19); x_58 = l_Lean_MapDeclarationExtension_insert___rarg(x_16, x_52, x_1, x_2); -x_59 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; +x_59 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; x_60 = lean_alloc_ctor(0, 7, 0); lean_ctor_set(x_60, 0, x_58); lean_ctor_set(x_60, 1, x_53); @@ -4039,7 +3949,7 @@ if (lean_is_exclusive(x_64)) { lean_dec_ref(x_64); x_70 = lean_box(0); } -x_71 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +x_71 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; if (lean_is_scalar(x_70)) { x_72 = lean_alloc_ctor(0, 5, 0); } else { @@ -4094,7 +4004,7 @@ x_81 = lean_ctor_get(x_79, 0); lean_inc(x_81); lean_dec(x_79); x_82 = l_Lean_instInhabitedDeclarationRanges; -x_83 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__1; +x_83 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__1; lean_inc(x_1); x_84 = l_Lean_MapDeclarationExtension_contains___rarg(x_82, x_83, x_81, x_1); lean_dec(x_81); @@ -4133,7 +4043,7 @@ if (lean_is_exclusive(x_86)) { x_94 = lean_box(0); } x_95 = l_Lean_MapDeclarationExtension_insert___rarg(x_83, x_88, x_1, x_2); -x_96 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; +x_96 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; if (lean_is_scalar(x_94)) { x_97 = lean_alloc_ctor(0, 7, 0); } else { @@ -4175,7 +4085,7 @@ if (lean_is_exclusive(x_101)) { lean_dec_ref(x_101); x_107 = lean_box(0); } -x_108 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +x_108 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; if (lean_is_scalar(x_107)) { x_109 = lean_alloc_ctor(0, 5, 0); } else { @@ -4221,7 +4131,104 @@ return x_116; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___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_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___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_inc(x_8); +x_11 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_2, 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; +lean_dec(x_8); +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 = lean_box(0); +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 = 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; +} +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_19 = lean_ctor_get(x_11, 1); +lean_inc(x_19); +lean_dec(x_11); +x_20 = lean_ctor_get(x_12, 0); +lean_inc(x_20); +lean_dec(x_12); +lean_inc(x_8); +x_21 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_19); +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_20); +lean_dec(x_8); +lean_dec(x_1); +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 = lean_box(0); +lean_ctor_set(x_21, 0, x_25); +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 = 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_26); +return x_28; +} +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +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); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_20); +lean_ctor_set(x_31, 1, x_30); +x_32 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5(x_1, x_31, x_4, x_5, x_6, x_7, x_8, x_9, x_29); +lean_dec(x_8); +return x_32; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___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) { _start: { lean_object* x_9; @@ -5041,7 +5048,7 @@ lean_dec(x_29); x_30 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___closed__1; lean_inc(x_2); x_31 = l_Lean_TagDeclarationExtension_tag(x_30, x_28, x_2); -x_32 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; +x_32 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; lean_ctor_set(x_25, 4, x_32); lean_ctor_set(x_25, 0, x_31); x_33 = lean_st_ref_set(x_11, x_25, x_26); @@ -5057,10 +5064,10 @@ lean_dec(x_35); 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; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; +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_39 = lean_ctor_get(x_36, 1); lean_dec(x_39); -x_40 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +x_40 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; lean_ctor_set(x_36, 1, x_40); x_41 = lean_st_ref_set(x_9, x_36, x_37); x_42 = lean_ctor_get(x_41, 1); @@ -5068,272 +5075,178 @@ lean_inc(x_42); lean_dec(x_41); x_43 = lean_ctor_get(x_10, 5); lean_inc(x_43); -lean_inc(x_10); -x_44 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_43, x_6, x_7, x_8, x_9, x_10, x_11, x_42); -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_10); -x_47 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_43, x_6, x_7, x_8, x_9, x_10, x_11, x_46); -lean_dec(x_43); -x_48 = !lean_is_exclusive(x_47); -if (x_48 == 0) -{ -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_47, 0); -x_50 = lean_ctor_get(x_47, 1); -lean_ctor_set(x_47, 1, x_49); -lean_ctor_set(x_47, 0, x_45); -x_51 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_2, x_47, x_6, x_7, x_8, x_9, x_10, x_11, x_50); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_6); -return x_51; -} -else -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_52 = lean_ctor_get(x_47, 0); -x_53 = lean_ctor_get(x_47, 1); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_47); -x_54 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_54, 0, x_45); -lean_ctor_set(x_54, 1, x_52); -x_55 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_2, x_54, x_6, x_7, x_8, x_9, x_10, x_11, x_53); +x_44 = l_Lean_Elab_addAuxDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_2, x_43, x_43, x_6, x_7, x_8, x_9, x_10, x_11, x_42); lean_dec(x_11); -lean_dec(x_10); lean_dec(x_6); -return x_55; -} +lean_dec(x_43); +return x_44; } 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; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_56 = lean_ctor_get(x_36, 0); -x_57 = lean_ctor_get(x_36, 2); -x_58 = lean_ctor_get(x_36, 3); -x_59 = lean_ctor_get(x_36, 4); -lean_inc(x_59); -lean_inc(x_58); -lean_inc(x_57); -lean_inc(x_56); +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_36, 0); +x_46 = lean_ctor_get(x_36, 2); +x_47 = lean_ctor_get(x_36, 3); +x_48 = lean_ctor_get(x_36, 4); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +lean_inc(x_45); lean_dec(x_36); -x_60 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; -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_9, x_61, x_37); -x_63 = lean_ctor_get(x_62, 1); -lean_inc(x_63); -lean_dec(x_62); -x_64 = lean_ctor_get(x_10, 5); -lean_inc(x_64); -lean_inc(x_10); -x_65 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_64, x_6, x_7, x_8, x_9, x_10, x_11, x_63); -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_10); -x_68 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_64, x_6, x_7, x_8, x_9, x_10, x_11, x_67); -lean_dec(x_64); -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); -} -if (lean_is_scalar(x_71)) { - x_72 = lean_alloc_ctor(0, 2, 0); -} else { - x_72 = x_71; -} -lean_ctor_set(x_72, 0, x_66); -lean_ctor_set(x_72, 1, x_69); -x_73 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_2, x_72, x_6, x_7, x_8, x_9, x_10, x_11, x_70); +x_49 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; +x_50 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_50, 0, x_45); +lean_ctor_set(x_50, 1, x_49); +lean_ctor_set(x_50, 2, x_46); +lean_ctor_set(x_50, 3, x_47); +lean_ctor_set(x_50, 4, x_48); +x_51 = lean_st_ref_set(x_9, x_50, x_37); +x_52 = lean_ctor_get(x_51, 1); +lean_inc(x_52); +lean_dec(x_51); +x_53 = lean_ctor_get(x_10, 5); +lean_inc(x_53); +x_54 = l_Lean_Elab_addAuxDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_2, x_53, x_53, x_6, x_7, x_8, x_9, x_10, x_11, x_52); lean_dec(x_11); -lean_dec(x_10); lean_dec(x_6); -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; 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_74 = lean_ctor_get(x_25, 0); -x_75 = lean_ctor_get(x_25, 1); -x_76 = lean_ctor_get(x_25, 2); -x_77 = lean_ctor_get(x_25, 3); -x_78 = lean_ctor_get(x_25, 5); -x_79 = lean_ctor_get(x_25, 6); -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_dec(x_25); -x_80 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___closed__1; -lean_inc(x_2); -x_81 = l_Lean_TagDeclarationExtension_tag(x_80, x_74, x_2); -x_82 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; -x_83 = lean_alloc_ctor(0, 7, 0); -lean_ctor_set(x_83, 0, x_81); -lean_ctor_set(x_83, 1, x_75); -lean_ctor_set(x_83, 2, x_76); -lean_ctor_set(x_83, 3, x_77); -lean_ctor_set(x_83, 4, x_82); -lean_ctor_set(x_83, 5, x_78); -lean_ctor_set(x_83, 6, x_79); -x_84 = lean_st_ref_set(x_11, x_83, x_26); -x_85 = lean_ctor_get(x_84, 1); -lean_inc(x_85); -lean_dec(x_84); -x_86 = lean_st_ref_take(x_9, x_85); -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, 2); -lean_inc(x_90); -x_91 = lean_ctor_get(x_87, 3); -lean_inc(x_91); -x_92 = lean_ctor_get(x_87, 4); -lean_inc(x_92); -if (lean_is_exclusive(x_87)) { - lean_ctor_release(x_87, 0); - lean_ctor_release(x_87, 1); - lean_ctor_release(x_87, 2); - lean_ctor_release(x_87, 3); - lean_ctor_release(x_87, 4); - x_93 = x_87; -} else { - lean_dec_ref(x_87); - x_93 = lean_box(0); +lean_dec(x_53); +return x_54; } -x_94 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; -if (lean_is_scalar(x_93)) { - x_95 = lean_alloc_ctor(0, 5, 0); -} else { - x_95 = x_93; -} -lean_ctor_set(x_95, 0, x_89); -lean_ctor_set(x_95, 1, x_94); -lean_ctor_set(x_95, 2, x_90); -lean_ctor_set(x_95, 3, x_91); -lean_ctor_set(x_95, 4, x_92); -x_96 = lean_st_ref_set(x_9, x_95, x_88); -x_97 = lean_ctor_get(x_96, 1); -lean_inc(x_97); -lean_dec(x_96); -x_98 = lean_ctor_get(x_10, 5); -lean_inc(x_98); -lean_inc(x_10); -x_99 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_98, x_6, x_7, x_8, x_9, x_10, x_11, x_97); -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); -lean_inc(x_10); -x_102 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_98, x_6, x_7, x_8, x_9, x_10, x_11, x_101); -lean_dec(x_98); -x_103 = lean_ctor_get(x_102, 0); -lean_inc(x_103); -x_104 = lean_ctor_get(x_102, 1); -lean_inc(x_104); -if (lean_is_exclusive(x_102)) { - lean_ctor_release(x_102, 0); - lean_ctor_release(x_102, 1); - x_105 = x_102; +} +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; 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_55 = lean_ctor_get(x_25, 0); +x_56 = lean_ctor_get(x_25, 1); +x_57 = lean_ctor_get(x_25, 2); +x_58 = lean_ctor_get(x_25, 3); +x_59 = lean_ctor_get(x_25, 5); +x_60 = lean_ctor_get(x_25, 6); +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_25); +x_61 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___closed__1; +lean_inc(x_2); +x_62 = l_Lean_TagDeclarationExtension_tag(x_61, x_55, x_2); +x_63 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; +x_64 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_64, 0, x_62); +lean_ctor_set(x_64, 1, x_56); +lean_ctor_set(x_64, 2, x_57); +lean_ctor_set(x_64, 3, x_58); +lean_ctor_set(x_64, 4, x_63); +lean_ctor_set(x_64, 5, x_59); +lean_ctor_set(x_64, 6, x_60); +x_65 = lean_st_ref_set(x_11, x_64, x_26); +x_66 = lean_ctor_get(x_65, 1); +lean_inc(x_66); +lean_dec(x_65); +x_67 = lean_st_ref_take(x_9, 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); +lean_dec(x_67); +x_70 = lean_ctor_get(x_68, 0); +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); +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); + x_74 = x_68; } else { - lean_dec_ref(x_102); - x_105 = lean_box(0); + lean_dec_ref(x_68); + x_74 = lean_box(0); } -if (lean_is_scalar(x_105)) { - x_106 = lean_alloc_ctor(0, 2, 0); +x_75 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; +if (lean_is_scalar(x_74)) { + x_76 = lean_alloc_ctor(0, 5, 0); } else { - x_106 = x_105; + x_76 = x_74; } -lean_ctor_set(x_106, 0, x_100); -lean_ctor_set(x_106, 1, x_103); -x_107 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_2, x_106, x_6, x_7, x_8, x_9, x_10, x_11, x_104); +lean_ctor_set(x_76, 0, x_70); +lean_ctor_set(x_76, 1, x_75); +lean_ctor_set(x_76, 2, x_71); +lean_ctor_set(x_76, 3, x_72); +lean_ctor_set(x_76, 4, x_73); +x_77 = lean_st_ref_set(x_9, x_76, x_69); +x_78 = lean_ctor_get(x_77, 1); +lean_inc(x_78); +lean_dec(x_77); +x_79 = lean_ctor_get(x_10, 5); +lean_inc(x_79); +x_80 = l_Lean_Elab_addAuxDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_2, x_79, x_79, x_6, x_7, x_8, x_9, x_10, x_11, x_78); lean_dec(x_11); -lean_dec(x_10); lean_dec(x_6); -return x_107; +lean_dec(x_79); +return x_80; } } else { -uint8_t x_108; +uint8_t x_81; lean_dec(x_11); lean_dec(x_10); lean_dec(x_6); lean_dec(x_2); -x_108 = !lean_is_exclusive(x_22); -if (x_108 == 0) +x_81 = !lean_is_exclusive(x_22); +if (x_81 == 0) { return x_22; } else { -lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_109 = lean_ctor_get(x_22, 0); -x_110 = lean_ctor_get(x_22, 1); -lean_inc(x_110); -lean_inc(x_109); +lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_82 = lean_ctor_get(x_22, 0); +x_83 = lean_ctor_get(x_22, 1); +lean_inc(x_83); +lean_inc(x_82); lean_dec(x_22); -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_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_112; +uint8_t x_85; lean_dec(x_11); lean_dec(x_10); lean_dec(x_6); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_112 = !lean_is_exclusive(x_13); -if (x_112 == 0) +x_85 = !lean_is_exclusive(x_13); +if (x_85 == 0) { return x_13; } else { -lean_object* x_113; lean_object* x_114; lean_object* x_115; -x_113 = lean_ctor_get(x_13, 0); -x_114 = lean_ctor_get(x_13, 1); -lean_inc(x_114); -lean_inc(x_113); +lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_86 = lean_ctor_get(x_13, 0); +x_87 = lean_ctor_get(x_13, 1); +lean_inc(x_87); +lean_inc(x_86); lean_dec(x_13); -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_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; } } } @@ -5658,7 +5571,7 @@ lean_inc(x_8); x_17 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); lean_closure_set(x_17, 0, x_8); lean_closure_set(x_17, 1, x_16); -x_18 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5), 8, 1); +x_18 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__6), 8, 1); lean_closure_set(x_18, 0, x_17); x_19 = l_Lean_Elab_Command_liftTermElabM___rarg(x_18, x_4, x_5, x_12); if (lean_obj_tag(x_19) == 0) @@ -5844,7 +5757,7 @@ lean_inc(x_8); x_66 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); lean_closure_set(x_66, 0, x_8); lean_closure_set(x_66, 1, x_65); -x_67 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5), 8, 1); +x_67 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__6), 8, 1); lean_closure_set(x_67, 0, x_66); x_68 = l_Lean_Elab_Command_liftTermElabM___rarg(x_67, x_4, x_5, x_61); if (lean_obj_tag(x_68) == 0) @@ -6119,11 +6032,11 @@ lean_dec(x_3); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___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_EXPORT lean_object* l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___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_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_getDeclarationRange_x3f___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___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_5); lean_dec(x_4); @@ -6133,11 +6046,11 @@ lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___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_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___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) { _start: { lean_object* x_10; -x_10 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__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); @@ -6147,6 +6060,21 @@ lean_dec(x_3); return x_10; } } +LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___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) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Elab_addAuxDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___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_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_Ext_realizeExtTheorem___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -7529,267 +7457,233 @@ return x_356; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___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; lean_object* x_14; uint8_t x_15; +lean_object* x_10; lean_object* x_11; x_10 = lean_ctor_get(x_7, 5); lean_inc(x_10); -lean_inc(x_7); -x_11 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_10, 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); -lean_inc(x_7); -x_14 = l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_13); +x_11 = l_Lean_Elab_addAuxDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__3(x_1, x_10, x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_10); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) -{ -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_ctor_set(x_14, 1, x_16); -lean_ctor_set(x_14, 0, x_12); -x_18 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_1, x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_17); -lean_dec(x_7); -return x_18; -} -else -{ -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_ctor_get(x_14, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_14); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_12); -lean_ctor_set(x_21, 1, x_19); -x_22 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4(x_1, x_21, x_3, x_4, x_5, x_6, x_7, x_8, x_20); -lean_dec(x_7); -return x_22; -} +return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___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_Elab_Tactic_Ext_realizeExtIffTheorem___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_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_Lean_ConstantInfo_levelParams(x_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; +x_14 = l_Lean_ConstantInfo_levelParams(x_1); lean_inc(x_2); -x_14 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_14, 0, x_2); -lean_ctor_set(x_14, 1, x_13); -lean_ctor_set(x_14, 2, x_3); -x_15 = lean_box(0); +x_15 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_15, 0, x_2); +lean_ctor_set(x_15, 1, x_14); +lean_ctor_set(x_15, 2, x_3); +x_16 = lean_box(0); lean_inc(x_2); -x_16 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_16, 0, x_2); -lean_ctor_set(x_16, 1, x_15); -x_17 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_17, 0, x_14); -lean_ctor_set(x_17, 1, x_4); -lean_ctor_set(x_17, 2, x_16); -x_18 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_18, 0, x_17); +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_alloc_ctor(0, 3, 0); +lean_ctor_set(x_18, 0, x_15); +lean_ctor_set(x_18, 1, x_4); +lean_ctor_set(x_18, 2, x_17); +x_19 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_19, 0, x_18); +lean_inc(x_12); lean_inc(x_11); -lean_inc(x_10); -x_19 = l_Lean_addDecl(x_18, x_10, x_11, x_12); -if (lean_obj_tag(x_19) == 0) +x_20 = l_Lean_addDecl(x_19, x_11, x_12, x_13); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_20; uint8_t x_21; -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); -x_21 = l_Lean_Name_isAtomic(x_2); -if (x_21 == 0) +lean_object* x_21; uint8_t x_22; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = l_Lean_Name_isAtomic(x_2); +if (x_22 == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_22 = lean_st_ref_take(x_11, x_20); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); +lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_23 = lean_st_ref_take(x_12, x_21); +x_24 = lean_ctor_get(x_23, 0); lean_inc(x_24); -lean_dec(x_22); -x_25 = !lean_is_exclusive(x_23); -if (x_25 == 0) +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_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; uint8_t x_36; -x_26 = lean_ctor_get(x_23, 0); -x_27 = lean_ctor_get(x_23, 4); -lean_dec(x_27); -x_28 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___closed__1; -lean_inc(x_2); -x_29 = l_Lean_TagDeclarationExtension_tag(x_28, x_26, x_2); -x_30 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; -lean_ctor_set(x_23, 4, x_30); -lean_ctor_set(x_23, 0, x_29); -x_31 = lean_st_ref_set(x_11, x_23, x_24); -x_32 = lean_ctor_get(x_31, 1); -lean_inc(x_32); -lean_dec(x_31); -x_33 = lean_st_ref_take(x_9, x_32); -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); +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_27 = lean_ctor_get(x_24, 0); +x_28 = lean_ctor_get(x_24, 4); +lean_dec(x_28); +x_29 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___closed__1; +x_30 = l_Lean_TagDeclarationExtension_tag(x_29, x_27, x_2); +x_31 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; +lean_ctor_set(x_24, 4, x_31); +lean_ctor_set(x_24, 0, x_30); +x_32 = lean_st_ref_set(x_12, x_24, x_25); +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); +x_34 = lean_st_ref_take(x_10, x_33); +x_35 = lean_ctor_get(x_34, 0); lean_inc(x_35); -lean_dec(x_33); -x_36 = !lean_is_exclusive(x_34); -if (x_36 == 0) +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); +lean_dec(x_34); +x_37 = !lean_is_exclusive(x_35); +if (x_37 == 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; -x_37 = lean_ctor_get(x_34, 1); -lean_dec(x_37); -x_38 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; -lean_ctor_set(x_34, 1, x_38); -x_39 = lean_st_ref_set(x_9, x_34, x_35); -x_40 = lean_ctor_get(x_39, 1); -lean_inc(x_40); -lean_dec(x_39); -x_41 = lean_box(0); -x_42 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2(x_2, x_41, x_6, x_7, x_8, x_9, x_10, x_11, x_40); -lean_dec(x_11); -return x_42; +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_35, 1); +lean_dec(x_38); +x_39 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; +lean_ctor_set(x_35, 1, x_39); +x_40 = lean_st_ref_set(x_10, x_35, x_36); +x_41 = lean_ctor_get(x_40, 1); +lean_inc(x_41); +lean_dec(x_40); +x_42 = lean_box(0); +x_43 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2(x_5, x_42, x_7, x_8, x_9, x_10, x_11, x_12, x_41); +lean_dec(x_12); +return x_43; } 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; -x_43 = lean_ctor_get(x_34, 0); -x_44 = lean_ctor_get(x_34, 2); -x_45 = lean_ctor_get(x_34, 3); -x_46 = lean_ctor_get(x_34, 4); +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_35, 0); +x_45 = lean_ctor_get(x_35, 2); +x_46 = lean_ctor_get(x_35, 3); +x_47 = lean_ctor_get(x_35, 4); +lean_inc(x_47); lean_inc(x_46); lean_inc(x_45); lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_34); -x_47 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; -x_48 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_48, 0, x_43); -lean_ctor_set(x_48, 1, x_47); -lean_ctor_set(x_48, 2, x_44); -lean_ctor_set(x_48, 3, x_45); -lean_ctor_set(x_48, 4, x_46); -x_49 = lean_st_ref_set(x_9, x_48, x_35); -x_50 = lean_ctor_get(x_49, 1); -lean_inc(x_50); -lean_dec(x_49); -x_51 = lean_box(0); -x_52 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2(x_2, x_51, x_6, x_7, x_8, x_9, x_10, x_11, x_50); -lean_dec(x_11); -return x_52; +lean_dec(x_35); +x_48 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; +x_49 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_49, 0, x_44); +lean_ctor_set(x_49, 1, x_48); +lean_ctor_set(x_49, 2, x_45); +lean_ctor_set(x_49, 3, x_46); +lean_ctor_set(x_49, 4, x_47); +x_50 = lean_st_ref_set(x_10, x_49, x_36); +x_51 = lean_ctor_get(x_50, 1); +lean_inc(x_51); +lean_dec(x_50); +x_52 = lean_box(0); +x_53 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2(x_5, x_52, x_7, x_8, x_9, x_10, x_11, x_12, x_51); +lean_dec(x_12); +return x_53; } } 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; -x_53 = lean_ctor_get(x_23, 0); -x_54 = lean_ctor_get(x_23, 1); -x_55 = lean_ctor_get(x_23, 2); -x_56 = lean_ctor_get(x_23, 3); -x_57 = lean_ctor_get(x_23, 5); -x_58 = lean_ctor_get(x_23, 6); +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_54 = lean_ctor_get(x_24, 0); +x_55 = lean_ctor_get(x_24, 1); +x_56 = lean_ctor_get(x_24, 2); +x_57 = lean_ctor_get(x_24, 3); +x_58 = lean_ctor_get(x_24, 5); +x_59 = lean_ctor_get(x_24, 6); +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_23); -x_59 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___closed__1; -lean_inc(x_2); -x_60 = l_Lean_TagDeclarationExtension_tag(x_59, x_53, x_2); -x_61 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; -x_62 = lean_alloc_ctor(0, 7, 0); -lean_ctor_set(x_62, 0, x_60); -lean_ctor_set(x_62, 1, x_54); -lean_ctor_set(x_62, 2, x_55); -lean_ctor_set(x_62, 3, x_56); -lean_ctor_set(x_62, 4, x_61); -lean_ctor_set(x_62, 5, x_57); -lean_ctor_set(x_62, 6, x_58); -x_63 = lean_st_ref_set(x_11, x_62, x_24); -x_64 = lean_ctor_get(x_63, 1); -lean_inc(x_64); -lean_dec(x_63); -x_65 = lean_st_ref_take(x_9, x_64); -x_66 = lean_ctor_get(x_65, 0); -lean_inc(x_66); -x_67 = lean_ctor_get(x_65, 1); +lean_dec(x_24); +x_60 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__3___closed__1; +x_61 = l_Lean_TagDeclarationExtension_tag(x_60, x_54, x_2); +x_62 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; +x_63 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_63, 0, x_61); +lean_ctor_set(x_63, 1, x_55); +lean_ctor_set(x_63, 2, x_56); +lean_ctor_set(x_63, 3, x_57); +lean_ctor_set(x_63, 4, x_62); +lean_ctor_set(x_63, 5, x_58); +lean_ctor_set(x_63, 6, x_59); +x_64 = lean_st_ref_set(x_12, x_63, x_25); +x_65 = lean_ctor_get(x_64, 1); +lean_inc(x_65); +lean_dec(x_64); +x_66 = lean_st_ref_take(x_10, x_65); +x_67 = lean_ctor_get(x_66, 0); lean_inc(x_67); -lean_dec(x_65); -x_68 = lean_ctor_get(x_66, 0); +x_68 = lean_ctor_get(x_66, 1); lean_inc(x_68); -x_69 = lean_ctor_get(x_66, 2); +lean_dec(x_66); +x_69 = lean_ctor_get(x_67, 0); lean_inc(x_69); -x_70 = lean_ctor_get(x_66, 3); +x_70 = lean_ctor_get(x_67, 2); lean_inc(x_70); -x_71 = lean_ctor_get(x_66, 4); +x_71 = lean_ctor_get(x_67, 3); lean_inc(x_71); -if (lean_is_exclusive(x_66)) { - lean_ctor_release(x_66, 0); - lean_ctor_release(x_66, 1); - lean_ctor_release(x_66, 2); - lean_ctor_release(x_66, 3); - lean_ctor_release(x_66, 4); - x_72 = x_66; +x_72 = lean_ctor_get(x_67, 4); +lean_inc(x_72); +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); + x_73 = x_67; } else { - lean_dec_ref(x_66); - x_72 = lean_box(0); + lean_dec_ref(x_67); + x_73 = lean_box(0); } -x_73 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; -if (lean_is_scalar(x_72)) { - x_74 = lean_alloc_ctor(0, 5, 0); +x_74 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; +if (lean_is_scalar(x_73)) { + x_75 = lean_alloc_ctor(0, 5, 0); } else { - x_74 = x_72; + x_75 = x_73; } -lean_ctor_set(x_74, 0, x_68); -lean_ctor_set(x_74, 1, x_73); -lean_ctor_set(x_74, 2, x_69); -lean_ctor_set(x_74, 3, x_70); -lean_ctor_set(x_74, 4, x_71); -x_75 = lean_st_ref_set(x_9, x_74, x_67); -x_76 = lean_ctor_get(x_75, 1); -lean_inc(x_76); -lean_dec(x_75); -x_77 = lean_box(0); -x_78 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2(x_2, x_77, x_6, x_7, x_8, x_9, x_10, x_11, x_76); -lean_dec(x_11); -return x_78; +lean_ctor_set(x_75, 0, x_69); +lean_ctor_set(x_75, 1, x_74); +lean_ctor_set(x_75, 2, x_70); +lean_ctor_set(x_75, 3, x_71); +lean_ctor_set(x_75, 4, x_72); +x_76 = lean_st_ref_set(x_10, x_75, x_68); +x_77 = lean_ctor_get(x_76, 1); +lean_inc(x_77); +lean_dec(x_76); +x_78 = lean_box(0); +x_79 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2(x_5, x_78, x_7, x_8, x_9, x_10, x_11, x_12, x_77); +lean_dec(x_12); +return x_79; } } else { -lean_object* x_79; lean_object* x_80; -x_79 = lean_box(0); -x_80 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2(x_2, x_79, x_6, x_7, x_8, x_9, x_10, x_11, x_20); -lean_dec(x_11); -return x_80; +lean_object* x_80; lean_object* x_81; +lean_dec(x_2); +x_80 = lean_box(0); +x_81 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__2(x_5, x_80, x_7, x_8, x_9, x_10, x_11, x_12, x_21); +lean_dec(x_12); +return x_81; } } else { -uint8_t x_81; +uint8_t x_82; +lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_5); lean_dec(x_2); -x_81 = !lean_is_exclusive(x_19); -if (x_81 == 0) +x_82 = !lean_is_exclusive(x_20); +if (x_82 == 0) { -return x_19; +return x_20; } else { -lean_object* x_82; lean_object* x_83; lean_object* x_84; -x_82 = lean_ctor_get(x_19, 0); -x_83 = lean_ctor_get(x_19, 1); +lean_object* x_83; lean_object* x_84; lean_object* x_85; +x_83 = lean_ctor_get(x_20, 0); +x_84 = lean_ctor_get(x_20, 1); +lean_inc(x_84); lean_inc(x_83); -lean_inc(x_82); -lean_dec(x_19); -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_dec(x_20); +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; } } } @@ -7830,6 +7724,7 @@ x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); lean_inc(x_12); +lean_inc(x_1); x_14 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__1), 9, 2); lean_closure_set(x_14, 0, x_1); lean_closure_set(x_14, 1, x_12); @@ -7862,7 +7757,7 @@ if (x_23 == 0) lean_object* x_24; lean_object* x_25; lean_free_object(x_19); x_24 = lean_box(0); -x_25 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__3(x_2, x_3, x_12, x_21, x_24, x_4, x_5, x_6, x_7, x_8, x_9, x_22); +x_25 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__3(x_2, x_3, x_12, x_21, x_1, x_24, x_4, x_5, x_6, x_7, x_8, x_9, x_22); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -7874,6 +7769,7 @@ 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; uint8_t x_32; lean_dec(x_12); lean_dec(x_3); +lean_dec(x_1); x_26 = l_Lean_MessageData_ofExpr(x_21); x_27 = l_Lean_indentD(x_26); x_28 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__4___closed__2; @@ -7923,7 +7819,7 @@ if (x_38 == 0) { lean_object* x_39; lean_object* x_40; x_39 = lean_box(0); -x_40 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__3(x_2, x_3, x_12, x_36, x_39, x_4, x_5, x_6, x_7, x_8, x_9, x_37); +x_40 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__3(x_2, x_3, x_12, x_36, x_1, x_39, x_4, x_5, x_6, x_7, x_8, x_9, x_37); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -7935,6 +7831,7 @@ 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; lean_dec(x_12); lean_dec(x_3); +lean_dec(x_1); x_41 = l_Lean_MessageData_ofExpr(x_36); x_42 = l_Lean_indentD(x_41); x_43 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___lambda__4___closed__2; @@ -7985,6 +7882,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_16); if (x_52 == 0) { @@ -8152,7 +8050,7 @@ lean_inc(x_6); x_16 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); lean_closure_set(x_16, 0, x_6); lean_closure_set(x_16, 1, x_15); -x_17 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5), 8, 1); +x_17 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__6), 8, 1); lean_closure_set(x_17, 0, x_16); x_18 = l_Lean_Elab_Command_liftTermElabM___rarg(x_17, x_2, x_3, x_14); if (lean_obj_tag(x_18) == 0) @@ -8471,7 +8369,7 @@ lean_inc(x_6); x_103 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withDeclName___rarg), 9, 2); lean_closure_set(x_103, 0, x_6); lean_closure_set(x_103, 1, x_102); -x_104 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5), 8, 1); +x_104 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutErrToSorry___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__6), 8, 1); lean_closure_set(x_104, 0, x_103); x_105 = l_Lean_Elab_Command_liftTermElabM___rarg(x_104, x_2, x_3, x_101); if (lean_obj_tag(x_105) == 0) @@ -8678,18 +8576,18 @@ lean_dec(x_2); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___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_Elab_Tactic_Ext_realizeExtIffTheorem___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_Elab_Tactic_Ext_realizeExtIffTheorem___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_object* x_14; +x_14 = l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___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_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_13; +return x_14; } } LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_realizeExtIffTheorem___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) { @@ -8732,7 +8630,7 @@ x_1 = l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorem___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l_repr___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_repr___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____spec__1(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -8741,7 +8639,7 @@ x_3 = l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_reprKey____x40 return x_3; } } -LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) @@ -8795,7 +8693,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____spec__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____spec__2(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -8829,13 +8727,13 @@ lean_inc(x_8); lean_dec(x_1); x_9 = lean_unsigned_to_nat(0u); x_10 = l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_reprKey____x40_Lean_Meta_DiscrTreeTypes___hyg_355_(x_8, x_9); -x_11 = l_List_foldl___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____spec__3(x_2, x_10, x_4); +x_11 = l_List_foldl___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____spec__3(x_2, x_10, x_4); return x_11; } } } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__1() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__1() { _start: { lean_object* x_1; @@ -8843,29 +8741,29 @@ x_1 = lean_mk_string_unchecked("declName", 8, 8); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__2() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__1; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____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_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__3() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____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_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__2; +x_2 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____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_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__4() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__4() { _start: { lean_object* x_1; @@ -8873,29 +8771,29 @@ x_1 = lean_mk_string_unchecked(" := ", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__5() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__4; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____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_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__6() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__3; -x_2 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__5; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__3; +x_2 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____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_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__7() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__7() { _start: { lean_object* x_1; lean_object* x_2; @@ -8904,7 +8802,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__8() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__8() { _start: { lean_object* x_1; lean_object* x_2; @@ -8914,7 +8812,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__9() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__9() { _start: { lean_object* x_1; @@ -8922,17 +8820,17 @@ x_1 = lean_mk_string_unchecked("priority", 8, 8); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__10() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__9; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____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___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__11() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__11() { _start: { lean_object* x_1; @@ -8940,17 +8838,17 @@ x_1 = lean_mk_string_unchecked("keys", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__12() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__11; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____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___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__13() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__13() { _start: { lean_object* x_1; lean_object* x_2; @@ -8959,7 +8857,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__14() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__14() { _start: { lean_object* x_1; @@ -8967,35 +8865,35 @@ x_1 = lean_mk_string_unchecked("{ ", 2, 2); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__15() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__15() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__14; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__14; x_2 = lean_string_length(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__16() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__16() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__15; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__15; x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__17() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__17() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__14; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____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_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__18() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__18() { _start: { lean_object* x_1; @@ -9003,21 +8901,21 @@ x_1 = lean_mk_string_unchecked(" }", 2, 2); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__19() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__19() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__18; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__18; 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_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__20() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__20() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__8; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__8; x_2 = lean_box(1); x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -9025,7 +8923,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__21() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__21() { _start: { lean_object* x_1; @@ -9033,35 +8931,35 @@ x_1 = lean_mk_string_unchecked("#[", 2, 2); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__22() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__22() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__21; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__21; x_2 = lean_string_length(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__23() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__23() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__22; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__22; x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__24() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__24() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__21; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__21; 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_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__25() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__25() { _start: { lean_object* x_1; @@ -9069,17 +8967,17 @@ x_1 = lean_mk_string_unchecked("]", 1, 1); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__26() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__26() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__25; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____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_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__27() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__27() { _start: { lean_object* x_1; @@ -9087,33 +8985,33 @@ x_1 = lean_mk_string_unchecked("#[]", 3, 3); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__28() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__28() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__27; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____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_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__29() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__29() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__13; -x_2 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__28; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__13; +x_2 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__28; 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_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__30() { +static lean_object* _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__30() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__29; +x_1 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__29; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -9121,7 +9019,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121_(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; uint8_t x_33; @@ -9129,7 +9027,7 @@ x_3 = lean_ctor_get(x_1, 0); lean_inc(x_3); x_4 = lean_unsigned_to_nat(0u); x_5 = l_Lean_Name_reprPrec(x_3, x_4); -x_6 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__7; +x_6 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____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); @@ -9137,11 +9035,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_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__6; +x_10 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____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_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__8; +x_12 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__8; x_13 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_13, 0, x_11); lean_ctor_set(x_13, 1, x_12); @@ -9149,11 +9047,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_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__10; +x_16 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__10; 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_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__5; +x_18 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____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); @@ -9177,7 +9075,7 @@ 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_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__12; +x_28 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__12; x_29 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_29, 0, x_27); lean_ctor_set(x_29, 1, x_28); @@ -9194,17 +9092,17 @@ 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; 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; x_34 = lean_array_to_list(x_31); -x_35 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__20; -x_36 = l_Std_Format_joinSep___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____spec__2(x_34, x_35); -x_37 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__24; +x_35 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__20; +x_36 = l_Std_Format_joinSep___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____spec__2(x_34, x_35); +x_37 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__24; x_38 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_38, 0, x_37); lean_ctor_set(x_38, 1, x_36); -x_39 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__26; +x_39 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__26; 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 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__23; +x_41 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__23; x_42 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_42, 0, x_41); lean_ctor_set(x_42, 1, x_40); @@ -9212,7 +9110,7 @@ x_43 = 1; x_44 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_44, 0, x_42); lean_ctor_set_uint8(x_44, sizeof(void*)*1, x_43); -x_45 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__13; +x_45 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__13; x_46 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_46, 0, x_45); lean_ctor_set(x_46, 1, x_44); @@ -9222,15 +9120,15 @@ lean_ctor_set_uint8(x_47, sizeof(void*)*1, x_8); x_48 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_48, 0, x_30); lean_ctor_set(x_48, 1, x_47); -x_49 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__17; +x_49 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__17; x_50 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_50, 0, x_49); lean_ctor_set(x_50, 1, x_48); -x_51 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__19; +x_51 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__19; x_52 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_52, 0, x_50); lean_ctor_set(x_52, 1, x_51); -x_53 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__16; +x_53 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__16; x_54 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_54, 0, x_53); lean_ctor_set(x_54, 1, x_52); @@ -9243,19 +9141,19 @@ 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_dec(x_31); -x_56 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__30; +x_56 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__30; x_57 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_57, 0, x_30); lean_ctor_set(x_57, 1, x_56); -x_58 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__17; +x_58 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__17; x_59 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_59, 0, x_58); lean_ctor_set(x_59, 1, x_57); -x_60 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__19; +x_60 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__19; x_61 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_61, 0, x_59); lean_ctor_set(x_61, 1, x_60); -x_62 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__16; +x_62 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__16; x_63 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_63, 0, x_62); lean_ctor_set(x_63, 1, x_61); @@ -9266,11 +9164,11 @@ return x_64; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191_(x_1, x_2); +x_3 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121_(x_1, x_2); lean_dec(x_2); return x_3; } @@ -9279,7 +9177,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_Ext_instReprExtTheorem___closed__1( _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____boxed), 2, 0); return x_1; } } @@ -9291,7 +9189,7 @@ x_1 = l_Lean_Elab_Tactic_Ext_instReprExtTheorem___closed__1; return x_1; } } -LEAN_EXPORT uint8_t l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269____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_EXPORT uint8_t l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3199____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_8; uint8_t x_9; @@ -9332,7 +9230,7 @@ return x_17; } } } -LEAN_EXPORT uint8_t l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3199_(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; uint8_t x_9; @@ -9376,18 +9274,18 @@ return x_16; else { uint8_t x_17; -x_17 = l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269____spec__1(x_5, x_8, lean_box(0), x_5, x_8, x_13, lean_box(0)); +x_17 = l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3199____spec__1(x_5, x_8, lean_box(0), x_5, x_8, x_13, lean_box(0)); return x_17; } } } } } -LEAN_EXPORT lean_object* l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269____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_EXPORT lean_object* l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3199____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: { uint8_t x_8; lean_object* x_9; -x_8 = l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269____spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Array_isEqvAux___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3199____spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); @@ -9396,11 +9294,11 @@ x_9 = lean_box(x_8); return x_9; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3199____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269_(x_1, x_2); +x_3 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3199_(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); @@ -9411,7 +9309,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_Ext_instBEqExtTheorem___closed__1() _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3199____boxed), 2, 0); return x_1; } } @@ -9423,7 +9321,7 @@ x_1 = l_Lean_Elab_Tactic_Ext_instBEqExtTheorem___closed__1; return x_1; } } -LEAN_EXPORT uint64_t l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359____spec__1(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_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3289____spec__1(lean_object* x_1, size_t x_2, size_t x_3, uint64_t x_4) { _start: { uint8_t x_5; @@ -9447,7 +9345,7 @@ return x_4; } } } -LEAN_EXPORT uint64_t l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359_(lean_object* x_1) { +LEAN_EXPORT uint64_t l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3289_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; uint64_t x_5; uint64_t x_6; uint64_t x_7; uint64_t x_8; uint64_t x_9; uint64_t x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -9487,14 +9385,14 @@ size_t x_17; size_t x_18; uint64_t x_19; uint64_t x_20; x_17 = 0; x_18 = lean_usize_of_nat(x_11); lean_dec(x_11); -x_19 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359____spec__1(x_4, x_17, x_18, x_10); +x_19 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3289____spec__1(x_4, x_17, x_18, x_10); x_20 = lean_uint64_mix_hash(x_9, x_19); return x_20; } } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359____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___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3289____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; uint64_t x_7; uint64_t x_8; lean_object* x_9; @@ -9504,17 +9402,17 @@ 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_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359____spec__1(x_1, x_5, x_6, x_7); +x_8 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3289____spec__1(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___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359____boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3289____boxed(lean_object* x_1) { _start: { uint64_t x_2; lean_object* x_3; -x_2 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359_(x_1); +x_2 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3289_(x_1); lean_dec(x_1); x_3 = lean_box_uint64(x_2); return x_3; @@ -9524,7 +9422,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_Ext_instHashableExtTheorem___closed _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3359____boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_hashExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3289____boxed), 1, 0); return x_1; } } @@ -9579,7 +9477,7 @@ x_1 = l_Lean_Elab_Tactic_Ext_extExt_config___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__4(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_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__4(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; @@ -9621,7 +9519,7 @@ return x_15; } } } -static size_t _init_l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__1() { +static size_t _init_l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3___closed__1() { _start: { size_t x_1; size_t x_2; size_t x_3; @@ -9631,17 +9529,17 @@ x_3 = lean_usize_shift_left(x_1, x_2); return x_3; } } -static size_t _init_l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__2() { +static size_t _init_l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3___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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__1; +x_2 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3___closed__1; x_3 = lean_usize_sub(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3(lean_object* x_1, size_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3(lean_object* x_1, size_t x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -9653,7 +9551,7 @@ 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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__2; +x_7 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3___closed__2; x_8 = lean_usize_land(x_2, x_7); x_9 = lean_usize_to_nat(x_8); x_10 = lean_box(2); @@ -9714,7 +9612,7 @@ 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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__2; +x_22 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3___closed__2; x_23 = lean_usize_land(x_2, x_22); x_24 = lean_usize_to_nat(x_23); x_25 = lean_box(2); @@ -9776,24 +9674,24 @@ 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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__4(x_36, x_37, lean_box(0), x_38, x_3); +x_39 = l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__4(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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__2(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_DiscrTree_Key_hash(x_2); x_4 = lean_uint64_to_usize(x_3); -x_5 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3(x_1, x_4, x_2); +x_5 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3(x_1, x_4, x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____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) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____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; @@ -9820,7 +9718,7 @@ 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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6(x_6, x_17, x_1, x_9, x_10); +x_20 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__6(x_6, x_17, x_1, x_9, x_10); x_4 = lean_box(0); x_5 = x_19; x_6 = x_20; @@ -9828,7 +9726,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____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; @@ -9920,7 +9818,7 @@ return x_29; } } } -static lean_object* _init_l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6___closed__1() { +static lean_object* _init_l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__6___closed__1() { _start: { lean_object* x_1; @@ -9928,7 +9826,7 @@ 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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____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) @@ -9941,7 +9839,7 @@ lean_object* x_7; size_t x_8; size_t x_9; size_t x_10; size_t x_11; lean_object* x_7 = lean_ctor_get(x_1, 0); x_8 = 1; x_9 = 5; -x_10 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__2; +x_10 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3___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); @@ -10041,7 +9939,7 @@ lean_object* x_35; size_t x_36; size_t x_37; lean_object* x_38; lean_object* x_3 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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6(x_35, x_36, x_37, x_4, x_5); +x_38 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__6(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); @@ -10056,7 +9954,7 @@ 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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6(x_40, x_41, x_42, x_4, x_5); +x_43 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__6(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); @@ -10087,7 +9985,7 @@ lean_inc(x_48); lean_dec(x_1); x_49 = 1; x_50 = 5; -x_51 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__2; +x_51 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3___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); @@ -10172,7 +10070,7 @@ if (lean_is_exclusive(x_57)) { } 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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6(x_71, x_73, x_74, x_4, x_5); +x_75 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__6(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 { @@ -10209,7 +10107,7 @@ 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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__8(x_1, x_83, x_4, x_5); +x_84 = l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__8(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) @@ -10227,8 +10125,8 @@ 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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6___closed__1; -x_93 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__7(x_3, x_90, x_91, lean_box(0), x_83, x_92); +x_92 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__6___closed__1; +x_93 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__7(x_3, x_90, x_91, lean_box(0), x_83, x_92); lean_dec(x_91); lean_dec(x_90); return x_93; @@ -10255,7 +10153,7 @@ 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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__8(x_96, x_97, x_4, x_5); +x_98 = l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__8(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) @@ -10273,8 +10171,8 @@ 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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6___closed__1; -x_107 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__7(x_3, x_104, x_105, lean_box(0), x_97, x_106); +x_106 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__6___closed__1; +x_107 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__7(x_3, x_104, x_105, lean_box(0), x_97, x_106); lean_dec(x_105); lean_dec(x_104); return x_107; @@ -10292,18 +10190,18 @@ return x_98; } } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__5(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_DiscrTree_Key_hash(x_2); x_5 = lean_uint64_to_usize(x_4); x_6 = 1; -x_7 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6(x_1, x_5, x_6, x_2, x_3); +x_7 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__6(x_1, x_5, x_6, x_2, x_3); return x_7; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal_loop___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal_loop___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; @@ -10321,7 +10219,7 @@ else { lean_object* x_7; uint8_t x_8; x_7 = lean_array_fget(x_1, x_3); -x_8 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3269_(x_2, x_7); +x_8 = l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_beqExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3199_(x_2, x_7); lean_dec(x_7); if (x_8 == 0) { @@ -10342,7 +10240,7 @@ return x_12; } } } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____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_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____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_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; uint8_t x_15; @@ -10395,7 +10293,7 @@ x_24 = lean_ctor_get(x_19, 0); lean_dec(x_24); x_25 = lean_unsigned_to_nat(1u); x_26 = lean_nat_add(x_3, x_25); -x_27 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(x_1, x_2, x_26, x_23); +x_27 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9(x_1, x_2, x_26, x_23); lean_dec(x_26); lean_ctor_set(x_19, 1, x_27); lean_ctor_set(x_19, 0, x_4); @@ -10411,7 +10309,7 @@ lean_inc(x_29); lean_dec(x_19); x_30 = lean_unsigned_to_nat(1u); x_31 = lean_nat_add(x_3, x_30); -x_32 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(x_1, x_2, x_31, x_29); +x_32 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9(x_1, x_2, x_31, x_29); lean_dec(x_31); x_33 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_33, 0, x_4); @@ -10462,7 +10360,7 @@ return x_43; } } } -LEAN_EXPORT lean_object* l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____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_EXPORT lean_object* l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____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) { _start: { uint8_t x_7; @@ -10513,7 +10411,7 @@ x_21 = lean_ctor_get(x_16, 0); lean_dec(x_21); x_22 = lean_unsigned_to_nat(1u); x_23 = lean_nat_add(x_3, x_22); -x_24 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(x_1, x_2, x_23, x_20); +x_24 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9(x_1, x_2, x_23, x_20); lean_dec(x_23); lean_ctor_set(x_16, 1, x_24); lean_ctor_set(x_16, 0, x_4); @@ -10528,7 +10426,7 @@ lean_inc(x_26); lean_dec(x_16); x_27 = lean_unsigned_to_nat(1u); x_28 = lean_nat_add(x_3, x_27); -x_29 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(x_1, x_2, x_28, x_26); +x_29 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9(x_1, x_2, x_28, x_26); lean_dec(x_28); x_30 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_30, 0, x_4); @@ -10583,7 +10481,7 @@ x_44 = lean_ctor_get(x_40, 1); x_45 = lean_ctor_get(x_40, 0); lean_dec(x_45); x_46 = lean_nat_add(x_3, x_37); -x_47 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(x_1, x_2, x_46, x_44); +x_47 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9(x_1, x_2, x_46, x_44); lean_dec(x_46); lean_ctor_set(x_40, 1, x_47); lean_ctor_set(x_40, 0, x_4); @@ -10598,7 +10496,7 @@ x_49 = lean_ctor_get(x_40, 1); lean_inc(x_49); lean_dec(x_40); x_50 = lean_nat_add(x_3, x_37); -x_51 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(x_1, x_2, x_50, x_49); +x_51 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9(x_1, x_2, x_50, x_49); lean_dec(x_50); x_52 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_52, 0, x_4); @@ -10616,7 +10514,7 @@ x_54 = lean_array_get_size(x_5); x_55 = lean_unsigned_to_nat(1u); x_56 = lean_nat_sub(x_54, x_55); lean_dec(x_54); -x_57 = l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__12(x_1, x_2, x_3, x_4, x_5, x_6, x_8, x_56); +x_57 = l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__12(x_1, x_2, x_3, x_4, x_5, x_6, x_8, x_56); return x_57; } } @@ -10671,7 +10569,7 @@ return x_72; } } } -static lean_object* _init_l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9___closed__1() { +static lean_object* _init_l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -10682,7 +10580,7 @@ lean_ctor_set(x_2, 1, x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -10699,7 +10597,7 @@ if (x_9 == 0) { lean_object* x_10; lean_object* x_11; x_10 = lean_unsigned_to_nat(0u); -x_11 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal_loop___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__10(x_6, x_2, x_10); +x_11 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal_loop___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__10(x_6, x_2, x_10); lean_ctor_set(x_4, 0, x_11); return x_4; } @@ -10707,12 +10605,12 @@ else { lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; x_12 = lean_array_fget(x_1, x_3); -x_13 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9___closed__1; +x_13 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9___closed__1; lean_inc(x_12); 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_15 = l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__11(x_1, x_2, x_3, x_12, x_7, x_14); +x_15 = l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__11(x_1, x_2, x_3, x_12, x_7, x_14); lean_ctor_set(x_4, 1, x_15); return x_4; } @@ -10732,7 +10630,7 @@ if (x_19 == 0) { lean_object* x_20; lean_object* x_21; lean_object* x_22; x_20 = lean_unsigned_to_nat(0u); -x_21 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal_loop___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__10(x_16, x_2, x_20); +x_21 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal_loop___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__10(x_16, x_2, 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_17); @@ -10742,12 +10640,12 @@ else { lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; x_23 = lean_array_fget(x_1, x_3); -x_24 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9___closed__1; +x_24 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9___closed__1; lean_inc(x_23); 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 = l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__11(x_1, x_2, x_3, x_23, x_17, x_25); +x_26 = l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__11(x_1, x_2, x_3, x_23, x_17, x_25); x_27 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_27, 0, x_16); lean_ctor_set(x_27, 1, x_26); @@ -10756,7 +10654,7 @@ return x_27; } } } -static lean_object* _init_l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__13___closed__1() { +static lean_object* _init_l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__13___closed__1() { _start: { lean_object* x_1; @@ -10764,16 +10662,16 @@ x_1 = l_Lean_Meta_DiscrTree_instInhabited(lean_box(0)); return x_1; } } -LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__13(lean_object* x_1) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__13(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__13___closed__1; +x_2 = l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__13___closed__1; x_3 = lean_panic_fn(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__1() { +static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__1() { _start: { lean_object* x_1; @@ -10781,7 +10679,7 @@ x_1 = lean_mk_string_unchecked("Lean.Meta.DiscrTree", 19, 19); return x_1; } } -static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__2() { +static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__2() { _start: { lean_object* x_1; @@ -10789,7 +10687,7 @@ x_1 = lean_mk_string_unchecked("Lean.Meta.DiscrTree.insertCore", 30, 30); return x_1; } } -static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__3() { +static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__3() { _start: { lean_object* x_1; @@ -10797,20 +10695,20 @@ x_1 = lean_mk_string_unchecked("invalid key sequence", 20, 20); return x_1; } } -static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__4() { +static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__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; -x_1 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__1; -x_2 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__2; +x_1 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__1; +x_2 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__2; x_3 = lean_unsigned_to_nat(484u); x_4 = lean_unsigned_to_nat(23u); -x_5 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__3; +x_5 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___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_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -10828,13 +10726,13 @@ lean_object* x_8; lean_object* x_9; lean_object* x_10; x_8 = l_Lean_Meta_DiscrTree_instInhabitedKey; x_9 = l_outOfBounds___rarg(x_8); lean_inc(x_1); -x_10 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__2(x_1, x_9); +x_10 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__2(x_1, x_9); if (lean_obj_tag(x_10) == 0) { lean_object* x_11; lean_object* x_12; lean_object* x_13; x_11 = lean_unsigned_to_nat(1u); x_12 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(x_2, x_3, x_11); -x_13 = l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__5(x_1, x_9, x_12); +x_13 = l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__5(x_1, x_9, x_12); return x_13; } else @@ -10844,8 +10742,8 @@ x_14 = lean_ctor_get(x_10, 0); lean_inc(x_14); lean_dec(x_10); x_15 = lean_unsigned_to_nat(1u); -x_16 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(x_2, x_3, x_15, x_14); -x_17 = l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__5(x_1, x_9, x_16); +x_16 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9(x_2, x_3, x_15, x_14); +x_17 = l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__5(x_1, x_9, x_16); return x_17; } } @@ -10854,13 +10752,13 @@ else lean_object* x_18; lean_object* x_19; x_18 = lean_array_fget(x_2, x_6); lean_inc(x_1); -x_19 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__2(x_1, x_18); +x_19 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__2(x_1, x_18); if (lean_obj_tag(x_19) == 0) { lean_object* x_20; lean_object* x_21; lean_object* x_22; x_20 = lean_unsigned_to_nat(1u); x_21 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(x_2, x_3, x_20); -x_22 = l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__5(x_1, x_18, x_21); +x_22 = l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__5(x_1, x_18, x_21); return x_22; } else @@ -10870,8 +10768,8 @@ x_23 = lean_ctor_get(x_19, 0); lean_inc(x_23); lean_dec(x_19); x_24 = lean_unsigned_to_nat(1u); -x_25 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(x_2, x_3, x_24, x_23); -x_26 = l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__5(x_1, x_18, x_25); +x_25 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9(x_2, x_3, x_24, x_23); +x_26 = l_Lean_PersistentHashMap_insert___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__5(x_1, x_18, x_25); return x_26; } } @@ -10881,13 +10779,13 @@ else lean_object* x_27; lean_object* x_28; lean_dec(x_3); lean_dec(x_1); -x_27 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__4; -x_28 = l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__13(x_27); +x_27 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__4; +x_28 = l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__13(x_27); return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____lambda__1(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; @@ -10900,7 +10798,7 @@ x_5 = lean_ctor_get(x_1, 1); x_6 = lean_ctor_get(x_2, 2); lean_inc(x_6); lean_inc(x_2); -x_7 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1(x_4, x_6, x_2); +x_7 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1(x_4, x_6, x_2); lean_dec(x_6); x_8 = lean_ctor_get(x_2, 0); lean_inc(x_8); @@ -10922,7 +10820,7 @@ lean_dec(x_1); x_12 = lean_ctor_get(x_2, 2); lean_inc(x_12); lean_inc(x_2); -x_13 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1(x_10, x_12, x_2); +x_13 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1(x_10, x_12, x_2); lean_dec(x_12); x_14 = lean_ctor_get(x_2, 0); lean_inc(x_14); @@ -10936,7 +10834,7 @@ return x_16; } } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__1() { _start: { lean_object* x_1; @@ -10944,7 +10842,7 @@ x_1 = lean_mk_string_unchecked("Elab", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__2() { _start: { lean_object* x_1; @@ -10952,7 +10850,7 @@ x_1 = lean_mk_string_unchecked("Ext", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__3() { _start: { lean_object* x_1; @@ -10960,28 +10858,28 @@ x_1 = lean_mk_string_unchecked("extExtension", 12, 12); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____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_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__1; x_3 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__10; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2; -x_5 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__3; +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__2; +x_5 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__3; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____lambda__1), 2, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____lambda__1), 2, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__6() { _start: { lean_object* x_1; @@ -10989,14 +10887,14 @@ x_1 = lean_alloc_closure((void*)(l_id___rarg___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__4; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__5; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__4; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__5; x_3 = l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorems___closed__1; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__6; +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__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); @@ -11005,59 +10903,59 @@ lean_ctor_set(x_5, 3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__7; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__7; x_3 = l_Lean_registerSimpleScopedEnvExtension___rarg(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__4___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_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____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_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__4(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_PersistentHashMap_findAtAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__4(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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3___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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3(x_1, x_4, x_3); +x_5 = l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3(x_1, x_4, x_3); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__2___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__2___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__2(x_1, x_2); +x_3 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__2(x_1, x_2); lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____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_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____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_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__7(x_7, x_2, x_3, x_4, x_5, x_6); +x_8 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____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_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6___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_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____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; @@ -11065,45 +10963,45 @@ 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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6(x_1, x_6, x_7, x_4, x_5); +x_8 = l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__6(x_1, x_6, x_7, x_4, x_5); return x_8; } } -LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____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___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____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) { _start: { lean_object* x_9; -x_9 = l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__12(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__12(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_3); lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____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_EXPORT lean_object* l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____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) { _start: { lean_object* x_7; -x_7 = l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__11(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Array_binInsertM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__11(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_3); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9___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_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9(x_1, x_2, x_3, x_4); +x_5 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_1); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1(x_1, x_2, x_3); +x_4 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1(x_1, x_2, x_3); lean_dec(x_2); return x_4; } @@ -11980,7 +11878,7 @@ x_7 = lean_box(x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__3(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; uint8_t x_11; @@ -12068,7 +11966,7 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__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_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; @@ -12087,7 +11985,7 @@ lean_object* x_11; lean_object* x_12; x_11 = lean_ctor_get(x_3, 6); lean_dec(x_11); lean_ctor_set(x_3, 6, x_9); -x_12 = l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__3(x_2, x_3, x_4, x_8); +x_12 = l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__3(x_2, x_3, x_4, x_8); return x_12; } else @@ -12125,12 +12023,12 @@ lean_ctor_set(x_23, 7, x_19); lean_ctor_set(x_23, 8, x_20); lean_ctor_set(x_23, 9, x_21); lean_ctor_set_uint8(x_23, sizeof(void*)*10, x_22); -x_24 = l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__3(x_2, x_23, x_4, x_8); +x_24 = l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__3(x_2, x_23, x_4, x_8); return x_24; } } } -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__1() { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__1() { _start: { lean_object* x_1; @@ -12138,7 +12036,7 @@ x_1 = lean_mk_string_unchecked("runtime", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__2() { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__2() { _start: { lean_object* x_1; @@ -12146,17 +12044,17 @@ x_1 = lean_mk_string_unchecked("maxRecDepth", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__3() { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__1; -x_2 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__2; +x_1 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__1; +x_2 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__2; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__4() { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__4() { _start: { lean_object* x_1; lean_object* x_2; @@ -12166,32 +12064,32 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__5() { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__4; +x_1 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__4; x_2 = l_Lean_MessageData_ofFormat(x_1); return x_2; } } -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__6() { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__3; -x_2 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__5; +x_1 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__3; +x_2 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__5; x_3 = lean_alloc_ctor(8, 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_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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; -x_5 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__6; +x_5 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__6; x_6 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_6, 0, x_1); lean_ctor_set(x_6, 1, x_5); @@ -12201,7 +12099,7 @@ lean_ctor_set(x_7, 1, x_4); return x_7; } } -static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__1() { +static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___rarg___closed__1() { _start: { lean_object* x_1; @@ -12209,38 +12107,38 @@ x_1 = l_Lean_Elab_unsupportedSyntaxExceptionId; return x_1; } } -static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__2() { +static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___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_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__1; +x_2 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___rarg___closed__1; 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_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___rarg(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__2; +x_2 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___rarg___closed__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; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg), 1, 0); +x_3 = lean_alloc_closure((void*)(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___rarg), 1, 0); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__1(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; @@ -12409,7 +12307,7 @@ return x_41; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___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_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { uint8_t x_5; lean_object* x_6; lean_object* x_7; @@ -12421,7 +12319,7 @@ lean_ctor_set(x_7, 1, x_4); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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) { _start: { lean_object* x_7; lean_object* x_8; @@ -12432,7 +12330,7 @@ lean_ctor_set(x_8, 1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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) { _start: { lean_object* x_7; lean_object* x_8; @@ -12443,7 +12341,7 @@ lean_ctor_set(x_8, 1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1(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_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; uint8_t x_35; @@ -12475,23 +12373,23 @@ x_16 = lean_ctor_get(x_14, 3); lean_inc(x_16); lean_dec(x_14); lean_inc(x_8); -x_17 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__1___boxed), 4, 1); +x_17 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__1___boxed), 4, 1); lean_closure_set(x_17, 0, x_8); lean_inc(x_12); x_18 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed), 3, 1); lean_closure_set(x_18, 0, x_12); lean_inc(x_8); -x_19 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__2___boxed), 4, 1); +x_19 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__2___boxed), 4, 1); lean_closure_set(x_19, 0, x_8); lean_inc(x_16); lean_inc(x_12); lean_inc(x_8); -x_20 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__3___boxed), 6, 3); +x_20 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__3___boxed), 6, 3); lean_closure_set(x_20, 0, x_8); lean_closure_set(x_20, 1, x_12); lean_closure_set(x_20, 2, x_16); lean_inc(x_8); -x_21 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__4___boxed), 6, 3); +x_21 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__4___boxed), 6, 3); lean_closure_set(x_21, 0, x_8); lean_closure_set(x_21, 1, x_12); lean_closure_set(x_21, 2, x_16); @@ -12679,7 +12577,7 @@ lean_object* x_81; lean_object* x_82; lean_object* x_83; x_81 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_81, 0, x_78); x_82 = l_Lean_MessageData_ofFormat(x_81); -x_83 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__2(x_77, x_82, x_2, x_3, x_37); +x_83 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__2(x_77, x_82, x_2, x_3, x_37); lean_dec(x_77); return x_83; } @@ -12687,7 +12585,7 @@ else { lean_object* x_84; lean_dec(x_78); -x_84 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4(x_77, x_2, x_3, x_37); +x_84 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4(x_77, x_2, x_3, x_37); lean_dec(x_2); return x_84; } @@ -12696,7 +12594,7 @@ else { lean_object* x_85; lean_dec(x_2); -x_85 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg(x_37); +x_85 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___rarg(x_37); return x_85; } } @@ -12833,7 +12731,7 @@ lean_object* x_122; lean_object* x_123; lean_object* x_124; x_122 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_122, 0, x_119); x_123 = l_Lean_MessageData_ofFormat(x_122); -x_124 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__2(x_118, x_123, x_2, x_3, x_87); +x_124 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__2(x_118, x_123, x_2, x_3, x_87); lean_dec(x_118); return x_124; } @@ -12841,7 +12739,7 @@ else { lean_object* x_125; lean_dec(x_119); -x_125 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4(x_118, x_2, x_3, x_87); +x_125 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4(x_118, x_2, x_3, x_87); lean_dec(x_2); return x_125; } @@ -12850,14 +12748,14 @@ else { lean_object* x_126; lean_dec(x_2); -x_126 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg(x_87); +x_126 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___rarg(x_87); return x_126; } } } } } -LEAN_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__6(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_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__6(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_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -12878,7 +12776,7 @@ x_14 = lean_ctor_get(x_11, 0); x_15 = lean_ctor_get(x_11, 4); lean_dec(x_15); x_16 = l_Lean_ScopedEnvExtension_addCore___rarg(x_14, x_1, x_2, x_3, x_9); -x_17 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; +x_17 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; lean_ctor_set(x_11, 4, x_17); lean_ctor_set(x_11, 0, x_16); x_18 = lean_st_ref_set(x_7, x_11, x_12); @@ -12897,7 +12795,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_21, 1); lean_dec(x_24); -x_25 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +x_25 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; lean_ctor_set(x_21, 1, x_25); x_26 = lean_st_ref_set(x_5, x_21, x_22); x_27 = !lean_is_exclusive(x_26); @@ -12935,7 +12833,7 @@ lean_inc(x_35); lean_inc(x_34); lean_inc(x_33); lean_dec(x_21); -x_37 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +x_37 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; x_38 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_38, 0, x_33); lean_ctor_set(x_38, 1, x_37); @@ -12981,7 +12879,7 @@ lean_inc(x_45); lean_inc(x_44); lean_dec(x_11); x_50 = l_Lean_ScopedEnvExtension_addCore___rarg(x_44, x_1, x_2, x_3, x_9); -x_51 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; +x_51 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; x_52 = lean_alloc_ctor(0, 7, 0); lean_ctor_set(x_52, 0, x_50); lean_ctor_set(x_52, 1, x_45); @@ -13019,7 +12917,7 @@ if (lean_is_exclusive(x_56)) { lean_dec_ref(x_56); x_62 = lean_box(0); } -x_63 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +x_63 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; if (lean_is_scalar(x_62)) { x_64 = lean_alloc_ctor(0, 5, 0); } else { @@ -13053,7 +12951,7 @@ return x_69; } } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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) { _start: { uint8_t x_8; @@ -13122,7 +13020,7 @@ return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8___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_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__8___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_object* x_8; @@ -13133,7 +13031,7 @@ lean_ctor_set(x_8, 1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8(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_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__8(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; uint8_t x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; @@ -13193,7 +13091,7 @@ if (x_24 == 0) { lean_object* x_25; lean_object* x_26; x_25 = lean_box(0); -x_26 = l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8___lambda__1(x_1, x_2, x_25, x_3, x_4, x_5); +x_26 = l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__8___lambda__1(x_1, x_2, x_25, x_3, x_4, x_5); return x_26; } else @@ -13232,7 +13130,7 @@ return x_36; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; @@ -13244,7 +13142,7 @@ lean_ctor_set(x_5, 1, x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; lean_object* x_6; @@ -13256,7 +13154,7 @@ lean_ctor_set(x_6, 1, x_3); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___closed__1() { _start: { lean_object* x_1; @@ -13264,17 +13162,17 @@ x_1 = lean_mk_string_unchecked("prioDefault", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__1; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___closed__3() { _start: { lean_object* x_1; @@ -13282,16 +13180,16 @@ x_1 = lean_mk_string_unchecked("default", 7, 7); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3(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; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__3; +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___closed__3; lean_inc(x_1); x_5 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_5, 0, x_1); lean_ctor_set(x_5, 1, x_4); -x_6 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__2; +x_6 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___closed__2; x_7 = l_Lean_Syntax_node1(x_1, x_6, x_5); x_8 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_8, 0, x_7); @@ -13299,7 +13197,7 @@ lean_ctor_set(x_8, 1, x_3); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_1) == 0) @@ -13320,7 +13218,7 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__5(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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__5(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; @@ -13382,7 +13280,7 @@ return x_24; } } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__1() { _start: { lean_object* x_1; @@ -13390,67 +13288,67 @@ x_1 = lean_alloc_closure((void*)(l_ReaderT_read___at_Lean_Macro_instMonadRefMacr return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__1___boxed), 3, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__1; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__2; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__1; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__2; x_3 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Macro_instMonadRefMacroM___spec__2___rarg), 4, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__4() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__2___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__2___boxed), 3, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__3; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__4; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__3; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__4; x_3 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Macro_instMonadRefMacroM___spec__2___rarg), 4, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__6() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___boxed), 3, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__5; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__6; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__5; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__6; x_3 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Macro_instMonadRefMacroM___spec__2___rarg), 4, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, uint8_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_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, uint8_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) { _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; uint8_t x_19; @@ -13497,13 +13395,13 @@ lean_inc(x_27); x_28 = lean_ctor_get(x_26, 1); lean_inc(x_28); lean_dec(x_26); -x_29 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__4), 4, 1); +x_29 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__4), 4, 1); lean_closure_set(x_29, 0, x_2); -x_30 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__7; +x_30 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__7; x_31 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Macro_instMonadRefMacroM___spec__2___rarg), 4, 2); lean_closure_set(x_31, 0, x_30); lean_closure_set(x_31, 1, x_29); -x_32 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___boxed), 4, 1); +x_32 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___boxed), 4, 1); lean_closure_set(x_32, 0, x_31); x_33 = l_Lean_liftCommandElabM___rarg(x_32, x_10, x_11, x_28); if (lean_obj_tag(x_33) == 0) @@ -13521,7 +13419,7 @@ lean_ctor_set(x_36, 1, x_34); lean_ctor_set(x_36, 2, x_27); x_37 = l_Lean_Elab_Tactic_Ext_getExtTheorems___closed__1; lean_inc(x_10); -x_38 = l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__6(x_37, x_36, x_4, x_8, x_9, x_10, x_11, x_35); +x_38 = l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__6(x_37, x_36, x_4, x_8, x_9, x_10, x_11, x_35); lean_dec(x_9); lean_dec(x_8); if (x_5 == 0) @@ -13560,7 +13458,7 @@ lean_object* x_45; lean_object* x_46; lean_object* x_47; x_45 = lean_ctor_get(x_38, 1); lean_inc(x_45); lean_dec(x_38); -x_46 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__5___boxed), 5, 2); +x_46 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__5___boxed), 5, 2); lean_closure_set(x_46, 0, x_6); lean_closure_set(x_46, 1, x_3); x_47 = l_Lean_liftCommandElabM___rarg(x_46, x_10, x_11, x_45); @@ -13732,13 +13630,13 @@ lean_inc(x_86); x_87 = lean_ctor_get(x_85, 1); lean_inc(x_87); lean_dec(x_85); -x_88 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__4), 4, 1); +x_88 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__4), 4, 1); lean_closure_set(x_88, 0, x_2); -x_89 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__7; +x_89 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__7; x_90 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Macro_instMonadRefMacroM___spec__2___rarg), 4, 2); lean_closure_set(x_90, 0, x_89); lean_closure_set(x_90, 1, x_88); -x_91 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___boxed), 4, 1); +x_91 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___boxed), 4, 1); lean_closure_set(x_91, 0, x_90); x_92 = l_Lean_liftCommandElabM___rarg(x_91, x_10, x_11, x_87); if (lean_obj_tag(x_92) == 0) @@ -13756,7 +13654,7 @@ lean_ctor_set(x_95, 1, x_93); lean_ctor_set(x_95, 2, x_86); x_96 = l_Lean_Elab_Tactic_Ext_getExtTheorems___closed__1; lean_inc(x_10); -x_97 = l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__6(x_96, x_95, x_4, x_8, x_9, x_10, x_11, x_94); +x_97 = l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__6(x_96, x_95, x_4, x_8, x_9, x_10, x_11, x_94); lean_dec(x_9); lean_dec(x_8); if (x_5 == 0) @@ -13792,7 +13690,7 @@ lean_object* x_102; lean_object* x_103; lean_object* x_104; x_102 = lean_ctor_get(x_97, 1); lean_inc(x_102); lean_dec(x_97); -x_103 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__5___boxed), 5, 2); +x_103 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__5___boxed), 5, 2); lean_closure_set(x_103, 0, x_6); lean_closure_set(x_103, 1, x_3); x_104 = l_Lean_liftCommandElabM___rarg(x_103, x_10, x_11, x_102); @@ -13913,7 +13811,7 @@ return x_120; } } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__7___closed__1() { _start: { lean_object* x_1; @@ -13921,16 +13819,16 @@ x_1 = lean_mk_string_unchecked("@[ext] attribute only applies to structures and return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__7___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__1; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__7___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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; @@ -14006,7 +13904,7 @@ lean_dec(x_38); lean_inc(x_37); x_39 = l_Lean_MessageData_ofExpr(x_37); x_40 = l_Lean_indentD(x_39); -x_41 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__2; +x_41 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__7___closed__2; lean_ctor_set_tag(x_33, 7); lean_ctor_set(x_33, 1, x_40); lean_ctor_set(x_33, 0, x_41); @@ -14117,7 +14015,7 @@ else lean_object* x_64; lean_object* x_65; lean_dec(x_31); x_64 = lean_box(0); -x_65 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6(x_49, x_2, x_6, x_3, x_4, x_5, x_64, x_8, x_9, x_10, x_11, x_35); +x_65 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6(x_49, x_2, x_6, x_3, x_4, x_5, x_64, x_8, x_9, x_10, x_11, x_35); return x_65; } } @@ -14132,7 +14030,7 @@ lean_dec(x_33); lean_inc(x_66); x_67 = l_Lean_MessageData_ofExpr(x_66); x_68 = l_Lean_indentD(x_67); -x_69 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__2; +x_69 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__7___closed__2; x_70 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_70, 0, x_69); lean_ctor_set(x_70, 1, x_68); @@ -14247,7 +14145,7 @@ else lean_object* x_93; lean_object* x_94; lean_dec(x_31); x_93 = lean_box(0); -x_94 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6(x_78, x_2, x_6, x_3, x_4, x_5, x_93, x_8, x_9, x_10, x_11, x_35); +x_94 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6(x_78, x_2, x_6, x_3, x_4, x_5, x_93, x_8, x_9, x_10, x_11, x_35); return x_94; } } @@ -14276,7 +14174,7 @@ if (lean_is_exclusive(x_95)) { lean_inc(x_97); x_99 = l_Lean_MessageData_ofExpr(x_97); x_100 = l_Lean_indentD(x_99); -x_101 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__2; +x_101 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__7___closed__2; if (lean_is_scalar(x_98)) { x_102 = lean_alloc_ctor(7, 2, 0); } else { @@ -14396,7 +14294,7 @@ else lean_object* x_126; lean_object* x_127; lean_dec(x_104); x_126 = lean_box(0); -x_127 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6(x_111, x_2, x_6, x_3, x_4, x_5, x_126, x_8, x_9, x_10, x_11, x_96); +x_127 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6(x_111, x_2, x_6, x_3, x_4, x_5, x_126, x_8, x_9, x_10, x_11, x_96); return x_127; } } @@ -14512,7 +14410,7 @@ if (lean_is_exclusive(x_153)) { lean_inc(x_156); x_158 = l_Lean_MessageData_ofExpr(x_156); x_159 = l_Lean_indentD(x_158); -x_160 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__2; +x_160 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__7___closed__2; if (lean_is_scalar(x_157)) { x_161 = lean_alloc_ctor(7, 2, 0); } else { @@ -14637,7 +14535,7 @@ else lean_object* x_185; lean_object* x_186; lean_dec(x_163); x_185 = lean_box(0); -x_186 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6(x_170, x_2, x_6, x_3, x_4, x_5, x_185, x_8, x_9, x_10, x_11, x_155); +x_186 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6(x_170, x_2, x_6, x_3, x_4, x_5, x_185, x_8, x_9, x_10, x_11, x_155); return x_186; } } @@ -14707,7 +14605,7 @@ return x_194; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__8(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_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__8(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; lean_object* x_9; lean_object* x_10; uint8_t x_11; @@ -14769,7 +14667,7 @@ return x_25; } } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__9___closed__1() { _start: { lean_object* x_1; @@ -14777,16 +14675,16 @@ x_1 = lean_mk_string_unchecked("unexpected 'flat' configuration on @[ext] theore return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__9___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__1; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__9___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9(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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__9(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) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; @@ -14876,7 +14774,7 @@ if (lean_obj_tag(x_7) == 0) { lean_object* x_24; lean_object* x_25; x_24 = lean_box(0); -x_25 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7(x_2, x_17, x_3, x_18, x_1, x_4, x_24, x_8, x_9, x_10, x_11, x_21); +x_25 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__7(x_2, x_17, x_3, x_18, x_1, x_4, x_24, x_8, x_9, x_10, x_11, x_21); lean_dec(x_2); return x_25; } @@ -14888,8 +14786,8 @@ lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); x_26 = lean_ctor_get(x_7, 0); -x_27 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__2; -x_28 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__7(x_26, x_27, x_8, x_9, x_10, x_11, x_21); +x_27 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__9___closed__2; +x_28 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__7(x_26, x_27, x_8, x_9, x_10, x_11, x_21); lean_dec(x_11); lean_dec(x_9); lean_dec(x_8); @@ -14918,7 +14816,7 @@ else lean_object* x_33; lean_object* x_34; lean_object* x_35; x_33 = lean_box(x_19); lean_inc(x_1); -x_34 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__8___boxed), 6, 3); +x_34 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__8___boxed), 6, 3); lean_closure_set(x_34, 0, x_1); lean_closure_set(x_34, 1, x_4); lean_closure_set(x_34, 2, x_33); @@ -14932,7 +14830,7 @@ 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_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7(x_2, x_17, x_3, x_18, x_1, x_36, x_38, x_8, x_9, x_10, x_11, x_37); +x_39 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__7(x_2, x_17, x_3, x_18, x_1, x_36, x_38, x_8, x_9, x_10, x_11, x_37); lean_dec(x_2); return x_39; } @@ -14971,7 +14869,7 @@ return x_43; } } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__1() { _start: { lean_object* x_1; @@ -14979,16 +14877,16 @@ x_1 = lean_mk_string_unchecked("invalid syntax for 'ext' attribute", 34, 34); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__1; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__3() { _start: { lean_object* x_1; @@ -14996,7 +14894,7 @@ x_1 = lean_mk_string_unchecked("Attr", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__4() { _start: { lean_object* x_1; @@ -15004,19 +14902,19 @@ x_1 = lean_mk_string_unchecked("extFlat", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___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_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; x_2 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__2; -x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__3; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__4; +x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__3; +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__4; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10(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_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10(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) { _start: { lean_object* x_12; lean_object* x_13; uint8_t x_14; @@ -15036,7 +14934,7 @@ lean_dec(x_13); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_17 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2; +x_17 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__2; x_18 = l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(x_17, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); @@ -15050,7 +14948,7 @@ lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; x_19 = lean_unsigned_to_nat(0u); x_20 = l_Lean_Syntax_getArg(x_13, x_19); lean_dec(x_13); -x_21 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__5; +x_21 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__5; lean_inc(x_20); x_22 = l_Lean_Syntax_isOfKind(x_20, x_21); if (x_22 == 0) @@ -15060,7 +14958,7 @@ lean_dec(x_20); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_23 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2; +x_23 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__2; x_24 = l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(x_23, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); @@ -15077,7 +14975,7 @@ lean_dec(x_20); x_27 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_27, 0, x_26); x_28 = lean_box(0); -x_29 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9(x_1, x_2, x_3, x_4, x_6, x_28, x_27, x_7, x_8, x_9, x_10, x_11); +x_29 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__9(x_1, x_2, x_3, x_4, x_6, x_28, x_27, x_7, x_8, x_9, x_10, x_11); lean_dec(x_27); return x_29; } @@ -15089,25 +14987,25 @@ lean_object* x_30; lean_object* x_31; lean_dec(x_13); x_30 = lean_box(0); lean_inc(x_2); -x_31 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9(x_1, x_2, x_3, x_4, x_6, x_30, x_2, x_7, x_8, x_9, x_10, x_11); +x_31 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__9(x_1, x_2, x_3, x_4, x_6, x_30, x_2, x_7, x_8, x_9, x_10, x_11); lean_dec(x_2); return x_31; } } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___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_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; x_2 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__2; -x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__3; +x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__3; x_4 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__5___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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__2() { _start: { uint8_t x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; @@ -15132,12 +15030,12 @@ lean_ctor_set_uint8(x_5, 12, x_2); return x_5; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__3() { _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; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__2; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__2; x_3 = l_Lean_Elab_Tactic_Ext_mkExtType___closed__6; x_4 = l_Lean_Elab_Tactic_Ext_withExtHyps___rarg___lambda__2___closed__1; x_5 = lean_unsigned_to_nat(0u); @@ -15154,7 +15052,7 @@ lean_ctor_set_uint8(x_7, sizeof(void*)*6 + 1, x_6); return x_7; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -15173,7 +15071,7 @@ lean_ctor_set(x_3, 8, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -15186,15 +15084,15 @@ lean_ctor_set(x_2, 3, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___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; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__4; -x_3 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__4; +x_3 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5; x_4 = l_Lean_Elab_Tactic_Ext_mkExtType___closed__5; -x_5 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__5; +x_5 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__5; x_6 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_6, 0, x_2); lean_ctor_set(x_6, 1, x_3); @@ -15204,7 +15102,7 @@ lean_ctor_set(x_6, 4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__7() { _start: { lean_object* x_1; @@ -15212,27 +15110,27 @@ x_1 = lean_mk_string_unchecked("extIff", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__8() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___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_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; x_2 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__2; -x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__3; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__7; +x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__3; +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__7; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11(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_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11(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; uint8_t 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_7 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__1; +x_7 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__1; lean_inc(x_2); x_8 = l_Lean_Syntax_isOfKind(x_2, x_7); x_9 = lean_box(0); -x_10 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__6; +x_10 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__6; x_11 = lean_st_mk_ref(x_10, x_6); if (x_8 == 0) { @@ -15269,8 +15167,8 @@ if (x_12 == 0) lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_dec(x_2); lean_dec(x_1); -x_15 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2; -x_16 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3; +x_15 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__2; +x_16 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__3; x_17 = l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(x_15, x_16, x_13, x_4, x_5, x_14); lean_dec(x_5); lean_dec(x_4); @@ -15311,8 +15209,8 @@ lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; lean_dec(x_23); lean_dec(x_2); lean_dec(x_1); -x_26 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2; -x_27 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3; +x_26 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__2; +x_27 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__3; x_28 = l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(x_26, x_27, x_13, x_4, x_5, x_14); lean_dec(x_5); lean_dec(x_4); @@ -15342,7 +15240,7 @@ lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; x_33 = lean_unsigned_to_nat(0u); x_34 = l_Lean_Syntax_getArg(x_23, x_33); lean_dec(x_23); -x_35 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__8; +x_35 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__8; lean_inc(x_34); x_36 = l_Lean_Syntax_isOfKind(x_34, x_35); if (x_36 == 0) @@ -15351,8 +15249,8 @@ lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; lean_dec(x_34); lean_dec(x_2); lean_dec(x_1); -x_37 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2; -x_38 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3; +x_37 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__2; +x_38 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__3; x_39 = l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(x_37, x_38, x_13, x_4, x_5, x_14); lean_dec(x_5); lean_dec(x_4); @@ -15385,9 +15283,9 @@ lean_dec(x_34); x_46 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_46, 0, x_45); x_47 = lean_box(0); -x_48 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3; +x_48 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__3; lean_inc(x_13); -x_49 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10(x_2, x_9, x_3, x_1, x_47, x_46, x_48, x_13, x_4, x_5, x_14); +x_49 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10(x_2, x_9, x_3, x_1, x_47, x_46, x_48, x_13, x_4, x_5, x_14); lean_dec(x_46); if (lean_obj_tag(x_49) == 0) { @@ -15451,9 +15349,9 @@ else lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_dec(x_23); x_61 = lean_box(0); -x_62 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3; +x_62 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__3; lean_inc(x_13); -x_63 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10(x_2, x_9, x_3, x_1, x_61, x_9, x_62, x_13, x_4, x_5, x_14); +x_63 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10(x_2, x_9, x_3, x_1, x_61, x_9, x_62, x_13, x_4, x_5, x_14); if (lean_obj_tag(x_63) == 0) { lean_object* x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; @@ -15513,14 +15411,14 @@ return x_74; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__12(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__12(lean_object* x_1, lean_object* x_2) { _start: { lean_inc(x_1); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__13(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; @@ -15537,7 +15435,7 @@ x_9 = l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorems; x_10 = l_Lean_Elab_Tactic_Ext_getExtTheorems___closed__1; x_11 = l_Lean_ScopedEnvExtension_getState___rarg(x_9, x_10, x_8); lean_dec(x_8); -x_12 = l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8(x_11, x_1, x_2, x_3, x_7); +x_12 = l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__8(x_11, x_1, x_2, x_3, x_7); 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; uint8_t x_18; @@ -15559,10 +15457,10 @@ lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean x_19 = lean_ctor_get(x_16, 0); x_20 = lean_ctor_get(x_16, 4); lean_dec(x_20); -x_21 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__12___boxed), 2, 1); +x_21 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__12___boxed), 2, 1); lean_closure_set(x_21, 0, x_13); x_22 = l_Lean_ScopedEnvExtension_modifyState___rarg(x_10, x_19, x_21); -x_23 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; +x_23 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; lean_ctor_set(x_16, 4, x_23); lean_ctor_set(x_16, 0, x_22); x_24 = lean_st_ref_set(x_3, x_16, x_17); @@ -15605,10 +15503,10 @@ lean_inc(x_33); lean_inc(x_32); lean_inc(x_31); lean_dec(x_16); -x_37 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__12___boxed), 2, 1); +x_37 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__12___boxed), 2, 1); lean_closure_set(x_37, 0, x_13); x_38 = l_Lean_ScopedEnvExtension_modifyState___rarg(x_10, x_31, x_37); -x_39 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2; +x_39 = l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2; x_40 = lean_alloc_ctor(0, 7, 0); lean_ctor_set(x_40, 0, x_38); lean_ctor_set(x_40, 1, x_32); @@ -15663,7 +15561,7 @@ return x_49; } } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -15673,37 +15571,37 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__1; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__1; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__2; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__2; x_2 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__10; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__3; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__3; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__5() { _start: { lean_object* x_1; @@ -15711,17 +15609,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__4; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__5; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__4; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__7() { _start: { lean_object* x_1; @@ -15729,57 +15627,57 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__8() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__6; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__7; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__6; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__9() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__8; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__8; x_2 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__10() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__9; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__9; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__11() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__10; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__10; x_2 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__10; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__12() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__11; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__11; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__13() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__13() { _start: { lean_object* x_1; @@ -15787,27 +15685,27 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__14() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__12; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__13; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__12; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__13; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__15() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__14; -x_2 = lean_unsigned_to_nat(3766u); +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__14; +x_2 = lean_unsigned_to_nat(3696u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__16() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -15817,7 +15715,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__17() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__17() { _start: { lean_object* x_1; @@ -15825,13 +15723,13 @@ x_1 = lean_mk_string_unchecked("Marks a theorem as an extensionality theorem", 4 return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__18() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__15; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__16; -x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__17; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__15; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__16; +x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__17; x_4 = 0; x_5 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_5, 0, x_1); @@ -15841,29 +15739,29 @@ lean_ctor_set_uint8(x_5, sizeof(void*)*3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__19() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__19() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___boxed), 6, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___boxed), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__20() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__20() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__13___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__13___boxed), 4, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__21() { +static lean_object* _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__21() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__18; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__19; -x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__20; +x_1 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__18; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__19; +x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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); @@ -15871,120 +15769,120 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__21; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__21; x_3 = l_Lean_registerBuiltinAttribute(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__3___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_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__3(x_1, x_2, x_3, x_4); +x_5 = l_Lean_throwError___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__3(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__2___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_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__2(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__2(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_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___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_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4(x_1, x_2, x_3, x_4); +x_5 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4(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_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5(x_1, x_2); +x_3 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5(x_1, x_2); lean_dec(x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__1___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_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_1); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___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_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___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_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__2(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__2(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_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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) { _start: { lean_object* x_7; -x_7 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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) { _start: { lean_object* x_7; -x_7 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1___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_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__1(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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: { uint8_t x_9; lean_object* x_10; x_9 = lean_unbox(x_3); lean_dec(x_3); -x_10 = l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__6(x_1, x_2, x_9, x_4, x_5, x_6, x_7, x_8); +x_10 = l_Lean_ScopedEnvExtension_add___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__6(x_1, x_2, x_9, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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) { _start: { lean_object* x_8; -x_8 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_4); lean_dec(x_3); @@ -15992,67 +15890,67 @@ lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8___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_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__8___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_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__8___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; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8___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_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__8___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_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__8(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__8(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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__1(x_1, x_2, x_3); lean_dec(x_2); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__2(x_1, x_2, x_3); +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__2(x_1, x_2, x_3); lean_dec(x_2); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3(x_1, x_2, x_3); +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3(x_1, x_2, x_3); lean_dec(x_2); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__5___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_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__5___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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__5(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__5(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_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -16060,12 +15958,12 @@ x_13 = lean_unbox(x_4); lean_dec(x_4); x_14 = lean_unbox(x_5); lean_dec(x_5); -x_15 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6(x_1, x_2, x_3, x_13, x_14, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6(x_1, x_2, x_3, x_13, x_14, x_6, 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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -16073,74 +15971,74 @@ x_13 = lean_unbox(x_3); lean_dec(x_3); x_14 = lean_unbox(x_4); lean_dec(x_4); -x_15 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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); +x_15 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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_1); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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) { _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_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__8(x_1, x_2, x_7, x_4, x_5, x_6); +x_8 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__8(x_1, x_2, x_7, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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) { _start: { uint8_t x_13; lean_object* x_14; x_13 = lean_unbox(x_3); lean_dec(x_3); -x_14 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9(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_14 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__9(x_1, x_2, x_13, x_4, 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_14; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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) { _start: { uint8_t x_12; lean_object* x_13; x_12 = lean_unbox(x_3); lean_dec(x_3); -x_13 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10(x_1, x_2, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_13 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10(x_1, x_2, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_6); lean_dec(x_5); return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____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_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____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) { _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_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11(x_1, x_2, x_7, x_4, x_5, x_6); +x_8 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11(x_1, x_2, x_7, x_4, x_5, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__12___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__12___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__12(x_1, x_2); +x_3 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__12(x_1, x_2); lean_dec(x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__13___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_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__13___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_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__13(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__13(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); return x_5; @@ -17662,9 +17560,9 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheore { 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_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__1; x_3 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__10; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2; +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__2; x_5 = l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem__1___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -17683,9 +17581,9 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheore { 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_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__1; x_3 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__10; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2; +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__2; x_5 = l___regBuiltin_Lean_Elab_Tactic_Ext_evalApplyExtTheorem__1___closed__3; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -20462,9 +20360,9 @@ static lean_object* _init_l_Lean_Elab_Tactic_Ext_evalExt___closed__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; x_1 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__1; x_3 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__10; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2; +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__2; x_5 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__5___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -20635,9 +20533,9 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt__1___close { 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_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1; -x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1; +x_2 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__1; x_3 = l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__10; -x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2; +x_4 = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__2; x_5 = l___regBuiltin_Lean_Elab_Tactic_Ext_evalExt__1___closed__1; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -20886,16 +20784,16 @@ l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1_ lean_mark_persistent(l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___closed__3); l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___closed__4 = _init_l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___closed__4(); lean_mark_persistent(l_Lean_getConstInfoInduct___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__1___closed__4); -l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__1 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__1(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__1); -l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__2); -l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__3 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__3(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__3); -l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__4 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__4(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__4); -l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5(); -lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__4___closed__5); +l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__1 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__1(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__1); +l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__2); +l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__3 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__3(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__3); +l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__4 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__4(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__4); +l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5 = _init_l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5(); +lean_mark_persistent(l_Lean_addDeclarationRanges___at_Lean_Elab_Tactic_Ext_realizeExtTheorem___spec__5___closed__5); l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__1); l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__2 = _init_l_Lean_Elab_Tactic_Ext_realizeExtTheorem___lambda__2___closed__2(); @@ -21130,66 +21028,66 @@ l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorem___closed__1 = _init_l_Lean_Elab_T lean_mark_persistent(l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorem___closed__1); l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorem = _init_l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorem(); lean_mark_persistent(l_Lean_Elab_Tactic_Ext_instInhabitedExtTheorem); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__1 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__1(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__1); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__2 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__2(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__2); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__3 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__3(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__3); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__4 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__4(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__4); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__5 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__5(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__5); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__6 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__6(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__6); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__7 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__7(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__7); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__8 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__8(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__8); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__9 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__9(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__9); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__10 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__10(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__10); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__11 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__11(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__11); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__12 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__12(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__12); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__13 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__13(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__13); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__14 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__14(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__14); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__15 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__15(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__15); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__16 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__16(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__16); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__17 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__17(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__17); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__18 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__18(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__18); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__19 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__19(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__19); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__20 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__20(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__20); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__21 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__21(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__21); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__22 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__22(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__22); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__23 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__23(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__23); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__24 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__24(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__24); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__25 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__25(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__25); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__26 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__26(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__26); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__27 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__27(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__27); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__28 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__28(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__28); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__29 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__29(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__29); -l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__30 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__30(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3191____closed__30); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__1 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__1(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__1); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__2 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__2(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__2); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__3 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__3(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__3); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__4 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__4(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__4); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__5 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__5(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__5); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__6 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__6(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__6); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__7 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__7(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__7); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__8 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__8(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__8); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__9 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__9(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__9); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__10 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__10(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__10); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__11 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__11(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__11); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__12 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__12(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__12); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__13 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__13(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__13); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__14 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__14(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__14); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__15 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__15(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__15); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__16 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__16(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__16); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__17 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__17(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__17); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__18 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__18(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__18); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__19 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__19(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__19); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__20 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__20(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__20); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__21 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__21(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__21); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__22 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__22(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__22); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__23 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__23(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__23); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__24 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__24(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__24); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__25 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__25(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__25); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__26 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__26(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__26); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__27 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__27(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__27); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__28 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__28(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__28); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__29 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__29(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__29); +l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__30 = _init_l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__30(); +lean_mark_persistent(l___private_Lean_Elab_Tactic_Ext_0__Lean_Elab_Tactic_Ext_reprExtTheorem____x40_Lean_Elab_Tactic_Ext___hyg_3121____closed__30); l_Lean_Elab_Tactic_Ext_instReprExtTheorem___closed__1 = _init_l_Lean_Elab_Tactic_Ext_instReprExtTheorem___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_Ext_instReprExtTheorem___closed__1); l_Lean_Elab_Tactic_Ext_instReprExtTheorem = _init_l_Lean_Elab_Tactic_Ext_instReprExtTheorem(); @@ -21210,37 +21108,37 @@ l_Lean_Elab_Tactic_Ext_extExt_config___closed__1 = _init_l_Lean_Elab_Tactic_Ext_ lean_mark_persistent(l_Lean_Elab_Tactic_Ext_extExt_config___closed__1); l_Lean_Elab_Tactic_Ext_extExt_config = _init_l_Lean_Elab_Tactic_Ext_extExt_config(); lean_mark_persistent(l_Lean_Elab_Tactic_Ext_extExt_config); -l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__1 = _init_l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__1(); -l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__2 = _init_l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__3___closed__2(); -l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6___closed__1 = _init_l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6___closed__1(); -lean_mark_persistent(l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__6___closed__1); -l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9___closed__1 = _init_l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9___closed__1(); -lean_mark_persistent(l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__9___closed__1); -l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__13___closed__1 = _init_l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__13___closed__1(); -lean_mark_persistent(l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__13___closed__1); -l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__1 = _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__1(); -lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__1); -l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__2 = _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__2(); -lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__2); -l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__3 = _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__3(); -lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__3); -l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__4 = _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__4(); -lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____spec__1___closed__4); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__1); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__2); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__3); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__4); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__5); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__6 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__6); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__7 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471____closed__7); -if (builtin) {res = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3471_(lean_io_mk_world()); +l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3___closed__1 = _init_l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3___closed__1(); +l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3___closed__2 = _init_l_Lean_PersistentHashMap_findAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__3___closed__2(); +l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__6___closed__1 = _init_l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__6___closed__1(); +lean_mark_persistent(l_Lean_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__6___closed__1); +l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9___closed__1 = _init_l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__9___closed__1); +l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__13___closed__1 = _init_l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__13___closed__1(); +lean_mark_persistent(l_panic___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__13___closed__1); +l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__1 = _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__1(); +lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__1); +l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__2 = _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__2(); +lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__2); +l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__3 = _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__3(); +lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__3); +l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__4 = _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__4(); +lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____spec__1___closed__4); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__1); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__2); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__3); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__4); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__5); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__6 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__6); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__7 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401____closed__7); +if (builtin) {res = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3401_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Elab_Tactic_Ext_extExtension = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_Tactic_Ext_extExtension); @@ -21253,119 +21151,119 @@ l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___closed__1 = _init_l_Lean_Elab_ lean_mark_persistent(l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___closed__1); l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___closed__2 = _init_l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___closed__2(); lean_mark_persistent(l_Lean_Elab_Tactic_Ext_ExtTheorems_erase___rarg___closed__2); -l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__1 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__1(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__1); -l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__2 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__2(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__2); -l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__3 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__3(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__3); -l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__4 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__4(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__4); -l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__5 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__5(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__5); -l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__6 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__6(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__4___closed__6); -l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__1 = _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__1(); -lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__1); -l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__2 = _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__2(); -lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____spec__5___rarg___closed__2); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__1); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__2); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__3___closed__3); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__1); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__2); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__3); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__4); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__5); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__6 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__6); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__7 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__6___closed__7); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__1); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__7___closed__2); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__1); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__9___closed__2); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__1); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__2); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__3); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__4); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__10___closed__5); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__1); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__2); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__3); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__4); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__5); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__6 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__6); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__7 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__7); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__8 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____lambda__11___closed__8); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__1); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__2); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__3); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__4); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__5); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__6 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__6); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__7 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__7); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__8 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__8); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__9 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__9(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__9); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__10 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__10(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__10); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__11 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__11(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__11); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__12 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__12(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__12); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__13 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__13(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__13); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__14 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__14(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__14); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__15 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__15(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__15); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__16 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__16(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__16); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__17 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__17(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__17); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__18 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__18(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__18); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__19 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__19(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__19); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__20 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__20(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__20); -l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__21 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__21(); -lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766____closed__21); -if (builtin) {res = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3766_(lean_io_mk_world()); +l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__1 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__1(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__1); +l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__2 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__2(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__2); +l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__3 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__3(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__3); +l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__4 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__4(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__4); +l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__5 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__5(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__5); +l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__6 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__6(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__4___closed__6); +l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___rarg___closed__1 = _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___rarg___closed__1(); +lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___rarg___closed__1); +l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___rarg___closed__2 = _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___rarg___closed__2(); +lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____spec__5___rarg___closed__2); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___closed__1); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___closed__2); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__3___closed__3); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__1); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__2); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__3); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__4); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__5); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__6 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__6); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__7 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__6___closed__7); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__7___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__7___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__7___closed__1); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__7___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__7___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__7___closed__2); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__9___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__9___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__9___closed__1); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__9___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__9___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__9___closed__2); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__1); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__2); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__3); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__4); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__10___closed__5); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__1); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__2); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__3); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__4); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__5); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__6 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__6); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__7 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__7); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__8 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____lambda__11___closed__8); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__1 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__1); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__2 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__2); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__3 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__3); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__4 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__4); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__5 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__5); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__6 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__6); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__7 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__7); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__8 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__8); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__9 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__9); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__10 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__10(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__10); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__11 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__11(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__11); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__12 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__12(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__12); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__13 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__13(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__13); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__14 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__14(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__14); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__15 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__15(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__15); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__16 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__16(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__16); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__17 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__17(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__17); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__18 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__18(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__18); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__19 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__19(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__19); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__20 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__20(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__20); +l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__21 = _init_l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__21(); +lean_mark_persistent(l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696____closed__21); +if (builtin) {res = l_Lean_Elab_Tactic_Ext_initFn____x40_Lean_Elab_Tactic_Ext___hyg_3696_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__1___lambda__1___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_Ext_applyExtTheoremAt___spec__1___lambda__1___closed__1(); diff --git a/stage0/stdlib/Lean/Elab/Tactic/Induction.c b/stage0/stdlib/Lean/Elab/Tactic/Induction.c index 3ae273f9dec0..7660191fa3c8 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Induction.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Induction.c @@ -19,7 +19,6 @@ lean_object* l_Lean_Elab_Tactic_tagUntaggedGoals(lean_object*, lean_object*, lea lean_object* l_Lean_Meta_getElimInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_isAssigned___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__3___closed__6; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137_(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_withAltsOfOptInductionAlts___rarg(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_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFields___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -31,23 +30,22 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tac LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_expandCases_x3f(lean_object*); lean_object* l_Lean_Meta_getElimExprInfo(lean_object*, 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*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__12; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___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_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltName(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp_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_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___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*); static lean_object* l_Lean_Elab_Tactic_ElimApp_setMotiveArg___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__1___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAlt___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_Elab_Tactic_evalInduction___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* l_Array_mapMUnsafe_map___at_Lean_LocalContext_getFVars___spec__1(size_t, size_t, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__1___closed__1; -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__1; static lean_object* l_Lean_Elab_Tactic_evalCases___lambda__4___closed__1; lean_object* l_Lean_Elab_Term_resolveId_x3f(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCases_declRange__1___closed__1; lean_object* l_Lean_Meta_throwTacticEx___rarg(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_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079_(lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__6; lean_object* l_Lean_Elab_CommandContextInfo_save___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___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___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getArgExpectedType(lean_object*); @@ -94,7 +92,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction_declRange__1__ lean_object* l_Lean_Elab_Tactic_evalTacticAt(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_withoutTacticIncrementality___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyPreTac___spec__1___closed__1; static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___closed__1; -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__10; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabCasesTargets___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*); LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromises___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___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_Elab_Tactic_evalCases___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*); @@ -108,6 +105,7 @@ lean_object* l_Lean_Syntax_getId(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeVars___spec__1___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeVars___spec__2(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*); extern lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; lean_object* l_Array_findIdx_x3f_loop___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__3; lean_object* l_Lean_Expr_sort___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorry___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_elabTermForElim___spec__2(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*); @@ -127,9 +125,9 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tac lean_object* l_Lean_Meta_generalizeTargetsEq(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_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFields___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_mkTacticInfo(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_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__16; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArgs(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeVars___spec__1___lambda__2___closed__3; lean_object* l___private_Lean_Meta_Tactic_Generalize_0__Lean_Meta_generalizeCore(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getFirstAltLhs(lean_object*); @@ -142,15 +140,14 @@ lean_object* l_Lean_MVarId_assign___at_Lean_Elab_Tactic_refineCore___spec__1(lea LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_checkAltsOfOptInductionAlts(lean_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_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___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* 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*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__6; lean_object* lean_array_fget(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_casesOnSuffix; static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___lambda__3___closed__4; static lean_object* l_Lean_Elab_Tactic_elabCasesTargets___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__1(lean_object*, uint8_t, 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_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_checkAltsOfOptInductionAlts___spec__1___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__6(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_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__14; 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*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_elabTermForElim___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_FVarSubst_get(lean_object*, lean_object*); @@ -159,7 +156,7 @@ LEAN_EXPORT lean_object* l_Lean_isInductive___at___private_Lean_Elab_Tactic_Indu uint8_t l_Lean_LocalDecl_hasValue(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFields___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_Expr_fvarId_x21(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAlt___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_Elab_Tactic_evalAlt___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_Elab_Tactic_evalInduction___lambda__5(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*); lean_object* lean_environment_find(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_withAltsOfOptInductionAlts(lean_object*); @@ -186,9 +183,9 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_ uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_expandMultiAlt_x3f(lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__10; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_withAltsOfOptInductionAlts___rarg___lambda__1___boxed(lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__8; lean_object* l_Lean_Expr_mvar___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts___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_Lean_Elab_Tactic_ElimApp_setMotiveArg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -205,8 +202,8 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction__1___closed__5 LEAN_EXPORT lean_object* l_Array_zipWithAux___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_panic___at_Lean_Elab_Tactic_elabCasesTargets___spec__3___closed__1; lean_object* l_Lean_Meta_appendTag(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__12; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_expandInductionAlts_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeTargets(lean_object*, 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_evalInduction___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*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyPreTac___spec__1(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -223,7 +220,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tac LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__6(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_evalCases___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*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_altHasExplicitModifier(lean_object*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__7; LEAN_EXPORT uint8_t l_Lean_Elab_Tactic_isHoleRHS(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___spec__5___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___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*); static lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__3___closed__7; @@ -234,7 +230,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_ static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltName___closed__5; static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___boxed(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_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___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*, lean_object*, lean_object*, lean_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_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___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*); uint8_t l_Lean_Expr_hasMVar(lean_object*); @@ -295,13 +290,13 @@ static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_g static lean_object* l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__2___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__1___at_Lean_Elab_Tactic_evalInduction_checkTargets___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_Lean_Elab_Tactic_ElimApp_evalAlts___boxed(lean_object**); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__3; LEAN_EXPORT lean_object* l_Lean_isInductive___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___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___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getNumExplicitFields(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___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_Array_zip___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalAlt___spec__1___closed__1; +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__13; static lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyPreTac___spec__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___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___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_elabTermForElim___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -319,6 +314,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalInduct LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltRHS___boxed(lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_setMotiveArg___closed__1; lean_object* l_Lean_registerTraceClass(lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__7; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithIncremental___spec__7___lambda__2___boxed__const__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__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_object* l_Lean_Meta_SavedState_restore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -342,6 +338,7 @@ LEAN_EXPORT uint8_t l_Std_Range_forIn_x27_loop___at_Lean_Elab_Tactic_ElimApp_eva lean_object* l_Lean_MessageData_ofFormat(lean_object*); lean_object* l_Lean_PersistentArray_append___rarg(lean_object*, lean_object*); lean_object* l_Lean_Elab_getBetterRef(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__11; 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_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___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*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltVars(lean_object*); @@ -367,6 +364,7 @@ lean_object* l_Lean_log___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__3(lean_o LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Elab_addBuiltinIncrementalElab(lean_object*, lean_object*); uint8_t l_List_isEmpty___rarg(lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__4; lean_object* lean_st_mk_ref(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore(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*); @@ -379,12 +377,14 @@ static lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__3__ lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_withMainContext___spec__1___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_Name_num___override(lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_elabTermEnsuringType(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_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___lambda__8___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withReuseContext___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_withAltsOfOptInductionAlts___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_ElimApp_mkElimApp___spec__3(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_Std_Range_forIn_x27_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithIncremental___spec__4___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAlt(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_levelZero; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161_(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_withAltsOfOptInductionAlts___rarg___lambda__1(lean_object*); lean_object* l_Lean_MVarId_revert(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedExpr; @@ -398,10 +398,11 @@ static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_E LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCases___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*); static lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabCasesTargets___boxed__const__1; -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__9; +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__9; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction_declRange__1___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeTargets___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_getMainTarget___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_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__5; lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___lambda__6___closed__1; lean_object* l_Lean_Syntax_getSepArgs(lean_object*); @@ -412,9 +413,9 @@ LEAN_EXPORT lean_object* l_Array_zipWithAux___at_Lean_Elab_Tactic_ElimApp_evalAl LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithIncremental___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*); uint8_t lean_name_eq(lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithIncremental___spec__4___closed__2; -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__4; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction__1___closed__1; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withReuseContext___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_withAltsOfOptInductionAlts___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*); LEAN_EXPORT lean_object* l_Lean_Elab_addConstInfo___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___spec__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_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeVars___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*); @@ -450,6 +451,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction_checkTargets___boxed(l LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___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_Elab_Tactic_ElimApp_evalAlts_applyAltStx(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, 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_Array_eraseIdx___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltLhses___boxed(lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___closed__2; extern lean_object* l_Std_Format_defWidth; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCases_declRange__1___closed__4; @@ -461,7 +463,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSa LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFields___spec__2(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*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__2; extern lean_object* l_Lean_instInhabitedFVarId; static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___lambda__3___closed__1; static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeTargets___closed__1; @@ -485,6 +486,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__3(lean_objec lean_object* l_Lean_Elab_Term_ensureHasType(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_evalInduction_declRange__1___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithIncremental___spec__3(lean_object*, lean_object*, lean_object*, 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_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__5; lean_object* l_Lean_Name_mkStr6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getUserGeneralizingFVarIds___closed__1; lean_object* l_Lean_Elab_Tactic_saveState___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -496,11 +498,12 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tac LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___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_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_closeUsingOrAdmit(lean_object*, 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_elabCasesTargets___lambda__2(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*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__6; +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__3; lean_object* l_Lean_Syntax_setArg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp_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* l_Lean_Meta_introNCore(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltName___closed__7; -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__5; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___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 uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__1(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__1___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -530,19 +533,20 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__2(lean_objec LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getArgExpectedType___boxed(lean_object*); lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCases__1___closed__3; +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__15; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___lambda__6___boxed(lean_object**); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__1(lean_object*, lean_object*, size_t, size_t, 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_MVarId_getDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction__2(lean_object*); lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Term_withDeclName___spec__3___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__11; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltDArrow(lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getUserGeneralizingFVarIds___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_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getOptPreTacOfOptInductionAlts(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeVars___spec__1___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__13(lean_object*, 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_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_checkAltsOfOptInductionAlts___spec__1(lean_object*, size_t, size_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_Lean_PersistentArray_mapM___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__9(lean_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_forInUnsafe_loop___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -574,6 +578,7 @@ lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMe LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__4___boxed(lean_object**); lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_evalTactic_handleEx___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___regBuiltin_Lean_Elab_Tactic_evalCases__1___closed__4; +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_ElimApp_mkElimApp___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isNone(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___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*); @@ -589,6 +594,7 @@ lean_object* lean_nat_sub(lean_object*, lean_object*); lean_object* l_Lean_MVarId_tryClear(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getAppFn(lean_object*); static lean_object* l_Lean_Elab_Tactic_elabCasesTargets___lambda__1___closed__1; +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__8; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getOptPreTacOfOptInductionAlts___boxed(lean_object*); lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts___lambda__1___boxed(lean_object**); @@ -605,7 +611,6 @@ lean_object* l_Lean_RBNode_insert___at_Lean_FVarIdSet_insert___spec__1(lean_obje static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCases_declRange__1___closed__5; static lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithIncremental___spec__4___closed__3; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Tactic_elabCasesTargets___spec__5(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_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__13; lean_object* lean_erase_macro_scopes(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getBindingName___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedArgTacticReuse___at_Lean_Elab_Tactic_evalInduction___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*); @@ -621,15 +626,13 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_withReuseContext___at___private_Lean_E LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getFType___boxed(lean_object*); static lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyPreTac___spec__1___closed__5; uint8_t l_Lean_Syntax_hasMissing(lean_object*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__15; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyPreTac___spec__1___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___boxed(lean_object**); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_checkAltsOfOptInductionAlts___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_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__3___boxed(lean_object**); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__14; static lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___closed__4; -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__16; static lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___lambda__8___closed__7; static lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___lambda__6___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_withAltsOfOptInductionAlts___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*); @@ -668,12 +671,10 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithIncremental___spec__7___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_object*); lean_object* l_Lean_Elab_Tactic_withTacticInfoContext___rarg(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_evalInduction_declRange__1___closed__7; -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithIncremental___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_object*); lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction_checkTargets(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCases__2(lean_object*); lean_object* l_Lean_Meta_mkFreshExprSyntheticOpaqueMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyAltStx___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*); @@ -687,8 +688,10 @@ static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_Tactic_I LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_isHoleRHS___boxed(lean_object*); static lean_object* l_Lean_Elab_Tactic_getInductiveValFromMajor___lambda__1___closed__2; lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getNumExplicitFields___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103_(lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); uint8_t l_Array_contains___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps_visit___spec__2(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_withAltsOfOptInductionAlts___rarg___lambda__1___closed__2; @@ -708,18 +711,18 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_ElimApp_mkElimA lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__3___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__1___boxed(lean_object**); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__5; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_mkElimApp___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_Term_withNarrowedTacticReuse___at_Lean_Elab_Tactic_evalInduction___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_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isFVar(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__7(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* l_Lean_Expr_mvarId_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCases___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*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___lambda__5___closed__2; -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__2; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__1___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithIncremental___spec__7(lean_object*, 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_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Tactic_withTacticInfoContext___spec__2___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltLhses(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction_declRange__1___closed__5; static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFields___lambda__1___closed__2; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); @@ -747,6 +750,24 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAlt___lambda__4(lean_object*, le LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getFType___rarg___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_ElimApp_evalAlts_goWithInfo___lambda__3___boxed(lean_object**); uint8_t l_Array_isEmpty___rarg(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltLhses(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l_Lean_Syntax_getArg(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltLhses___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltLhses(x_1); +lean_dec(x_1); +return x_2; +} +} LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getFirstAltLhs(lean_object* x_1) { _start: { @@ -1216,31 +1237,51 @@ return x_18; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAlt___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_Lean_Elab_Tactic_evalAlt___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_14; uint8_t x_15; -x_14 = l_Lean_Elab_Tactic_getGoals___rarg(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_15; uint8_t x_16; +x_15 = l_Lean_Elab_Tactic_getGoals___rarg(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_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_14, 0); -x_17 = lean_ctor_get(x_14, 1); -x_18 = lean_box(0); -lean_ctor_set_tag(x_14, 1); -lean_ctor_set(x_14, 1, x_18); -lean_ctor_set(x_14, 0, x_1); -x_19 = l_Lean_Elab_Tactic_setGoals(x_14, 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, 1); -lean_inc(x_20); -lean_dec(x_19); -x_21 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalAlt___lambda__1), 11, 2); -lean_closure_set(x_21, 0, x_2); -lean_closure_set(x_21, 1, x_3); -x_22 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); -lean_closure_set(x_22, 0, x_4); -lean_closure_set(x_22, 1, x_21); +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_box(0); +lean_ctor_set_tag(x_15, 1); +lean_ctor_set(x_15, 1, x_19); +lean_ctor_set(x_15, 0, x_1); +x_20 = l_Lean_Elab_Tactic_setGoals(x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_18); +x_21 = !lean_is_exclusive(x_20); +if (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; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_22 = lean_ctor_get(x_20, 1); +x_23 = lean_ctor_get(x_20, 0); +lean_dec(x_23); +x_24 = lean_unsigned_to_nat(0u); +x_25 = l_Lean_Syntax_getArg(x_2, x_24); +lean_ctor_set_tag(x_20, 1); +lean_ctor_set(x_20, 1, x_19); +lean_ctor_set(x_20, 0, x_3); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_20); +x_27 = lean_array_mk(x_26); +x_28 = lean_box(2); +x_29 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalAlt___spec__1___closed__2; +x_30 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +lean_ctor_set(x_30, 2, x_27); +x_31 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalAlt___lambda__1), 11, 2); +lean_closure_set(x_31, 0, x_4); +lean_closure_set(x_31, 1, x_5); +x_32 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_32, 0, x_30); +lean_closure_set(x_32, 1, x_31); +lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); @@ -1248,17 +1289,17 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -x_23 = l_Lean_Elab_Tactic_closeUsingOrAdmit(x_22, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_20); -if (lean_obj_tag(x_23) == 0) +x_33 = l_Lean_Elab_Tactic_closeUsingOrAdmit(x_32, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_22); +if (lean_obj_tag(x_33) == 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 = l_Lean_Elab_Tactic_setGoals(x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_25); +lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t 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 = l_Lean_Elab_Tactic_setGoals(x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_35); +lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -1266,37 +1307,37 @@ 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_26); -if (x_27 == 0) +x_37 = !lean_is_exclusive(x_36); +if (x_37 == 0) { -lean_object* x_28; -x_28 = lean_ctor_get(x_26, 0); -lean_dec(x_28); -lean_ctor_set(x_26, 0, x_24); -return x_26; +lean_object* x_38; +x_38 = lean_ctor_get(x_36, 0); +lean_dec(x_38); +lean_ctor_set(x_36, 0, x_34); +return x_36; } else { -lean_object* x_29; lean_object* x_30; -x_29 = lean_ctor_get(x_26, 1); -lean_inc(x_29); -lean_dec(x_26); -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_24); -lean_ctor_set(x_30, 1, x_29); -return x_30; +lean_object* x_39; lean_object* x_40; +x_39 = lean_ctor_get(x_36, 1); +lean_inc(x_39); +lean_dec(x_36); +x_40 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_40, 0, x_34); +lean_ctor_set(x_40, 1, x_39); +return x_40; } } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; -x_31 = lean_ctor_get(x_23, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_23, 1); -lean_inc(x_32); -lean_dec(x_23); -x_33 = l_Lean_Elab_Tactic_setGoals(x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_32); +lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_41 = lean_ctor_get(x_33, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_33, 1); +lean_inc(x_42); +lean_dec(x_33); +x_43 = l_Lean_Elab_Tactic_setGoals(x_17, x_6, x_7, 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); @@ -1304,52 +1345,57 @@ lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -x_34 = !lean_is_exclusive(x_33); -if (x_34 == 0) +x_44 = !lean_is_exclusive(x_43); +if (x_44 == 0) { -lean_object* x_35; -x_35 = lean_ctor_get(x_33, 0); -lean_dec(x_35); -lean_ctor_set_tag(x_33, 1); -lean_ctor_set(x_33, 0, x_31); -return x_33; +lean_object* x_45; +x_45 = lean_ctor_get(x_43, 0); +lean_dec(x_45); +lean_ctor_set_tag(x_43, 1); +lean_ctor_set(x_43, 0, x_41); +return x_43; } 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(1, 2, 0); -lean_ctor_set(x_37, 0, x_31); -lean_ctor_set(x_37, 1, x_36); -return x_37; +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(1, 2, 0); +lean_ctor_set(x_47, 0, x_41); +lean_ctor_set(x_47, 1, x_46); +return x_47; } } } 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; -x_38 = lean_ctor_get(x_14, 0); -x_39 = lean_ctor_get(x_14, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_14); -x_40 = lean_box(0); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_1); -lean_ctor_set(x_41, 1, x_40); -x_42 = l_Lean_Elab_Tactic_setGoals(x_41, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_39); -x_43 = lean_ctor_get(x_42, 1); -lean_inc(x_43); -lean_dec(x_42); -x_44 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalAlt___lambda__1), 11, 2); -lean_closure_set(x_44, 0, x_2); -lean_closure_set(x_44, 1, x_3); -x_45 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); -lean_closure_set(x_45, 0, x_4); -lean_closure_set(x_45, 1, x_44); +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_48 = lean_ctor_get(x_20, 1); +lean_inc(x_48); +lean_dec(x_20); +x_49 = lean_unsigned_to_nat(0u); +x_50 = l_Lean_Syntax_getArg(x_2, x_49); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_3); +lean_ctor_set(x_51, 1, x_19); +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_box(2); +x_55 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalAlt___spec__1___closed__2; +x_56 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_55); +lean_ctor_set(x_56, 2, x_53); +x_57 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalAlt___lambda__1), 11, 2); +lean_closure_set(x_57, 0, x_4); +lean_closure_set(x_57, 1, x_5); +x_58 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_58, 0, x_56); +lean_closure_set(x_58, 1, x_57); +lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); @@ -1357,17 +1403,17 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -x_46 = l_Lean_Elab_Tactic_closeUsingOrAdmit(x_45, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_43); -if (lean_obj_tag(x_46) == 0) +x_59 = l_Lean_Elab_Tactic_closeUsingOrAdmit(x_58, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_48); +if (lean_obj_tag(x_59) == 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_Elab_Tactic_setGoals(x_38, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_48); +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_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_setGoals(x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_61); +lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -1375,35 +1421,35 @@ lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -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; +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_49); - x_51 = lean_box(0); + lean_dec_ref(x_62); + x_64 = lean_box(0); } -if (lean_is_scalar(x_51)) { - x_52 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_64)) { + x_65 = lean_alloc_ctor(0, 2, 0); } else { - x_52 = x_51; + x_65 = x_64; } -lean_ctor_set(x_52, 0, x_47); -lean_ctor_set(x_52, 1, x_50); -return x_52; +lean_ctor_set(x_65, 0, x_60); +lean_ctor_set(x_65, 1, x_63); +return x_65; } 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; -x_53 = lean_ctor_get(x_46, 0); -lean_inc(x_53); -x_54 = lean_ctor_get(x_46, 1); -lean_inc(x_54); -lean_dec(x_46); -x_55 = l_Lean_Elab_Tactic_setGoals(x_38, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_54); +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_59, 0); +lean_inc(x_66); +x_67 = lean_ctor_get(x_59, 1); +lean_inc(x_67); +lean_dec(x_59); +x_68 = l_Lean_Elab_Tactic_setGoals(x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_67); +lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -1411,26 +1457,158 @@ lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -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; +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_55); - x_57 = lean_box(0); + lean_dec_ref(x_68); + x_70 = lean_box(0); } -if (lean_is_scalar(x_57)) { - x_58 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_70)) { + x_71 = lean_alloc_ctor(1, 2, 0); } else { - x_58 = x_57; - lean_ctor_set_tag(x_58, 1); + x_71 = x_70; + lean_ctor_set_tag(x_71, 1); +} +lean_ctor_set(x_71, 0, x_66); +lean_ctor_set(x_71, 1, x_69); +return x_71; } -lean_ctor_set(x_58, 0, x_53); -lean_ctor_set(x_58, 1, x_56); -return x_58; +} +} +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; 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_72 = lean_ctor_get(x_15, 0); +x_73 = lean_ctor_get(x_15, 1); +lean_inc(x_73); +lean_inc(x_72); +lean_dec(x_15); +x_74 = lean_box(0); +x_75 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_75, 0, x_1); +lean_ctor_set(x_75, 1, x_74); +x_76 = l_Lean_Elab_Tactic_setGoals(x_75, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_73); +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_76); + x_78 = lean_box(0); +} +x_79 = lean_unsigned_to_nat(0u); +x_80 = l_Lean_Syntax_getArg(x_2, x_79); +if (lean_is_scalar(x_78)) { + x_81 = lean_alloc_ctor(1, 2, 0); +} else { + x_81 = x_78; + lean_ctor_set_tag(x_81, 1); +} +lean_ctor_set(x_81, 0, x_3); +lean_ctor_set(x_81, 1, x_74); +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 = lean_box(2); +x_85 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalAlt___spec__1___closed__2; +x_86 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_86, 0, x_84); +lean_ctor_set(x_86, 1, x_85); +lean_ctor_set(x_86, 2, x_83); +x_87 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalAlt___lambda__1), 11, 2); +lean_closure_set(x_87, 0, x_4); +lean_closure_set(x_87, 1, x_5); +x_88 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg), 11, 2); +lean_closure_set(x_88, 0, x_86); +lean_closure_set(x_88, 1, x_87); +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_89 = l_Lean_Elab_Tactic_closeUsingOrAdmit(x_88, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_77); +if (lean_obj_tag(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; +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 = l_Lean_Elab_Tactic_setGoals(x_72, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_91); +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); +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_90); +lean_ctor_set(x_95, 1, x_93); +return x_95; +} +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; +x_96 = lean_ctor_get(x_89, 0); +lean_inc(x_96); +x_97 = lean_ctor_get(x_89, 1); +lean_inc(x_97); +lean_dec(x_89); +x_98 = l_Lean_Elab_Tactic_setGoals(x_72, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_97); +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); +x_99 = lean_ctor_get(x_98, 1); +lean_inc(x_99); +if (lean_is_exclusive(x_98)) { + lean_ctor_release(x_98, 0); + lean_ctor_release(x_98, 1); + x_100 = x_98; +} else { + lean_dec_ref(x_98); + 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_tag(x_101, 1); +} +lean_ctor_set(x_101, 0, x_96); +lean_ctor_set(x_101, 1, x_99); +return x_101; } } } @@ -1671,11 +1849,13 @@ if (x_17 == 0) { lean_object* x_18; lean_object* x_19; lean_inc(x_14); -x_18 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalAlt___lambda__2), 13, 4); +lean_inc(x_16); +x_18 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalAlt___lambda__2___boxed), 14, 5); lean_closure_set(x_18, 0, x_1); -lean_closure_set(x_18, 1, x_3); -lean_closure_set(x_18, 2, x_14); -lean_closure_set(x_18, 3, x_2); +lean_closure_set(x_18, 1, x_2); +lean_closure_set(x_18, 2, x_16); +lean_closure_set(x_18, 3, x_3); +lean_closure_set(x_18, 4, x_14); x_19 = l_Lean_Elab_Tactic_withCaseRef___at_Lean_Elab_Tactic_evalAlt___spec__1(x_16, x_14, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); return x_19; } @@ -1693,6 +1873,15 @@ return x_21; } } } +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAlt___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_evalAlt___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_2); +return x_15; +} +} static lean_object* _init_l_Lean_Elab_Tactic_ElimApp_instInhabitedAlt___closed__1() { _start: { @@ -16186,7 +16375,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___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_8; uint8_t x_9; @@ -16775,7 +16964,7 @@ lean_inc(x_35); lean_dec(x_34); x_36 = lean_array_get_size(x_11); x_37 = lean_mk_empty_array_with_capacity(x_36); -x_38 = l_Array_mapIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2(x_3, x_11, x_11, x_36, x_27, lean_box(0), x_37); +x_38 = l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2(x_3, x_11, x_11, x_36, x_27, lean_box(0), x_37); lean_inc(x_19); lean_inc(x_18); lean_inc(x_17); @@ -17034,11 +17223,11 @@ lean_dec(x_1); return x_5; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___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_8; -x_8 = l_Array_mapIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Array_mapFinIdxM_map___at_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_3); lean_dec(x_2); return x_8; @@ -21775,7 +21964,7 @@ lean_dec(x_2); return x_10; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__1() { _start: { lean_object* x_1; @@ -21783,7 +21972,7 @@ x_1 = lean_mk_string_unchecked("tactic", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__2() { _start: { lean_object* x_1; @@ -21791,17 +21980,17 @@ x_1 = lean_mk_string_unchecked("customEliminators", 17, 17); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__1; -x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__2; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__1; +x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__2; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__4() { _start: { lean_object* x_1; @@ -21809,13 +21998,13 @@ x_1 = lean_mk_string_unchecked("enable using custom eliminators in the 'inductio return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____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 = 1; -x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__1; -x_3 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__4; +x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__1; +x_3 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__4; x_4 = lean_box(x_1); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_4); @@ -21824,26 +22013,26 @@ lean_ctor_set(x_5, 2, x_3); return x_5; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____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; x_1 = l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltName___closed__1; x_2 = l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyPreTac___spec__1___closed__2; x_3 = l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__3___closed__1; -x_4 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__1; -x_5 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__2; +x_4 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__1; +x_5 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____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_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103_(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_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__3; -x_3 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__5; -x_4 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__6; +x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__3; +x_3 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__5; +x_4 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__6; 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; } @@ -27306,7 +27495,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_elabCasesTargets___lambda__1___clos 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_Tactic_elabCasesTargets___lambda__1___closed__4; x_2 = l_Lean_Elab_Tactic_elabCasesTargets___lambda__1___closed__5; -x_3 = lean_unsigned_to_nat(713u); +x_3 = lean_unsigned_to_nat(717u); x_4 = lean_unsigned_to_nat(8u); x_5 = l_Lean_Elab_Tactic_elabCasesTargets___lambda__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -29653,7 +29842,7 @@ x_3 = l_Lean_Elab_addBuiltinIncrementalElab(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -29663,7 +29852,7 @@ x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -29673,27 +29862,27 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__2; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__2; x_2 = l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyPreTac___spec__1___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__3; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__3; x_2 = l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__3___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__5() { _start: { lean_object* x_1; @@ -29701,17 +29890,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__4; -x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__5; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__4; +x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__7() { _start: { lean_object* x_1; @@ -29719,47 +29908,47 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__8() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__6; -x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__7; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__6; +x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__9() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__8; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__8; x_2 = l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltName___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__10() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__9; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__9; x_2 = l_Lean_Elab_Term_withoutTacticIncrementality___at_Lean_Elab_Tactic_ElimApp_evalAlts_applyPreTac___spec__1___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__11() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__10; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__10; x_2 = l_Lean_Elab_Tactic_ElimApp_evalAlts_goWithInfo___lambda__3___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__12() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__12() { _start: { lean_object* x_1; @@ -29767,17 +29956,17 @@ x_1 = lean_mk_string_unchecked("Induction", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__13() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__11; -x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__12; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__11; +x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__14() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__14() { _start: { lean_object* x_1; @@ -29785,33 +29974,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__15() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__13; -x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__14; +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__13; +x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__14; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__16() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__15; -x_2 = lean_unsigned_to_nat(11137u); +x_1 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__15; +x_2 = lean_unsigned_to_nat(11161u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161_(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_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__1; +x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__1; x_3 = 0; -x_4 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__16; +x_4 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__16; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); if (lean_obj_tag(x_5) == 0) { @@ -30086,19 +30275,19 @@ l_Lean_Elab_Tactic_getInductiveValFromMajor___lambda__1___closed__2 = _init_l_Le lean_mark_persistent(l_Lean_Elab_Tactic_getInductiveValFromMajor___lambda__1___closed__2); l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_elabTermForElim___closed__1 = _init_l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_elabTermForElim___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_elabTermForElim___closed__1); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__1 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__1); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__2 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__2); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__3 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__3); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__4 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__4); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__5 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__5); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__6 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079____closed__6); -if (builtin) {res = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8079_(lean_io_mk_world()); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__1 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__1); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__2 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__2); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__3 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__3); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__4 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__4); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__5 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__5); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__6 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103____closed__6); +if (builtin) {res = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8103_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Elab_Tactic_tactic_customEliminators = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_Tactic_tactic_customEliminators); @@ -30227,39 +30416,39 @@ lean_dec_ref(res); }if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_evalCases__2(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__1 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__1); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__2 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__2); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__3 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__3); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__4 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__4); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__5 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__5); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__6 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__6); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__7 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__7); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__8 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__8); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__9 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__9(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__9); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__10 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__10(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__10); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__11 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__11(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__11); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__12 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__12(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__12); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__13 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__13(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__13); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__14 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__14(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__14); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__15 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__15(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__15); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__16 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__16(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137____closed__16); -if (builtin) {res = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11137_(lean_io_mk_world()); +}l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__1 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__1); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__2 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__2); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__3 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__3); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__4 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__4); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__5 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__5); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__6 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__6); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__7 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__7); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__8 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__8); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__9 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__9); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__10 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__10(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__10); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__11 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__11(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__11); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__12 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__12(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__12); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__13 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__13(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__13); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__14 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__14(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__14); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__15 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__15(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__15); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__16 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__16(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161____closed__16); +if (builtin) {res = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_11161_(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/SolveByElim.c b/stage0/stdlib/Lean/Elab/Tactic/SolveByElim.c index e79d6443eb49..2ea2ccd5c9b9 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/SolveByElim.c +++ b/stage0/stdlib/Lean/Elab/Tactic/SolveByElim.c @@ -173,6 +173,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_SolveByElim_evalApplyRu static lean_object* l_Lean_Elab_Tactic_SolveByElim_elabConfig___closed__1; lean_object* l_Sum_getLeft_x3f___rarg(lean_object*); lean_object* l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5___boxed(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_SolveByElim_evalApplyAssumption_declRange__1___closed__1; static lean_object* l_Lean_Elab_Tactic_SolveByElim_elabConfig___closed__8; static lean_object* l___regBuiltin_Lean_Elab_Tactic_SolveByElim_evalApplyRules_declRange__1___closed__4; @@ -212,7 +213,6 @@ static lean_object* l_Lean_Elab_Tactic_SolveByElim_evalApplyRules___closed__2; LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at_Lean_Elab_Tactic_SolveByElim_elabConfig___spec__9(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_Lean_Elab_Tactic_SolveByElim_elabConfig___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SolveByElim_evalSolveByElim___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*, lean_object*, lean_object*, lean_object*); static size_t l_Lean_Elab_Tactic_SolveByElim_parseArgs___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_SolveByElim_evalApplyAssumption_declRange__1___closed__2; @@ -226,7 +226,6 @@ size_t lean_usize_add(size_t, size_t); static lean_object* l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Tactic_SolveByElim_elabConfig___spec__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_SolveByElim_evalApplyAssumption_declRange__1___closed__6; static lean_object* l_Lean_Elab_Tactic_SolveByElim_parseUsing___closed__1; -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withoutModifyingStateWithInfoAndMessages___at_Lean_Elab_Tactic_SolveByElim_elabConfig___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SolveByElim_processSyntax(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_Lean_Elab_Tactic_SolveByElim_elabApplyRulesConfig(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -242,6 +241,7 @@ static lean_object* l_Lean_Elab_Tactic_SolveByElim_elabConfig___closed__13; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SolveByElim_processSyntax___boxed(lean_object*, 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_evalExpr_x27___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_SolveByElim_evalUnsafe____x40_Lean_Elab_Tactic_SolveByElim___hyg_8____closed__4; +LEAN_EXPORT uint8_t l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5(lean_object*, lean_object*); extern lean_object* l_Lean_Elab_unsupportedSyntaxExceptionId; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SolveByElim_evalUnsafe____x40_Lean_Elab_Tactic_SolveByElim___hyg_8____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); @@ -3612,7 +3612,7 @@ goto _start; } } } -LEAN_EXPORT uint8_t l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -3700,7 +3700,7 @@ lean_dec(x_1); x_7 = lean_ctor_get(x_2, 0); lean_inc(x_7); lean_dec(x_2); -x_8 = l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5(x_6, x_7); +x_8 = l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5(x_6, x_7); return x_8; } } @@ -3988,11 +3988,11 @@ x_6 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec_ return x_6; } } -LEAN_EXPORT lean_object* l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Init_Data_Sum_0__Sum_beqSum____x40_Init_Data_Sum___hyg_242____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5(x_1, x_2); +x_3 = l___private_Init_Data_Sum_Basic_0__Sum_beqSum____x40_Init_Data_Sum_Basic___hyg_243____at_Lean_Elab_Tactic_SolveByElim_parseArgs___spec__5(x_1, x_2); x_4 = lean_box(x_3); return x_4; } diff --git a/stage0/stdlib/Lean/Elab/Term.c b/stage0/stdlib/Lean/Elab/Term.c index af6f01980ae7..b8427267ed07 100644 --- a/stage0/stdlib/Lean/Elab/Term.c +++ b/stage0/stdlib/Lean/Elab/Term.c @@ -22,6 +22,7 @@ static lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Term_0__Lean LEAN_EXPORT lean_object* l_Lean_MVarId_isAssigned___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__2(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_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2___closed__1; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Term_exposeLevelMVars___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_hasNoImplicitLambdaAnnotation___closed__1; lean_object* l_Lean_Meta_mkSorry(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -46,7 +47,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_setLevelNames___boxed(lean_object*, le LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorryImp(lean_object*); static lean_object* l_Lean_Elab_Term_mkExplicitBinder___closed__11; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__2(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274_(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Core_transform___at_Lean_Elab_Term_exposeLevelMVars___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instInhabitedTermElabM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -54,7 +54,6 @@ lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Metava static lean_object* l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Term_expandDeclId___spec__10___closed__1; static lean_object* l_Lean_Elab_Term_getInfoTreeWithContext_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveLocalName___boxed(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_Term___hyg_17274____closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLocalContextImp___rarg(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_throwMVarError___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -65,7 +64,6 @@ static lean_object* l_Lean_Elab_Term_getFVarLocalDecl_x21___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabUsingElabFnsAux___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*); static lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___lambda__3___closed__1; static lean_object* l_Lean_Elab_Term_mkAuxName___closed__1; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__1; extern lean_object* l_Lean_instMonadExceptOfExceptionCoreM; LEAN_EXPORT lean_object* l_Lean_Elab_Term_getInfoTreeWithContext_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveId_x3f(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -97,7 +95,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_TacticParsedSnapshot_data(lean_objec LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorCustomInfo(lean_object*, 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_assign___at_Lean_Elab_Term_exprToSyntax___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_Array_mapMUnsafe_map___at_Lean_Elab_Term_withDeclName___spec__8(lean_object*, 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_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__2; static lean_object* l_Lean_Linter_checkDeprecated___at_Lean_Elab_Term_mkConst___spec__3___closed__7; static lean_object* l_Lean_Elab_Term_withExpectedType___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_exposeLevelMVars___spec__4(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*); @@ -117,6 +114,8 @@ LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_v LEAN_EXPORT lean_object* l_Lean_Elab_Term_instAddErrorMessageContextTermElabM(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_MetavarContext_0__Lean_DependsOn_dep_visit___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__10(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_commitIfNoErrors_x3f(lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__11; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__2; LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__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_Lean_Core_transform_visit___at_Lean_Elab_Term_exposeLevelMVars___spec__2___boxed__const__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withSavedContext(lean_object*); @@ -133,12 +132,12 @@ static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabUsingElabFn LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Term_isLetRecAuxMVar___spec__3(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_LevelMVarErrorInfo_logError___lambda__1___closed__4; lean_object* l_Lean_Elab_Level_elabLevel(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadMacroAdapterTermElabM; LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at_Lean_Elab_Term_withDeclName___spec__2___rarg___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_Term_getInfoTreeWithContext_x3f___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_Core_transform___at_Lean_Elab_Term_exposeLevelMVars___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkTacticMVar___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_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Term_isLetRecAuxMVar___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_find___at_Lean_Elab_Term_resolveLocalName___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkExplicitBinder___closed__6; @@ -153,14 +152,13 @@ lean_object* l_Lean_profileitIOUnsafe___rarg(lean_object*, lean_object*, lean_ob LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instInhabitedSyntheticMVarDecl; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__1; LEAN_EXPORT 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*); lean_object* l_Lean_RBNode_findCore___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimApp___spec__4(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instInhabitedTacticParsedSnapshot; LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerSyntheticMVar___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_Elab_Term_registerSyntheticMVarWithCurrRef(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_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__4(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_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withLevelNames(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__34___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars___closed__4; @@ -170,6 +168,7 @@ static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_expandDeclId___ static lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_847____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutHeedElabAsElim(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__6; uint8_t l_Array_contains___at_Lean_Meta_arrowDomainsN___spec__2(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_instToStringMVarErrorKind___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveLocalName_go___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -178,8 +177,8 @@ lean_object* l_Lean_Meta_isProp(lean_object*, lean_object*, lean_object*, lean_o lean_object* l_Lean_ConstantInfo_levelParams(lean_object*); lean_object* l_Lean_indentD(lean_object*); double lean_float_div(double, double); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__7; static lean_object* l_Lean_Elab_Tactic_instBEqCacheKey___closed__1; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__6; static lean_object* l_Lean_Elab_Term_levelMVarToParam___closed__2; LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___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_Term_synthesizeInstMVarCore___lambda__3___closed__2; @@ -188,8 +187,8 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAu static lean_object* l_Lean_Elab_Tactic_instInhabitedCache___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_useImplicitLambda___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_addDocString___at_Lean_Elab_Term_expandDeclId___spec__9___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_of_nat(lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__1; uint64_t lean_uint64_mix_hash(uint64_t, uint64_t); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__41(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__7(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -218,7 +217,6 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwTypeMismatch LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Elab_Term_resolveId_x3f___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___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_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticReuse___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__4; static lean_object* l_Lean_Elab_Term_mkCoe___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_instMonadTermElabM___closed__3; @@ -235,8 +233,9 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkCoe___lambda__1(lean_object*, lean_o LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_expandDeclId___spec__4(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* l_Lean_MetavarContext_getDelayedMVarAssignmentCore_x3f(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___rarg___closed__3; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__3; lean_object* l_Lean_Syntax_getId(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabTermEnsuringType(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_findSomeRevM_x3f_find___at_Lean_Elab_Term_resolveLocalName___spec__5(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); @@ -245,7 +244,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorHoleInfo___boxed(lean LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__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_Elab_Term_isLocalIdent_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__41___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__2; lean_object* l_Lean_Expr_sort___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadMacroAdapterTermElabM___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Term_expandDeclId___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -263,25 +261,27 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkConst___lambda__1___boxed(lean_objec LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Term_logUnassignedLevelMVarsUsingErrorInfos___spec__4(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_Array_mapMUnsafe_map___at_Lean_Elab_Term_withDeclName___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_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Term_addAutoBoundImplicits_x27___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_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__4; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2___boxed__const__1; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_mkConst___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isNoImplicitLambda___closed__2; lean_object* l_String_removeLeadingSpaces(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveLocalName(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_expandDeclId___spec__4___closed__1; -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__10; lean_object* l_Lean_Core_getMessageLog___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_expandDeclId___closed__1; lean_object* l_Lean_Core_checkSystem(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Term_resolveId_x3f___spec__3(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeRevMAux___at_Lean_Elab_Term_resolveLocalName___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_liftExcept___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__8(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20064____closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static double l_Lean_withTraceNode___at_Lean_Elab_Term_mkCoe___spec__1___lambda__4___closed__5; LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__36___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveId_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_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___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_TacticParsedSnapshot_data___boxed(lean_object*); static lean_object* l_Lean_Elab_Term_ensureType___lambda__1___closed__1; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__5; LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_addTraceNode___at_Lean_Elab_Term_mkCoe___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_mk_array(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_traceAtCmdPos___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -294,6 +294,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_throwAutoBoundImplicitLocal___at_Lean_Elab_ LEAN_EXPORT lean_object* l_Lean_Elab_Term_instToStringMVarErrorKind___boxed(lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveLocalName___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Term_isExplicit(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_TermElabM_toIO___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2___closed__2; @@ -301,7 +302,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_CommandContextInfo_saveNoFileMap___at_Lean_ static lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Term_withDeclName___spec__3___rarg___closed__2; static lean_object* l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__4; static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2___lambda__2___closed__1; -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadTermElabM; lean_object* l_Lean_instMonadQuotationOfMonadFunctorOfMonadLift___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyM___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__5(lean_object*, lean_object*); @@ -315,6 +315,7 @@ lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_hasNoImplicitLambdaAnnotation___boxed(lean_object*); lean_object* l_Lean_Level_isMVar___boxed(lean_object*); static lean_object* l_Lean_Elab_CommandContextInfo_saveNoFileMap___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__3___rarg___closed__1; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedTacticReuse___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeRevMAux___at_Lean_Elab_Term_resolveLocalName___spec__4(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkAuxName___closed__2; @@ -372,7 +373,7 @@ lean_object* l_Lean_Expr_fvarId_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__38___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_transform_visit___at_Lean_Elab_Term_exposeLevelMVars___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_ReaderT_pure___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__12___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__5; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__15; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_useImplicitLambda___lambda__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_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Term_withDeclName___spec__3___rarg___closed__1; @@ -405,7 +406,6 @@ static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_dropTermParens_ LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_921____boxed(lean_object*); static lean_object* l_Lean_Elab_Term_extraMsgToMsg___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutHeedElabAsElim___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__2; static lean_object* l_Lean_Elab_Term_instMonadBacktrackSavedStateTermElabM___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_useImplicitLambda(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Linter_getLinterValue(lean_object*, lean_object*); @@ -426,7 +426,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVa lean_object* l_Lean_Expr_setPPUniverses(lean_object*, uint8_t); static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError___closed__3; static lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___rarg___closed__14; -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__3; lean_object* lean_io_get_num_heartbeats(lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); static lean_object* l_Lean_Linter_checkDeprecated___at_Lean_Elab_Term_mkConst___spec__3___closed__4; @@ -456,7 +455,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutHeedElabAsElim___rarg___lambda_ static lean_object* l_Lean_Elab_Term_instInhabitedMVarErrorKind___closed__7; lean_object* l_Lean_PersistentArray_toList___rarg(lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Term_getFVarLocalDecl_x21___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__4; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_resolveName_x27___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_List_any___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___closed__5; @@ -492,7 +490,6 @@ LEAN_EXPORT lean_object* l_Lean_Core_transform_visit_visitPost___at_Lean_Elab_Te static lean_object* l_Lean_Elab_Term_instInhabitedLevelMVarErrorInfo___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__10___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 l_Lean_Name_isPrefixOf(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__8; LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__30___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplicitLambda_loop___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_Term_instMonadMacroAdapterTermElabM___closed__2; @@ -519,6 +516,7 @@ LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Term_logUnassignedUsin LEAN_EXPORT lean_object* l_Lean_mkAuxName___at_Lean_Elab_Term_mkAuxName___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___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplicitLambdaAux___closed__2; static lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Term_0__Lean_Elab_Term_isLambdaWithImplicit___spec__1___closed__3; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__3; static lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars___closed__3; static lean_object* l_Lean_Elab_addBuiltinIncrementalElab___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_tryPostpone___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -532,7 +530,7 @@ lean_object* l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(lean_o LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkExplicitBinder(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_instToStringSyntheticMVarKind___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__7; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__2; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__40___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_isLocalIdent_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -542,6 +540,7 @@ static lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___lambda__3___closed LEAN_EXPORT lean_object* l_Lean_Elab_Term_withPushMacroExpansionStack___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Kernel_isDiagnosticsEnabled(lean_object*); static lean_object* l_Lean_Elab_Term_mkTypeMismatchError___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850_(lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_Term_resolveName_x27___spec__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_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Term_expandDeclId___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT 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*); @@ -550,11 +549,12 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplic uint8_t l_Lean_Expr_hasMVar(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instInhabitedCacheKey; uint8_t l_Lean_isReservedName(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_withMacroExpansionInfo___at_Lean_Elab_Term_withMacroExpansion___spec__1___rarg___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_initFn____x40_Lean_Elab_Term___hyg_19578____closed__1; static lean_object* l_Lean_Elab_Tactic_instInhabitedTacticFinishedSnapshot___closed__2; static lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Term_TermElabM_run(lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__9; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTypeAscription(lean_object*); LEAN_EXPORT uint8_t l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2___lambda__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -579,7 +579,6 @@ static lean_object* l_Lean_Elab_Term_instInhabitedSyntheticMVarDecl___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___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*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutHeedElabAsElimImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars___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_initFn____x40_Lean_Elab_Term___hyg_19578____closed__8; static lean_object* l_Lean_Elab_Term_instMonadMacroAdapterTermElabM___closed__3; lean_object* lean_io_promise_resolve(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabUsingElabFnsAux___lambda__1___closed__1; @@ -627,6 +626,7 @@ static lean_object* l_Lean_Linter_checkDeprecated___at_Lean_Elab_Term_mkConst___ LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__8(lean_object*); uint8_t l_List_elem___at_Lean_addAliasEntry___spec__16(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyM___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__13(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Term_applyResult___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_withoutHeedElabAsElim___rarg___closed__1; static lean_object* l_Lean_Elab_Term_isLetRecAuxMVar___closed__2; @@ -647,15 +647,14 @@ lean_object* lean_st_ref_take(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_getLetRecsToLift(lean_object*); lean_object* l_Lean_Meta_withRestoreOrSaveFull___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_saveContext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withReuseContext___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Term_resolveLocalName_loop___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_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Term_expandDeclId___spec__6___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___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at_Lean_Elab_Term_withDeclName___spec__2___rarg___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_initFn____x40_Lean_Elab_Term___hyg_19617____closed__4; lean_object* l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Term_withMacroExpansion___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorry___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_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__5; static lean_object* l_Lean_Elab_Term_collectUnassignedMVars_go___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedTacticReuse___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_expandMacroImpl_x3f(lean_object*, lean_object*, lean_object*, lean_object*); @@ -663,6 +662,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_TermElabM_toIO___rarg___lambda__1(lean LEAN_EXPORT 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*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_847_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__14___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__2; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__31___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); lean_object* l_Lean_declareBuiltin(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -671,7 +671,6 @@ lean_object* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lea lean_object* l_Lean_mkPrivateName(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_exposeLevelMVars___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Term_addDotCompletionInfo___spec__2___boxed(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_Term___hyg_17274____closed__4; LEAN_EXPORT lean_object* l_Lean_logWarning___at_Lean_Elab_Term_mkConst___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars_x3f___boxed(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_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__11(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -687,24 +686,27 @@ uint64_t lean_uint64_shift_right(uint64_t, uint64_t); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___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_instantiateMVars___at___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___spec__7(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withMacroExpansion(lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__1; lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); static lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_exposeLevelMVars___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__13; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__40(lean_object*, lean_object*, size_t, size_t); uint8_t l_Lean_TagAttribute_hasTag(lean_object*, lean_object*, lean_object*); lean_object* l_List_findSome_x3f___rarg(lean_object*, lean_object*); lean_object* l_Lean_Meta_isType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofSyntax(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveName_process(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_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__3; LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__28___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732_(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__9(lean_object*, lean_object*, size_t, size_t); 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_Term_getLevelNames(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_logUnassignedLevelMVarsUsingErrorInfos___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_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedLevelMVarsUsingErrorInfos___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__14; LEAN_EXPORT 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_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___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___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__4___boxed(lean_object*, lean_object*, lean_object*); @@ -713,8 +715,8 @@ LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyMAux___at_Lean_Elab_Term_addAutoBo LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedArgTacticReuse(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instInhabitedCache; LEAN_EXPORT lean_object* l_Lean_Core_transform_visit___at_Lean_Elab_Term_exposeLevelMVars___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*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__2; lean_object* l_Lean_Option_get___at_Lean_profiler_threshold_getSecs___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__9; static lean_object* l_Lean_getConstInfo___at_Lean_Elab_Term_mkConst___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutErrToSorryImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -731,6 +733,7 @@ LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Term lean_object* l_Lean_registerTraceClass(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabUsingElabFnsAux___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_Lean_Elab_Tactic_instToSnapshotTreeTacticFinishedSnapshot(lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__10; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_useImplicitLambda___lambda__4___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_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Term_mkCoe___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_log___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__9(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -741,7 +744,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_TermElabM_toIO(lean_object*); lean_object* l_Lean_Meta_SavedState_restore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLocalDeclImp___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Term_ppGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars_x3f___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_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__10___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*); @@ -752,7 +754,6 @@ static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTer static lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___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*); static lean_object* l_Lean_Elab_Term_mkExplicitBinder___closed__10; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabTerm___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_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__23(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Term_expandDeclId___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -767,6 +768,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerSyntheticMVarWithCurrRef___box LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__29___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__52(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_Term_withoutMacroStackAtErr___rarg(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_Term___hyg_17313____closed__12; lean_object* l_Lean_Syntax_getKind(lean_object*); static lean_object* l_Lean_Elab_Term_exposeLevelMVars___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_collectUnassignedMVars_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -795,7 +797,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_decorateEr LEAN_EXPORT lean_object* l_Lean_Elab_Term_withAuxDecl(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__5___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instToSnapshotTreeTacticParsedSnapshot_go___lambda__1(lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__11; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_addTermInfo___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_Lean_FVarId_getDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -827,7 +829,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_withPushMacroExpansionStack(lean_objec LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Term_mkCoe___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*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_throwMVarError(lean_object*); lean_object* l_Lean_throwError___at_Lean_registerTagAttribute___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__6; uint64_t l___private_Lean_Expr_0__Lean_hashMVarId____x40_Lean_Expr___hyg_1976_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___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_Elab_Term_MVarErrorInfo_logError_appendExtra___boxed(lean_object*, lean_object*); @@ -839,16 +840,16 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerCustomErrorIfMVar___boxed(lean LEAN_EXPORT lean_object* l_Lean_profileitM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___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_EXPORT 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*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_TermElabM_run_x27___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___boxed__const__1; LEAN_EXPORT lean_object* l_Lean_Elab_addBuiltinIncrementalElab(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkFreshBinderName___rarg___closed__1; static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___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*); uint8_t l_List_isEmpty___rarg(lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__3; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__4; static lean_object* l_Lean_Elab_Term_instMonadTermElabM___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_traceAtCmdPos(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__6; static uint8_t l_Lean_Elab_Term_collectUnassignedMVars_go___closed__1; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_mkSyntheticSorryFor___closed__1; static lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg___closed__1; @@ -875,13 +876,13 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_termElabAttribute; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplicitLambdaAux___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, 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*); uint8_t l_Lean_MessageData_hasTag(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__2; static lean_object* l_Lean_Elab_Term_instToStringSyntheticMVarKind___closed__2; static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2___lambda__2___closed__2; static lean_object* l_Lean_Elab_Tactic_instToSnapshotTreeTacticFinishedSnapshot___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_saveState___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___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* l_Lean_Name_num___override(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__1; static lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1___closed__1; LEAN_EXPORT uint8_t l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__1(uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -897,8 +898,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_liftLevelM___rarg___boxed(lean_object* LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__1(lean_object*); lean_object* l_Lean_RBNode_insert___at_Lean_MVarIdMap_insert___spec__1___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeRevMAux___at_Lean_Elab_Term_resolveLocalName___spec__9___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__6; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___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_Elab_Term_instMonadTermElabM___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -912,6 +911,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_dropTermPa static lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___rarg___closed__12; lean_object* lean_io_mono_nanos_now(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeRevM_x3f___at_Lean_Elab_Term_resolveLocalName___spec__7___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19797_(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabUsingElabFns(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_Term_MVarErrorInfo_logError___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Term_LevelMVarErrorInfo_logError___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -939,7 +939,7 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_tryPostponeIfHasM LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabUsingElabFns___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20103_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Option_set___at_Lean_Elab_Term_withoutMacroStackAtErr___spec__1(lean_object*, lean_object*, uint8_t); uint64_t l_Lean_Expr_hash(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -950,7 +950,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_expandDecl uint8_t l_Lean_BinderInfo_isInstImplicit(uint8_t); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withDeclName___spec__13(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* l_Lean_mkAnnotation(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withLogging___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instToStringSyntheticMVarKind(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -992,6 +991,8 @@ lean_object* l_Lean_RBNode_insert___at_Lean_FVarIdMap_insert___spec__1___rarg(le LEAN_EXPORT lean_object* l_Lean_Elab_isIncrementalElab___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_decorateErrorMessageWithLambdaImplicitVars___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__4; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__7; LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__2(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__24(lean_object*, lean_object*, size_t, size_t); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__3___closed__2; @@ -1009,12 +1010,14 @@ extern lean_object* l_Lean_warningAsError; static lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars___closed__1; extern lean_object* l_Lean_Elab_pp_macroStack; static lean_object* l_Lean_Elab_Term_mkConst___lambda__1___closed__2; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadTermElabM___lambda__1(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_Elab_Term_0__Lean_Elab_Term_isNoImplicitLambda(lean_object*); static lean_object* l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__10; LEAN_EXPORT lean_object* l_Lean_Elab_Term_isSaveInfoAnnotation_x3f___boxed(lean_object*); lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__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*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__1; static lean_object* l_Lean_Elab_Term_TermElabM_toIO___rarg___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Term_expandDeclId___spec__7___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_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__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*); @@ -1059,6 +1062,7 @@ extern lean_object* l_Lean_diagnostics; uint8_t l_Lean_Syntax_isIdent(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplicitLambdaAux(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_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__9(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_Term___hyg_17313____closed__10; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_resolveId_x3f___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_Term_postponeElabTerm(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_anyMAux___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__46___boxed(lean_object*, lean_object*); @@ -1066,6 +1070,7 @@ lean_object* l_Lean_LocalDecl_fvarId(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTacticBlock___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2___lambda__2___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_postponeElabTerm___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_initFn____x40_Lean_Elab_Term___hyg_19771_(lean_object*); extern lean_object* l_Lean_Elab_abortTermExceptionId; LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_ensureType___spec__1___rarg(lean_object*); static lean_object* l_Lean_Elab_Term_resolveId_x3f___lambda__2___closed__3; @@ -1074,9 +1079,8 @@ LEAN_EXPORT lean_object* l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandD LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutMacroStackAtErr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkTacticMVar(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_withoutErrToSorry___rarg___closed__1; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__3; static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_exposeLevelMVars___spec__7___rarg___closed__4; -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__2; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__12; uint8_t l_Lean_LocalDecl_isAuxDecl(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveLocalName_go___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Term_resolveLocalName_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1109,16 +1113,15 @@ LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTacticBlock(l LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__34(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_containsPendingMVar___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__2; static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Term_mkCoe___spec__1___lambda__3___closed__2; uint8_t l_Lean_PersistentHashMap_contains___at_Lean_MVarId_isAssigned___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__7; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__4___lambda__1(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_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_instToSnapshotTreeTacticParsedSnapshot_go___spec__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_resolveName_process___closed__3; static lean_object* l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2___lambda__2___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MVarId_assign___at_Lean_Elab_Term_exprToSyntax___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_initFn____x40_Lean_Elab_Term___hyg_19811____closed__4; static lean_object* l_Lean_Elab_Term_throwErrorIfErrors___closed__2; LEAN_EXPORT lean_object* l_Lean_addDocString_x27___at_Lean_Elab_Term_expandDeclId___spec__8(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_resolveName_process___closed__1; @@ -1131,7 +1134,6 @@ LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyMAux___at_Lean_Elab_Term_addAutoBo uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); static size_t l_Lean_Elab_Term_instInhabitedMVarErrorKind___closed__5; static lean_object* l_List_forIn_loop___at_Lean_Elab_Term_logUnassignedLevelMVarsUsingErrorInfos___spec__4___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627_(lean_object*); extern lean_object* l_Lean_inheritedTraceOptions; LEAN_EXPORT lean_object* l_Lean_Elab_isIncrementalElab___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_exposeLevelMVars___spec__7(lean_object*); @@ -1142,6 +1144,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_exposeLevelMVars___spec__7___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_profileitM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__11(lean_object*); lean_object* l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_addAutoBoundImplicits_go(lean_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_findSomeRevM_x3f_find___at_Lean_Elab_Term_resolveLocalName___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTypeAscription___closed__1; @@ -1164,7 +1167,9 @@ static lean_object* l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___sp LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withDeclName___spec__12(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_Term_withAutoBoundImplicit___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___closed__1; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkConst___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_initFn____x40_Lean_Elab_Term___hyg_19617____closed__8; static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwTypeMismatchError___spec__1(lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isHole___closed__1; @@ -1177,7 +1182,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_ensureHasType(lean_object*, lean_objec lean_object* l_Lean_LocalDecl_userName(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_addTermInfo___lambda__1(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*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTacticBlock___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__11(lean_object*, 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_MVarErrorInfo_logError_appendExtra(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_setElabConfig(lean_object*); @@ -1185,6 +1189,7 @@ static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_decorateErrorMe LEAN_EXPORT lean_object* l_Lean_log___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__9___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_Term_registerMVarErrorHoleInfo(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_exposeLevelMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__5; static lean_object* l_Lean_Elab_Tactic_instInhabitedTacticFinishedSnapshot___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkTermElabAttributeUnsafe(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1194,6 +1199,7 @@ static lean_object* l_Lean_Elab_Term_instMonadBacktrackSavedStateTermElabM___clo extern lean_object* l_Lean_Linter_deprecatedAttr; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadMacroAdapterTermElabM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Core_interruptExceptionId; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___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_Linter_checkDeprecated___at_Lean_Elab_Term_mkConst___spec__3___closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Term_isSaveInfoAnnotation_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1201,6 +1207,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Lean_Elab_Term_resolveLocalName___spec__8(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__1; static lean_object* l_Lean_Elab_Term_resolveName___closed__4; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__7; LEAN_EXPORT 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*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_mkAuxName___spec__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_Term_0__Lean_Elab_Term_applyAttributesCore___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*); @@ -1212,7 +1219,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_throwTypeMismatchError(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkCoe___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_Elab_Term_mkFreshIdent___rarg___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*); static lean_object* l_Lean_Elab_Term_mkCoe___closed__1; -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__3; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__6; lean_object* l_Lean_instAddErrorMessageContextOfAddMessageContextOfMonad___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Lean_Elab_Term_resolveLocalName___spec__6___boxed(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_Elab_Term_addAutoBoundImplicits_go___spec__22(lean_object*, lean_object*); @@ -1222,7 +1229,6 @@ static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError___lambda__1___closed static double l_Lean_addTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__2___closed__1; static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Term_mkCoe___spec__1___lambda__4___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_universeConstraintsCheckpoint___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19758_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadMacroAdapterTermElabM___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Name_hasMacroScopes(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isNoImplicitLambda___boxed(lean_object*); @@ -1248,7 +1254,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadTermElabM___lambda__1___boxed static lean_object* l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapM___at_Lean_Elab_Term_withDeclName___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_Elab_Term_collectUnassignedMVars(lean_object*, 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_initFn____x40_Lean_Elab_Term___hyg_19732____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__11; uint8_t l_Lean_Name_isAtomic(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instInhabitedTermElabM___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1324,10 +1329,10 @@ static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_exposeLevelMVa static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_expandDeclId___spec__4___closed__4; lean_object* l_Lean_ParametricAttribute_getParam_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_CommandContextInfo_save___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__2___boxed(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_Term___hyg_17313_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_saveState___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_indentExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Term_mkCoe___spec__1___lambda__2___boxed(lean_object**); -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_BinderInfo_isExplicit(uint8_t); static lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___rarg___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instInhabitedTacticFinishedSnapshot; @@ -1336,6 +1341,7 @@ static lean_object* l_Lean_Linter_checkDeprecated___at_Lean_Elab_Term_mkConst___ static lean_object* l_Lean_Elab_Term_exposeLevelMVars___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__14(lean_object*, 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_Lean_Elab_Term_isLetRecAuxMVar___lambda__3___closed__1; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__5; LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__12(lean_object*, lean_object*, 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_Elab_Term_addAutoBoundImplicits_go___spec__3___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_isLetRecAuxMVar___closed__1; @@ -1367,10 +1373,9 @@ static lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instInhabitedMVarErrorInfo; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isExplicit___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName(lean_object*, 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_initFn____x40_Lean_Elab_Term___hyg_19771____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__13___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__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_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__4; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__10; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Term_logUnassignedLevelMVarsUsingErrorInfos___spec__4___lambda__1(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_Term_mkCoe___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_getDelayedMVarRoot___at_Lean_Elab_Term_isLetRecAuxMVar___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1406,7 +1411,6 @@ LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTypeAscriptio static lean_object* l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_exposeLevelMVars___spec__7___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__3; static lean_object* l_Lean_Elab_Term_throwTypeMismatchError___rarg___closed__1; lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectLevelMVars_visitExpr___spec__2(lean_object*); static lean_object* l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__3; @@ -1432,6 +1436,7 @@ lean_object* lean_nat_mul(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withDeclName___spec__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_Elab_Term_registerLevelMVarErrorExprInfo(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_resetMessageLog(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__2; static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_exposeLevelMVars___spec__7___rarg___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars(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_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1454,6 +1459,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveName___lambda__2___boxed(lean_o LEAN_EXPORT lean_object* l_Lean_Elab_Term_checkDeprecated___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_Term_tryPostponeIfHasMVars_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Elab_Term_ContainsPendingMVar_visit___spec__2___boxed(lean_object*, lean_object*); uint8_t l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withInfoContext_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1499,6 +1505,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkCoe(lean_object*, lean_object*, lean static lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars___closed__6; lean_object* l_Lean_registerBuiltinAttribute(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwPostpone___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_incrementalAttr; LEAN_EXPORT lean_object* l_Lean_Elab_Term_saveState___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_useImplicitLambda___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1507,7 +1514,6 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_resolveName_x27__ static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2___closed__1; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isNoImplicitLambda___closed__1; static lean_object* l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811_(lean_object*); lean_object* l_List_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Term_withMacroExpansion___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_Term_withAuxDecl___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1519,19 +1525,20 @@ lean_object* l___private_Lean_ToExpr_0__Lean_Name_toExprAux(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerLevelMVarErrorInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withNarrowedArgTacticReuse___rarg___lambda__1(lean_object*, lean_object*); lean_object* l___private_Lean_MonadEnv_0__Lean_mkAuxNameAux(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instBEqCacheKey; static lean_object* l_List_foldl___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__2___closed__1; static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadParentDeclTermElabM; static lean_object* l_Lean_Elab_Term_extraMsgToMsg___closed__1; size_t lean_usize_sub(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__47(lean_object*, lean_object*, size_t, size_t); lean_object* l_Lean_PersistentArray_get_x21___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__9; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTypeAscription___lambda__1___boxed(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__15(lean_object*, lean_object*, size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666_(lean_object*); static lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_observing___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_find___at_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___spec__1___boxed(lean_object*, lean_object*); @@ -1567,7 +1574,6 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImpli uint8_t l_Lean_Expr_hasFVar(lean_object*); static lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___rarg___closed__8; static lean_object* l_Lean_Elab_isIncrementalElab___rarg___lambda__3___closed__1; -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__9; LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__11(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_withRestoreOrSaveFull___rarg___closed__6; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTypeAscription___closed__4; @@ -1576,16 +1582,13 @@ LEAN_EXPORT lean_object* l_Lean_logAt___at___private_Lean_Elab_Term_0__Lean_Elab static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__7___closed__1; lean_object* l_Lean_MessageLog_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_withAutoBoundImplicit_loop___spec__1___rarg(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_Term___hyg_17274____closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instInhabitedTacticParsedSnapshotData(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__2(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveName___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*); uint8_t l_Lean_Level_isMVar(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__4___rarg___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_initFn____x40_Lean_Elab_Term___hyg_19811____closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withLevelNames___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_Term_mkExplicitBinder___closed__2; -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__1; LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Term_isExplicitApp(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_throwMVarError___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_resolveName_x27___closed__2; @@ -1598,6 +1601,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_addTermInfo(lean_object*, lean_object* static lean_object* l_Lean_Core_transform___at_Lean_Elab_Term_exposeLevelMVars___spec__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_extraMsgToMsg(lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTermCore___closed__1; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__2; extern lean_object* l_Lean_trace_profiler; LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2___lambda__3(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_Elab_Term_withoutErrToSorry___rarg(lean_object*, lean_object*); @@ -1633,7 +1637,6 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBound lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAux___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_localDeclDependsOn___at_Lean_Elab_Term_addAutoBoundImplicits_go___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_Lean_Elab_Term_withRestoreOrSaveFull___rarg___closed__17; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__14; extern lean_object* l_Lean_KVMap_empty; LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapMAux___at_Lean_Elab_Term_withDeclName___spec__10(lean_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_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -1691,7 +1694,6 @@ LEAN_EXPORT lean_object* l_Lean_PersistentArray_mapM___at_Lean_Elab_Term_without uint8_t lean_usize_dec_lt(size_t, size_t); static lean_object* l_Lean_Elab_Term_exposeLevelMVars___lambda__1___closed__1; lean_object* l_Lean_RBNode_find___at_Lean_NameMap_find_x3f___spec__1___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withAuxDecl___rarg___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_findSomeRevM_x3f_find___at_Lean_Elab_Term_resolveLocalName___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeRevMAux___at_Lean_Elab_Term_resolveLocalName___spec__9(lean_object*, lean_object*); @@ -1701,22 +1703,24 @@ LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Lean_Elab_Term_resol LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__13(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_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__4___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_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2___closed__4; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__2; lean_object* l_Lean_getExprMVarAssignment_x3f___at___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_getResetInfoTrees___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__5___rarg___boxed(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* l_Lean_realizeGlobalName(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20103____closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withAutoBoundImplicitForbiddenPred___rarg___lambda__1(lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__13; static lean_object* l_Lean_Elab_Term_instToStringSyntheticMVarKind___closed__1; static lean_object* l_Lean_Elab_Term_getInfoTreeWithContext_x3f___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_withMacroExpansionInfo___at_Lean_Elab_Term_withMacroExpansion___spec__1(lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instInhabitedMVarErrorKind; LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_withAutoBoundImplicit_loop___spec__1(lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__15; LEAN_EXPORT lean_object* l_Lean_Elab_Term_observing(lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__1; uint8_t l_Lean_Exception_isRuntime(lean_object*); lean_object* l_Lean_Expr_lam___override(lean_object*, lean_object*, lean_object*, uint8_t); static lean_object* l_Lean_Elab_Term_exposeLevelMVars___lambda__2___closed__5; @@ -1730,7 +1734,6 @@ LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_v LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2___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_Term_0__Lean_Elab_Term_mkConsts___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_Term_withNarrowedArgTacticReuse___rarg(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_Term___hyg_10627____closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_Elab_Term_addDotCompletionInfo___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTacticBlock___closed__3; static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError___lambda__1___closed__6; @@ -1741,7 +1744,6 @@ uint8_t l_Lean_Expr_isFVar(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_exprToSyntax___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_Elab_InfoTree_Main_0__Lean_Elab_withSavedPartialInfoContext___at_Lean_Elab_Term_withDeclName___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_Term_SavedState_restore___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_initFn____x40_Lean_Elab_Term___hyg_19578____closed__3; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__7___closed__2; static lean_object* l_Lean_Elab_Term_expandDeclId___closed__2; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabUsingElabFns___closed__1; @@ -1758,17 +1760,19 @@ lean_object* l_Lean_getStructureFieldsFlattened(lean_object*, lean_object*, uint lean_object* l_Lean_Expr_mvarId_x21(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplicitLambda_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_EXPORT lean_object* l_Lean_Elab_throwPostpone___at_Lean_Elab_Term_tryPostpone___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___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_Lean_addDocString_x27___at_Lean_Elab_Term_expandDeclId___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_Elab_Term_instInhabitedState___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg(lean_object*); uint8_t l_Lean_Elab_isValidAutoBoundImplicitName(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Core_withIncRecDepth___at_Lean_Elab_Term_exposeLevelMVars___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Attribute_Builtin_ensureNoArgs___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__6; LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__10___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_throwAutoBoundImplicitLocal___at_Lean_Elab_Term_resolveName_process___spec__1___closed__2; lean_object* l_String_toSubstring_x27(lean_object*); LEAN_EXPORT lean_object* l_Lean_getDelayedMVarAssignment_x3f___at_Lean_Elab_Term_ContainsPendingMVar_visit___spec__4(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_Term___hyg_17313____closed__8; static lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___lambda__3___closed__4; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__9(lean_object*, 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_Lean_Elab_Term_mkCoe___lambda__2___closed__2; @@ -1793,6 +1797,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_tryPostpone(lean_object*, lean_object* lean_object* l_List_filterTR_loop___at_Lean_filterFieldList___spec__1(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyMAux___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__38(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Lean_Elab_Term_resolveLocalName___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Message_0__Lean_beqMessageSeverity____x40_Lean_Message___hyg_106_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Term_removeSaveInfoAnnotation(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___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*); @@ -1800,13 +1805,11 @@ static lean_object* l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_getLetRecsToLift___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticReuse___rarg___lambda__1(uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__10___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_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__5; static lean_object* l_Lean_addDocString___at_Lean_Elab_Term_expandDeclId___spec__9___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__4___boxed(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_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__7(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_Term_registerLevelMVarErrorExprInfo___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_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Term_expandDeclId___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20064_(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_expandDeclId___spec__4___closed__5; static lean_object* l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__8; static lean_object* l_Lean_Elab_Term_mkExplicitBinder___closed__8; @@ -1830,8 +1833,8 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_debug_byAsSorry; static lean_object* l_Lean_Elab_Tactic_instToSnapshotTreeTacticParsedSnapshot_go___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_useImplicitLambda___lambda__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_Lean_Elab_Term_withAutoBoundImplicit_loop___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_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__5; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isLambdaWithImplicit___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617_(lean_object*); static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwTypeMismatchError___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_contains___at_Lean_Elab_Term_logUnassignedLevelMVarsUsingErrorInfos___spec__1(lean_object*, lean_object*); @@ -1840,7 +1843,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutTacticReuse___rarg___lambda__2( LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Term_mkCoe___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*); double lean_float_sub(double, double); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ContainsPendingMVar_visit___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578_(lean_object*); LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_hasExprMVar(lean_object*); lean_object* l_Lean_Meta_processPostponed(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -34168,15 +34170,7 @@ return x_22; } } } -static lean_object* _init_l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("attribute application", 21, 21); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___boxed__const__1() { +static lean_object* _init_l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2___boxed__const__1() { _start: { size_t x_1; lean_object* x_2; @@ -34185,6 +34179,32 @@ x_2 = lean_box_usize(x_1); return x_2; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___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: +{ +size_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_12 = lean_array_size(x_1); +x_13 = lean_box_usize(x_12); +x_14 = l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2___boxed__const__1; +lean_inc(x_2); +x_15 = lean_alloc_closure((void*)(l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__1___boxed), 12, 5); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, x_3); +lean_closure_set(x_15, 2, x_1); +lean_closure_set(x_15, 3, x_13); +lean_closure_set(x_15, 4, x_14); +x_16 = l_Lean_Elab_Term_withDeclName___rarg(x_2, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_16; +} +} +static lean_object* _init_l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("attribute application", 21, 21); +return x_1; +} +} LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, 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: { @@ -34195,34 +34215,31 @@ x_12 = lean_box(0); x_13 = lean_name_eq(x_1, x_12); if (x_13 == 0) { -size_t 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_array_size(x_2); -x_15 = lean_box_usize(x_14); -x_16 = l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___boxed__const__1; -x_17 = lean_alloc_closure((void*)(l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__1___boxed), 12, 5); -lean_closure_set(x_17, 0, x_1); -lean_closure_set(x_17, 1, x_3); -lean_closure_set(x_17, 2, x_2); -lean_closure_set(x_17, 3, x_15); -lean_closure_set(x_17, 4, x_16); -x_18 = l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___closed__1; -x_19 = l_Lean_profileitM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__11___rarg(x_18, x_11, x_17, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_box(0); +x_15 = lean_alloc_closure((void*)(l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2___boxed), 11, 4); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, x_1); +lean_closure_set(x_15, 2, x_3); +lean_closure_set(x_15, 3, x_14); +x_16 = l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___closed__1; +x_17 = l_Lean_profileitM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__11___rarg(x_16, x_11, x_15, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_11); -return x_19; +return x_17; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_20 = lean_box(0); -x_21 = lean_alloc_closure((void*)(l_ReaderT_pure___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__12___rarg___boxed), 8, 1); -lean_closure_set(x_21, 0, x_20); -x_22 = l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___closed__1; -x_23 = l_Lean_profileitM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__11___rarg(x_22, x_11, x_21, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_18 = lean_box(0); +x_19 = lean_alloc_closure((void*)(l_ReaderT_pure___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__12___rarg___boxed), 8, 1); +lean_closure_set(x_19, 0, x_18); +x_20 = l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___closed__1; +x_21 = l_Lean_profileitM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__11___rarg(x_20, x_11, x_19, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_11); -return x_23; +return x_21; } } } @@ -34415,6 +34432,15 @@ lean_dec(x_3); return x_15; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___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___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___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); +return x_12; +} +} LEAN_EXPORT lean_object* l_Lean_Elab_Term_applyAttributesAt(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) { _start: { @@ -45448,7 +45474,7 @@ lean_dec(x_1); return x_9; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__1() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__1() { _start: { lean_object* x_1; @@ -45456,7 +45482,7 @@ x_1 = lean_mk_string_unchecked("debug", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__2() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__2() { _start: { lean_object* x_1; @@ -45464,17 +45490,17 @@ x_1 = lean_mk_string_unchecked("byAsSorry", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__3() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____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_Term___hyg_10627____closed__1; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__2; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__1; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__2; 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_Term___hyg_10627____closed__4() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__4() { _start: { lean_object* x_1; @@ -45482,13 +45508,13 @@ x_1 = lean_mk_string_unchecked("replace `by ..` blocks with `sorry` IF the expec return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__5() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____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_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__1; -x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__4; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__1; +x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__4; x_4 = lean_box(x_1); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_4); @@ -45497,26 +45523,26 @@ lean_ctor_set(x_5, 2, x_3); return x_5; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__6() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____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; x_1 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__5; x_2 = l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__2; x_3 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__7; -x_4 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__1; -x_5 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__2; +x_4 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__1; +x_5 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____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_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666_(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_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__3; -x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__5; -x_4 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__6; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__3; +x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__5; +x_4 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__6; 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; } @@ -68129,7 +68155,7 @@ lean_dec(x_3); return x_9; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__1() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__1() { _start: { lean_object* x_1; @@ -68137,17 +68163,17 @@ x_1 = lean_mk_string_unchecked("letrec", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__2() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__2; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__1; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__1; 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_Term___hyg_17274____closed__3() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -68157,27 +68183,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_Term___hyg_17274____closed__4() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____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_Term___hyg_17274____closed__3; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__3; x_2 = l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__2; 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_Term___hyg_17274____closed__5() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__4; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__4; x_2 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___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_Term___hyg_17274____closed__6() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__6() { _start: { lean_object* x_1; @@ -68185,17 +68211,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_Term___hyg_17274____closed__7() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__5; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__6; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__5; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__6; 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_Term___hyg_17274____closed__8() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__8() { _start: { lean_object* x_1; @@ -68203,47 +68229,47 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__9() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____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_Term___hyg_17274____closed__7; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__8; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__7; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__8; 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_Term___hyg_17274____closed__10() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____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_Term___hyg_17274____closed__9; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__9; x_2 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___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_Term___hyg_17274____closed__11() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__10; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__10; x_2 = l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__2; 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_Term___hyg_17274____closed__12() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____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_Term___hyg_17274____closed__11; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__11; x_2 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___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_Term___hyg_17274____closed__13() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__13() { _start: { lean_object* x_1; @@ -68251,33 +68277,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_Term___hyg_17274____closed__14() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____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_Term___hyg_17274____closed__12; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__13; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__12; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____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_Term___hyg_17274____closed__15() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____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_Term___hyg_17274____closed__14; -x_2 = lean_unsigned_to_nat(17274u); +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__14; +x_2 = lean_unsigned_to_nat(17313u); 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_Term___hyg_17274_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313_(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_Term___hyg_17274____closed__2; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__2; x_3 = 0; -x_4 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__15; +x_4 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__15; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -68684,7 +68710,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_isLetRecAuxMVar(lean_object* x_1, lean _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_9 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__2; +x_9 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__2; x_10 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_traceAtCmdPos___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); @@ -76094,7 +76120,7 @@ lean_object* x_14; uint8_t x_15; lean_object* x_16; x_14 = lean_ctor_get(x_13, 1); lean_inc(x_14); lean_dec(x_13); -x_15 = lean_ctor_get_uint8(x_2, sizeof(void*)*2); +x_15 = lean_ctor_get_uint8(x_2, sizeof(void*)*3); lean_inc(x_6); x_16 = l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___spec__5(x_15, x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_14); if (lean_obj_tag(x_16) == 0) @@ -77154,7 +77180,7 @@ lean_inc(x_32); x_33 = lean_ctor_get(x_30, 1); lean_inc(x_33); lean_dec(x_30); -x_34 = lean_ctor_get(x_3, 0); +x_34 = lean_ctor_get(x_3, 1); lean_inc(x_34); lean_dec(x_3); lean_inc(x_32); @@ -78495,87 +78521,87 @@ x_3 = lean_alloc_closure((void*)(l_Lean_Elab_withoutModifyingStateWithInfoAndMes return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__1() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__4; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__6; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__4; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__2() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__1; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__8; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__1; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__8; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__3() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__2; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__2; x_2 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__4() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__3; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__3; x_2 = l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__5() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__4; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__4; x_2 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__6() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__5; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__13; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__5; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__13; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__7() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__6; -x_2 = lean_unsigned_to_nat(19578u); +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__6; +x_2 = lean_unsigned_to_nat(19617u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__8() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__2; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__1; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__1; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__9() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -78585,13 +78611,13 @@ x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617_(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_Elab_Term_0__Lean_Elab_Term_postponeElabTermCore___closed__2; x_3 = 0; -x_4 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__7; +x_4 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__7; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); if (lean_obj_tag(x_5) == 0) { @@ -78607,7 +78633,7 @@ lean_object* x_9; lean_object* x_10; lean_object* x_11; x_9 = lean_ctor_get(x_8, 1); lean_inc(x_9); lean_dec(x_8); -x_10 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__8; +x_10 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__8; x_11 = l_Lean_registerTraceClass(x_10, x_3, x_4, x_9); if (lean_obj_tag(x_11) == 0) { @@ -78615,7 +78641,7 @@ lean_object* x_12; lean_object* x_13; lean_object* x_14; x_12 = lean_ctor_get(x_11, 1); lean_inc(x_12); lean_dec(x_11); -x_13 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__9; +x_13 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__9; x_14 = l_Lean_registerTraceClass(x_13, x_3, x_4, x_12); return x_14; } @@ -78689,7 +78715,7 @@ return x_26; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____lambda__1(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; @@ -78700,7 +78726,7 @@ lean_ctor_set(x_6, 1, x_4); return x_6; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__1() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__1() { _start: { lean_object* x_1; @@ -78708,17 +78734,17 @@ x_1 = lean_mk_string_unchecked("incremental", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__2() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____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_initFn____x40_Lean_Elab_Term___hyg_19732____closed__1; +x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__3() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__3() { _start: { lean_object* x_1; @@ -78726,18 +78752,18 @@ x_1 = lean_mk_string_unchecked("incrementalAttr", 15, 15); return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__4() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__5; x_2 = l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__2; -x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__3; +x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__3; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__5() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__5() { _start: { lean_object* x_1; @@ -78745,39 +78771,39 @@ x_1 = lean_mk_string_unchecked("Marks an elaborator (tactic or command, currentl return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__6() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__6() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____lambda__1___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____lambda__1___boxed), 4, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; uint8_t x_6; lean_object* x_7; -x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__2; -x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__5; -x_4 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__6; -x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__4; +x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__2; +x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__5; +x_4 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__6; +x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__4; x_6 = 0; x_7 = l_Lean_registerTagAttribute(x_2, x_3, x_4, x_5, x_6, x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____lambda__1___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_initFn____x40_Lean_Elab_Term___hyg_19732____lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19758_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19797_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; uint8_t x_4; @@ -78845,7 +78871,7 @@ return x_13; } } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -78853,40 +78879,40 @@ x_1 = lean_mk_string_unchecked("addBuiltinIncrementalElab", 25, 25); return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__5; x_2 = l_Lean_Elab_Term_withoutTacticIncrementality___rarg___lambda__3___closed__2; -x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__1; +x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____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_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____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_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__2; +x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____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_initFn____x40_Lean_Elab_Term___hyg_19811____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_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____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; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_inc(x_1); x_6 = l___private_Lean_ToExpr_0__Lean_Name_toExprAux(x_1); -x_7 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__3; +x_7 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__3; x_8 = l_Lean_Expr_app___override(x_7, x_6); x_9 = l_Lean_declareBuiltin(x_1, x_8, x_3, x_4, x_5); return x_9; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__1() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__1() { _start: { lean_object* x_1; @@ -78894,16 +78920,16 @@ x_1 = lean_mk_string_unchecked("invalid attribute 'builtin_incremental', must be return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__2() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__1; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2(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_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2(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; @@ -78921,7 +78947,7 @@ if (x_10 == 0) { 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_19811____lambda__2___closed__2; +x_11 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____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_4); x_13 = !lean_is_exclusive(x_12); @@ -78947,7 +78973,7 @@ 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_19811____lambda__1(x_1, x_17, x_4, x_5, x_8); +x_18 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1(x_1, x_17, x_4, x_5, x_8); lean_dec(x_4); return x_18; } @@ -78978,7 +79004,7 @@ return x_22; } } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__1() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__1() { _start: { lean_object* x_1; @@ -78986,35 +79012,35 @@ x_1 = lean_mk_string_unchecked("attribute cannot be erased", 26, 26); return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__2() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__1; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3(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_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__2; +x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___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_initFn____x40_Lean_Elab_Term___hyg_19811____closed__1() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__6; -x_2 = lean_unsigned_to_nat(19811u); +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__6; +x_2 = lean_unsigned_to_nat(19850u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__2() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__2() { _start: { lean_object* x_1; @@ -79022,17 +79048,17 @@ x_1 = lean_mk_string_unchecked("builtin_incremental", 19, 19); return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__3() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____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_initFn____x40_Lean_Elab_Term___hyg_19811____closed__2; +x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__4() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__4() { _start: { lean_object* x_1; @@ -79040,7 +79066,7 @@ x_1 = lean_mk_string_unchecked("(builtin) ", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__5() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____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; @@ -79053,29 +79079,29 @@ lean_dec(x_2); x_4 = lean_ctor_get(x_3, 2); lean_inc(x_4); lean_dec(x_3); -x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__4; +x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__4; x_6 = lean_string_append(x_5, x_4); lean_dec(x_4); return x_6; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__6() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__5; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__5; x_2 = l_Lean_Elab_Term_extraMsgToMsg___closed__3; x_3 = lean_string_append(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__7() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__7() { _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_initFn____x40_Lean_Elab_Term___hyg_19811____closed__1; -x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__3; -x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__6; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__1; +x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__3; +x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__6; x_4 = 1; x_5 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_5, 0, x_1); @@ -79085,29 +79111,29 @@ lean_ctor_set_uint8(x_5, sizeof(void*)*3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__8() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__8() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___boxed), 6, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___boxed), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__9() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__9() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___boxed), 4, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__10() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__7; -x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__8; -x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__9; +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__7; +x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__8; +x_3 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__9; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -79115,42 +79141,42 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__10; +x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__10; x_3 = l_Lean_registerBuiltinAttribute(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____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_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____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_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____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_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____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_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____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: { 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_19811____lambda__2(x_1, x_2, x_7, x_4, x_5, x_6); +x_8 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2(x_1, x_2, x_7, x_4, x_5, x_6); lean_dec(x_5); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___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_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); @@ -79327,23 +79353,23 @@ x_7 = l_Lean_Elab_isIncrementalElab___rarg___lambda__4(x_1, x_2, x_3, x_4, x_6); return x_7; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20064____closed__1() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20103____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__6; -x_2 = lean_unsigned_to_nat(20064u); +x_1 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__6; +x_2 = lean_unsigned_to_nat(20103u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20064_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20103_(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_Elab_Term_0__Lean_Elab_Term_elabImplicitLambdaAux___closed__2; x_3 = 0; -x_4 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20064____closed__1; +x_4 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20103____closed__1; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -79821,10 +79847,10 @@ l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAt lean_mark_persistent(l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__7___closed__2); l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__7___closed__3 = _init_l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__7___closed__3(); lean_mark_persistent(l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__7___closed__3); +l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2___boxed__const__1 = _init_l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2___boxed__const__1(); +lean_mark_persistent(l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___lambda__2___boxed__const__1); l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___closed__1 = _init_l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___closed__1); -l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___boxed__const__1 = _init_l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___boxed__const__1(); -lean_mark_persistent(l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___boxed__const__1); l_Lean_Elab_Term_mkTypeMismatchError___closed__1 = _init_l_Lean_Elab_Term_mkTypeMismatchError___closed__1(); lean_mark_persistent(l_Lean_Elab_Term_mkTypeMismatchError___closed__1); l_Lean_Elab_Term_mkTypeMismatchError___closed__2 = _init_l_Lean_Elab_Term_mkTypeMismatchError___closed__2(); @@ -79929,19 +79955,19 @@ l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTermCore___closed__4 = lean_mark_persistent(l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTermCore___closed__4); l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTermCore___closed__5 = _init_l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTermCore___closed__5(); lean_mark_persistent(l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTermCore___closed__5); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__1(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__1); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__2(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__2); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__3 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__3(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__3); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__4 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__4(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__4); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__5 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__5(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__5); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__6 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__6(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627____closed__6); -if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10627_(lean_io_mk_world()); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__1(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__1); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__2(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__2); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__3 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__3(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__3); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__4 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__4(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__4); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__5 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__5(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__5); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__6 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__6(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666____closed__6); +if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_10666_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Elab_Term_debug_byAsSorry = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_Term_debug_byAsSorry); @@ -80101,37 +80127,37 @@ l_Lean_Elab_Term_mkAuxName___closed__1 = _init_l_Lean_Elab_Term_mkAuxName___clos lean_mark_persistent(l_Lean_Elab_Term_mkAuxName___closed__1); l_Lean_Elab_Term_mkAuxName___closed__2 = _init_l_Lean_Elab_Term_mkAuxName___closed__2(); lean_mark_persistent(l_Lean_Elab_Term_mkAuxName___closed__2); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__1(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__1); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__2(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__2); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__3 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__3(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__3); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__4 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__4(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__4); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__5 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__5(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__5); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__6 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__6(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__6); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__7 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__7(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__7); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__8 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__8(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__8); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__9 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__9(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__9); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__10 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__10(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__10); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__11 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__11(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__11); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__12 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__12(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__12); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__13 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__13(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__13); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__14 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__14(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__14); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__15 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__15(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274____closed__15); -if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17274_(lean_io_mk_world()); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__1(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__1); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__2(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__2); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__3 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__3(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__3); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__4 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__4(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__4); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__5 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__5(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__5); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__6 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__6(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__6); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__7 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__7(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__7); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__8 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__8(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__8); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__9 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__9(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__9); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__10 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__10(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__10); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__11 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__11(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__11); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__12 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__12(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__12); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__13 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__13(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__13); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__14 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__14(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__14); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__15 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__15(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313____closed__15); +if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_17313_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Lean_Elab_Term_isLetRecAuxMVar___lambda__3___closed__1 = _init_l_Lean_Elab_Term_isLetRecAuxMVar___lambda__3___closed__1(); @@ -80290,95 +80316,95 @@ l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__3 = _init_l_Lean_Elab_Term_e lean_mark_persistent(l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__3); l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__4 = _init_l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__4(); lean_mark_persistent(l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__4); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__1(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__1); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__2(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__2); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__3 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__3(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__3); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__4 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__4(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__4); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__5 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__5(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__5); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__6 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__6(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__6); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__7 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__7(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__7); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__8 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__8(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__8); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__9 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__9(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578____closed__9); -if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19578_(lean_io_mk_world()); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__1(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__1); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__2(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__2); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__3 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__3(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__3); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__4 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__4(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__4); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__5 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__5(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__5); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__6 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__6(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__6); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__7 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__7(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__7); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__8 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__8(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__8); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__9 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__9(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617____closed__9); +if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19617_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__1(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__1); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__2(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__2); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__3 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__3(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__3); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__4 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__4(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__4); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__5 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__5(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__5); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__6 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__6(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732____closed__6); -if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19732_(lean_io_mk_world()); +}l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__1(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__1); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__2(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__2); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__3 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__3(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__3); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__4 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__4(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__4); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__5 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__5(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__5); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__6 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__6(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771____closed__6); +if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19771_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Elab_incrementalAttr = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_incrementalAttr); lean_dec_ref(res); -}if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19758_(lean_io_mk_world()); +}if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19797_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Elab_builtinIncrementalElabs = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_builtinIncrementalElabs); lean_dec_ref(res); }l_Lean_Elab_addBuiltinIncrementalElab___closed__1 = _init_l_Lean_Elab_addBuiltinIncrementalElab___closed__1(); lean_mark_persistent(l_Lean_Elab_addBuiltinIncrementalElab___closed__1); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__1); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__2); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__3 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__1___closed__3); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__1); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__2___closed__2); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__1); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____lambda__3___closed__2); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__1(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__1); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__2(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__2); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__3 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__3(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__3); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__4 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__4(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__4); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__5 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__5(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__5); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__6 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__6(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__6); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__7 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__7(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__7); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__8 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__8(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__8); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__9 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__9(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__9); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__10 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__10(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811____closed__10); -if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19811_(lean_io_mk_world()); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__1); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__2); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__3 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__1___closed__3); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__1); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__2___closed__2); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__1); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____lambda__3___closed__2); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__1(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__1); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__2(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__2); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__3 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__3(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__3); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__4 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__4(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__4); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__5 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__5(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__5); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__6 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__6(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__6); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__7 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__7(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__7); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__8 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__8(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__8); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__9 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__9(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__9); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__10 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__10(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850____closed__10); +if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_19850_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Lean_Elab_isIncrementalElab___rarg___lambda__3___closed__1 = _init_l_Lean_Elab_isIncrementalElab___rarg___lambda__3___closed__1(); lean_mark_persistent(l_Lean_Elab_isIncrementalElab___rarg___lambda__3___closed__1); l_Lean_Elab_isIncrementalElab___rarg___closed__1 = _init_l_Lean_Elab_isIncrementalElab___rarg___closed__1(); lean_mark_persistent(l_Lean_Elab_isIncrementalElab___rarg___closed__1); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20064____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20064____closed__1(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20064____closed__1); -if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20064_(lean_io_mk_world()); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20103____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20103____closed__1(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20103____closed__1); +if (builtin) {res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20103_(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/Language/Basic.c b/stage0/stdlib/Lean/Language/Basic.c index 36aad633d8d7..e42c30ce744c 100644 --- a/stage0/stdlib/Lean/Language/Basic.c +++ b/stage0/stdlib/Lean/Language/Basic.c @@ -24,7 +24,6 @@ LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Language_SnapshotTree_tr lean_object* l_Lean_Json_compress(lean_object*); extern lean_object* l_Lean_profiler; LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Language_SnapshotTree_trace_go___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__5; LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTask_cancel___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Language_withAlwaysResolvedPromises___spec__2___rarg___lambda__1___boxed(lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); @@ -66,7 +65,6 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Language_reportMess LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTask_ofIO(lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); -static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__3; static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__40; LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_toTyped_x3f(lean_object*); static lean_object* l_Lean_Language_SnapshotTree_trace_go___lambda__2___closed__1; @@ -78,6 +76,7 @@ static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__23; static lean_object* l_Lean_Language_reportMessages___closed__1; lean_object* l_Lean_Elab_InfoTree_format(lean_object*, lean_object*, lean_object*); uint8_t lean_float_decLt(double, double); +static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__4; static lean_object* l_Lean_Language_SnapshotTree_trace_go___closed__10; LEAN_EXPORT lean_object* l_Lean_Language_instToSnapshotTreeDynamicSnapshot(lean_object*); static lean_object* l_Lean_Language_SnapshotTree_trace_go___closed__6; @@ -104,7 +103,6 @@ lean_object* lean_string_utf8_byte_size(lean_object*); static lean_object* l_Lean_Language_SnapshotTree_trace_go___closed__7; LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Language_SnapshotTree_trace_go___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_withHeaderExceptions___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__1; static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__20; lean_object* l_IO_Promise_resolve___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); @@ -124,6 +122,8 @@ LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTree_runAndReport___boxed(lean_ static lean_object* l_Lean_Language_instInhabitedSnapshotTree___closed__1; static lean_object* l_Lean_Language_diagnosticsOfHeaderError___closed__1; LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTree_trace_go___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__3; +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTask_pure(lean_object*); LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Language_SnapshotTree_trace_go___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__21; @@ -161,6 +161,7 @@ lean_object* l_Lean_addMessageContextPartial___at_Lean_Core_instAddMessageContex LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Language_SnapshotTree_trace_go___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTree_forM___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Language_Snapshot_instInhabitedDiagnostics___closed__5; +static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__2; LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromise___rarg___lambda__2___boxed(lean_object*); static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__1; static lean_object* l_Lean_Language_instInhabitedDynamicSnapshot___closed__3; @@ -170,6 +171,7 @@ static lean_object* l_Lean_Language_instInhabitedDynamicSnapshot___closed__1; LEAN_EXPORT lean_object* l_Lean_PersistentArray_forMAux___at_Lean_Language_reportMessages___spec__3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Language_SnapshotTree_trace_go___closed__5; LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Language_SnapshotTree_trace_go___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_thunk_get_own(lean_object*); static double l_Lean_withTraceNode___at_Lean_Language_SnapshotTree_trace_go___spec__5___lambda__4___closed__5; LEAN_EXPORT lean_object* l_Lean_MessageLog_forM___at_Lean_Language_reportMessages___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__22; @@ -179,7 +181,6 @@ extern lean_object* l_Task_Priority_default; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Language_withAlwaysResolvedPromises___spec__2___rarg___lambda__2(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_instInhabitedSnapshotTask___rarg(lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057_(lean_object*); static lean_object* l_Lean_Language_SnapshotTree_trace_go___closed__11; static lean_object* l_Lean_Language_Snapshot_instInhabitedDiagnostics___closed__1; extern lean_object* l_Lean_MessageLog_empty; @@ -207,6 +208,7 @@ static lean_object* l_Lean_Language_instInhabitedDynamicSnapshot___closed__4; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Language_reportMessages___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromises___rarg___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_Language_mkIncrementalProcessor___elambda__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_mk_thunk(lean_object*); LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Language_SnapshotTree_trace_go___spec__5___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_Array_foldlMUnsafe_fold___at_Lean_Language_SnapshotTree_getAll___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*); lean_object* l___private_Lean_Util_Trace_0__Lean_addTraceNode___at_Lean_compileDecl___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -218,6 +220,7 @@ LEAN_EXPORT lean_object* l_Lean_Language_mkIncrementalProcessor___elambda__1(lea double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); static lean_object* l_Lean_withTraceNode___at_Lean_Language_SnapshotTree_trace_go___spec__5___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Language_SnapshotTree_getAll___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__5; static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__8; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Language_withAlwaysResolvedPromises___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Language_reportMessages___lambda__2___closed__1; @@ -225,6 +228,7 @@ LEAN_EXPORT lean_object* l_Functor_mapRev___at_Lean_Language_reportMessages___sp LEAN_EXPORT lean_object* l_Lean_MessageLog_forM___at_Lean_Language_reportMessages___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_instMonadLiftProcessingMProcessingTIO___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__4; +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Language_reportMessages___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Language_SnapshotTree_trace_go___spec__5___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_forInUnsafe_loop___at_Lean_Language_withAlwaysResolvedPromises___spec__2(lean_object*, lean_object*); @@ -238,7 +242,6 @@ lean_object* l_IO_println___at_Lean_Environment_displayStats___spec__3(lean_obje LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromise(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Language_withHeaderExceptions___rarg___closed__1; static lean_object* l_Lean_Language_SnapshotTree_trace_go___lambda__3___closed__2; -static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__2; static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__37; static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__41; LEAN_EXPORT lean_object* l_Lean_Language_withHeaderExceptions(lean_object*); @@ -246,6 +249,7 @@ uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__27; LEAN_EXPORT lean_object* l_Lean_Language_withAlwaysResolvedPromises___rarg___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__25; +static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__1; LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Language_SnapshotTree_trace_go___spec__5___lambda__2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, double, double, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_forMAux___at_Lean_Language_reportMessages___spec__3___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); @@ -275,6 +279,7 @@ lean_object* l_List_reverse___rarg(lean_object*); static lean_object* l_Lean_Language_withAlwaysResolvedPromise___rarg___closed__1; lean_object* lean_array_mk(lean_object*); static lean_object* l_Lean_Language_SnapshotTree_trace_go___closed__8; +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Language_withAlwaysResolvedPromises___spec__2___rarg___lambda__1(lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__18; @@ -287,8 +292,8 @@ extern lean_object* l_Lean_trace_profiler; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Language_withAlwaysResolvedPromises___spec__1___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTask_get___rarg(lean_object*); lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_compileDecl___spec__4___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTree_trace(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__4; LEAN_EXPORT lean_object* l_Lean_Language_mkIncrementalProcessor___elambda__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_io_error_to_string(lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); @@ -313,6 +318,7 @@ static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__32; LEAN_EXPORT lean_object* l_Std_Format_prefixJoin___at_Lean_Language_SnapshotTree_trace_go___spec__2(lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTask_bindIO___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1___lambda__1(lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); static lean_object* l___auto____x40_Lean_Language_Basic___hyg_62____closed__6; LEAN_EXPORT lean_object* l_Lean_Language_SnapshotTask_cancel(lean_object*); @@ -4984,10 +4990,10 @@ return x_3; LEAN_EXPORT lean_object* l_Lean_Language_instToSnapshotTreeDynamicSnapshot(lean_object* x_1) { _start: { -lean_object* x_2; +lean_object* x_2; lean_object* x_3; x_2 = lean_ctor_get(x_1, 1); -lean_inc(x_2); -return x_2; +x_3 = lean_thunk_get_own(x_2); +return x_3; } } LEAN_EXPORT lean_object* l_Lean_Language_instToSnapshotTreeDynamicSnapshot___boxed(lean_object* x_1) { @@ -4999,19 +5005,30 @@ lean_dec(x_1); return x_2; } } +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_apply_1(x_1, x_2); +return x_4; +} +} LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___rarg(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_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_inc(x_3); x_4 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_3); -x_5 = lean_apply_1(x_2, x_3); -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_4); -lean_ctor_set(x_6, 1, x_5); -return x_6; +x_5 = lean_alloc_closure((void*)(l_Lean_Language_DynamicSnapshot_ofTyped___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_5, 0, x_2); +lean_closure_set(x_5, 1, x_3); +x_6 = lean_mk_thunk(x_5); +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_4); +lean_ctor_set(x_7, 1, x_6); +return x_7; } } LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped(lean_object* x_1) { @@ -5022,6 +5039,15 @@ x_2 = lean_alloc_closure((void*)(l_Lean_Language_DynamicSnapshot_ofTyped___rarg) return x_2; } } +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_Language_DynamicSnapshot_ofTyped___rarg___lambda__1(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_toTyped_x3f___rarg(lean_object* x_1, lean_object* x_2) { _start: { @@ -5049,6 +5075,17 @@ lean_dec(x_1); return x_3; } } +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; +x_3 = l_Lean_addTrace___at_Lean_Language_SnapshotTree_trace_go___spec__7___closed__1; +x_4 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_3); +return x_4; +} +} LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1(lean_object* x_1, lean_object* x_2) { _start: { @@ -5057,10 +5094,9 @@ lean_inc(x_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); -x_4 = l_Lean_addTrace___at_Lean_Language_SnapshotTree_trace_go___spec__7___closed__1; -x_5 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_5, 0, x_2); -lean_ctor_set(x_5, 1, x_4); +x_4 = lean_alloc_closure((void*)(l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1___lambda__1___boxed), 2, 1); +lean_closure_set(x_4, 0, x_2); +x_5 = lean_mk_thunk(x_4); x_6 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_6, 0, x_3); lean_ctor_set(x_6, 1, x_5); @@ -5139,6 +5175,15 @@ x_3 = l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDy return x_3; } } +LEAN_EXPORT lean_object* l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Language_DynamicSnapshot_ofTyped___at_Lean_Language_instInhabitedDynamicSnapshot___spec__1___lambda__1(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} LEAN_EXPORT lean_object* l_Lean_Language_instInhabitedDynamicSnapshot___lambda__1___boxed(lean_object* x_1) { _start: { @@ -5265,7 +5310,7 @@ lean_dec(x_4); return x_5; } } -static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__1() { +static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__1() { _start: { lean_object* x_1; @@ -5273,17 +5318,17 @@ x_1 = lean_mk_string_unchecked("printMessageEndPos", 18, 18); return x_1; } } -static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__2() { +static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__1; +x_2 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__3() { +static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__3() { _start: { lean_object* x_1; @@ -5291,13 +5336,13 @@ x_1 = lean_mk_string_unchecked("print end position of each message in addition t return x_1; } } -static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__4() { +static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____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_Language_instInhabitedSnapshot___closed__1; -x_3 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__3; +x_3 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__3; x_4 = lean_box(x_1); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_4); @@ -5306,24 +5351,24 @@ lean_ctor_set(x_5, 2, x_3); return x_5; } } -static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__5() { +static lean_object* _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l___auto____x40_Lean_Language_Basic___hyg_62____closed__1; x_2 = l_Lean_Language_instImpl____x40_Lean_Language_Basic___hyg_1850____closed__1; -x_3 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__1; +x_3 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058_(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_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__2; -x_3 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__4; -x_4 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__5; +x_2 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__2; +x_3 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__4; +x_4 = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__5; x_5 = l_Lean_Option_register___at_Lean_initFn____x40_Lean_Util_Profile___hyg_5____spec__1(x_2, x_3, x_4, x_1); return x_5; } @@ -7162,17 +7207,17 @@ l_Lean_Language_instInhabitedDynamicSnapshot___closed__5 = _init_l_Lean_Language lean_mark_persistent(l_Lean_Language_instInhabitedDynamicSnapshot___closed__5); l_Lean_Language_instInhabitedDynamicSnapshot = _init_l_Lean_Language_instInhabitedDynamicSnapshot(); lean_mark_persistent(l_Lean_Language_instInhabitedDynamicSnapshot); -l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__1 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__1(); -lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__1); -l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__2 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__2(); -lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__2); -l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__3 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__3(); -lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__3); -l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__4 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__4(); -lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__4); -l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__5 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__5(); -lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057____closed__5); -if (builtin) {res = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2057_(lean_io_mk_world()); +l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__1 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__1(); +lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__1); +l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__2 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__2(); +lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__2); +l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__3 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__3(); +lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__3); +l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__4 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__4(); +lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__4); +l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__5 = _init_l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__5(); +lean_mark_persistent(l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058____closed__5); +if (builtin) {res = l_Lean_Language_initFn____x40_Lean_Language_Basic___hyg_2058_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Language_printMessageEndPos = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Language_printMessageEndPos); diff --git a/stage0/stdlib/Lean/Language/Lean/Types.c b/stage0/stdlib/Lean/Language/Lean/Types.c index d6c494f83544..242bce031457 100644 --- a/stage0/stdlib/Lean/Language/Lean/Types.c +++ b/stage0/stdlib/Lean/Language/Lean/Types.c @@ -27,6 +27,7 @@ LEAN_EXPORT lean_object* l_Lean_Language_Lean_HeaderParsedSnapshot_processedResu static lean_object* l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go___closed__3; static lean_object* l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go___closed__2; LEAN_EXPORT lean_object* l_Lean_Language_Lean_CommandParsedSnapshot_nextCmdSnap_x3f___boxed(lean_object*); +lean_object* lean_thunk_get_own(lean_object*); LEAN_EXPORT lean_object* l_Lean_Language_Lean_HeaderParsedSnapshot_processedResult___lambda__1___boxed(lean_object*); static lean_object* l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go___closed__1; LEAN_EXPORT lean_object* l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go___lambda__2(lean_object*); @@ -144,10 +145,10 @@ return x_2; LEAN_EXPORT lean_object* l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go___lambda__1(lean_object* x_1) { _start: { -lean_object* x_2; +lean_object* x_2; lean_object* x_3; x_2 = lean_ctor_get(x_1, 1); -lean_inc(x_2); -return x_2; +x_3 = lean_thunk_get_own(x_2); +return x_3; } } LEAN_EXPORT lean_object* l_Lean_Language_Lean_instToSnapshotTreeCommandParsedSnapshot_go___lambda__2(lean_object* x_1) { diff --git a/stage0/stdlib/Lean/LazyInitExtension.c b/stage0/stdlib/Lean/LazyInitExtension.c deleted file mode 100644 index fd852129ca29..000000000000 --- a/stage0/stdlib/Lean/LazyInitExtension.c +++ /dev/null @@ -1,322 +0,0 @@ -// Lean compiler output -// Module: Lean.LazyInitExtension -// Imports: Lean.MonadEnv -#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_instInhabitedLazyInitExtensionOfMonad(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_EnvExtensionInterfaceUnsafe_registerExt___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_registerLazyInitExtension___rarg(lean_object*, lean_object*); -lean_object* l_Lean_EnvExtensionInterfaceUnsafe_instInhabitedExt___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_EnvExtension_getState___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_registerLazyInitExtension___rarg___closed__1; -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_EStateM_pure___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_registerLazyInitExtension(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__2(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__2; -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get(lean_object*, lean_object*); -lean_object* l_Lean_EnvExtension_setState___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__1; -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* _init_l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_EnvExtensionInterfaceUnsafe_instInhabitedExt___lambda__1), 1, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(0u); -x_2 = l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___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_Lean_instInhabitedLazyInitExtensionOfMonad___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; -x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); -lean_dec(x_1); -x_4 = lean_ctor_get(x_3, 1); -lean_inc(x_4); -lean_dec(x_3); -x_5 = lean_apply_2(x_4, lean_box(0), x_2); -x_6 = l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__2; -x_7 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_5); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Lean_instInhabitedLazyInitExtensionOfMonad(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg), 2, 0); -return x_3; -} -} -static lean_object* _init_l_Lean_registerLazyInitExtension___rarg___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_alloc_closure((void*)(l_EStateM_pure___rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_registerLazyInitExtension___rarg(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; lean_object* x_4; -x_3 = l_Lean_registerLazyInitExtension___rarg___closed__1; -x_4 = l_Lean_EnvExtensionInterfaceUnsafe_registerExt___rarg(x_3, x_2); -if (lean_obj_tag(x_4) == 0) -{ -uint8_t x_5; -x_5 = !lean_is_exclusive(x_4); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; -x_6 = lean_ctor_get(x_4, 0); -x_7 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_1); -lean_ctor_set(x_4, 0, x_7); -return x_4; -} -else -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_8 = lean_ctor_get(x_4, 0); -x_9 = lean_ctor_get(x_4, 1); -lean_inc(x_9); -lean_inc(x_8); -lean_dec(x_4); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, 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; -} -} -else -{ -uint8_t x_12; -lean_dec(x_1); -x_12 = !lean_is_exclusive(x_4); -if (x_12 == 0) -{ -return x_4; -} -else -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_4, 0); -x_14 = lean_ctor_get(x_4, 1); -lean_inc(x_14); -lean_inc(x_13); -lean_dec(x_4); -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_Lean_registerLazyInitExtension(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_registerLazyInitExtension___rarg), 2, 0); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___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(1, 1, 0); -lean_ctor_set(x_4, 0, x_1); -x_5 = l_Lean_EnvExtension_setState___rarg(x_2, x_3, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__2(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 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -lean_dec(x_1); -x_5 = lean_ctor_get(x_4, 1); -lean_inc(x_5); -lean_dec(x_4); -x_6 = lean_apply_2(x_5, lean_box(0), x_2); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___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; -x_6 = lean_ctor_get(x_1, 1); -lean_inc(x_6); -lean_dec(x_1); -lean_inc(x_5); -x_7 = lean_alloc_closure((void*)(l_Lean_LazyInitExtension_get___rarg___lambda__1___boxed), 3, 2); -lean_closure_set(x_7, 0, x_5); -lean_closure_set(x_7, 1, x_2); -x_8 = lean_apply_1(x_6, x_7); -x_9 = lean_alloc_closure((void*)(l_Lean_LazyInitExtension_get___rarg___lambda__2___boxed), 3, 2); -lean_closure_set(x_9, 0, x_3); -lean_closure_set(x_9, 1, x_5); -x_10 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_8, x_9); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__4(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; -x_6 = lean_box(0); -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); -x_8 = l_Lean_EnvExtension_getState___rarg(x_6, x_7, x_5); -if (lean_obj_tag(x_8) == 0) -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = lean_ctor_get(x_1, 1); -lean_inc(x_9); -lean_dec(x_1); -lean_inc(x_4); -x_10 = lean_alloc_closure((void*)(l_Lean_LazyInitExtension_get___rarg___lambda__3), 5, 4); -lean_closure_set(x_10, 0, x_2); -lean_closure_set(x_10, 1, x_7); -lean_closure_set(x_10, 2, x_3); -lean_closure_set(x_10, 3, x_4); -x_11 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_9, x_10); -return x_11; -} -else -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -lean_dec(x_7); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_12 = lean_ctor_get(x_8, 0); -lean_inc(x_12); -lean_dec(x_8); -x_13 = lean_ctor_get(x_3, 0); -lean_inc(x_13); -lean_dec(x_3); -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -lean_dec(x_13); -x_15 = lean_apply_2(x_14, lean_box(0), x_12); -return x_15; -} -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg(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; -x_4 = lean_ctor_get(x_2, 1); -lean_inc(x_4); -x_5 = lean_ctor_get(x_1, 0); -lean_inc(x_5); -lean_inc(x_4); -x_6 = lean_alloc_closure((void*)(l_Lean_LazyInitExtension_get___rarg___lambda__4___boxed), 5, 4); -lean_closure_set(x_6, 0, x_3); -lean_closure_set(x_6, 1, x_1); -lean_closure_set(x_6, 2, x_2); -lean_closure_set(x_6, 3, x_4); -x_7 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_5, x_6); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_LazyInitExtension_get___rarg), 3, 0); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_LazyInitExtension_get___rarg___lambda__1(x_1, x_2, x_3); -lean_dec(x_2); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_LazyInitExtension_get___rarg___lambda__2(x_1, x_2, x_3); -lean_dec(x_3); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___rarg___lambda__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_LazyInitExtension_get___rarg___lambda__4(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_5); -return x_6; -} -} -lean_object* initialize_Lean_MonadEnv(uint8_t builtin, lean_object*); -static bool _G_initialized = false; -LEAN_EXPORT lean_object* initialize_Lean_LazyInitExtension(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_MonadEnv(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__1 = _init_l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__1(); -lean_mark_persistent(l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__1); -l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__2 = _init_l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__2(); -lean_mark_persistent(l_Lean_instInhabitedLazyInitExtensionOfMonad___rarg___closed__2); -l_Lean_registerLazyInitExtension___rarg___closed__1 = _init_l_Lean_registerLazyInitExtension___rarg___closed__1(); -lean_mark_persistent(l_Lean_registerLazyInitExtension___rarg___closed__1); -return lean_io_result_mk_ok(lean_box(0)); -} -#ifdef __cplusplus -} -#endif diff --git a/stage0/stdlib/Lean/Linter/ConstructorAsVariable.c b/stage0/stdlib/Lean/Linter/ConstructorAsVariable.c index ac66853ba0a9..19048351e0c2 100644 --- a/stage0/stdlib/Lean/Linter/ConstructorAsVariable.c +++ b/stage0/stdlib/Lean/Linter/ConstructorAsVariable.c @@ -13,126 +13,123 @@ #ifdef __cplusplus extern "C" { #endif -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__2; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__4; static lean_object* l_Lean_Linter_constructorNameAsVariable___closed__1; -LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__4(lean_object*, lean_object*); lean_object* l_Lean_PersistentArray_toArray___rarg(lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__5; lean_object* lean_whnf(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getHeadInfo(lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___boxed(lean_object*, lean_object*); uint64_t l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__4; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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*); size_t lean_uint64_to_usize(uint64_t); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_constructorNameAsVariable___elambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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_Syntax_getId(lean_object*); uint8_t l___private_Lean_Syntax_0__String_beqRange____x40_Lean_Syntax___hyg_95_(lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7___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_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_qpartition___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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_mk_array(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); -static lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__17(lean_object*, size_t, size_t, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___closed__1; lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_constructorNameAsVariable___closed__3; LEAN_EXPORT lean_object* l_Lean_Linter_linter_constructorNameAsVariable; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__5(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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*); lean_object* lean_environment_find(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_logAt___at_Lean_Elab_Command_runLinters___spec__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__1; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__8; +LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(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_stringToMessageData(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__8; lean_object* l_Lean_PersistentArray_toList___rarg(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__6___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 uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__4; -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__7; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__4; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__2(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_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__1___boxed(lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); lean_object* lean_local_ctx_find(lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__2; +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__6___lambda__1___closed__1; uint64_t lean_uint64_shift_right(uint64_t, uint64_t); -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__9; lean_object* lean_nat_div(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__2; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__2; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__11; lean_object* l_Lean_Elab_Info_updateContext_x3f(lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__6; +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__5; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__2; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(lean_object*, lean_object*); static lean_object* l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofFormat(lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__3; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__10; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__6; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7___lambda__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*); -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__7; lean_object* lean_st_mk_ref(lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1; -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__12; -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__4; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_inferType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Command_instMonadCommandElabM; LEAN_EXPORT lean_object* l_Lean_Linter_constructorNameAsVariable___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__4; 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_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__3; -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11(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_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__12; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__10; lean_object* l_Lean_Elab_Command_addLinter(lean_object*, lean_object*); lean_object* l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__2; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__3; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__2(lean_object*); lean_object* l_Lean_LocalDecl_userName(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4(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_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__3; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Name_hasMacroScopes(lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__5; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___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*); uint8_t l_String_Range_contains(lean_object*, lean_object*, uint8_t); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12(lean_object*, lean_object*); 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_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__9; -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__6; +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__2; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__3; static lean_object* l_Lean_Linter_constructorNameAsVariable___closed__2; -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__6; -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getAppFn_x27(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__3(lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_xor(uint64_t, uint64_t); lean_object* lean_panic_fn(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__1; lean_object* lean_nat_sub(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___boxed(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_Syntax_getRange_x3f(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8_(lean_object*); @@ -140,42 +137,44 @@ lean_object* l_Lean_Elab_TermInfo_runMetaM___rarg(lean_object*, lean_object*, le static lean_object* l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__1; lean_object* l_Lean_Elab_Info_range_x3f(lean_object*); lean_object* l_List_reverse___rarg(lean_object*); +static lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1; size_t lean_usize_sub(size_t, size_t); lean_object* lean_array_mk(lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5(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); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__11; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__7; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__7; lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__9; lean_object* lean_io_error_to_string(lean_object*); lean_object* l_instInhabitedOfMonad___rarg(lean_object*, lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); -static lean_object* l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10___closed__1; -LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___boxed(lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); static lean_object* l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__2; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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*, lean_object*); static lean_object* l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__4; uint8_t lean_nat_dec_le(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__4; lean_object* lean_nat_add(lean_object*, lean_object*); +static lean_object* l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1; lean_object* l_Lean_Elab_Info_stx(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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_Lean_Linter_constructorNameAsVariable___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_1340_(lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__3; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__5; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__6; size_t lean_usize_land(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Linter_constructorNameAsVariable; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__6___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_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__5; -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__3; static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_ConstructorAsVariable___hyg_8____closed__1() { _start: @@ -1199,7 +1198,7 @@ goto _start; } } } -static lean_object* _init_l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10___closed__1() { +static lean_object* _init_l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -1209,17 +1208,17 @@ x_3 = l_instInhabitedOfMonad___rarg(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9(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; -x_5 = l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10___closed__1; +x_5 = l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1; x_6 = lean_panic_fn(x_5, x_1); x_7 = lean_apply_3(x_6, x_2, x_3, x_4); return x_7; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___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, lean_object* x_8) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___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, lean_object* x_8) { _start: { if (lean_obj_tag(x_4) == 0) @@ -1250,7 +1249,7 @@ lean_inc(x_6); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9(x_1, x_2, x_3, x_12, x_6, x_7, x_8); +x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8(x_1, x_2, x_3, x_12, x_6, x_7, x_8); if (lean_obj_tag(x_14) == 0) { lean_object* x_15; lean_object* x_16; @@ -1315,7 +1314,7 @@ lean_inc(x_6); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_24 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9(x_1, x_2, x_3, x_22, x_6, x_7, x_8); +x_24 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8(x_1, x_2, x_3, x_22, 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; @@ -1367,7 +1366,7 @@ return x_32; } } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__1() { _start: { lean_object* x_1; @@ -1375,7 +1374,7 @@ x_1 = lean_mk_string_unchecked("Lean.Server.InfoUtils", 21, 21); return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__2() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__2() { _start: { lean_object* x_1; @@ -1383,7 +1382,7 @@ x_1 = lean_mk_string_unchecked("Lean.Elab.InfoTree.visitM.go", 28, 28); return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__3() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__3() { _start: { lean_object* x_1; @@ -1391,20 +1390,20 @@ x_1 = lean_mk_string_unchecked("unexpected context-free info tree node", 38, 38) return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__4() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___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_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1; -x_2 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__2; -x_3 = lean_unsigned_to_nat(56u); +x_1 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__1; +x_2 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__2; +x_3 = lean_unsigned_to_nat(62u); x_4 = lean_unsigned_to_nat(21u); -x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__3; +x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___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_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___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) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___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) { _start: { if (lean_obj_tag(x_3) == 0) @@ -1429,8 +1428,8 @@ lean_object* x_12; lean_object* x_13; lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__4; -x_13 = l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10(x_12, x_5, x_6, x_7); +x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__4; +x_13 = l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9(x_12, x_5, x_6, x_7); return x_13; } default: @@ -1487,111 +1486,179 @@ lean_inc(x_21); x_24 = lean_apply_6(x_1, x_21, x_22, x_23, x_5, x_6, x_7); 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, 1); +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) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_dec(x_1); +x_27 = lean_ctor_get(x_24, 1); +lean_inc(x_27); lean_dec(x_24); -lean_inc(x_21); -x_26 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_22); -x_27 = l_Lean_PersistentArray_toList___rarg(x_23); x_28 = lean_box(0); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_2); -x_29 = l_List_mapM_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11(x_1, x_2, x_26, x_27, x_28, x_5, x_6, x_25); +x_29 = lean_apply_7(x_2, x_21, x_22, x_23, x_28, x_5, x_6, x_27); if (lean_obj_tag(x_29) == 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); +uint8_t x_30; +x_30 = !lean_is_exclusive(x_29); +if (x_30 == 0) +{ +lean_object* x_31; +x_31 = lean_ctor_get(x_29, 0); +lean_ctor_set(x_3, 0, x_31); +lean_ctor_set(x_29, 0, x_3); +return x_29; +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_29, 0); +x_33 = lean_ctor_get(x_29, 1); +lean_inc(x_33); +lean_inc(x_32); lean_dec(x_29); -x_32 = lean_apply_7(x_2, x_21, x_22, x_23, x_30, x_5, x_6, x_31); -if (lean_obj_tag(x_32) == 0) +lean_ctor_set(x_3, 0, x_32); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_3); +lean_ctor_set(x_34, 1, x_33); +return x_34; +} +} +else { -uint8_t x_33; -x_33 = !lean_is_exclusive(x_32); -if (x_33 == 0) +uint8_t x_35; +lean_free_object(x_3); +x_35 = !lean_is_exclusive(x_29); +if (x_35 == 0) { -lean_object* x_34; lean_object* x_35; -x_34 = lean_ctor_get(x_32, 0); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_32, 0, x_35); -return x_32; +return x_29; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_36 = lean_ctor_get(x_32, 0); -x_37 = lean_ctor_get(x_32, 1); +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_29, 0); +x_37 = lean_ctor_get(x_29, 1); lean_inc(x_37); lean_inc(x_36); -lean_dec(x_32); -x_38 = lean_alloc_ctor(1, 1, 0); +lean_dec(x_29); +x_38 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_38, 0, x_36); -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; +lean_ctor_set(x_38, 1, x_37); +return x_38; +} } } else { -uint8_t x_40; -x_40 = !lean_is_exclusive(x_32); -if (x_40 == 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_24, 1); +lean_inc(x_39); +lean_dec(x_24); +lean_inc(x_21); +x_40 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_22); +x_41 = l_Lean_PersistentArray_toList___rarg(x_23); +x_42 = lean_box(0); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_2); +x_43 = l_List_mapM_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10(x_1, x_2, x_40, x_41, x_42, x_5, x_6, x_39); +if (lean_obj_tag(x_43) == 0) { -return x_32; +lean_object* x_44; lean_object* x_45; lean_object* x_46; +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_apply_7(x_2, x_21, x_22, x_23, x_44, x_5, x_6, x_45); +if (lean_obj_tag(x_46) == 0) +{ +uint8_t x_47; +x_47 = !lean_is_exclusive(x_46); +if (x_47 == 0) +{ +lean_object* x_48; lean_object* x_49; +x_48 = lean_ctor_get(x_46, 0); +x_49 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_46, 0, x_49); +return x_46; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_32, 0); -x_42 = lean_ctor_get(x_32, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_32); -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_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +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, 1, 0); +lean_ctor_set(x_52, 0, x_50); +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 +{ +uint8_t x_54; +x_54 = !lean_is_exclusive(x_46); +if (x_54 == 0) +{ +return x_46; +} +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_46, 0); +x_56 = lean_ctor_get(x_46, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_46); +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_44; +uint8_t x_58; lean_dec(x_23); lean_dec(x_22); lean_dec(x_21); lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); -x_44 = !lean_is_exclusive(x_29); -if (x_44 == 0) +x_58 = !lean_is_exclusive(x_43); +if (x_58 == 0) { -return x_29; +return x_43; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_29, 0); -x_46 = lean_ctor_get(x_29, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_29); -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_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_43, 0); +x_60 = lean_ctor_get(x_43, 1); +lean_inc(x_60); +lean_inc(x_59); +lean_dec(x_43); +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 { -uint8_t x_48; +uint8_t x_62; lean_dec(x_23); lean_dec(x_22); lean_free_object(x_3); @@ -1600,210 +1667,269 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); -x_48 = !lean_is_exclusive(x_24); -if (x_48 == 0) +x_62 = !lean_is_exclusive(x_24); +if (x_62 == 0) { return x_24; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_24, 0); -x_50 = lean_ctor_get(x_24, 1); -lean_inc(x_50); -lean_inc(x_49); +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_24, 0); +x_64 = lean_ctor_get(x_24, 1); +lean_inc(x_64); +lean_inc(x_63); lean_dec(x_24); -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; +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_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_52 = lean_ctor_get(x_3, 0); -lean_inc(x_52); +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_66 = lean_ctor_get(x_3, 0); +lean_inc(x_66); lean_dec(x_3); -x_53 = lean_ctor_get(x_4, 0); -lean_inc(x_53); -x_54 = lean_ctor_get(x_4, 1); -lean_inc(x_54); +x_67 = lean_ctor_get(x_4, 0); +lean_inc(x_67); +x_68 = lean_ctor_get(x_4, 1); +lean_inc(x_68); lean_dec(x_4); lean_inc(x_1); lean_inc(x_6); lean_inc(x_5); -lean_inc(x_54); -lean_inc(x_53); -lean_inc(x_52); -x_55 = lean_apply_6(x_1, x_52, x_53, x_54, x_5, x_6, x_7); -if (lean_obj_tag(x_55) == 0) +lean_inc(x_68); +lean_inc(x_67); +lean_inc(x_66); +x_69 = lean_apply_6(x_1, x_66, x_67, x_68, x_5, x_6, x_7); +if (lean_obj_tag(x_69) == 0) { -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_55, 1); -lean_inc(x_56); -lean_dec(x_55); -lean_inc(x_52); -x_57 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_57, 0, x_52); -x_58 = l_Lean_Elab_Info_updateContext_x3f(x_57, x_53); -x_59 = l_Lean_PersistentArray_toList___rarg(x_54); -x_60 = lean_box(0); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_2); -x_61 = l_List_mapM_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11(x_1, x_2, x_58, x_59, x_60, x_5, x_6, x_56); -if (lean_obj_tag(x_61) == 0) +lean_object* x_70; uint8_t x_71; +x_70 = lean_ctor_get(x_69, 0); +lean_inc(x_70); +x_71 = lean_unbox(x_70); +lean_dec(x_70); +if (x_71 == 0) { -lean_object* x_62; lean_object* x_63; lean_object* x_64; -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_apply_7(x_2, x_52, x_53, x_54, x_62, x_5, x_6, x_63); -if (lean_obj_tag(x_64) == 0) +lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_dec(x_1); +x_72 = lean_ctor_get(x_69, 1); +lean_inc(x_72); +lean_dec(x_69); +x_73 = lean_box(0); +x_74 = lean_apply_7(x_2, x_66, x_67, x_68, x_73, x_5, x_6, x_72); +if (lean_obj_tag(x_74) == 0) { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_65 = lean_ctor_get(x_64, 0); -lean_inc(x_65); -x_66 = lean_ctor_get(x_64, 1); +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_74); + x_77 = lean_box(0); +} +x_78 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_78, 0, x_75); +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; +x_80 = lean_ctor_get(x_74, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_74, 1); +lean_inc(x_81); +if (lean_is_exclusive(x_74)) { + lean_ctor_release(x_74, 0); + lean_ctor_release(x_74, 1); + x_82 = x_74; +} else { + lean_dec_ref(x_74); + 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; +x_84 = lean_ctor_get(x_69, 1); +lean_inc(x_84); +lean_dec(x_69); 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; +x_85 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_85, 0, x_66); +x_86 = l_Lean_Elab_Info_updateContext_x3f(x_85, x_67); +x_87 = l_Lean_PersistentArray_toList___rarg(x_68); +x_88 = lean_box(0); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_2); +x_89 = l_List_mapM_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10(x_1, x_2, x_86, x_87, x_88, x_5, x_6, x_84); +if (lean_obj_tag(x_89) == 0) +{ +lean_object* x_90; lean_object* x_91; lean_object* x_92; +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_7(x_2, x_66, x_67, x_68, x_90, x_5, x_6, x_91); +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_64); - x_67 = lean_box(0); + lean_dec_ref(x_92); + x_95 = lean_box(0); } -x_68 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_68, 0, x_65); -if (lean_is_scalar(x_67)) { - x_69 = lean_alloc_ctor(0, 2, 0); +x_96 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_96, 0, x_93); +if (lean_is_scalar(x_95)) { + x_97 = lean_alloc_ctor(0, 2, 0); } else { - x_69 = x_67; + x_97 = x_95; } -lean_ctor_set(x_69, 0, x_68); -lean_ctor_set(x_69, 1, x_66); -return x_69; +lean_ctor_set(x_97, 0, x_96); +lean_ctor_set(x_97, 1, x_94); +return x_97; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_70 = lean_ctor_get(x_64, 0); -lean_inc(x_70); -x_71 = lean_ctor_get(x_64, 1); -lean_inc(x_71); -if (lean_is_exclusive(x_64)) { - lean_ctor_release(x_64, 0); - lean_ctor_release(x_64, 1); - x_72 = x_64; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; +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_64); - x_72 = lean_box(0); + lean_dec_ref(x_92); + x_100 = lean_box(0); } -if (lean_is_scalar(x_72)) { - x_73 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_100)) { + x_101 = lean_alloc_ctor(1, 2, 0); } else { - x_73 = x_72; + x_101 = x_100; } -lean_ctor_set(x_73, 0, x_70); -lean_ctor_set(x_73, 1, x_71); -return x_73; +lean_ctor_set(x_101, 0, x_98); +lean_ctor_set(x_101, 1, x_99); +return x_101; } } else { -lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -lean_dec(x_54); -lean_dec(x_53); -lean_dec(x_52); +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +lean_dec(x_68); +lean_dec(x_67); +lean_dec(x_66); lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); -x_74 = lean_ctor_get(x_61, 0); -lean_inc(x_74); -x_75 = lean_ctor_get(x_61, 1); -lean_inc(x_75); -if (lean_is_exclusive(x_61)) { - lean_ctor_release(x_61, 0); - lean_ctor_release(x_61, 1); - x_76 = x_61; +x_102 = lean_ctor_get(x_89, 0); +lean_inc(x_102); +x_103 = lean_ctor_get(x_89, 1); +lean_inc(x_103); +if (lean_is_exclusive(x_89)) { + lean_ctor_release(x_89, 0); + lean_ctor_release(x_89, 1); + x_104 = x_89; } else { - lean_dec_ref(x_61); - x_76 = lean_box(0); + lean_dec_ref(x_89); + x_104 = lean_box(0); } -if (lean_is_scalar(x_76)) { - x_77 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_104)) { + x_105 = lean_alloc_ctor(1, 2, 0); } else { - x_77 = x_76; + x_105 = x_104; +} +lean_ctor_set(x_105, 0, x_102); +lean_ctor_set(x_105, 1, x_103); +return x_105; } -lean_ctor_set(x_77, 0, x_74); -lean_ctor_set(x_77, 1, x_75); -return x_77; } } else { -lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -lean_dec(x_54); -lean_dec(x_53); -lean_dec(x_52); +lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; +lean_dec(x_68); +lean_dec(x_67); +lean_dec(x_66); lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); -x_78 = lean_ctor_get(x_55, 0); -lean_inc(x_78); -x_79 = lean_ctor_get(x_55, 1); -lean_inc(x_79); -if (lean_is_exclusive(x_55)) { - lean_ctor_release(x_55, 0); - lean_ctor_release(x_55, 1); - x_80 = x_55; +x_106 = lean_ctor_get(x_69, 0); +lean_inc(x_106); +x_107 = lean_ctor_get(x_69, 1); +lean_inc(x_107); +if (lean_is_exclusive(x_69)) { + lean_ctor_release(x_69, 0); + lean_ctor_release(x_69, 1); + x_108 = x_69; } else { - lean_dec_ref(x_55); - x_80 = lean_box(0); + lean_dec_ref(x_69); + x_108 = lean_box(0); } -if (lean_is_scalar(x_80)) { - x_81 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_108)) { + x_109 = lean_alloc_ctor(1, 2, 0); } else { - x_81 = x_80; + x_109 = x_108; } -lean_ctor_set(x_81, 0, x_78); -lean_ctor_set(x_81, 1, x_79); -return x_81; +lean_ctor_set(x_109, 0, x_106); +lean_ctor_set(x_109, 1, x_107); +return x_109; } } } default: { -lean_object* x_82; lean_object* x_83; +lean_object* x_110; lean_object* x_111; 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_82 = lean_box(0); -x_83 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_83, 0, x_82); -lean_ctor_set(x_83, 1, x_7); -return x_83; -} -} +x_110 = lean_box(0); +x_111 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_111, 0, x_110); +lean_ctor_set(x_111, 1, x_7); +return x_111; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_constructorNameAsVariable___elambda__1___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) { -_start: -{ -lean_object* x_7; lean_object* x_8; -x_7 = lean_box(0); -x_8 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9(x_1, x_2, x_7, x_3, x_4, x_5, x_6); -return x_8; } } LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___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) { @@ -1814,64 +1940,76 @@ x_9 = lean_apply_6(x_1, x_2, x_3, x_4, x_6, x_7, x_8); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___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_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___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) { _start: { -lean_object* x_7; lean_object* x_8; -x_7 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7___lambda__1___boxed), 8, 1); -lean_closure_set(x_7, 0, x_2); -x_8 = l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8(x_1, x_7, x_3, x_4, x_5, x_6); -if (lean_obj_tag(x_8) == 0) +lean_object* x_8; lean_object* x_9; +x_8 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7___lambda__1___boxed), 8, 1); +lean_closure_set(x_8, 0, x_2); +x_9 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8(x_1, x_8, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_9) == 0) { -uint8_t x_9; -x_9 = !lean_is_exclusive(x_8); -if (x_9 == 0) +uint8_t x_10; +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) { -lean_object* x_10; lean_object* x_11; -x_10 = lean_ctor_get(x_8, 0); -lean_dec(x_10); -x_11 = lean_box(0); -lean_ctor_set(x_8, 0, x_11); -return x_8; +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +lean_dec(x_11); +x_12 = lean_box(0); +lean_ctor_set(x_9, 0, x_12); +return x_9; } else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_8, 1); -lean_inc(x_12); -lean_dec(x_8); -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_12); -return x_14; +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_9, 1); +lean_inc(x_13); +lean_dec(x_9); +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 { -uint8_t x_15; -x_15 = !lean_is_exclusive(x_8); -if (x_15 == 0) +uint8_t x_16; +x_16 = !lean_is_exclusive(x_9); +if (x_16 == 0) { -return x_8; +return x_9; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_8, 0); -x_17 = lean_ctor_get(x_8, 1); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_9, 0); +x_18 = lean_ctor_get(x_9, 1); +lean_inc(x_18); lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_8); -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_dec(x_9); +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_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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: +{ +uint8_t x_7; lean_object* x_8; lean_object* x_9; +x_7 = 1; +x_8 = lean_box(x_7); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_6); +return x_9; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___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_object* x_6) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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; lean_object* x_9; lean_object* x_10; @@ -1885,11 +2023,11 @@ x_10 = lean_whnf(x_8, x_2, x_3, x_4, x_5, x_9); return x_10; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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; -x_13 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__1), 6, 1); +x_13 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__2), 6, 1); lean_closure_set(x_13, 0, x_9); x_14 = l_Lean_Elab_TermInfo_runMetaM___rarg(x_1, x_2, x_13, x_12); if (lean_obj_tag(x_14) == 0) @@ -2248,7 +2386,7 @@ return x_92; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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; @@ -2281,7 +2419,7 @@ lean_inc(x_18); x_19 = lean_ctor_get(x_17, 1); lean_inc(x_19); lean_dec(x_17); -x_20 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__2(x_2, x_3, x_4, x_5, x_6, x_1, x_12, x_15, x_18, x_9, x_10, x_19); +x_20 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__3(x_2, x_3, x_4, x_5, x_6, x_1, x_12, x_15, x_18, x_9, x_10, x_19); lean_dec(x_15); return x_20; } @@ -2345,7 +2483,7 @@ lean_inc(x_36); x_37 = lean_ctor_get(x_14, 0); lean_inc(x_37); lean_dec(x_14); -x_38 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__2(x_2, x_3, x_4, x_5, x_6, x_1, x_12, x_36, x_37, x_9, x_10, x_11); +x_38 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__3(x_2, x_3, x_4, x_5, x_6, x_1, x_12, x_36, x_37, x_9, x_10, x_11); lean_dec(x_36); return x_38; } @@ -2386,7 +2524,7 @@ return x_42; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1() { _start: { lean_object* x_1; @@ -2394,7 +2532,7 @@ x_1 = l_Lean_Linter_linter_constructorNameAsVariable; return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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; lean_object* x_14; uint8_t x_15; @@ -2403,7 +2541,7 @@ lean_inc(x_12); x_13 = lean_ctor_get(x_12, 3); lean_inc(x_13); lean_dec(x_12); -x_14 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1; +x_14 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1; x_15 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_13, x_14); lean_dec(x_13); if (x_15 == 0) @@ -2425,12 +2563,12 @@ else { lean_object* x_18; lean_object* x_19; x_18 = lean_box(0); -x_19 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__3(x_2, x_3, x_1, x_4, x_5, x_6, x_7, x_18, x_9, x_10, x_11); +x_19 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__4(x_2, x_3, x_1, x_4, x_5, x_6, x_7, x_18, x_9, x_10, x_11); return x_19; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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_object* x_12, lean_object* x_13) { _start: { lean_object* x_14; lean_object* x_15; @@ -2516,7 +2654,7 @@ if (x_30 == 0) { lean_object* x_31; lean_object* x_32; x_31 = lean_box(0); -x_32 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4(x_4, x_14, x_2, x_5, x_6, x_7, x_8, x_31, x_11, x_12, x_13); +x_32 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5(x_4, x_14, x_2, x_5, x_6, x_7, x_8, x_31, x_11, x_12, x_13); return x_32; } else @@ -2557,7 +2695,7 @@ return x_36; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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) { _start: { if (lean_obj_tag(x_5) == 1) @@ -2627,7 +2765,7 @@ if (x_36 == 0) lean_object* x_37; lean_object* x_38; lean_free_object(x_17); x_37 = lean_box(0); -x_38 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__5(x_5, x_10, x_12, x_4, x_2, x_1, x_16, x_11, x_3, x_37, x_7, x_8, x_20); +x_38 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__6(x_5, x_10, x_12, x_4, x_2, x_1, x_16, x_11, x_3, x_37, x_7, x_8, x_20); lean_dec(x_5); return x_38; } @@ -2679,7 +2817,7 @@ if (x_57 == 0) { lean_object* x_58; lean_object* x_59; x_58 = lean_box(0); -x_59 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__5(x_5, x_10, x_12, x_4, x_2, x_1, x_16, x_11, x_3, x_58, x_7, x_8, x_41); +x_59 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__6(x_5, x_10, x_12, x_4, x_2, x_1, x_16, x_11, x_3, x_58, x_7, x_8, x_41); lean_dec(x_5); return x_59; } @@ -2731,26 +2869,15 @@ return x_65; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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) { -_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_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__7___boxed), 6, 0); +x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__1___boxed), 6, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___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_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11(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) { _start: { uint8_t x_11; @@ -2770,65 +2897,66 @@ return x_12; } else { -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; lean_dec(x_7); x_13 = lean_array_uget(x_4, x_6); lean_inc(x_1); lean_inc(x_2); lean_inc(x_3); -x_14 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__6___boxed), 9, 3); +x_14 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__7___boxed), 9, 3); lean_closure_set(x_14, 0, x_3); lean_closure_set(x_14, 1, x_2); lean_closure_set(x_14, 2, x_1); -x_15 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___closed__1; +x_15 = lean_box(0); +x_16 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___closed__1; lean_inc(x_9); lean_inc(x_8); -x_16 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7(x_14, x_15, x_13, x_8, x_9, x_10); -if (lean_obj_tag(x_16) == 0) +x_17 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__7(x_16, x_14, x_15, x_13, x_8, x_9, x_10); +if (lean_obj_tag(x_17) == 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_10 = x_17; +lean_object* x_18; size_t x_19; size_t x_20; lean_object* x_21; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_19 = 1; +x_20 = lean_usize_add(x_6, x_19); +x_21 = lean_box(0); +x_6 = x_20; +x_7 = x_21; +x_10 = x_18; goto _start; } else { -uint8_t x_22; +uint8_t x_23; lean_dec(x_9); lean_dec(x_8); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_22 = !lean_is_exclusive(x_16); -if (x_22 == 0) +x_23 = !lean_is_exclusive(x_17); +if (x_23 == 0) { -return x_16; +return x_17; } 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_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_17, 0); +x_25 = lean_ctor_get(x_17, 1); +lean_inc(x_25); 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; +lean_dec(x_17); +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_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -2853,7 +2981,7 @@ goto _start; } } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__1() { _start: { lean_object* x_1; @@ -2861,16 +2989,16 @@ x_1 = lean_mk_string_unchecked("note: this linter can be disabled with `set_opti return x_1; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__2() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1; +x_1 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__3() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__3() { _start: { lean_object* x_1; @@ -2878,16 +3006,16 @@ x_1 = lean_mk_string_unchecked(" false`", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__4() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__3; +x_1 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__5() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -2896,7 +3024,7 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__6() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__6() { _start: { lean_object* x_1; @@ -2904,16 +3032,16 @@ x_1 = lean_mk_string_unchecked("\n", 1, 1); return x_1; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__7() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__6; +x_1 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__6; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__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) { +LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__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) { _start: { uint8_t x_7; @@ -2926,19 +3054,19 @@ x_9 = lean_ctor_get(x_1, 1); lean_dec(x_9); lean_inc(x_8); x_10 = l_Lean_MessageData_ofName(x_8); -x_11 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__2; +x_11 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__2; lean_ctor_set_tag(x_1, 7); lean_ctor_set(x_1, 1, x_10); lean_ctor_set(x_1, 0, x_11); -x_12 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__4; +x_12 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__4; x_13 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_13, 0, x_1); lean_ctor_set(x_13, 1, x_12); -x_14 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__5; +x_14 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__5; x_15 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_3); -x_16 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__7; +x_16 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__7; x_17 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); @@ -2963,19 +3091,19 @@ lean_inc(x_23); lean_dec(x_1); lean_inc(x_23); x_24 = l_Lean_MessageData_ofName(x_23); -x_25 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__2; +x_25 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__2; x_26 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_26, 0, x_25); lean_ctor_set(x_26, 1, x_24); -x_27 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__4; +x_27 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__4; 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_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__5; +x_29 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__5; x_30 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_30, 0, x_29); lean_ctor_set(x_30, 1, x_3); -x_31 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__7; +x_31 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___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); @@ -2994,7 +3122,7 @@ return x_37; } } } -LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___lambda__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; uint8_t x_7; @@ -3006,15 +3134,15 @@ x_7 = lean_nat_dec_lt(x_4, x_6); return x_7; } } -static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1() { +static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___lambda__1___boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___lambda__1___boxed), 2, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -3027,7 +3155,7 @@ return x_1; else { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_5 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1; +x_5 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1; lean_inc(x_2); x_6 = l_Array_qpartition___rarg(x_1, x_5, x_2, x_3); x_7 = lean_ctor_get(x_6, 0); @@ -3039,7 +3167,7 @@ x_9 = lean_nat_dec_le(x_3, x_7); if (x_9 == 0) { lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(x_8, x_2, x_7); +x_10 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_8, x_2, x_7); x_11 = lean_unsigned_to_nat(1u); x_12 = lean_nat_add(x_7, x_11); lean_dec(x_7); @@ -3056,7 +3184,7 @@ return x_8; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1() { _start: { lean_object* x_1; @@ -3064,16 +3192,16 @@ x_1 = lean_mk_string_unchecked("Local variable '", 16, 16); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__1; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__3() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__3() { _start: { lean_object* x_1; @@ -3081,16 +3209,16 @@ x_1 = lean_mk_string_unchecked("' resembles constructor '", 25, 25); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__4() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__3; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__5() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__5() { _start: { lean_object* x_1; @@ -3098,16 +3226,16 @@ x_1 = lean_mk_string_unchecked("' - ", 4, 4); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__6() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__5; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__5; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__7() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__7() { _start: { lean_object* x_1; @@ -3115,16 +3243,16 @@ x_1 = lean_mk_string_unchecked("write '.", 8, 8); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__8() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__7; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__7; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__9() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__9() { _start: { lean_object* x_1; @@ -3132,16 +3260,16 @@ x_1 = lean_mk_string_unchecked("' (with a dot) or '", 19, 19); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__10() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__9; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__9; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__11() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__11() { _start: { lean_object* x_1; @@ -3149,16 +3277,16 @@ x_1 = lean_mk_string_unchecked("' to use the constructor.", 25, 25); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__12() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__11; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__11; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(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) { _start: { uint8_t x_8; @@ -3197,12 +3325,12 @@ x_17 = lean_ctor_get(x_12, 0); x_18 = lean_ctor_get(x_15, 0); x_19 = lean_ctor_get(x_15, 1); x_20 = l_Lean_MessageData_ofName(x_18); -x_21 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__2; +x_21 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__2; lean_inc(x_20); lean_ctor_set_tag(x_15, 7); lean_ctor_set(x_15, 1, x_20); lean_ctor_set(x_15, 0, x_21); -x_22 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__4; +x_22 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__4; lean_ctor_set_tag(x_12, 7); lean_ctor_set(x_12, 1, x_22); lean_ctor_set(x_12, 0, x_15); @@ -3211,31 +3339,31 @@ lean_inc(x_23); lean_ctor_set_tag(x_10, 7); lean_ctor_set(x_10, 1, x_23); lean_ctor_set(x_10, 0, x_12); -x_24 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__6; +x_24 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__6; x_25 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_25, 0, x_10); lean_ctor_set(x_25, 1, x_24); -x_26 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__8; +x_26 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__8; 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_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__10; +x_28 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__10; 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_alloc_ctor(7, 2, 0); lean_ctor_set(x_30, 0, x_29); lean_ctor_set(x_30, 1, x_23); -x_31 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__12; +x_31 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__12; 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 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_33, 0, x_25); lean_ctor_set(x_33, 1, x_32); -x_34 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1; +x_34 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1; lean_inc(x_5); -x_35 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_34, x_17, x_33, x_5, x_6, x_7); +x_35 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(x_34, x_17, x_33, x_5, x_6, x_7); lean_dec(x_17); x_36 = lean_ctor_get(x_35, 1); lean_inc(x_36); @@ -3258,12 +3386,12 @@ lean_inc(x_43); lean_inc(x_42); lean_dec(x_15); x_44 = l_Lean_MessageData_ofName(x_42); -x_45 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__2; +x_45 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__2; lean_inc(x_44); x_46 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_46, 0, x_45); lean_ctor_set(x_46, 1, x_44); -x_47 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__4; +x_47 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__4; lean_ctor_set_tag(x_12, 7); lean_ctor_set(x_12, 1, x_47); lean_ctor_set(x_12, 0, x_46); @@ -3272,31 +3400,31 @@ lean_inc(x_48); lean_ctor_set_tag(x_10, 7); lean_ctor_set(x_10, 1, x_48); lean_ctor_set(x_10, 0, x_12); -x_49 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__6; +x_49 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__6; x_50 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_50, 0, x_10); lean_ctor_set(x_50, 1, x_49); -x_51 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__8; +x_51 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__8; x_52 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_52, 0, x_51); lean_ctor_set(x_52, 1, x_44); -x_53 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__10; +x_53 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__10; 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 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_55, 0, x_54); lean_ctor_set(x_55, 1, x_48); -x_56 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__12; +x_56 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__12; x_57 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_57, 0, x_55); lean_ctor_set(x_57, 1, x_56); x_58 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_58, 0, x_50); lean_ctor_set(x_58, 1, x_57); -x_59 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1; +x_59 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1; lean_inc(x_5); -x_60 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_59, x_41, x_58, x_5, x_6, x_7); +x_60 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(x_59, x_41, x_58, x_5, x_6, x_7); lean_dec(x_41); x_61 = lean_ctor_get(x_60, 1); lean_inc(x_61); @@ -3331,7 +3459,7 @@ if (lean_is_exclusive(x_66)) { x_70 = lean_box(0); } x_71 = l_Lean_MessageData_ofName(x_68); -x_72 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__2; +x_72 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__2; lean_inc(x_71); if (lean_is_scalar(x_70)) { x_73 = lean_alloc_ctor(7, 2, 0); @@ -3341,7 +3469,7 @@ if (lean_is_scalar(x_70)) { } lean_ctor_set(x_73, 0, x_72); lean_ctor_set(x_73, 1, x_71); -x_74 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__4; +x_74 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__4; x_75 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_75, 0, x_73); lean_ctor_set(x_75, 1, x_74); @@ -3350,31 +3478,31 @@ lean_inc(x_76); lean_ctor_set_tag(x_10, 7); lean_ctor_set(x_10, 1, x_76); lean_ctor_set(x_10, 0, x_75); -x_77 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__6; +x_77 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__6; x_78 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_78, 0, x_10); lean_ctor_set(x_78, 1, x_77); -x_79 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__8; +x_79 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__8; x_80 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_80, 0, x_79); lean_ctor_set(x_80, 1, x_71); -x_81 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__10; +x_81 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__10; 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 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_83, 0, x_82); lean_ctor_set(x_83, 1, x_76); -x_84 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__12; +x_84 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__12; x_85 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_85, 0, x_83); lean_ctor_set(x_85, 1, x_84); x_86 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_86, 0, x_78); lean_ctor_set(x_86, 1, x_85); -x_87 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1; +x_87 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1; lean_inc(x_5); -x_88 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_87, x_67, x_86, x_5, x_6, x_7); +x_88 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(x_87, x_67, x_86, x_5, x_6, x_7); lean_dec(x_67); x_89 = lean_ctor_get(x_88, 1); lean_inc(x_89); @@ -3419,7 +3547,7 @@ if (lean_is_exclusive(x_95)) { x_100 = lean_box(0); } x_101 = l_Lean_MessageData_ofName(x_98); -x_102 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__2; +x_102 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__2; lean_inc(x_101); if (lean_is_scalar(x_100)) { x_103 = lean_alloc_ctor(7, 2, 0); @@ -3429,7 +3557,7 @@ if (lean_is_scalar(x_100)) { } lean_ctor_set(x_103, 0, x_102); lean_ctor_set(x_103, 1, x_101); -x_104 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__4; +x_104 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__4; if (lean_is_scalar(x_97)) { x_105 = lean_alloc_ctor(7, 2, 0); } else { @@ -3443,31 +3571,31 @@ lean_inc(x_106); x_107 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_107, 0, x_105); lean_ctor_set(x_107, 1, x_106); -x_108 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__6; +x_108 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__6; 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 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__8; +x_110 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__8; x_111 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_111, 0, x_110); lean_ctor_set(x_111, 1, x_101); -x_112 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__10; +x_112 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__10; 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 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_114, 0, x_113); lean_ctor_set(x_114, 1, x_106); -x_115 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__12; +x_115 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__12; x_116 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_116, 0, x_114); lean_ctor_set(x_116, 1, x_115); x_117 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_117, 0, x_109); lean_ctor_set(x_117, 1, x_116); -x_118 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1; +x_118 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1; lean_inc(x_5); -x_119 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_118, x_96, x_117, x_5, x_6, x_7); +x_119 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(x_118, x_96, x_117, x_5, x_6, x_7); lean_dec(x_96); x_120 = lean_ctor_get(x_119, 1); lean_inc(x_120); @@ -3483,7 +3611,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__17(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_Linter_constructorNameAsVariable___elambda__1___spec__16(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -3492,7 +3620,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_Linter_constructorNameAsVariable___elambda__1___spec__13(x_4, x_6); +x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12(x_4, x_6); lean_dec(x_6); x_8 = 1; x_9 = lean_usize_add(x_2, x_8); @@ -3617,7 +3745,7 @@ x_23 = lean_box(0); lean_inc(x_3); lean_inc(x_2); lean_inc(x_19); -x_24 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12(x_9, x_16, x_19, x_15, x_21, x_22, x_23, x_2, x_3, x_20); +x_24 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11(x_9, x_16, x_19, x_15, x_21, x_22, x_23, x_2, x_3, x_20); lean_dec(x_15); if (lean_obj_tag(x_24) == 0) { @@ -3645,9 +3773,9 @@ lean_dec(x_30); lean_dec(x_29); x_33 = l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__4; x_34 = l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__6; -x_35 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(x_33, x_31, x_34); +x_35 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_33, x_31, x_34); x_36 = lean_array_size(x_35); -x_37 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(x_35, x_36, x_22, x_23, x_2, x_3, x_28); +x_37 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(x_35, x_36, x_22, x_23, x_2, x_3, x_28); lean_dec(x_3); lean_dec(x_35); x_38 = !lean_is_exclusive(x_37); @@ -3682,9 +3810,9 @@ lean_dec(x_30); lean_dec(x_29); x_43 = l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__4; x_44 = l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__6; -x_45 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(x_43, x_31, x_44); +x_45 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_43, x_31, x_44); x_46 = lean_array_size(x_45); -x_47 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(x_45, x_46, x_22, x_23, x_2, x_3, x_28); +x_47 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(x_45, x_46, x_22, x_23, x_2, x_3, x_28); lean_dec(x_3); lean_dec(x_45); x_48 = !lean_is_exclusive(x_47); @@ -3714,16 +3842,16 @@ size_t x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_objec x_52 = lean_usize_of_nat(x_30); lean_dec(x_30); x_53 = l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__4; -x_54 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__17(x_29, x_22, x_52, x_53); +x_54 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(x_29, x_22, x_52, x_53); lean_dec(x_29); x_55 = lean_array_get_size(x_54); x_56 = lean_unsigned_to_nat(1u); x_57 = lean_nat_sub(x_55, x_56); lean_dec(x_55); -x_58 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(x_54, x_31, x_57); +x_58 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_54, x_31, x_57); lean_dec(x_57); x_59 = lean_array_size(x_58); -x_60 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(x_58, x_59, x_22, x_23, x_2, x_3, x_28); +x_60 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(x_58, x_59, x_22, x_23, x_2, x_3, x_28); lean_dec(x_3); lean_dec(x_58); x_61 = !lean_is_exclusive(x_60); @@ -3861,11 +3989,24 @@ lean_dec(x_5); return x_9; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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_8); @@ -3873,11 +4014,11 @@ lean_dec(x_4); return x_13; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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_10); lean_dec(x_9); lean_dec(x_8); @@ -3885,11 +4026,11 @@ lean_dec(x_5); return x_12; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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_10); lean_dec(x_9); lean_dec(x_8); @@ -3897,11 +4038,11 @@ lean_dec(x_5); return x_12; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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_object* x_13) { _start: { lean_object* x_14; -x_14 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__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); +x_14 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__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_12); lean_dec(x_11); lean_dec(x_10); @@ -3911,11 +4052,11 @@ lean_dec(x_1); return x_14; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___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) { _start: { lean_object* x_10; -x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__7(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); @@ -3924,20 +4065,7 @@ lean_dec(x_1); return x_10; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___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) { -_start: -{ -lean_object* x_7; -x_7 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__7(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_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___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_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___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) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -3945,51 +4073,51 @@ 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_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12(x_1, x_2, x_3, x_4, x_11, x_12, x_7, x_8, x_9, x_10); +x_13 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11(x_1, x_2, x_3, x_4, x_11, x_12, x_7, x_8, x_9, x_10); lean_dec(x_4); return x_13; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(x_1, x_2); +x_3 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12(x_1, x_2); lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___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_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___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) { _start: { lean_object* x_7; -x_7 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_2); return x_7; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___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_Linter_constructorNameAsVariable___elambda__1___spec__15___lambda__1(x_1, x_2); +x_3 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___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_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(x_1, x_2, x_3); +x_4 = l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14(x_1, x_2, x_3); lean_dec(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___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) { _start: { size_t x_8; size_t x_9; lean_object* x_10; @@ -3997,13 +4125,13 @@ x_8 = lean_unbox_usize(x_2); lean_dec(x_2); x_9 = lean_unbox_usize(x_3); lean_dec(x_3); -x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(x_1, x_8, x_9, x_4, x_5, x_6, x_7); +x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15(x_1, x_8, x_9, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_1); return x_10; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__17___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_Linter_constructorNameAsVariable___elambda__1___spec__16___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; @@ -4011,7 +4139,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_Linter_constructorNameAsVariable___elambda__1___spec__17(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } @@ -4072,60 +4200,60 @@ lean_mark_persistent(l_Lean_Linter_linter_constructorNameAsVariable); lean_dec_ref(res); }l_List_forIn_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__6___lambda__1___closed__1 = _init_l_List_forIn_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__6___lambda__1___closed__1(); lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__6___lambda__1___closed__1); -l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10___closed__1 = _init_l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10___closed__1(); -lean_mark_persistent(l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__10___closed__1); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__2(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__2); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__3(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__3); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__4(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__4); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___lambda__4___closed__1); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__12___closed__1); -l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1); -l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__2 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__2(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__2); -l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__3 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__3(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__3); -l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__4 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__4(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__4); -l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__5 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__5(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__5); -l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__6 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__6(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__6); -l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__7 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__7(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__7); -l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1 = _init_l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1(); -lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__1); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__2); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__3(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__3); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__4(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__4); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__5 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__5(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__5); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__6 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__6(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__6); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__7 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__7(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__7); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__8 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__8(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__8); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__9 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__9(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__9); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__10 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__10(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__10); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__11 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__11(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__11); -l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__12 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__12(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__16___closed__12); +l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1 = _init_l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1(); +lean_mark_persistent(l_panic___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__9___closed__1); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__1(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__1); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__2(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__2); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__3(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__3); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__4(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__8___closed__4); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___lambda__5___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__11___closed__1); +l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__1 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__1(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__1); +l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__2 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__2(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__2); +l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__3 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__3(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__3); +l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__4 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__4(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__4); +l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__5 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__5(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__5); +l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__6 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__6(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__6); +l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__7 = _init_l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__7(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__13___closed__7); +l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1 = _init_l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1(); +lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__14___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__2); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__3(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__3); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__4(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__4); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__5 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__5(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__5); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__6 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__6(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__6); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__7 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__7(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__7); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__8 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__8(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__8); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__9 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__9(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__9); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__10 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__10(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__10); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__11 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__11(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__11); +l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__12 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__12(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_constructorNameAsVariable___elambda__1___spec__15___closed__12); l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__1 = _init_l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__1); l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__2 = _init_l_Lean_Linter_constructorNameAsVariable___elambda__1___closed__2(); diff --git a/stage0/stdlib/Lean/Linter/UnusedVariables.c b/stage0/stdlib/Lean/Linter/UnusedVariables.c index cb150692a468..5666c1ef7969 100644 --- a/stage0/stdlib/Lean/Linter/UnusedVariables.c +++ b/stage0/stdlib/Lean/Linter/UnusedVariables.c @@ -13,652 +13,712 @@ #ifdef __cplusplus extern "C" { #endif -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__31(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316_(lean_object*); +static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__3; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent___closed__1; -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__6; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__32(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_followAliases(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__5; -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__9; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__2; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences___spec__1(lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__10; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__9; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_insertObjImpl___rarg___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__8; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__17(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_insertObjImpl___spec__2(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__22; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__6; lean_object* lean_mk_empty_array_with_capacity(lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__8; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231_(lean_object*); +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14(lean_object*, size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__11___boxed(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__2; +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__1; uint8_t l_Lean_Syntax_matchesIdent(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__3; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__10; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__11; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__1; -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__1(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__9; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__6; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__7; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690_(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Linter_getUnusedVariablesIgnoreFns(lean_object*); +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__1(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_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentArray_toArray___rarg(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107_(lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__1___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__9; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987_(lean_object*); lean_object* l_Lean_ConstantInfo_type(lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments_visitEntry___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__1; +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getHeadInfo(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__9; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__10; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__2(lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__6; uint64_t l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__4; LEAN_EXPORT lean_object* l_Lean_Linter_getUnusedVariablesIgnoreFns___boxed(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__11; -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__8; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences___spec__1___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___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*); uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_ForEachExpr_visit___spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_insertObjImpl___spec__3(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__4; size_t lean_uint64_to_usize(uint64_t); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments_visitNode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__2; LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_insertObjImpl___spec__1(size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_initFn____x40_Lean_Linter_UnusedVariables___hyg_5794_(lean_object*); -LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__18; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__5; lean_object* l_Lean_Syntax_getId(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__19; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__1; uint8_t l___private_Lean_Syntax_0__String_beqRange____x40_Lean_Syntax___hyg_95_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_getLinterUnusedVariables___boxed(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__4; +LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___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_array_push(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__3(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__12; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___closed__1; lean_object* l_Array_qpartition___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__2; -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__21; -static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___closed__1; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__2(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__16; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__8; lean_object* lean_mk_array(lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__3; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11___boxed(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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__13; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__2; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArgs(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__11; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__13; uint8_t l_String_Range_includes(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__12; -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* l_Lean_Elab_InfoTree_hasSorry(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__3(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*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__3; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(lean_object*, lean_object*, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__10; static lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___closed__3; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__7(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments_visitExpr___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_UnusedVariables_visitAssignments___closed__2; -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__4; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__10; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_getLinterUnusedVariablesFunArgs___boxed(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__19; +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__1; lean_object* lean_environment_find(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__1; lean_object* l_Lean_Attribute_Builtin_ensureNoArgs(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__4; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_logAt___at_Lean_Elab_Command_runLinters___spec__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__22; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__30___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__2; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__5___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_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__7; uint8_t l_Lean_Linter_getLinterValue(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__8; +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__9; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__3___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__8___boxed(lean_object*, lean_object*, 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_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__1; +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); lean_object* l_Lean_stringToMessageData(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences___spec__16___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_EStateM_instMonad(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_insertObjImpl(lean_object*); lean_object* l_Lean_PersistentArray_toList___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3___boxed(lean_object**); uint8_t l_List_any___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); lean_object* l_List_head_x21___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments_visitNode___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__4; -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__8(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__17; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_getUnusedVariablesIgnoreFns___rarg___closed__1; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_getLinterUnusedVariablesFunArgs(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5___closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5___closed__1; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__6; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_insertObjImpl___spec__1___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__7; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__3; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__2; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__18(lean_object*, lean_object*); lean_object* lean_string_utf8_byte_size(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__10; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__12(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__5; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__4; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__3; +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2(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_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___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*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__12(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_mkIgnoreFnImpl___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences___spec__5(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__8; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___boxed(lean_object**); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__8; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25(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*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__13; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__2; -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__11; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__1(lean_object*); static lean_object* l_Lean_Linter_mkIgnoreFnImpl___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__2; size_t lean_ptr_addr(lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__5; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__7; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__4; +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__7(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ForEachExpr_visit___at_Lean_Linter_UnusedVariables_visitAssignments_visitExpr___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_getLinterUnusedVariablesPatternVars(lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_47____closed__2; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__6; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__7; -static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__7; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__7; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__9; +LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__6; +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__4; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__18; +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__4; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__10; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_visitAssignments_visitNode___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__6; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariablesIgnoreFnsExt; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__4; static lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___closed__2; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__3; lean_object* lean_local_ctx_find(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__7; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__29___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__1; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__8; lean_object* lean_st_ref_take(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__24; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__11; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_ForEachExpr_visit___spec__3(lean_object*); static lean_object* l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent___closed__2; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3(lean_object*, size_t, size_t); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__6; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_86_(lean_object*); lean_object* l_Lean_declareBuiltin(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__2; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_insertObjImpl___spec__4(lean_object*, lean_object*, lean_object*); lean_object* l_List_filterMapTR_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__3; lean_object* l_Lean_registerPersistentEnvExtensionUnsafe___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments_visitExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1(lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_shift_right(uint64_t, uint64_t); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__11; +static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__4; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7___boxed(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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__2; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__14; +static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__6; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4___boxed(lean_object**); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1; lean_object* lean_nat_div(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___closed__1; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19(lean_object*, lean_object*, lean_object*, uint8_t, 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_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__12; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379_(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__7; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__7; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Info_updateContext_x3f(lean_object*, lean_object*); -static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__2___boxed(lean_object*, lean_object*, lean_object*); uint64_t l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(lean_object*); lean_object* l_Lean_PersistentEnvExtension_addEntry___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__6; uint8_t l_Lean_Syntax_Stack_matches(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__8; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_47____closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__7; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__9; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__1___boxed(lean_object*, lean_object*); +static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentEnvExtension_getState___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__7; lean_object* lean_eval_const(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__8; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__2; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15___boxed(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_linter_unusedVariables_patternVars; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_86____closed__2; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__8(lean_object*); -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__2; lean_object* l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__20; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__2; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__6; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__5; -LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___lambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__2; lean_object* l_Lean_MessageData_ofFormat(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences___spec__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__1; lean_object* l_Lean_setEnv___at_Lean_registerParametricAttribute___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555_(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__2; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__24; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences_go(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__13; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____closed__1; -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__9___boxed(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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__8; lean_object* l_Lean_throwError___at_Lean_registerTagAttribute___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_filterMapTR_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__2(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__13; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948_(lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__4(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__11; lean_object* lean_st_mk_ref(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____closed__1; static lean_object* l_Lean_Linter_UnusedVariables_visitAssignments___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__6; -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__4; uint8_t l_Lean_MessageData_hasTag(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___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, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601_(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125_(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__8; LEAN_EXPORT lean_object* l_Lean_Linter_mkIgnoreFnImpl___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__3; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_visitAssignments___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_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__7; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__3; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__11(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l_Lean_Linter_mkIgnoreFnImpl___closed__5; -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__5; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__7; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__2; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__2; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__4; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__10; -static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__2; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__5; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__1; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__9; +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__6; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__32___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__6; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__1; uint64_t l_Lean_Expr_hash(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__3; -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__20(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__9; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__6; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__4; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__8; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__6; +LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__1___boxed(lean_object*, lean_object*); lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__4(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_mkIgnoreFnImpl___closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__13; -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(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*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Command_instMonadCommandElabM; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__1; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__4; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___closed__1; uint8_t lean_name_eq(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__5; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___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_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__8; +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__23(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_MessageData_isUnusedVariableWarning___lambda__1(lean_object*); -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_visitAssignments___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__4; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__1; -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences___spec__14(lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__16; +static lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__1; +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_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__7; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__3; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__8; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__3; static lean_object* l_Lean_Linter_mkIgnoreFnImpl___closed__4; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__1; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__16(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__21; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__1; uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); static lean_object* l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__7(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l_Lean_Linter_mkIgnoreFnImpl___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__15; LEAN_EXPORT lean_object* l_Lean_Linter_builtinUnusedVariablesIgnoreFnsRef; -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15(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_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(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*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__2; -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__7(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; uint8_t l_Lean_Syntax_isIdent(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__6; -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__5; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__12; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments_visitExpr___lambda__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__3(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__9; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__3; -LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__7___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__2; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__5(lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__11; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__3; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__7; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__20; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__7; +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__2; static lean_object* l_Lean_Linter_getLinterUnusedVariables___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__2; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__9; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__11; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_visitAssignments_visitNode___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_linter_unusedVariables_analyzeTactics; lean_object* l_Lean_Elab_Command_addLinter(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___lambda__1___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__3___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_ForEachExpr_visit___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_insertObjImpl___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__15; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__5; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___lambda__1___boxed(lean_object*, lean_object*); lean_object* l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__1; -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__7; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__4; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475_(lean_object*); +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__4; LEAN_EXPORT uint8_t l_Lean_MessageData_isUnusedVariableWarning(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_visitAssignments_visitNode___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_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__6; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, uint8_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_userName(lean_object*); lean_object* l_Substring_nextn(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277_(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__4; -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__3; -static lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____closed__1; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__1; lean_object* l_panic___at_Lean_Parser_ParserState_mkUnexpectedTokenErrors___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__7; LEAN_EXPORT lean_object* l_IO_ofExcept___at_Lean_Linter_mkIgnoreFnImpl___spec__1(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__10; +static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__7; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_followAliases___boxed(lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__4(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__9; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___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*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static size_t l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____closed__1; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__1; uint8_t l_Lean_Name_hasMacroScopes(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__4; -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__2(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____closed__1; static lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__2___closed__1; lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_ForEachExpr_visit___spec__6(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_linter_unusedVariables; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____closed__1; uint8_t l_String_Range_contains(lean_object*, lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4___boxed(lean_object**); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__8; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__5; lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); static lean_object* l_Lean_Linter_mkIgnoreFnImpl___closed__6; lean_object* lean_string_length(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__4; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__5(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20___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_Linter_UnusedVariables_collectReferences(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____closed__1; uint8_t l_Lean_Syntax_hasArgs(lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_getLinterUnusedVariables(lean_object*); -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__2; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__5; -static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640_(lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_findStack_x3f(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_MessageData_isUnusedVariableWarning___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_getUnusedVariablesIgnoreFns___rarg___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__1; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__1; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982_(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__3; static lean_object* l_Lean_MessageData_isUnusedVariableWarning___closed__1; -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____closed__1; +LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__1(lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__9; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__9(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_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments_visitExpr___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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* l_Lean_Syntax_isOfKind___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_getUnusedVariablesIgnoreFns___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__3; +static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__2; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__3; +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___boxed(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*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__8; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__12; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__4(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__4; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____closed__1; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__8(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_initFn____x40_Lean_Linter_UnusedVariables___hyg_6304_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__6___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021_(lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__2; +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___lambda__1(lean_object*); uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__8; +LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyMAux___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__12(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__9; LEAN_EXPORT lean_object* l_Lean_MessageData_isUnusedVariableWarning___boxed(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__6; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__10; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__5; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__7; uint64_t lean_uint64_xor(uint64_t, uint64_t); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); uint8_t l_Lean_Syntax_isNone(lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_86____closed__4; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_visitAssignments_visitNode___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_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703_(lean_object*); -static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__4; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___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_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192_(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__9; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___lambda__1___boxed(lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___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_Linter_UnusedVariables_unusedVariables___elambda__1___spec__2(lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387_(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__29(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__7; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__14; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6(lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__10; +static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__2; lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); +static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Linter_mkIgnoreFnImpl___lambda__1___boxed(lean_object*); lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__2; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__12; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__13___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__4; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__4; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___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* l_Lean_Elab_Info_range_x3f(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__3; +static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__5; +lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_registerBuiltinAttribute(lean_object*, lean_object*); +static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__10; lean_object* l_List_reverse___rarg(lean_object*); -static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__3; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3(lean_object*, size_t, size_t); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__12; uint8_t l___private_Lean_Attributes_0__Lean_beqAttributeKind____x40_Lean_Attributes___hyg_162_(uint8_t, uint8_t); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__9; -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__4; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__12; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_86____closed__1; size_t lean_usize_sub(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Command_instInhabitedScope; lean_object* lean_array_mk(lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22(lean_object*, uint8_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__5(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443_(lean_object*); static lean_object* l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8___closed__1; -static lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2___closed__1; -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__17; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_instantiateMVarsCore(lean_object*, lean_object*); uint8_t l_Substring_beq(lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__5; size_t lean_usize_add(size_t, size_t); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__13(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_hasFVar(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__3; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016_(lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences___spec__10(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__4; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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*); lean_object* l_Lean_KVMap_findCore(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__9(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__2; lean_object* lean_array_uget(lean_object*, size_t); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__14; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__9(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); size_t lean_array_size(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_47_(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__7; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__6; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8_(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15(lean_object*, lean_object*); lean_object* lean_io_error_to_string(lean_object*); lean_object* l_instInhabitedOfMonad___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_insertObjImpl___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__14; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___boxed(lean_object*); -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__2___boxed(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_InfoTree_findInfo_x3f(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__6; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__6; +static lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__4; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__12; LEAN_EXPORT lean_object* l_Lean_Linter_getLinterUnusedVariablesPatternVars___boxed(lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__6; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_47____closed__5; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__2; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__6; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__9; +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__5; +static lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___closed__1; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_47____closed__1; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_UnusedVariables_visitAssignments___closed__3; -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__11; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ForEachExpr_visit___at_Lean_Linter_UnusedVariables_visitAssignments_visitExpr___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_mkIgnoreFnImpl___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__5; lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_insertObjImpl___spec__4___at_Lean_Linter_UnusedVariables_insertObjImpl___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_followAliases___spec__1___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__11; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__10(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_mkIgnoreFnImpl___closed__7; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__11; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1(lean_object*, lean_object*, lean_object*); lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1(lean_object*, size_t, size_t, lean_object*); lean_object* lean_array_get_size(lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__7___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__2(lean_object*, lean_object*); uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__8; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_47____closed__4; LEAN_EXPORT lean_object* l_Lean_Linter_mkIgnoreFnImpl(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__7; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__5; +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__13(lean_object*, size_t, size_t); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__3; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__7; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742_(lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); -static lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__2; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11___boxed(lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__5; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__3; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___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_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__23; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__30(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_followAliases___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_86____closed__5; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__2; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__9; lean_object* lean_nat_add(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__2; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__4; lean_object* l_Lean_Elab_Info_stx(lean_object*); lean_object* l_EStateM_bind___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__3; -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__4; +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_visitAssignments_visitEntry(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__6; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__6___boxed(lean_object**); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5___boxed(lean_object**); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__1___boxed(lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___lambda__1(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__3; +LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__12___boxed(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); -static lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__5; +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Attribute_Builtin_ensureNoArgs___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__6; -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651_(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__23; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__31___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_Linter_UnusedVariables_collectReferences_go___spec__19(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__4; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_linter_unusedVariables_funArgs; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_UnusedVariables_collectReferences___spec__17(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__11(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__10; lean_object* l_Lean_MessageData_ofName(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__2; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__1; lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__5; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__4; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__4; +static lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_insertObjImpl___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__10; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__12; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__7; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__4; +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_86____closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences___spec__16___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__5; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___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_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__3; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__1___boxed(lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____closed__1; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__3(lean_object*); lean_object* l_List_get_x3f___rarg(lean_object*, lean_object*); lean_object* l_ReaderT_instMonad___rarg(lean_object*); size_t lean_usize_land(size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__5; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__9; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__5; LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__9; -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__3; uint8_t l_Lean_Elab_Info_contains(lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___boxed(lean_object**); +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____closed__1; uint8_t l_Lean_MessageLog_hasErrors(lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__5; static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__1() { _start: { @@ -887,6 +947,72 @@ x_5 = l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___ return x_5; } } +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("analyzeTactics", 14, 14); +return x_1; +} +} +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__2; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__1; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("enable analysis of local variables in presence of tactic proofs\n\nBy default, the linter will limit itself to linting a declaration's parameters whenever tactic proofs are present as these can be expensive to analyze. Enabling this option extends linting to local variables both inside and outside tactic proofs, though it can also lead to some false negatives as intermediate tactic states may reference some variables without the declaration ultimately depending on them.", 472, 472); +return x_1; +} +} +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__3; +x_4 = lean_box(x_1); +x_5 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_2); +lean_ctor_set(x_5, 2, x_3); +return x_5; +} +} +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__8; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__2; +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__1; +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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125_(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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__2; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__4; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____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; +} +} static lean_object* _init_l_Lean_Linter_getLinterUnusedVariables___closed__1() { _start: { @@ -1340,7 +1466,7 @@ lean_dec(x_1); return x_7; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -1349,11 +1475,11 @@ x_2 = lean_array_mk(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; uint8_t x_4; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; x_3 = lean_st_mk_ref(x_2, x_1); x_4 = !lean_is_exclusive(x_3); if (x_4 == 0) @@ -1416,7 +1542,7 @@ return x_12; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____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) { _start: { uint8_t x_7; @@ -1479,7 +1605,7 @@ return x_20; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__2(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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; @@ -1522,7 +1648,7 @@ x_19 = 0; x_20 = lean_usize_of_nat(x_9); lean_dec(x_9); lean_inc(x_5); -x_21 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__1(x_8, x_19, x_20, x_4, x_5, x_6); +x_21 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__1(x_8, x_19, x_20, x_4, x_5, x_6); lean_dec(x_8); if (lean_obj_tag(x_21) == 0) { @@ -1576,7 +1702,7 @@ return x_31; } } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__1(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; uint8_t x_4; @@ -1602,7 +1728,7 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__2(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; @@ -1616,7 +1742,7 @@ lean_ctor_set(x_5, 1, x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__3(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; @@ -1666,7 +1792,7 @@ lean_free_object(x_5); x_17 = 0; x_18 = lean_usize_of_nat(x_9); lean_dec(x_9); -x_19 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__2(x_1, x_17, x_18, x_7, x_2, x_8); +x_19 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__2(x_1, x_17, x_18, x_7, x_2, x_8); if (lean_obj_tag(x_19) == 0) { uint8_t x_20; @@ -1774,7 +1900,7 @@ size_t x_45; size_t x_46; lean_object* x_47; x_45 = 0; x_46 = lean_usize_of_nat(x_35); lean_dec(x_35); -x_47 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__2(x_1, x_45, x_46, x_33, x_2, x_34); +x_47 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__2(x_1, x_45, x_46, x_33, x_2, x_34); 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; @@ -1832,7 +1958,7 @@ return x_57; } } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__4(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__4(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; @@ -1911,7 +2037,7 @@ return x_23; } } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__5(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__5(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; @@ -1923,7 +2049,7 @@ x_4 = lean_array_mk(x_3); return x_4; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__1() { _start: { lean_object* x_1; @@ -1931,17 +2057,17 @@ x_1 = lean_mk_string_unchecked("number of local entries: ", 25, 25); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__1; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6(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; @@ -1951,14 +2077,14 @@ x_4 = l_List_lengthTRAux___rarg(x_2, x_3); x_5 = l___private_Init_Data_Repr_0__Nat_reprFast(x_4); x_6 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_6, 0, x_5); -x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__2; +x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__2; x_8 = lean_alloc_ctor(5, 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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__1() { _start: { lean_object* x_1; @@ -1966,87 +2092,87 @@ x_1 = lean_mk_string_unchecked("unusedVariablesIgnoreFnsExt", 27, 27); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__8; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__1; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__3() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__1), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__4() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__2), 2, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__2), 2, 0); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__4; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__4; x_3 = lean_alloc_closure((void*)(l_EStateM_bind___rarg), 3, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__6() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__3___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__3___boxed), 3, 0); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__7() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__4), 2, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__4), 2, 0); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__8() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__5), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__5), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__9() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__10() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____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; lean_object* x_7; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__2; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__5; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__6; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__7; -x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__8; -x_6 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__9; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__2; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__5; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__6; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__7; +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__8; +x_6 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__9; x_7 = lean_alloc_ctor(0, 6, 0); lean_ctor_set(x_7, 0, x_1); lean_ctor_set(x_7, 1, x_2); @@ -2057,16 +2183,16 @@ lean_ctor_set(x_7, 5, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__10; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__10; x_3 = l_Lean_registerPersistentEnvExtensionUnsafe___rarg(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____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) { _start: { size_t x_7; size_t x_8; lean_object* x_9; @@ -2074,12 +2200,12 @@ x_7 = lean_unbox_usize(x_2); lean_dec(x_2); x_8 = lean_unbox_usize(x_3); lean_dec(x_3); -x_9 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__1(x_1, x_7, x_8, x_4, x_5, x_6); +x_9 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__1(x_1, x_7, x_8, x_4, x_5, x_6); lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____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: { size_t x_7; size_t x_8; lean_object* x_9; @@ -2087,30 +2213,30 @@ x_7 = lean_unbox_usize(x_2); lean_dec(x_2); x_8 = lean_unbox_usize(x_3); lean_dec(x_3); -x_9 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____spec__2(x_1, x_7, x_8, x_4, x_5, x_6); +x_9 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____spec__2(x_1, x_7, x_8, x_4, x_5, x_6); lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__3(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__3(x_1, x_2, x_3); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6(x_1); +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6(x_1); lean_dec(x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -2118,28 +2244,28 @@ x_1 = lean_mk_string_unchecked("addBuiltinUnusedVariablesIgnoreFn", 33, 33); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__8; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__1; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__2; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__2; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____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; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; @@ -2150,13 +2276,13 @@ lean_dec(x_6); x_8 = lean_box(0); lean_inc(x_1); x_9 = l_Lean_Expr_const___override(x_1, x_8); -x_10 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__3; +x_10 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__3; x_11 = l_Lean_Expr_app___override(x_10, x_9); x_12 = l_Lean_declareBuiltin(x_1, x_11, x_3, x_4, x_7); return x_12; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__1() { _start: { lean_object* x_1; @@ -2164,16 +2290,16 @@ x_1 = lean_mk_string_unchecked("invalid attribute '", 19, 19); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__1; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__3() { _start: { lean_object* x_1; lean_object* x_2; @@ -2182,7 +2308,7 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____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_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____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; @@ -2206,11 +2332,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; uint8_t x_19; lean_dec(x_1); x_13 = l_Lean_MessageData_ofName(x_2); -x_14 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__2; +x_14 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__2; 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 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__3; +x_16 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__3; x_17 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); @@ -2239,7 +2365,7 @@ else lean_object* x_23; lean_object* x_24; lean_dec(x_2); x_23 = lean_box(0); -x_24 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1(x_1, x_23, x_4, x_5, x_9); +x_24 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1(x_1, x_23, x_4, x_5, x_9); return x_24; } } @@ -2269,7 +2395,7 @@ return x_28; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__1() { _start: { lean_object* x_1; @@ -2277,16 +2403,16 @@ x_1 = lean_mk_string_unchecked("', must be global", 17, 17); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__1; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____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_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____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) { _start: { lean_object* x_8; @@ -2305,11 +2431,11 @@ 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; uint8_t x_18; lean_dec(x_2); x_12 = l_Lean_MessageData_ofName(x_1); -x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__2; +x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__2; +x_15 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__2; x_16 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); @@ -2338,7 +2464,7 @@ 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_601____lambda__2(x_2, x_1, x_22, x_5, x_6, x_9); +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; } @@ -2370,7 +2496,7 @@ return x_27; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__1() { _start: { lean_object* x_1; @@ -2378,25 +2504,25 @@ x_1 = lean_mk_string_unchecked("attribute cannot be erased", 26, 26); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__1; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__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; -x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__2; +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1() { _start: { lean_object* x_1; @@ -2404,7 +2530,7 @@ x_1 = l_Lean_Linter_unusedVariablesIgnoreFnsExt; return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5(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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5(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; @@ -2445,7 +2571,7 @@ lean_inc(x_20); lean_dec(x_18); lean_ctor_set(x_6, 1, x_19); lean_ctor_set(x_6, 0, x_1); -x_21 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1; +x_21 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1; x_22 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_21, x_10, x_6); x_23 = l_Lean_setEnv___at_Lean_registerParametricAttribute___spec__3(x_22, x_3, x_4, x_20); return x_23; @@ -2521,7 +2647,7 @@ lean_inc(x_43); lean_dec(x_41); lean_ctor_set(x_6, 1, x_42); lean_ctor_set(x_6, 0, x_1); -x_44 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1; +x_44 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1; x_45 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_44, x_10, x_6); x_46 = l_Lean_setEnv___at_Lean_registerParametricAttribute___spec__3(x_45, x_3, x_4, x_43); return x_46; @@ -2611,7 +2737,7 @@ lean_dec(x_65); x_68 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_68, 0, x_1); lean_ctor_set(x_68, 1, x_66); -x_69 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1; +x_69 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1; x_70 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_69, x_56, x_68); x_71 = l_Lean_setEnv___at_Lean_registerParametricAttribute___spec__3(x_70, x_3, x_4, x_67); return x_71; @@ -2653,7 +2779,7 @@ return x_79; } } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____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_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____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) { _start: { lean_object* x_7; @@ -2677,11 +2803,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; uint8_t x_19; lean_dec(x_1); x_13 = l_Lean_MessageData_ofName(x_2); -x_14 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__2; +x_14 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__2; 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 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__3; +x_16 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__3; x_17 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); @@ -2710,7 +2836,7 @@ else lean_object* x_23; lean_object* x_24; lean_dec(x_2); x_23 = lean_box(0); -x_24 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5(x_1, x_23, x_4, x_5, x_9); +x_24 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5(x_1, x_23, x_4, x_5, x_9); return x_24; } } @@ -2740,7 +2866,7 @@ return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____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_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____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) { _start: { lean_object* x_8; @@ -2759,11 +2885,11 @@ 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; uint8_t x_18; lean_dec(x_2); x_12 = l_Lean_MessageData_ofName(x_1); -x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__2; +x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__2; +x_15 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__2; x_16 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); @@ -2792,7 +2918,7 @@ 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_601____lambda__6(x_2, x_1, x_22, x_5, x_6, x_9); +x_23 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__6(x_2, x_1, x_22, x_5, x_6, x_9); lean_dec(x_5); return x_23; } @@ -2824,7 +2950,7 @@ return x_27; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__1() { _start: { lean_object* x_1; @@ -2832,17 +2958,17 @@ x_1 = lean_mk_string_unchecked("builtin_unused_variables_ignore_fn", 34, 34); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -2852,17 +2978,17 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__3; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__3; x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__8; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__5() { _start: { lean_object* x_1; @@ -2870,17 +2996,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__4; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__5; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__4; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__7() { _start: { lean_object* x_1; @@ -2888,37 +3014,37 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__6; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__7; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__6; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__8; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__8; x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__10() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__9; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__9; x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__8; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__11() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__11() { _start: { lean_object* x_1; @@ -2926,17 +3052,17 @@ x_1 = lean_mk_string_unchecked("UnusedVariables", 15, 15); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__12() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__10; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__11; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__10; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__11; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__13() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__13() { _start: { lean_object* x_1; @@ -2944,27 +3070,27 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__14() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__12; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__13; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__12; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__13; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__15() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__14; -x_2 = lean_unsigned_to_nat(601u); +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__14; +x_2 = lean_unsigned_to_nat(640u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__16() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__16() { _start: { lean_object* x_1; @@ -2972,7 +3098,7 @@ x_1 = lean_mk_string_unchecked("(builtin) ", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__17() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__17() { _start: { lean_object* x_1; @@ -2980,23 +3106,23 @@ x_1 = lean_mk_string_unchecked("Marks a function of type `Lean.Linter.IgnoreFunc return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__18() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__16; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__17; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__16; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__17; x_3 = lean_string_append(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__19() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__19() { _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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__15; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__2; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__18; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__15; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__2; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__18; x_4 = 1; x_5 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_5, 0, x_1); @@ -3006,15 +3132,15 @@ lean_ctor_set_uint8(x_5, sizeof(void*)*3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__20() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__20() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___boxed), 4, 0); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__21() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__21() { _start: { lean_object* x_1; @@ -3022,33 +3148,33 @@ x_1 = lean_mk_string_unchecked("unused_variables_ignore_fn", 26, 26); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__22() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__22() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__21; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__21; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__23() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__23() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__4; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__17; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__17; x_3 = lean_string_append(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__24() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__24() { _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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__15; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__22; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__23; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__15; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__22; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__23; x_4 = 1; x_5 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_5, 0, x_1); @@ -3058,15 +3184,15 @@ lean_ctor_set_uint8(x_5, sizeof(void*)*3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640_(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; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__2; -x_3 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___boxed), 7, 1); +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__2; +x_3 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___boxed), 7, 1); lean_closure_set(x_3, 0, x_2); -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__19; -x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__20; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__19; +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__20; x_6 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_6, 0, x_4); lean_ctor_set(x_6, 1, x_3); @@ -3078,10 +3204,10 @@ lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_o x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); lean_dec(x_7); -x_9 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__22; -x_10 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__7___boxed), 7, 1); +x_9 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__22; +x_10 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__7___boxed), 7, 1); lean_closure_set(x_10, 0, x_9); -x_11 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__24; +x_11 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__24; x_12 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_12, 0, x_11); lean_ctor_set(x_12, 1, x_10); @@ -3113,84 +3239,84 @@ return x_17; } } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1(x_1, x_2, x_3, x_4, x_5); +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; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____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_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2(x_1, x_2, x_3, x_4, x_5, x_6); +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; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____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_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____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) { _start: { 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_601____lambda__3(x_1, x_2, x_3, x_8, x_5, x_6, x_7); +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; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5(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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____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_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____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) { _start: { lean_object* x_7; -x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__6(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__6(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; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____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_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____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) { _start: { 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_601____lambda__7(x_1, x_2, x_3, x_8, x_5, x_6, x_7); +x_9 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__7(x_1, x_2, x_3, x_8, x_5, x_6, x_7); lean_dec(x_6); return x_9; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -3198,27 +3324,27 @@ x_1 = lean_mk_string_unchecked("null", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4() { _start: { lean_object* x_1; @@ -3226,7 +3352,7 @@ x_1 = lean_mk_string_unchecked("Parser", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5() { _start: { lean_object* x_1; @@ -3234,7 +3360,7 @@ x_1 = lean_mk_string_unchecked("Command", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__6() { _start: { lean_object* x_1; @@ -3242,114 +3368,114 @@ x_1 = lean_mk_string_unchecked("variable", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____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; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__6; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__7; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__7; 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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__8; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__8; 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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__10() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__9; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__11() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__10; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__12() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__11; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___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; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1(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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__12; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__12; x_5 = l_Lean_Syntax_Stack_matches(x_2, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -3357,114 +3483,114 @@ x_1 = lean_mk_string_unchecked("structure", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__4; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__5; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__6; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___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; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1(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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__7; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__7; x_5 = l_Lean_Syntax_Stack_matches(x_2, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -3472,89 +3598,89 @@ x_1 = lean_mk_string_unchecked("inductive", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__4; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__5; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__6; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__7; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__9() { _start: { lean_object* x_1; @@ -3562,19 +3688,19 @@ x_1 = lean_mk_string_unchecked("optDeclSig", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__10() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____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; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__9; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__11() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__11() { _start: { lean_object* x_1; @@ -3582,47 +3708,47 @@ x_1 = lean_mk_string_unchecked("declSig", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__12() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__11; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__13() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__12; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__12; 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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__14() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__10; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__13; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__10; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___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_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1(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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__8; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__8; lean_inc(x_2); x_5 = l_Lean_Syntax_Stack_matches(x_2, x_4); if (x_5 == 0) @@ -3670,7 +3796,7 @@ else lean_object* x_16; lean_object* x_17; uint8_t x_18; x_16 = lean_alloc_closure((void*)(l_Lean_Syntax_isOfKind___boxed), 2, 1); lean_closure_set(x_16, 0, x_11); -x_17 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__14; +x_17 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__14; x_18 = l_List_any___rarg(x_17, x_16); return x_18; } @@ -3678,45 +3804,45 @@ return x_18; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__1() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__10; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__10; 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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -3728,55 +3854,55 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__1; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__2; 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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__3; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__4; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__5; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__7() { _start: { lean_object* x_1; @@ -3784,19 +3910,19 @@ x_1 = lean_mk_string_unchecked("ctor", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__7; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__7; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__9() { _start: { lean_object* x_1; @@ -3804,47 +3930,47 @@ x_1 = lean_mk_string_unchecked("structSimpleBinder", 18, 18); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__10() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____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; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__9; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__11() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__10; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__10; 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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__12() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__8; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__11; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__8; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___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; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1(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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__6; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__6; lean_inc(x_2); x_5 = l_Lean_Syntax_Stack_matches(x_2, x_4); if (x_5 == 0) @@ -3877,100 +4003,100 @@ lean_inc(x_11); lean_dec(x_10); x_12 = lean_alloc_closure((void*)(l_Lean_Syntax_isOfKind___boxed), 2, 1); lean_closure_set(x_12, 0, x_11); -x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__12; +x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__12; x_14 = l_List_any___rarg(x_13, x_12); return x_14; } } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__1() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__12; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__12; 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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__1; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__2; 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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__2; 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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__4; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__6() { _start: { lean_object* x_1; @@ -3978,19 +4104,19 @@ x_1 = lean_mk_string_unchecked("opaque", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____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; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__6; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__8() { _start: { lean_object* x_1; @@ -3998,47 +4124,47 @@ x_1 = lean_mk_string_unchecked("axiom", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__8; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__10() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__9; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__9; 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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__11() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__10; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__7; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___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; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1(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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__5; lean_inc(x_2); x_5 = l_Lean_Syntax_Stack_matches(x_2, x_4); if (x_5 == 0) @@ -4071,42 +4197,42 @@ lean_inc(x_11); lean_dec(x_10); x_12 = lean_alloc_closure((void*)(l_Lean_Syntax_isOfKind___boxed), 2, 1); lean_closure_set(x_12, 0, x_11); -x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__11; +x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__11; x_14 = l_List_any___rarg(x_13, x_12); return x_14; } } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__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_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____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; uint8_t x_7; @@ -4175,18 +4301,18 @@ return x_20; } } } -LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__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; x_3 = lean_array_get_size(x_1); x_4 = lean_mk_empty_array_with_capacity(x_3); x_5 = lean_unsigned_to_nat(0u); -x_6 = l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__2(x_1, x_2, x_3, x_5, x_4); +x_6 = l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__2(x_1, x_2, x_3, x_5, x_4); return x_6; } } -static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__1() { +static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__1() { _start: { lean_object* x_1; @@ -4194,7 +4320,7 @@ x_1 = lean_mk_string_unchecked("Attr", 4, 4); return x_1; } } -static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__2() { +static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__2() { _start: { lean_object* x_1; @@ -4202,19 +4328,19 @@ x_1 = lean_mk_string_unchecked("extern", 6, 6); return x_1; } } -static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__3() { +static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__1; -x_4 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__2; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__1; +x_4 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__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_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__4() { +static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__4() { _start: { lean_object* x_1; @@ -4222,19 +4348,19 @@ x_1 = lean_mk_string_unchecked("simple", 6, 6); return x_1; } } -static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__5() { +static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__1; -x_4 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__4; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__1; +x_4 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__4; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__6() { +static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__6() { _start: { lean_object* x_1; @@ -4242,17 +4368,17 @@ x_1 = lean_mk_string_unchecked("implemented_by", 14, 14); return x_1; } } -static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__7() { +static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__6; +x_2 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3(lean_object* x_1, size_t x_2, size_t x_3) { +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3(lean_object* x_1, size_t x_2, size_t x_3) { _start: { uint8_t x_4; @@ -4261,13 +4387,13 @@ if (x_4 == 0) { lean_object* x_5; lean_object* x_6; uint8_t x_7; x_5 = lean_array_uget(x_1, x_2); -x_6 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__3; +x_6 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__3; lean_inc(x_5); x_7 = l_Lean_Syntax_isOfKind(x_5, x_6); if (x_7 == 0) { lean_object* x_8; uint8_t x_9; -x_8 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__5; +x_8 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__5; lean_inc(x_5); x_9 = l_Lean_Syntax_isOfKind(x_5, x_8); if (x_9 == 0) @@ -4284,7 +4410,7 @@ 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_5, x_13); -x_15 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__7; +x_15 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__7; x_16 = l_Lean_Syntax_matchesIdent(x_14, x_15); lean_dec(x_14); if (x_16 == 0) @@ -4336,7 +4462,7 @@ return x_28; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -4344,7 +4470,7 @@ x_1 = lean_mk_string_unchecked("Term", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__2() { _start: { lean_object* x_1; @@ -4352,19 +4478,19 @@ x_1 = lean_mk_string_unchecked("attrInstance", 12, 12); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____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; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__2; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__4() { _start: { lean_object* x_1; @@ -4372,23 +4498,23 @@ x_1 = lean_mk_string_unchecked("attrKind", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__4; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__4; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__3; lean_inc(x_1); x_3 = l_Lean_Syntax_isOfKind(x_1, x_2); if (x_3 == 0) @@ -4403,7 +4529,7 @@ else lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; x_5 = lean_unsigned_to_nat(0u); x_6 = l_Lean_Syntax_getArg(x_1, x_5); -x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__5; +x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__5; lean_inc(x_6); x_8 = l_Lean_Syntax_isOfKind(x_6, x_7); if (x_8 == 0) @@ -4441,7 +4567,7 @@ return x_15; } } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__2(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; uint8_t x_7; @@ -4485,14 +4611,14 @@ size_t x_16; size_t x_17; uint8_t x_18; x_16 = 0; x_17 = lean_usize_of_nat(x_13); lean_dec(x_13); -x_18 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3(x_2, x_16, x_17); +x_18 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3(x_2, x_16, x_17); return x_18; } } } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__1() { _start: { lean_object* x_1; @@ -4500,19 +4626,19 @@ x_1 = lean_mk_string_unchecked("noncomputable", 13, 13); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3(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; uint8_t x_7; @@ -4538,7 +4664,7 @@ lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; x_11 = lean_unsigned_to_nat(0u); x_12 = l_Lean_Syntax_getArg(x_6, x_11); lean_dec(x_6); -x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__2; +x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__2; x_14 = l_Lean_Syntax_isOfKind(x_12, x_13); if (x_14 == 0) { @@ -4550,7 +4676,7 @@ else { lean_object* x_16; uint8_t x_17; x_16 = lean_box(0); -x_17 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__2(x_1, x_2, x_16); +x_17 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__2(x_1, x_2, x_16); return x_17; } } @@ -4560,12 +4686,12 @@ else lean_object* x_18; uint8_t x_19; lean_dec(x_6); x_18 = lean_box(0); -x_19 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__2(x_1, x_2, x_18); +x_19 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__2(x_1, x_2, x_18); return x_19; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__1() { _start: { lean_object* x_1; @@ -4573,19 +4699,19 @@ x_1 = lean_mk_string_unchecked("attributes", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__3() { _start: { lean_object* x_1; lean_object* x_2; @@ -4594,12 +4720,12 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__4() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = 1; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__3; x_3 = lean_box(x_1); x_4 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_4, 0, x_3); @@ -4607,15 +4733,15 @@ lean_ctor_set(x_4, 1, x_2); return x_4; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1), 1, 0); return x_1; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; uint8_t x_5; @@ -4636,7 +4762,7 @@ lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; x_7 = lean_unsigned_to_nat(0u); x_8 = l_Lean_Syntax_getArg(x_4, x_7); lean_dec(x_4); -x_9 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__2; +x_9 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__2; lean_inc(x_8); x_10 = l_Lean_Syntax_isOfKind(x_8, x_9); if (x_10 == 0) @@ -4660,7 +4786,7 @@ if (x_15 == 0) lean_object* x_47; lean_dec(x_14); lean_dec(x_13); -x_47 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__3; +x_47 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__3; x_16 = x_47; goto block_46; } @@ -4673,7 +4799,7 @@ if (x_48 == 0) lean_object* x_49; lean_dec(x_14); lean_dec(x_13); -x_49 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__3; +x_49 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__3; x_16 = x_49; goto block_46; } @@ -4683,7 +4809,7 @@ size_t x_50; size_t x_51; lean_object* x_52; lean_object* x_53; lean_object* x_5 x_50 = 0; x_51 = lean_usize_of_nat(x_14); lean_dec(x_14); -x_52 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__4; +x_52 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__4; x_53 = l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1(x_13, x_50, x_51, x_52); lean_dec(x_13); x_54 = lean_ctor_get(x_53, 1); @@ -4696,8 +4822,8 @@ goto block_46; block_46: { lean_object* x_17; lean_object* x_18; -x_17 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__5; -x_18 = l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__1(x_16, x_17); +x_17 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__5; +x_18 = l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__1(x_16, x_17); lean_dec(x_16); if (lean_obj_tag(x_18) == 0) { @@ -4737,7 +4863,7 @@ x_27 = l_Lean_Syntax_getArg(x_23, x_7); lean_dec(x_23); lean_ctor_set(x_18, 0, x_27); x_28 = lean_box(0); -x_29 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3(x_1, x_21, x_28, x_18); +x_29 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3(x_1, x_21, x_28, x_18); lean_dec(x_18); lean_dec(x_21); return x_29; @@ -4750,7 +4876,7 @@ lean_dec(x_23); lean_free_object(x_18); x_30 = lean_box(0); x_31 = lean_box(0); -x_32 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3(x_1, x_21, x_31, x_30); +x_32 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3(x_1, x_21, x_31, x_30); lean_dec(x_21); return x_32; } @@ -4785,7 +4911,7 @@ lean_dec(x_35); x_40 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_40, 0, x_39); x_41 = lean_box(0); -x_42 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3(x_1, x_33, x_41, x_40); +x_42 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3(x_1, x_33, x_41, x_40); lean_dec(x_40); lean_dec(x_33); return x_42; @@ -4797,7 +4923,7 @@ lean_object* x_43; lean_object* x_44; uint8_t x_45; lean_dec(x_35); x_43 = lean_box(0); x_44 = lean_box(0); -x_45 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3(x_1, x_33, x_44, x_43); +x_45 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3(x_1, x_33, x_44, x_43); lean_dec(x_33); return x_45; } @@ -4808,7 +4934,7 @@ return x_45; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__1() { _start: { lean_object* x_1; @@ -4816,19 +4942,19 @@ x_1 = lean_mk_string_unchecked("declModifiers", 13, 13); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__3() { _start: { lean_object* x_1; @@ -4836,19 +4962,19 @@ x_1 = lean_mk_string_unchecked("docComment", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__5() { _start: { lean_object* x_1; @@ -4856,105 +4982,105 @@ x_1 = lean_mk_string_unchecked("declaration", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__5; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__6; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__6; 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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__7; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__7; 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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__8; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__10() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__9; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__11() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__10; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__12() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__11; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__13() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__12; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___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_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_29; uint8_t x_30; -x_29 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__13; +x_29 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__13; lean_inc(x_2); x_30 = l_Lean_Syntax_Stack_matches(x_2, x_29); if (x_30 == 0) @@ -4985,13 +5111,13 @@ lean_dec(x_33); x_36 = lean_ctor_get(x_35, 0); lean_inc(x_36); lean_dec(x_35); -x_37 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__10; +x_37 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__10; lean_inc(x_36); x_38 = l_Lean_Syntax_isOfKind(x_36, x_37); if (x_38 == 0) { lean_object* x_39; uint8_t x_40; -x_39 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__12; +x_39 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__12; x_40 = l_Lean_Syntax_isOfKind(x_36, x_39); if (x_40 == 0) { @@ -5043,7 +5169,7 @@ lean_dec(x_8); x_10 = lean_unsigned_to_nat(0u); x_11 = l_Lean_Syntax_getArg(x_9, x_10); lean_dec(x_9); -x_12 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__2; +x_12 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__2; lean_inc(x_11); x_13 = l_Lean_Syntax_isOfKind(x_11, x_12); if (x_13 == 0) @@ -5077,7 +5203,7 @@ else lean_object* x_20; lean_object* x_21; uint8_t x_22; x_20 = l_Lean_Syntax_getArg(x_15, x_10); lean_dec(x_15); -x_21 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__4; +x_21 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__4; x_22 = l_Lean_Syntax_isOfKind(x_20, x_21); if (x_22 == 0) { @@ -5090,7 +5216,7 @@ else { lean_object* x_24; uint8_t x_25; x_24 = lean_box(0); -x_25 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4(x_11, x_24); +x_25 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4(x_11, x_24); lean_dec(x_11); return x_25; } @@ -5101,7 +5227,7 @@ else lean_object* x_26; uint8_t x_27; lean_dec(x_15); x_26 = lean_box(0); -x_27 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4(x_11, x_26); +x_27 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4(x_11, x_26); lean_dec(x_11); return x_27; } @@ -5110,42 +5236,42 @@ return x_27; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__2___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_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____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_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__2(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Array_sequenceMap_loop___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__2(x_1, x_2, x_3, x_4, x_5); lean_dec(x_1); return x_6; } } -LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__1(x_1, x_2); +x_3 = l_Array_sequenceMap___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__1(x_1, x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; uint8_t x_6; lean_object* x_7; @@ -5153,17 +5279,17 @@ x_4 = lean_unbox_usize(x_2); lean_dec(x_2); x_5 = lean_unbox_usize(x_3); lean_dec(x_3); -x_6 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3(x_1, x_4, x_5); +x_6 = l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3(x_1, x_4, x_5); lean_dec(x_1); x_7 = lean_box(x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__2(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__2(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); @@ -5171,11 +5297,11 @@ x_5 = lean_box(x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { uint8_t x_5; lean_object* x_6; -x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3(x_1, x_2, x_3, x_4); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -5184,29 +5310,29 @@ x_6 = lean_box(x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4(x_1, x_2); +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4(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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -5214,29 +5340,29 @@ x_1 = lean_mk_string_unchecked("explicitBinder", 14, 14); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__4() { _start: { lean_object* x_1; @@ -5244,102 +5370,102 @@ x_1 = lean_mk_string_unchecked("depArrow", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__4; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__5; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__5; 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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__6; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__7; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__8; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___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; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1(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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__9; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__9; x_5 = l_Lean_Syntax_Stack_matches(x_2, x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -5347,77 +5473,77 @@ x_1 = lean_mk_string_unchecked("letIdDecl", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__2; 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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__4; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__5; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__6; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__8() { _start: { lean_object* x_1; @@ -5425,19 +5551,19 @@ x_1 = lean_mk_string_unchecked("whereStructField", 16, 16); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__8; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__8; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -5445,7 +5571,7 @@ x_4 = l_Lean_Linter_getLinterUnusedVariablesFunArgs(x_3); if (x_4 == 0) { lean_object* x_5; uint8_t x_6; -x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__7; +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__7; lean_inc(x_2); x_6 = l_Lean_Syntax_Stack_matches(x_2, x_5); if (x_6 == 0) @@ -5507,7 +5633,7 @@ lean_dec(x_17); x_20 = lean_ctor_get(x_19, 0); lean_inc(x_20); lean_dec(x_19); -x_21 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__9; +x_21 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__9; x_22 = l_Lean_Syntax_isOfKind(x_20, x_21); if (x_22 == 0) { @@ -5535,71 +5661,71 @@ return x_25; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__2; 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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__1; 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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__2; 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_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -5607,7 +5733,7 @@ x_4 = l_Lean_Linter_getLinterUnusedVariablesFunArgs(x_3); if (x_4 == 0) { lean_object* x_5; uint8_t x_6; -x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__3; +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__3; lean_inc(x_2); x_6 = l_Lean_Syntax_Stack_matches(x_2, x_5); if (x_6 == 0) @@ -5655,7 +5781,7 @@ else lean_object* x_17; lean_object* x_18; uint8_t x_19; x_17 = lean_alloc_closure((void*)(l_Lean_Syntax_isOfKind___boxed), 2, 1); lean_closure_set(x_17, 0, x_12); -x_18 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__14; +x_18 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__14; x_19 = l_List_any___rarg(x_18, x_17); return x_19; } @@ -5671,35 +5797,35 @@ return x_20; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -5707,53 +5833,53 @@ x_1 = lean_mk_string_unchecked("basicFun", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__4; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__6() { _start: { lean_object* x_1; @@ -5761,41 +5887,41 @@ x_1 = lean_mk_string_unchecked("typeAscription", 14, 14); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____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; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__6; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__8() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__7; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__7; 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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__9() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__8; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__5; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__8; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___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_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -5803,13 +5929,13 @@ x_4 = l_Lean_Linter_getLinterUnusedVariablesFunArgs(x_3); if (x_4 == 0) { lean_object* x_5; uint8_t x_6; -x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__5; +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__5; lean_inc(x_2); x_6 = l_Lean_Syntax_Stack_matches(x_2, x_5); if (x_6 == 0) { lean_object* x_7; uint8_t x_8; -x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__9; +x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__9; x_8 = l_Lean_Syntax_Stack_matches(x_2, x_7); return x_8; } @@ -5830,35 +5956,35 @@ return x_10; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); return x_5; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -5866,19 +5992,19 @@ x_1 = lean_mk_string_unchecked("matchAlt", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____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_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__3() { _start: { lean_object* x_1; @@ -5886,7 +6012,7 @@ x_1 = lean_mk_string_unchecked("Tactic", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__4() { _start: { lean_object* x_1; @@ -5894,19 +6020,19 @@ x_1 = lean_mk_string_unchecked("inductionAltLHS", 15, 15); return x_1; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____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_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__3; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__4; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__3; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__4; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1(lean_object* x_1) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; uint8_t x_5; @@ -5915,13 +6041,13 @@ lean_inc(x_2); x_3 = lean_ctor_get(x_1, 1); lean_inc(x_3); lean_dec(x_1); -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__2; +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__2; lean_inc(x_2); x_5 = l_Lean_Syntax_isOfKind(x_2, x_4); if (x_5 == 0) { lean_object* x_6; uint8_t x_7; -x_6 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__5; +x_6 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__5; x_7 = l_Lean_Syntax_isOfKind(x_2, x_6); if (x_7 == 0) { @@ -5947,7 +6073,7 @@ x_12 = lean_nat_dec_eq(x_3, x_11); if (x_12 == 0) { lean_object* x_13; uint8_t x_14; -x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__5; +x_13 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__5; x_14 = l_Lean_Syntax_isOfKind(x_2, x_13); if (x_14 == 0) { @@ -5976,15 +6102,15 @@ return x_18; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2___closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___boxed), 1, 0); return x_1; } } -LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -5992,7 +6118,7 @@ x_4 = l_Lean_Linter_getLinterUnusedVariablesPatternVars(x_3); if (x_4 == 0) { lean_object* x_5; uint8_t x_6; -x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2___closed__1; +x_5 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2___closed__1; x_6 = l_List_any___rarg(x_2, x_5); return x_6; } @@ -6005,37 +6131,37 @@ return x_7; } } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2___boxed), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____closed__1; x_3 = l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___boxed(lean_object* x_1) { _start: { uint8_t x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1(x_1); +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1(x_1); x_3 = lean_box(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2(x_1, x_2, x_3); +x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_1); x_5 = lean_box(x_4); @@ -6047,7 +6173,7 @@ static lean_object* _init_l_Lean_Linter_getUnusedVariablesIgnoreFns___rarg___clo { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__3; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___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); @@ -6068,7 +6194,7 @@ x_6 = lean_ctor_get(x_5, 0); lean_inc(x_6); lean_dec(x_5); x_7 = l_Lean_Linter_getUnusedVariablesIgnoreFns___rarg___closed__1; -x_8 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1; +x_8 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1; x_9 = l_Lean_PersistentEnvExtension_getState___rarg(x_7, x_8, x_6); lean_dec(x_6); x_10 = lean_ctor_get(x_9, 1); @@ -6089,7 +6215,7 @@ x_13 = lean_ctor_get(x_11, 0); lean_inc(x_13); lean_dec(x_11); x_14 = l_Lean_Linter_getUnusedVariablesIgnoreFns___rarg___closed__1; -x_15 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1; +x_15 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1; x_16 = l_Lean_PersistentEnvExtension_getState___rarg(x_14, x_15, x_13); lean_dec(x_13); x_17 = lean_ctor_get(x_16, 1); @@ -9316,8 +9442,8 @@ static lean_object* _init_l_Lean_Linter_UnusedVariables_collectReferences_skipDe { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5; x_4 = l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; @@ -9344,7 +9470,7 @@ return x_5; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences___spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -9376,7 +9502,7 @@ return x_9; } } } -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -9405,7 +9531,7 @@ return x_8; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences___spec__5(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__5(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -9479,7 +9605,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__4(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_Linter_UnusedVariables_collectReferences_go___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; @@ -9498,7 +9624,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_Linter_UnusedVariables_collectReferences___spec__5(x_3, x_6); +x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences_go___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); @@ -9509,7 +9635,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__3(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___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; @@ -9520,11 +9646,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_Linter_UnusedVariables_collectReferences___spec__4(x_7, x_1, x_6); +x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__4(x_7, x_1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) @@ -9549,7 +9675,7 @@ x_9 = l___private_Lean_Syntax_0__String_beqRange____x40_Lean_Syntax___hyg_95_(x_ if (x_9 == 0) { lean_object* x_10; -x_10 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(x_1, x_2, x_8); +x_10 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(x_1, x_2, x_8); lean_ctor_set(x_3, 2, x_10); return x_3; } @@ -9576,7 +9702,7 @@ x_14 = l___private_Lean_Syntax_0__String_beqRange____x40_Lean_Syntax___hyg_95_(x if (x_14 == 0) { lean_object* x_15; lean_object* x_16; -x_15 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(x_1, x_2, x_13); +x_15 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(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); @@ -9598,7 +9724,7 @@ return x_17; } } } -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__7(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__7(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -9627,7 +9753,7 @@ return x_8; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences___spec__10(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__10(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -9701,7 +9827,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__9(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_Linter_UnusedVariables_collectReferences_go___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; @@ -9720,7 +9846,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_Linter_UnusedVariables_collectReferences___spec__10(x_3, x_6); +x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__10(x_3, x_6); x_10 = lean_unsigned_to_nat(1u); x_11 = lean_nat_add(x_1, x_10); lean_dec(x_1); @@ -9731,7 +9857,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__8(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__8(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; @@ -9742,11 +9868,194 @@ 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_Linter_UnusedVariables_collectReferences___spec__9(x_7, x_1, x_6); +x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__9(x_7, x_1, x_6); +return x_8; +} +} +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__13(lean_object* x_1, size_t x_2, size_t x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_eq(x_2, x_3); +if (x_4 == 0) +{ +lean_object* x_5; uint8_t x_6; +x_5 = lean_array_uget(x_1, x_2); +x_6 = l_Lean_PersistentArray_anyMAux___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__12(x_5); +lean_dec(x_5); +if (x_6 == 0) +{ +size_t x_7; size_t x_8; +x_7 = 1; +x_8 = lean_usize_add(x_2, x_7); +x_2 = x_8; +goto _start; +} +else +{ +uint8_t x_10; +x_10 = 1; +return x_10; +} +} +else +{ +uint8_t x_11; +x_11 = 0; +return x_11; +} +} +} +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___lambda__1(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +uint8_t x_2; +x_2 = 1; +return x_2; +} +else +{ +uint8_t x_3; +x_3 = 0; +return x_3; +} +} +} +static lean_object* _init_l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___lambda__1___boxed), 1, 0); +return x_1; +} +} +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14(lean_object* x_1, size_t x_2, size_t x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_eq(x_2, x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_array_uget(x_1, x_2); +x_6 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___closed__1; +x_7 = l_Lean_Elab_InfoTree_findInfo_x3f(x_6, x_5); +if (lean_obj_tag(x_7) == 0) +{ +size_t x_8; size_t x_9; +x_8 = 1; +x_9 = lean_usize_add(x_2, x_8); +x_2 = x_9; +goto _start; +} +else +{ +uint8_t x_11; +lean_dec(x_7); +x_11 = 1; +return x_11; +} +} +else +{ +uint8_t x_12; +x_12 = 0; +return x_12; +} +} +} +LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyMAux___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__12(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; uint8_t x_5; +x_2 = lean_ctor_get(x_1, 0); +x_3 = lean_array_get_size(x_2); +x_4 = lean_unsigned_to_nat(0u); +x_5 = lean_nat_dec_lt(x_4, x_3); +if (x_5 == 0) +{ +uint8_t x_6; +lean_dec(x_3); +x_6 = 0; +return x_6; +} +else +{ +size_t x_7; size_t x_8; uint8_t x_9; +x_7 = 0; +x_8 = lean_usize_of_nat(x_3); +lean_dec(x_3); +x_9 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__13(x_2, x_7, x_8); +return x_9; +} +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = lean_ctor_get(x_1, 0); +x_11 = lean_array_get_size(x_10); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_nat_dec_lt(x_12, x_11); +if (x_13 == 0) +{ +uint8_t x_14; +lean_dec(x_11); +x_14 = 0; +return x_14; +} +else +{ +size_t x_15; size_t x_16; uint8_t x_17; +x_15 = 0; +x_16 = lean_usize_of_nat(x_11); +lean_dec(x_11); +x_17 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14(x_10, x_15, x_16); +return x_17; +} +} +} +} +LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__11(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; +x_2 = lean_ctor_get(x_1, 0); +x_3 = l_Lean_PersistentArray_anyMAux___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__12(x_2); +if (x_3 == 0) +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_array_get_size(x_4); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_nat_dec_lt(x_6, x_5); +if (x_7 == 0) +{ +uint8_t x_8; +lean_dec(x_5); +x_8 = 0; return x_8; } +else +{ +size_t x_9; size_t x_10; uint8_t x_11; +x_9 = 0; +x_10 = lean_usize_of_nat(x_5); +lean_dec(x_5); +x_11 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14(x_4, x_9, x_10); +return x_11; +} +} +else +{ +return x_3; +} +} } -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -9775,7 +10084,7 @@ return x_8; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences___spec__14(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__18(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -9849,7 +10158,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__13(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_Linter_UnusedVariables_collectReferences_go___spec__17(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; @@ -9868,7 +10177,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_Linter_UnusedVariables_collectReferences___spec__14(x_3, x_6); +x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__18(x_3, x_6); x_10 = lean_unsigned_to_nat(1u); x_11 = lean_nat_add(x_1, x_10); lean_dec(x_1); @@ -9879,7 +10188,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__12(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__16(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; @@ -9890,11 +10199,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_Linter_UnusedVariables_collectReferences___spec__13(x_7, x_1, x_6); +x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__17(x_7, x_1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) @@ -9919,7 +10228,7 @@ x_9 = lean_name_eq(x_6, x_1); if (x_9 == 0) { lean_object* x_10; -x_10 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(x_1, x_2, x_8); +x_10 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(x_1, x_2, x_8); lean_ctor_set(x_3, 2, x_10); return x_3; } @@ -9946,7 +10255,7 @@ x_14 = lean_name_eq(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_Linter_UnusedVariables_collectReferences___spec__15(x_1, x_2, x_13); +x_15 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(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); @@ -9968,7 +10277,7 @@ return x_17; } } } -static lean_object* _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__1() { +static lean_object* _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__1() { _start: { lean_object* x_1; @@ -9976,179 +10285,189 @@ x_1 = l_EStateM_instMonad(lean_box(0), lean_box(0)); return x_1; } } -static lean_object* _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__2() { +static lean_object* _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__1; +x_2 = l_ReaderT_instMonad___rarg(x_1); +return x_2; +} +} +static lean_object* _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__1; +x_1 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__2; x_2 = l_ReaderT_instMonad___rarg(x_1); return x_2; } } -static lean_object* _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__3() { +static lean_object* _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__2; +x_2 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__3; x_3 = l_instInhabitedOfMonad___rarg(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_4 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__3; -x_5 = lean_panic_fn(x_4, x_1); -x_6 = lean_apply_2(x_5, x_2, x_3); -return x_6; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__4; +x_6 = lean_panic_fn(x_5, x_1); +x_7 = lean_box(x_2); +x_8 = lean_apply_3(x_6, x_7, x_3, x_4); +return x_8; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__20(lean_object* x_1, lean_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_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__23(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) { _start: { if (lean_obj_tag(x_4) == 0) { -lean_object* x_8; lean_object* x_9; -lean_dec(x_6); +lean_object* x_9; lean_object* x_10; +lean_dec(x_7); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_8 = l_List_reverse___rarg(x_5); -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; +x_9 = l_List_reverse___rarg(x_5); +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_10; -x_10 = !lean_is_exclusive(x_4); -if (x_10 == 0) +uint8_t x_11; +x_11 = !lean_is_exclusive(x_4); +if (x_11 == 0) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_4, 0); -x_12 = lean_ctor_get(x_4, 1); -lean_inc(x_6); +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_4, 0); +x_13 = lean_ctor_get(x_4, 1); +lean_inc(x_7); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_13 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18(x_1, x_2, x_3, x_11, x_6, x_7); -if (lean_obj_tag(x_13) == 0) +x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21(x_1, x_2, x_3, x_12, x_6, x_7, x_8); +if (lean_obj_tag(x_14) == 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_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); -lean_dec(x_13); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); lean_ctor_set(x_4, 1, x_5); -lean_ctor_set(x_4, 0, x_14); +lean_ctor_set(x_4, 0, x_15); { -lean_object* _tmp_3 = x_12; +lean_object* _tmp_3 = x_13; lean_object* _tmp_4 = x_4; -lean_object* _tmp_6 = x_15; +lean_object* _tmp_7 = x_16; x_4 = _tmp_3; x_5 = _tmp_4; -x_7 = _tmp_6; +x_8 = _tmp_7; } goto _start; } else { -uint8_t x_17; +uint8_t x_18; lean_free_object(x_4); -lean_dec(x_12); -lean_dec(x_6); -lean_dec(x_5); +lean_dec(x_13); +lean_dec(x_7); +lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_17 = !lean_is_exclusive(x_13); -if (x_17 == 0) +x_18 = !lean_is_exclusive(x_14); +if (x_18 == 0) { -return x_13; +return x_14; } else { -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_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_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; +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_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_4, 0); -x_22 = lean_ctor_get(x_4, 1); +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_4, 0); +x_23 = lean_ctor_get(x_4, 1); +lean_inc(x_23); lean_inc(x_22); -lean_inc(x_21); lean_dec(x_4); -lean_inc(x_6); +lean_inc(x_7); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_23 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18(x_1, x_2, x_3, x_21, x_6, x_7); -if (lean_obj_tag(x_23) == 0) +x_24 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21(x_1, x_2, x_3, x_22, x_6, x_7, x_8); +if (lean_obj_tag(x_24) == 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_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_5); -x_4 = x_22; -x_5 = x_26; -x_7 = 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_5); +x_4 = x_23; +x_5 = x_27; +x_8 = x_26; goto _start; } else { -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_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_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_28 = lean_ctor_get(x_23, 0); -lean_inc(x_28); -x_29 = lean_ctor_get(x_23, 1); +x_29 = lean_ctor_get(x_24, 0); 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; +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_23); - x_30 = lean_box(0); + lean_dec_ref(x_24); + x_31 = lean_box(0); } -if (lean_is_scalar(x_30)) { - x_31 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_31)) { + x_32 = lean_alloc_ctor(1, 2, 0); } else { - x_31 = x_30; + x_32 = x_31; } -lean_ctor_set(x_31, 0, x_28); -lean_ctor_set(x_31, 1, x_29); -return 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_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__1() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__1() { _start: { lean_object* x_1; @@ -10156,7 +10475,7 @@ x_1 = lean_mk_string_unchecked("Lean.Server.InfoUtils", 21, 21); return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__2() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__2() { _start: { lean_object* x_1; @@ -10164,7 +10483,7 @@ x_1 = lean_mk_string_unchecked("Lean.Elab.InfoTree.visitM.go", 28, 28); return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__3() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__3() { _start: { lean_object* x_1; @@ -10172,20 +10491,20 @@ x_1 = lean_mk_string_unchecked("unexpected context-free info tree node", 38, 38) return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__4() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___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_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__1; -x_2 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__2; -x_3 = lean_unsigned_to_nat(56u); +x_1 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__1; +x_2 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__2; +x_3 = lean_unsigned_to_nat(62u); x_4 = lean_unsigned_to_nat(21u); -x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__3; +x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___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_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18(lean_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_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21(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) { _start: { if (lean_obj_tag(x_3) == 0) @@ -10193,39 +10512,39 @@ if (lean_obj_tag(x_3) == 0) switch (lean_obj_tag(x_4)) { case 0: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = lean_ctor_get(x_4, 0); -lean_inc(x_7); -x_8 = lean_ctor_get(x_4, 1); +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_ctor_get(x_4, 0); lean_inc(x_8); +x_9 = lean_ctor_get(x_4, 1); +lean_inc(x_9); lean_dec(x_4); -x_9 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_7, x_3); -x_3 = x_9; -x_4 = x_8; +x_10 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_8, x_3); +x_3 = x_10; +x_4 = x_9; goto _start; } case 1: { -lean_object* x_11; lean_object* x_12; +lean_object* x_12; lean_object* x_13; lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_11 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__4; -x_12 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19(x_11, x_5, x_6); -return x_12; +x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__4; +x_13 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22(x_12, x_5, x_6, x_7); +return x_13; } default: { -lean_object* x_13; lean_object* x_14; -lean_dec(x_5); +lean_object* x_14; lean_object* x_15; +lean_dec(x_6); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -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_6); -return x_14; +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; } } } @@ -10234,554 +10553,766 @@ else switch (lean_obj_tag(x_4)) { case 0: { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_4, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_4, 1); +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_4, 0); lean_inc(x_16); +x_17 = lean_ctor_get(x_4, 1); +lean_inc(x_17); lean_dec(x_4); -x_17 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_15, x_3); -x_3 = x_17; -x_4 = x_16; +x_18 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_16, x_3); +x_3 = x_18; +x_4 = x_17; goto _start; } case 1: { -uint8_t x_19; -x_19 = !lean_is_exclusive(x_3); -if (x_19 == 0) +uint8_t x_20; +x_20 = !lean_is_exclusive(x_3); +if (x_20 == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_20 = lean_ctor_get(x_3, 0); -x_21 = lean_ctor_get(x_4, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_4, 1); +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_21 = lean_ctor_get(x_3, 0); +x_22 = lean_ctor_get(x_4, 0); lean_inc(x_22); +x_23 = lean_ctor_get(x_4, 1); +lean_inc(x_23); lean_dec(x_4); +x_24 = lean_box(x_5); lean_inc(x_1); -lean_inc(x_5); +lean_inc(x_6); +lean_inc(x_23); lean_inc(x_22); lean_inc(x_21); -lean_inc(x_20); -x_23 = lean_apply_5(x_1, x_20, x_21, x_22, x_5, x_6); -if (lean_obj_tag(x_23) == 0) +x_25 = lean_apply_6(x_1, x_21, x_22, x_23, x_24, x_6, x_7); +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_20); -x_25 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_21); -x_26 = l_Lean_PersistentArray_toList___rarg(x_22); -x_27 = lean_box(0); -lean_inc(x_5); -lean_inc(x_2); -x_28 = l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__20(x_1, x_2, x_25, x_26, x_27, x_5, x_24); -if (lean_obj_tag(x_28) == 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_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 = lean_apply_6(x_2, x_20, x_21, x_22, x_29, x_5, x_30); +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +lean_dec(x_1); +x_28 = lean_ctor_get(x_25, 1); +lean_inc(x_28); +lean_dec(x_25); +x_29 = lean_box(0); +x_30 = lean_box(x_5); +x_31 = lean_apply_7(x_2, x_21, x_22, x_23, x_29, x_30, x_6, x_28); if (lean_obj_tag(x_31) == 0) { uint8_t x_32; x_32 = !lean_is_exclusive(x_31); if (x_32 == 0) { -lean_object* x_33; lean_object* x_34; +lean_object* x_33; x_33 = lean_ctor_get(x_31, 0); -x_34 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_34, 0, x_33); -lean_ctor_set(x_31, 0, x_34); +lean_ctor_set(x_3, 0, x_33); +lean_ctor_set(x_31, 0, x_3); return x_31; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_35 = lean_ctor_get(x_31, 0); -x_36 = lean_ctor_get(x_31, 1); -lean_inc(x_36); +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_31, 0); +x_35 = lean_ctor_get(x_31, 1); lean_inc(x_35); +lean_inc(x_34); lean_dec(x_31); -x_37 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_37, 0, x_35); -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; +lean_ctor_set(x_3, 0, x_34); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_3); +lean_ctor_set(x_36, 1, x_35); +return x_36; } } else { -uint8_t x_39; -x_39 = !lean_is_exclusive(x_31); -if (x_39 == 0) +uint8_t x_37; +lean_free_object(x_3); +x_37 = !lean_is_exclusive(x_31); +if (x_37 == 0) { return x_31; } else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; -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_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_inc(x_38); lean_dec(x_31); -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; +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; +x_41 = lean_ctor_get(x_25, 1); +lean_inc(x_41); +lean_dec(x_25); +lean_inc(x_21); +x_42 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_22); +x_43 = l_Lean_PersistentArray_toList___rarg(x_23); +x_44 = lean_box(0); +lean_inc(x_6); +lean_inc(x_2); +x_45 = l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__23(x_1, x_2, x_42, x_43, x_44, x_5, x_6, x_41); +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 = 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_box(x_5); +x_49 = lean_apply_7(x_2, x_21, x_22, x_23, x_46, x_48, x_6, x_47); +if (lean_obj_tag(x_49) == 0) +{ +uint8_t x_50; +x_50 = !lean_is_exclusive(x_49); +if (x_50 == 0) +{ +lean_object* x_51; lean_object* x_52; +x_51 = lean_ctor_get(x_49, 0); +x_52 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_49, 0, x_52); +return x_49; +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_53 = lean_ctor_get(x_49, 0); +x_54 = lean_ctor_get(x_49, 1); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_49); +x_55 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_55, 0, x_53); +x_56 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_56, 0, x_55); +lean_ctor_set(x_56, 1, x_54); +return x_56; +} +} +else +{ +uint8_t x_57; +x_57 = !lean_is_exclusive(x_49); +if (x_57 == 0) +{ +return x_49; +} +else +{ +lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_58 = lean_ctor_get(x_49, 0); +x_59 = lean_ctor_get(x_49, 1); +lean_inc(x_59); +lean_inc(x_58); +lean_dec(x_49); +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_43; +uint8_t x_61; +lean_dec(x_23); lean_dec(x_22); lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_5); +lean_dec(x_6); lean_dec(x_2); -x_43 = !lean_is_exclusive(x_28); -if (x_43 == 0) +x_61 = !lean_is_exclusive(x_45); +if (x_61 == 0) { -return x_28; +return x_45; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_28, 0); -x_45 = lean_ctor_get(x_28, 1); -lean_inc(x_45); -lean_inc(x_44); -lean_dec(x_28); -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_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; +} } } } else { -uint8_t x_47; +uint8_t x_65; +lean_dec(x_23); lean_dec(x_22); -lean_dec(x_21); lean_free_object(x_3); -lean_dec(x_20); -lean_dec(x_5); +lean_dec(x_21); +lean_dec(x_6); lean_dec(x_2); lean_dec(x_1); -x_47 = !lean_is_exclusive(x_23); -if (x_47 == 0) +x_65 = !lean_is_exclusive(x_25); +if (x_65 == 0) { -return x_23; +return x_25; } 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_66; lean_object* x_67; lean_object* x_68; +x_66 = lean_ctor_get(x_25, 0); +x_67 = lean_ctor_get(x_25, 1); +lean_inc(x_67); +lean_inc(x_66); +lean_dec(x_25); +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_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_51 = lean_ctor_get(x_3, 0); -lean_inc(x_51); +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_3, 0); +lean_inc(x_69); lean_dec(x_3); -x_52 = lean_ctor_get(x_4, 0); -lean_inc(x_52); -x_53 = lean_ctor_get(x_4, 1); -lean_inc(x_53); +x_70 = lean_ctor_get(x_4, 0); +lean_inc(x_70); +x_71 = lean_ctor_get(x_4, 1); +lean_inc(x_71); lean_dec(x_4); +x_72 = lean_box(x_5); lean_inc(x_1); -lean_inc(x_5); -lean_inc(x_53); -lean_inc(x_52); -lean_inc(x_51); -x_54 = lean_apply_5(x_1, x_51, x_52, x_53, x_5, x_6); -if (lean_obj_tag(x_54) == 0) +lean_inc(x_6); +lean_inc(x_71); +lean_inc(x_70); +lean_inc(x_69); +x_73 = lean_apply_6(x_1, x_69, x_70, x_71, x_72, x_6, x_7); +if (lean_obj_tag(x_73) == 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; -x_55 = lean_ctor_get(x_54, 1); -lean_inc(x_55); -lean_dec(x_54); -lean_inc(x_51); -x_56 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_56, 0, x_51); -x_57 = l_Lean_Elab_Info_updateContext_x3f(x_56, x_52); -x_58 = l_Lean_PersistentArray_toList___rarg(x_53); -x_59 = lean_box(0); -lean_inc(x_5); -lean_inc(x_2); -x_60 = l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__20(x_1, x_2, x_57, x_58, x_59, x_5, x_55); -if (lean_obj_tag(x_60) == 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_61; lean_object* x_62; lean_object* x_63; -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 = lean_apply_6(x_2, x_51, x_52, x_53, x_61, x_5, x_62); -if (lean_obj_tag(x_63) == 0) +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +lean_dec(x_1); +x_76 = lean_ctor_get(x_73, 1); +lean_inc(x_76); +lean_dec(x_73); +x_77 = lean_box(0); +x_78 = lean_box(x_5); +x_79 = lean_apply_7(x_2, x_69, x_70, x_71, x_77, x_78, x_6, x_76); +if (lean_obj_tag(x_79) == 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_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_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; +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_63); - x_66 = lean_box(0); + lean_dec_ref(x_79); + x_82 = 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_83 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_83, 0, x_80); +if (lean_is_scalar(x_82)) { + x_84 = lean_alloc_ctor(0, 2, 0); } else { - x_68 = x_66; + 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_object* x_88; +x_85 = lean_ctor_get(x_79, 0); +lean_inc(x_85); +x_86 = lean_ctor_get(x_79, 1); +lean_inc(x_86); +if (lean_is_exclusive(x_79)) { + lean_ctor_release(x_79, 0); + lean_ctor_release(x_79, 1); + x_87 = x_79; +} else { + lean_dec_ref(x_79); + 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; } -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; -x_69 = lean_ctor_get(x_63, 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; +x_89 = lean_ctor_get(x_73, 1); +lean_inc(x_89); +lean_dec(x_73); 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; +x_90 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_90, 0, x_69); +x_91 = l_Lean_Elab_Info_updateContext_x3f(x_90, x_70); +x_92 = l_Lean_PersistentArray_toList___rarg(x_71); +x_93 = lean_box(0); +lean_inc(x_6); +lean_inc(x_2); +x_94 = l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__23(x_1, x_2, x_91, x_92, x_93, x_5, x_6, 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; +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_box(x_5); +x_98 = lean_apply_7(x_2, x_69, x_70, x_71, x_95, x_97, x_6, x_96); +if (lean_obj_tag(x_98) == 0) +{ +lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +x_100 = lean_ctor_get(x_98, 1); +lean_inc(x_100); +if (lean_is_exclusive(x_98)) { + lean_ctor_release(x_98, 0); + lean_ctor_release(x_98, 1); + x_101 = x_98; +} else { + lean_dec_ref(x_98); + x_101 = lean_box(0); +} +x_102 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_102, 0, x_99); +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; +} +else +{ +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); +if (lean_is_exclusive(x_98)) { + lean_ctor_release(x_98, 0); + lean_ctor_release(x_98, 1); + x_106 = x_98; } else { - lean_dec_ref(x_63); - x_71 = lean_box(0); + lean_dec_ref(x_98); + x_106 = lean_box(0); } -if (lean_is_scalar(x_71)) { - x_72 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_106)) { + x_107 = lean_alloc_ctor(1, 2, 0); } else { - x_72 = x_71; + x_107 = x_106; } -lean_ctor_set(x_72, 0, x_69); -lean_ctor_set(x_72, 1, x_70); -return x_72; +lean_ctor_set(x_107, 0, x_104); +lean_ctor_set(x_107, 1, x_105); +return x_107; } } else { -lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; -lean_dec(x_53); -lean_dec(x_52); -lean_dec(x_51); -lean_dec(x_5); +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +lean_dec(x_71); +lean_dec(x_70); +lean_dec(x_69); +lean_dec(x_6); lean_dec(x_2); -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_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_60); - x_75 = lean_box(0); + lean_dec_ref(x_94); + x_110 = lean_box(0); } -if (lean_is_scalar(x_75)) { - x_76 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_110)) { + x_111 = lean_alloc_ctor(1, 2, 0); } else { - x_76 = x_75; + x_111 = x_110; +} +lean_ctor_set(x_111, 0, x_108); +lean_ctor_set(x_111, 1, x_109); +return x_111; } -lean_ctor_set(x_76, 0, x_73); -lean_ctor_set(x_76, 1, x_74); -return x_76; } } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; -lean_dec(x_53); -lean_dec(x_52); -lean_dec(x_51); -lean_dec(x_5); +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +lean_dec(x_71); +lean_dec(x_70); +lean_dec(x_69); +lean_dec(x_6); lean_dec(x_2); lean_dec(x_1); -x_77 = lean_ctor_get(x_54, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_54, 1); -lean_inc(x_78); -if (lean_is_exclusive(x_54)) { - lean_ctor_release(x_54, 0); - lean_ctor_release(x_54, 1); - x_79 = x_54; +x_112 = lean_ctor_get(x_73, 0); +lean_inc(x_112); +x_113 = lean_ctor_get(x_73, 1); +lean_inc(x_113); +if (lean_is_exclusive(x_73)) { + lean_ctor_release(x_73, 0); + lean_ctor_release(x_73, 1); + x_114 = x_73; } else { - lean_dec_ref(x_54); - x_79 = lean_box(0); + lean_dec_ref(x_73); + x_114 = lean_box(0); } -if (lean_is_scalar(x_79)) { - x_80 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_114)) { + x_115 = lean_alloc_ctor(1, 2, 0); } else { - x_80 = x_79; + x_115 = x_114; } -lean_ctor_set(x_80, 0, x_77); -lean_ctor_set(x_80, 1, x_78); -return x_80; +lean_ctor_set(x_115, 0, x_112); +lean_ctor_set(x_115, 1, x_113); +return x_115; } } } default: { -lean_object* x_81; lean_object* x_82; -lean_dec(x_5); +lean_object* x_116; lean_object* x_117; +lean_dec(x_6); 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_6); -return x_82; -} -} +x_116 = lean_box(0); +x_117 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_117, 0, x_116); +lean_ctor_set(x_117, 1, x_7); +return x_117; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_UnusedVariables_collectReferences___spec__17(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_box(0); -x_7 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18(x_1, x_2, x_6, x_3, x_4, x_5); -return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences___spec__16___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_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20___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) { _start: { -lean_object* x_8; -x_8 = lean_apply_5(x_1, x_2, x_3, x_4, x_6, x_7); -return x_8; +lean_object* x_9; lean_object* x_10; +x_9 = lean_box(x_6); +x_10 = lean_apply_6(x_1, x_2, x_3, x_4, x_9, x_7, x_8); +return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences___spec__16(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_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20(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) { _start: { -lean_object* x_6; lean_object* x_7; -x_6 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences___spec__16___lambda__1___boxed), 7, 1); -lean_closure_set(x_6, 0, x_2); -x_7 = l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_UnusedVariables_collectReferences___spec__17(x_1, x_6, x_3, x_4, x_5); -if (lean_obj_tag(x_7) == 0) +lean_object* x_8; lean_object* x_9; +x_8 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20___lambda__1___boxed), 8, 1); +lean_closure_set(x_8, 0, x_2); +x_9 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21(x_1, x_8, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_9) == 0) { -uint8_t x_8; -x_8 = !lean_is_exclusive(x_7); -if (x_8 == 0) +uint8_t x_10; +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) { -lean_object* x_9; lean_object* x_10; -x_9 = lean_ctor_get(x_7, 0); -lean_dec(x_9); -x_10 = lean_box(0); -lean_ctor_set(x_7, 0, x_10); -return x_7; +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +lean_dec(x_11); +x_12 = lean_box(0); +lean_ctor_set(x_9, 0, x_12); +return x_9; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_7, 1); -lean_inc(x_11); -lean_dec(x_7); -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; +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_9, 1); +lean_inc(x_13); +lean_dec(x_9); +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 { -uint8_t x_14; -x_14 = !lean_is_exclusive(x_7); -if (x_14 == 0) +uint8_t x_16; +x_16 = !lean_is_exclusive(x_9); +if (x_16 == 0) { -return x_7; +return x_9; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_7, 0); -x_16 = lean_ctor_get(x_7, 1); -lean_inc(x_16); -lean_inc(x_15); -lean_dec(x_7); -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_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_9, 0); +x_18 = lean_ctor_get(x_9, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_9); +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_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__1(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_9 = lean_st_ref_take(x_7, x_8); -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -x_11 = lean_ctor_get(x_10, 1); -lean_inc(x_11); -x_12 = !lean_is_exclusive(x_9); -if (x_12 == 0) +lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_6 = lean_st_ref_take(x_4, x_5); +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_is_exclusive(x_7); +if (x_9 == 0) { -lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_13 = lean_ctor_get(x_9, 1); -x_14 = lean_ctor_get(x_9, 0); -lean_dec(x_14); -x_15 = !lean_is_exclusive(x_11); +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_7, 4); +x_11 = lean_ctor_get(x_1, 3); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 7); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_array_push(x_10, x_12); +lean_ctor_set(x_7, 4, x_13); +x_14 = lean_st_ref_set(x_4, x_7, x_8); +x_15 = !lean_is_exclusive(x_14); if (x_15 == 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; 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_16 = lean_ctor_get(x_11, 0); -x_17 = lean_ctor_get(x_11, 1); -x_18 = lean_array_get_size(x_17); -x_19 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_1); -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); -x_32 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences___spec__1(x_1, x_31); -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; uint8_t x_41; -x_33 = lean_ctor_get(x_10, 0); -lean_inc(x_33); -x_34 = l_Lean_LocalDecl_userName(x_2); -x_35 = lean_box(0); -lean_ctor_set_tag(x_9, 1); -lean_ctor_set(x_9, 1, x_35); -lean_ctor_set(x_9, 0, x_3); -x_36 = lean_array_mk(x_9); -x_37 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_37, 0, x_34); -lean_ctor_set(x_37, 1, x_4); -lean_ctor_set(x_37, 2, x_5); -lean_ctor_set(x_37, 3, x_36); -x_38 = lean_ctor_get(x_10, 2); -lean_inc(x_38); -x_39 = lean_ctor_get(x_10, 3); -lean_inc(x_39); -x_40 = lean_ctor_get(x_10, 4); -lean_inc(x_40); -lean_dec(x_10); -x_41 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2(x_1, x_31); -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; uint8_t x_51; -x_42 = lean_unsigned_to_nat(1u); -x_43 = lean_nat_add(x_16, x_42); +lean_object* x_16; uint8_t x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_14, 0); lean_dec(x_16); -x_44 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_44, 0, x_1); -lean_ctor_set(x_44, 1, x_37); -lean_ctor_set(x_44, 2, x_31); -x_45 = lean_array_uset(x_17, x_30, 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_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; -x_52 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__3(x_45); -lean_ctor_set(x_11, 1, x_52); -lean_ctor_set(x_11, 0, x_43); -x_53 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_53, 0, x_33); -lean_ctor_set(x_53, 1, x_11); -lean_ctor_set(x_53, 2, x_38); -lean_ctor_set(x_53, 3, x_39); -lean_ctor_set(x_53, 4, x_40); -x_54 = lean_st_ref_set(x_7, x_53, x_13); -x_55 = !lean_is_exclusive(x_54); -if (x_55 == 0) -{ -lean_object* x_56; lean_object* x_57; -x_56 = lean_ctor_get(x_54, 0); -lean_dec(x_56); -x_57 = lean_box(0); -lean_ctor_set(x_54, 0, x_57); -return x_54; +x_17 = 1; +x_18 = lean_box(x_17); +lean_ctor_set(x_14, 0, x_18); +return x_14; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_58 = lean_ctor_get(x_54, 1); -lean_inc(x_58); -lean_dec(x_54); -x_59 = lean_box(0); -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_object* x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; +x_19 = lean_ctor_get(x_14, 1); +lean_inc(x_19); +lean_dec(x_14); +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 { -lean_object* x_61; lean_object* x_62; uint8_t x_63; -lean_ctor_set(x_11, 1, x_45); -lean_ctor_set(x_11, 0, x_43); -x_61 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_61, 0, x_33); -lean_ctor_set(x_61, 1, x_11); -lean_ctor_set(x_61, 2, x_38); -lean_ctor_set(x_61, 3, x_39); -lean_ctor_set(x_61, 4, x_40); -x_62 = lean_st_ref_set(x_7, x_61, x_13); -x_63 = !lean_is_exclusive(x_62); -if (x_63 == 0) -{ -lean_object* x_64; lean_object* x_65; -x_64 = lean_ctor_get(x_62, 0); -lean_dec(x_64); -x_65 = lean_box(0); -lean_ctor_set(x_62, 0, x_65); -return x_62; -} +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; uint8_t x_35; lean_object* x_36; lean_object* x_37; +x_23 = lean_ctor_get(x_7, 0); +x_24 = lean_ctor_get(x_7, 1); +x_25 = lean_ctor_get(x_7, 2); +x_26 = lean_ctor_get(x_7, 3); +x_27 = lean_ctor_get(x_7, 4); +lean_inc(x_27); +lean_inc(x_26); +lean_inc(x_25); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_7); +x_28 = lean_ctor_get(x_1, 3); +lean_inc(x_28); +lean_dec(x_1); +x_29 = lean_ctor_get(x_28, 7); +lean_inc(x_29); +lean_dec(x_28); +x_30 = lean_array_push(x_27, x_29); +x_31 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_31, 0, x_23); +lean_ctor_set(x_31, 1, x_24); +lean_ctor_set(x_31, 2, x_25); +lean_ctor_set(x_31, 3, x_26); +lean_ctor_set(x_31, 4, x_30); +x_32 = lean_st_ref_set(x_4, x_31, x_8); +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +if (lean_is_exclusive(x_32)) { + lean_ctor_release(x_32, 0); + lean_ctor_release(x_32, 1); + x_34 = x_32; +} else { + lean_dec_ref(x_32); + x_34 = lean_box(0); +} +x_35 = 1; +x_36 = lean_box(x_35); +if (lean_is_scalar(x_34)) { + x_37 = lean_alloc_ctor(0, 2, 0); +} else { + x_37 = x_34; +} +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_33); +return x_37; +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__2(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; lean_object* x_6; lean_object* x_7; +x_5 = 1; +x_6 = lean_box(x_5); +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___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, uint8_t x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_17 = lean_st_ref_take(x_9, x_10); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +x_20 = !lean_is_exclusive(x_17); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = lean_ctor_get(x_17, 1); +x_22 = lean_ctor_get(x_17, 0); +lean_dec(x_22); +x_23 = !lean_is_exclusive(x_19); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; uint64_t x_27; uint64_t x_28; uint64_t x_29; uint64_t x_30; uint64_t x_31; uint64_t x_32; uint64_t x_33; size_t x_34; size_t x_35; size_t x_36; size_t x_37; size_t x_38; lean_object* x_39; lean_object* x_40; +x_24 = lean_ctor_get(x_19, 0); +x_25 = lean_ctor_get(x_19, 1); +x_26 = lean_array_get_size(x_25); +x_27 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_2); +x_28 = 32; +x_29 = lean_uint64_shift_right(x_27, x_28); +x_30 = lean_uint64_xor(x_27, x_29); +x_31 = 16; +x_32 = lean_uint64_shift_right(x_30, x_31); +x_33 = lean_uint64_xor(x_30, x_32); +x_34 = lean_uint64_to_usize(x_33); +x_35 = lean_usize_of_nat(x_26); +lean_dec(x_26); +x_36 = 1; +x_37 = lean_usize_sub(x_35, x_36); +x_38 = lean_usize_land(x_34, x_37); +x_39 = lean_array_uget(x_25, x_38); +x_40 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__1(x_2, 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; lean_object* x_47; lean_object* x_48; uint8_t x_49; +x_41 = lean_ctor_get(x_18, 0); +lean_inc(x_41); +x_42 = l_Lean_LocalDecl_userName(x_3); +x_43 = lean_box(0); +lean_ctor_set_tag(x_17, 1); +lean_ctor_set(x_17, 1, x_43); +lean_ctor_set(x_17, 0, x_4); +x_44 = lean_array_mk(x_17); +x_45 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_45, 0, x_42); +lean_ctor_set(x_45, 1, x_5); +lean_ctor_set(x_45, 2, x_6); +lean_ctor_set(x_45, 3, x_44); +x_46 = lean_ctor_get(x_18, 2); +lean_inc(x_46); +x_47 = lean_ctor_get(x_18, 3); +lean_inc(x_47); +x_48 = lean_ctor_get(x_18, 4); +lean_inc(x_48); +lean_dec(x_18); +x_49 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2(x_2, x_39); +if (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; uint8_t x_59; +x_50 = lean_unsigned_to_nat(1u); +x_51 = lean_nat_add(x_24, x_50); +lean_dec(x_24); +x_52 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_52, 0, x_2); +lean_ctor_set(x_52, 1, x_45); +lean_ctor_set(x_52, 2, x_39); +x_53 = lean_array_uset(x_25, x_38, x_52); +x_54 = lean_unsigned_to_nat(4u); +x_55 = lean_nat_mul(x_51, x_54); +x_56 = lean_unsigned_to_nat(3u); +x_57 = lean_nat_div(x_55, x_56); +lean_dec(x_55); +x_58 = lean_array_get_size(x_53); +x_59 = lean_nat_dec_le(x_57, x_58); +lean_dec(x_58); +lean_dec(x_57); +if (x_59 == 0) +{ +lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_60 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__3(x_53); +lean_ctor_set(x_19, 1, x_60); +lean_ctor_set(x_19, 0, x_51); +x_61 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_61, 0, x_41); +lean_ctor_set(x_61, 1, x_19); +lean_ctor_set(x_61, 2, x_46); +lean_ctor_set(x_61, 3, x_47); +lean_ctor_set(x_61, 4, x_48); +x_62 = lean_st_ref_set(x_9, x_61, x_21); +x_63 = !lean_is_exclusive(x_62); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; +x_64 = lean_ctor_get(x_62, 0); +lean_dec(x_64); +x_65 = lean_box(0); +lean_ctor_set(x_62, 0, x_65); +x_11 = x_62; +goto block_16; +} else { lean_object* x_66; lean_object* x_67; lean_object* x_68; @@ -10792,151 +11323,156 @@ x_67 = lean_box(0); x_68 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_68, 0, x_67); lean_ctor_set(x_68, 1, x_66); -return x_68; -} +x_11 = x_68; +goto block_16; } } 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; uint8_t x_75; -x_69 = lean_box(0); -x_70 = lean_array_uset(x_17, x_30, x_69); -x_71 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(x_1, x_37, x_31); -x_72 = lean_array_uset(x_70, x_30, x_71); -lean_ctor_set(x_11, 1, x_72); -x_73 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_73, 0, x_33); -lean_ctor_set(x_73, 1, x_11); -lean_ctor_set(x_73, 2, x_38); -lean_ctor_set(x_73, 3, x_39); -lean_ctor_set(x_73, 4, x_40); -x_74 = lean_st_ref_set(x_7, x_73, x_13); -x_75 = !lean_is_exclusive(x_74); -if (x_75 == 0) +lean_object* x_69; lean_object* x_70; uint8_t x_71; +lean_ctor_set(x_19, 1, x_53); +lean_ctor_set(x_19, 0, x_51); +x_69 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_69, 0, x_41); +lean_ctor_set(x_69, 1, x_19); +lean_ctor_set(x_69, 2, x_46); +lean_ctor_set(x_69, 3, x_47); +lean_ctor_set(x_69, 4, x_48); +x_70 = lean_st_ref_set(x_9, x_69, x_21); +x_71 = !lean_is_exclusive(x_70); +if (x_71 == 0) { -lean_object* x_76; lean_object* x_77; -x_76 = lean_ctor_get(x_74, 0); -lean_dec(x_76); -x_77 = lean_box(0); -lean_ctor_set(x_74, 0, x_77); -return x_74; +lean_object* x_72; lean_object* x_73; +x_72 = lean_ctor_get(x_70, 0); +lean_dec(x_72); +x_73 = lean_box(0); +lean_ctor_set(x_70, 0, x_73); +x_11 = x_70; +goto block_16; } else { -lean_object* x_78; lean_object* x_79; lean_object* x_80; -x_78 = lean_ctor_get(x_74, 1); -lean_inc(x_78); -lean_dec(x_74); -x_79 = lean_box(0); -x_80 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_80, 0, x_79); -lean_ctor_set(x_80, 1, x_78); -return x_80; +lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_74 = lean_ctor_get(x_70, 1); +lean_inc(x_74); +lean_dec(x_70); +x_75 = lean_box(0); +x_76 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_76, 1, x_74); +x_11 = x_76; +goto block_16; } } } 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; uint8_t x_92; -lean_free_object(x_9); -lean_dec(x_5); -lean_dec(x_4); -x_81 = lean_ctor_get(x_32, 0); -lean_inc(x_81); -lean_dec(x_32); -x_82 = lean_ctor_get(x_10, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_81, 0); -lean_inc(x_83); -x_84 = lean_ctor_get(x_81, 1); -lean_inc(x_84); -x_85 = lean_ctor_get(x_81, 2); -lean_inc(x_85); -x_86 = lean_ctor_get(x_81, 3); -lean_inc(x_86); -lean_dec(x_81); -x_87 = lean_array_push(x_86, x_3); -x_88 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_88, 0, x_83); -lean_ctor_set(x_88, 1, x_84); -lean_ctor_set(x_88, 2, x_85); -lean_ctor_set(x_88, 3, x_87); -x_89 = lean_ctor_get(x_10, 2); -lean_inc(x_89); -x_90 = lean_ctor_get(x_10, 3); -lean_inc(x_90); -x_91 = lean_ctor_get(x_10, 4); -lean_inc(x_91); -lean_dec(x_10); -x_92 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2(x_1, x_31); -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_16, x_93); -lean_dec(x_16); -x_95 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_95, 0, x_1); -lean_ctor_set(x_95, 1, x_88); -lean_ctor_set(x_95, 2, x_31); -x_96 = lean_array_uset(x_17, x_30, 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_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_77 = lean_box(0); +x_78 = lean_array_uset(x_25, x_38, x_77); +x_79 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(x_2, x_45, x_39); +x_80 = lean_array_uset(x_78, x_38, x_79); +lean_ctor_set(x_19, 1, x_80); +x_81 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_81, 0, x_41); +lean_ctor_set(x_81, 1, x_19); +lean_ctor_set(x_81, 2, x_46); +lean_ctor_set(x_81, 3, x_47); +lean_ctor_set(x_81, 4, x_48); +x_82 = lean_st_ref_set(x_9, x_81, x_21); +x_83 = !lean_is_exclusive(x_82); +if (x_83 == 0) { -lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; -x_103 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__3(x_96); -lean_ctor_set(x_11, 1, x_103); -lean_ctor_set(x_11, 0, x_94); -x_104 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_104, 0, x_82); -lean_ctor_set(x_104, 1, x_11); -lean_ctor_set(x_104, 2, x_89); -lean_ctor_set(x_104, 3, x_90); -lean_ctor_set(x_104, 4, x_91); -x_105 = lean_st_ref_set(x_7, x_104, x_13); -x_106 = !lean_is_exclusive(x_105); -if (x_106 == 0) -{ -lean_object* x_107; lean_object* x_108; -x_107 = lean_ctor_get(x_105, 0); -lean_dec(x_107); -x_108 = lean_box(0); -lean_ctor_set(x_105, 0, x_108); -return x_105; +lean_object* x_84; lean_object* x_85; +x_84 = lean_ctor_get(x_82, 0); +lean_dec(x_84); +x_85 = lean_box(0); +lean_ctor_set(x_82, 0, x_85); +x_11 = x_82; +goto block_16; } else { -lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_109 = lean_ctor_get(x_105, 1); -lean_inc(x_109); -lean_dec(x_105); -x_110 = lean_box(0); -x_111 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_111, 0, x_110); -lean_ctor_set(x_111, 1, x_109); -return x_111; +lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_86 = lean_ctor_get(x_82, 1); +lean_inc(x_86); +lean_dec(x_82); +x_87 = lean_box(0); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_87); +lean_ctor_set(x_88, 1, x_86); +x_11 = x_88; +goto block_16; +} } } else { -lean_object* x_112; lean_object* x_113; uint8_t x_114; -lean_ctor_set(x_11, 1, x_96); -lean_ctor_set(x_11, 0, x_94); +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; uint8_t x_100; +lean_free_object(x_17); +lean_dec(x_6); +lean_dec(x_5); +x_89 = lean_ctor_get(x_40, 0); +lean_inc(x_89); +lean_dec(x_40); +x_90 = lean_ctor_get(x_18, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_89, 0); +lean_inc(x_91); +x_92 = lean_ctor_get(x_89, 1); +lean_inc(x_92); +x_93 = lean_ctor_get(x_89, 2); +lean_inc(x_93); +x_94 = lean_ctor_get(x_89, 3); +lean_inc(x_94); +lean_dec(x_89); +x_95 = lean_array_push(x_94, x_4); +x_96 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_96, 0, x_91); +lean_ctor_set(x_96, 1, x_92); +lean_ctor_set(x_96, 2, x_93); +lean_ctor_set(x_96, 3, x_95); +x_97 = lean_ctor_get(x_18, 2); +lean_inc(x_97); +x_98 = lean_ctor_get(x_18, 3); +lean_inc(x_98); +x_99 = lean_ctor_get(x_18, 4); +lean_inc(x_99); +lean_dec(x_18); +x_100 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2(x_2, x_39); +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; +x_101 = lean_unsigned_to_nat(1u); +x_102 = lean_nat_add(x_24, x_101); +lean_dec(x_24); +x_103 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_103, 0, x_2); +lean_ctor_set(x_103, 1, x_96); +lean_ctor_set(x_103, 2, x_39); +x_104 = lean_array_uset(x_25, x_38, 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; lean_object* x_113; uint8_t x_114; +x_111 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__3(x_104); +lean_ctor_set(x_19, 1, x_111); +lean_ctor_set(x_19, 0, x_102); x_112 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_112, 0, x_82); -lean_ctor_set(x_112, 1, x_11); -lean_ctor_set(x_112, 2, x_89); -lean_ctor_set(x_112, 3, x_90); -lean_ctor_set(x_112, 4, x_91); -x_113 = lean_st_ref_set(x_7, x_112, x_13); +lean_ctor_set(x_112, 0, x_90); +lean_ctor_set(x_112, 1, x_19); +lean_ctor_set(x_112, 2, x_97); +lean_ctor_set(x_112, 3, x_98); +lean_ctor_set(x_112, 4, x_99); +x_113 = lean_st_ref_set(x_9, x_112, x_21); x_114 = !lean_is_exclusive(x_113); if (x_114 == 0) { @@ -10945,7 +11481,8 @@ x_115 = lean_ctor_get(x_113, 0); lean_dec(x_115); x_116 = lean_box(0); lean_ctor_set(x_113, 0, x_116); -return x_113; +x_11 = x_113; +goto block_16; } else { @@ -10957,757 +11494,821 @@ x_118 = lean_box(0); x_119 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_119, 0, x_118); lean_ctor_set(x_119, 1, x_117); -return x_119; -} +x_11 = x_119; +goto block_16; } } else { -lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; uint8_t x_126; -x_120 = lean_box(0); -x_121 = lean_array_uset(x_17, x_30, x_120); -x_122 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(x_1, x_88, x_31); -x_123 = lean_array_uset(x_121, x_30, x_122); -lean_ctor_set(x_11, 1, x_123); -x_124 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_124, 0, x_82); -lean_ctor_set(x_124, 1, x_11); -lean_ctor_set(x_124, 2, x_89); -lean_ctor_set(x_124, 3, x_90); -lean_ctor_set(x_124, 4, x_91); -x_125 = lean_st_ref_set(x_7, x_124, x_13); -x_126 = !lean_is_exclusive(x_125); -if (x_126 == 0) -{ -lean_object* x_127; lean_object* x_128; -x_127 = lean_ctor_get(x_125, 0); -lean_dec(x_127); -x_128 = lean_box(0); -lean_ctor_set(x_125, 0, x_128); -return x_125; +lean_object* x_120; lean_object* x_121; uint8_t x_122; +lean_ctor_set(x_19, 1, x_104); +lean_ctor_set(x_19, 0, x_102); +x_120 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_120, 0, x_90); +lean_ctor_set(x_120, 1, x_19); +lean_ctor_set(x_120, 2, x_97); +lean_ctor_set(x_120, 3, x_98); +lean_ctor_set(x_120, 4, x_99); +x_121 = lean_st_ref_set(x_9, x_120, x_21); +x_122 = !lean_is_exclusive(x_121); +if (x_122 == 0) +{ +lean_object* x_123; lean_object* x_124; +x_123 = lean_ctor_get(x_121, 0); +lean_dec(x_123); +x_124 = lean_box(0); +lean_ctor_set(x_121, 0, x_124); +x_11 = x_121; +goto block_16; } else { -lean_object* x_129; lean_object* x_130; lean_object* x_131; -x_129 = lean_ctor_get(x_125, 1); -lean_inc(x_129); -lean_dec(x_125); -x_130 = lean_box(0); -x_131 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_131, 0, x_130); -lean_ctor_set(x_131, 1, x_129); -return x_131; -} +lean_object* x_125; lean_object* x_126; lean_object* x_127; +x_125 = lean_ctor_get(x_121, 1); +lean_inc(x_125); +lean_dec(x_121); +x_126 = lean_box(0); +x_127 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_127, 0, x_126); +lean_ctor_set(x_127, 1, x_125); +x_11 = x_127; +goto block_16; } } } else { -lean_object* x_132; lean_object* x_133; lean_object* x_134; uint64_t 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; size_t x_142; size_t x_143; size_t x_144; size_t x_145; size_t x_146; lean_object* x_147; lean_object* x_148; -x_132 = lean_ctor_get(x_11, 0); -x_133 = lean_ctor_get(x_11, 1); -lean_inc(x_133); -lean_inc(x_132); -lean_dec(x_11); -x_134 = lean_array_get_size(x_133); -x_135 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_1); -x_136 = 32; -x_137 = lean_uint64_shift_right(x_135, x_136); -x_138 = lean_uint64_xor(x_135, x_137); -x_139 = 16; -x_140 = lean_uint64_shift_right(x_138, x_139); -x_141 = lean_uint64_xor(x_138, x_140); -x_142 = lean_uint64_to_usize(x_141); -x_143 = lean_usize_of_nat(x_134); -lean_dec(x_134); -x_144 = 1; -x_145 = lean_usize_sub(x_143, x_144); -x_146 = lean_usize_land(x_142, x_145); -x_147 = lean_array_uget(x_133, x_146); -x_148 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences___spec__1(x_1, 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; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; uint8_t x_157; -x_149 = lean_ctor_get(x_10, 0); -lean_inc(x_149); -x_150 = l_Lean_LocalDecl_userName(x_2); -x_151 = lean_box(0); -lean_ctor_set_tag(x_9, 1); -lean_ctor_set(x_9, 1, x_151); -lean_ctor_set(x_9, 0, x_3); -x_152 = lean_array_mk(x_9); -x_153 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_153, 0, x_150); -lean_ctor_set(x_153, 1, x_4); -lean_ctor_set(x_153, 2, x_5); -lean_ctor_set(x_153, 3, x_152); -x_154 = lean_ctor_get(x_10, 2); -lean_inc(x_154); -x_155 = lean_ctor_get(x_10, 3); -lean_inc(x_155); -x_156 = lean_ctor_get(x_10, 4); -lean_inc(x_156); -lean_dec(x_10); -x_157 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2(x_1, x_147); -if (x_157 == 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; lean_object* x_165; lean_object* x_166; uint8_t x_167; -x_158 = lean_unsigned_to_nat(1u); -x_159 = lean_nat_add(x_132, x_158); -lean_dec(x_132); -x_160 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_160, 0, x_1); -lean_ctor_set(x_160, 1, x_153); -lean_ctor_set(x_160, 2, x_147); -x_161 = lean_array_uset(x_133, x_146, x_160); -x_162 = lean_unsigned_to_nat(4u); -x_163 = lean_nat_mul(x_159, x_162); -x_164 = lean_unsigned_to_nat(3u); -x_165 = lean_nat_div(x_163, x_164); -lean_dec(x_163); -x_166 = lean_array_get_size(x_161); -x_167 = lean_nat_dec_le(x_165, x_166); -lean_dec(x_166); -lean_dec(x_165); -if (x_167 == 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; uint8_t x_134; +x_128 = lean_box(0); +x_129 = lean_array_uset(x_25, x_38, x_128); +x_130 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(x_2, x_96, x_39); +x_131 = lean_array_uset(x_129, x_38, x_130); +lean_ctor_set(x_19, 1, x_131); +x_132 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_132, 0, x_90); +lean_ctor_set(x_132, 1, x_19); +lean_ctor_set(x_132, 2, x_97); +lean_ctor_set(x_132, 3, x_98); +lean_ctor_set(x_132, 4, x_99); +x_133 = lean_st_ref_set(x_9, x_132, x_21); +x_134 = !lean_is_exclusive(x_133); +if (x_134 == 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; lean_object* x_175; -x_168 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__3(x_161); -x_169 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_169, 0, x_159); -lean_ctor_set(x_169, 1, x_168); -x_170 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_170, 0, x_149); -lean_ctor_set(x_170, 1, x_169); -lean_ctor_set(x_170, 2, x_154); -lean_ctor_set(x_170, 3, x_155); -lean_ctor_set(x_170, 4, x_156); -x_171 = lean_st_ref_set(x_7, x_170, x_13); -x_172 = lean_ctor_get(x_171, 1); -lean_inc(x_172); -if (lean_is_exclusive(x_171)) { - lean_ctor_release(x_171, 0); - lean_ctor_release(x_171, 1); - x_173 = x_171; -} else { - lean_dec_ref(x_171); - x_173 = lean_box(0); +lean_object* x_135; lean_object* x_136; +x_135 = lean_ctor_get(x_133, 0); +lean_dec(x_135); +x_136 = lean_box(0); +lean_ctor_set(x_133, 0, x_136); +x_11 = x_133; +goto block_16; +} +else +{ +lean_object* x_137; lean_object* x_138; lean_object* x_139; +x_137 = lean_ctor_get(x_133, 1); +lean_inc(x_137); +lean_dec(x_133); +x_138 = lean_box(0); +x_139 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_139, 0, x_138); +lean_ctor_set(x_139, 1, x_137); +x_11 = x_139; +goto block_16; +} } -x_174 = lean_box(0); -if (lean_is_scalar(x_173)) { - x_175 = lean_alloc_ctor(0, 2, 0); -} else { - x_175 = x_173; } -lean_ctor_set(x_175, 0, x_174); -lean_ctor_set(x_175, 1, x_172); -return x_175; } else { -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_176 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_176, 0, x_159); -lean_ctor_set(x_176, 1, x_161); -x_177 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_177, 0, x_149); +lean_object* x_140; lean_object* x_141; lean_object* x_142; uint64_t x_143; uint64_t x_144; uint64_t x_145; uint64_t x_146; uint64_t x_147; uint64_t x_148; uint64_t x_149; size_t x_150; size_t x_151; size_t x_152; size_t x_153; size_t x_154; lean_object* x_155; lean_object* x_156; +x_140 = lean_ctor_get(x_19, 0); +x_141 = lean_ctor_get(x_19, 1); +lean_inc(x_141); +lean_inc(x_140); +lean_dec(x_19); +x_142 = lean_array_get_size(x_141); +x_143 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_2); +x_144 = 32; +x_145 = lean_uint64_shift_right(x_143, x_144); +x_146 = lean_uint64_xor(x_143, x_145); +x_147 = 16; +x_148 = lean_uint64_shift_right(x_146, x_147); +x_149 = lean_uint64_xor(x_146, x_148); +x_150 = lean_uint64_to_usize(x_149); +x_151 = lean_usize_of_nat(x_142); +lean_dec(x_142); +x_152 = 1; +x_153 = lean_usize_sub(x_151, x_152); +x_154 = lean_usize_land(x_150, x_153); +x_155 = lean_array_uget(x_141, x_154); +x_156 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__1(x_2, x_155); +if (lean_obj_tag(x_156) == 0) +{ +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; uint8_t x_165; +x_157 = lean_ctor_get(x_18, 0); +lean_inc(x_157); +x_158 = l_Lean_LocalDecl_userName(x_3); +x_159 = lean_box(0); +lean_ctor_set_tag(x_17, 1); +lean_ctor_set(x_17, 1, x_159); +lean_ctor_set(x_17, 0, x_4); +x_160 = lean_array_mk(x_17); +x_161 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_161, 0, x_158); +lean_ctor_set(x_161, 1, x_5); +lean_ctor_set(x_161, 2, x_6); +lean_ctor_set(x_161, 3, x_160); +x_162 = lean_ctor_get(x_18, 2); +lean_inc(x_162); +x_163 = lean_ctor_get(x_18, 3); +lean_inc(x_163); +x_164 = lean_ctor_get(x_18, 4); +lean_inc(x_164); +lean_dec(x_18); +x_165 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2(x_2, x_155); +if (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; uint8_t x_175; +x_166 = lean_unsigned_to_nat(1u); +x_167 = lean_nat_add(x_140, x_166); +lean_dec(x_140); +x_168 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_168, 0, x_2); +lean_ctor_set(x_168, 1, x_161); +lean_ctor_set(x_168, 2, x_155); +x_169 = lean_array_uset(x_141, x_154, x_168); +x_170 = lean_unsigned_to_nat(4u); +x_171 = lean_nat_mul(x_167, x_170); +x_172 = lean_unsigned_to_nat(3u); +x_173 = lean_nat_div(x_171, x_172); +lean_dec(x_171); +x_174 = lean_array_get_size(x_169); +x_175 = lean_nat_dec_le(x_173, x_174); +lean_dec(x_174); +lean_dec(x_173); +if (x_175 == 0) +{ +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_176 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__3(x_169); +x_177 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_177, 0, x_167); lean_ctor_set(x_177, 1, x_176); -lean_ctor_set(x_177, 2, x_154); -lean_ctor_set(x_177, 3, x_155); -lean_ctor_set(x_177, 4, x_156); -x_178 = lean_st_ref_set(x_7, x_177, x_13); -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; +x_178 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_178, 0, x_157); +lean_ctor_set(x_178, 1, x_177); +lean_ctor_set(x_178, 2, x_162); +lean_ctor_set(x_178, 3, x_163); +lean_ctor_set(x_178, 4, x_164); +x_179 = lean_st_ref_set(x_9, x_178, x_21); +x_180 = lean_ctor_get(x_179, 1); +lean_inc(x_180); +if (lean_is_exclusive(x_179)) { + lean_ctor_release(x_179, 0); + lean_ctor_release(x_179, 1); + x_181 = x_179; +} else { + lean_dec_ref(x_179); + x_181 = lean_box(0); +} +x_182 = lean_box(0); +if (lean_is_scalar(x_181)) { + x_183 = lean_alloc_ctor(0, 2, 0); +} else { + x_183 = x_181; +} +lean_ctor_set(x_183, 0, x_182); +lean_ctor_set(x_183, 1, x_180); +x_11 = x_183; +goto block_16; +} +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_alloc_ctor(0, 2, 0); +lean_ctor_set(x_184, 0, x_167); +lean_ctor_set(x_184, 1, x_169); +x_185 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_185, 0, x_157); +lean_ctor_set(x_185, 1, x_184); +lean_ctor_set(x_185, 2, x_162); +lean_ctor_set(x_185, 3, x_163); +lean_ctor_set(x_185, 4, x_164); +x_186 = lean_st_ref_set(x_9, x_185, x_21); +x_187 = lean_ctor_get(x_186, 1); +lean_inc(x_187); +if (lean_is_exclusive(x_186)) { + lean_ctor_release(x_186, 0); + lean_ctor_release(x_186, 1); + x_188 = x_186; } else { - lean_dec_ref(x_178); - x_180 = lean_box(0); + lean_dec_ref(x_186); + x_188 = lean_box(0); } -x_181 = lean_box(0); -if (lean_is_scalar(x_180)) { - x_182 = lean_alloc_ctor(0, 2, 0); +x_189 = lean_box(0); +if (lean_is_scalar(x_188)) { + x_190 = lean_alloc_ctor(0, 2, 0); } else { - x_182 = x_180; -} -lean_ctor_set(x_182, 0, x_181); -lean_ctor_set(x_182, 1, x_179); -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; -x_183 = lean_box(0); -x_184 = lean_array_uset(x_133, x_146, x_183); -x_185 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(x_1, x_153, x_147); -x_186 = lean_array_uset(x_184, x_146, x_185); -x_187 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_187, 0, x_132); -lean_ctor_set(x_187, 1, x_186); -x_188 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_188, 0, x_149); -lean_ctor_set(x_188, 1, x_187); -lean_ctor_set(x_188, 2, x_154); -lean_ctor_set(x_188, 3, x_155); -lean_ctor_set(x_188, 4, x_156); -x_189 = lean_st_ref_set(x_7, x_188, x_13); -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; + x_190 = x_188; +} +lean_ctor_set(x_190, 0, x_189); +lean_ctor_set(x_190, 1, x_187); +x_11 = x_190; +goto block_16; +} +} +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; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; +x_191 = lean_box(0); +x_192 = lean_array_uset(x_141, x_154, x_191); +x_193 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(x_2, x_161, x_155); +x_194 = lean_array_uset(x_192, x_154, x_193); +x_195 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_195, 0, x_140); +lean_ctor_set(x_195, 1, x_194); +x_196 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_196, 0, x_157); +lean_ctor_set(x_196, 1, x_195); +lean_ctor_set(x_196, 2, x_162); +lean_ctor_set(x_196, 3, x_163); +lean_ctor_set(x_196, 4, x_164); +x_197 = lean_st_ref_set(x_9, x_196, x_21); +x_198 = lean_ctor_get(x_197, 1); +lean_inc(x_198); +if (lean_is_exclusive(x_197)) { + lean_ctor_release(x_197, 0); + lean_ctor_release(x_197, 1); + x_199 = x_197; } else { - lean_dec_ref(x_189); - x_191 = lean_box(0); + lean_dec_ref(x_197); + x_199 = lean_box(0); } -x_192 = lean_box(0); -if (lean_is_scalar(x_191)) { - x_193 = lean_alloc_ctor(0, 2, 0); +x_200 = lean_box(0); +if (lean_is_scalar(x_199)) { + x_201 = lean_alloc_ctor(0, 2, 0); } else { - x_193 = x_191; + x_201 = x_199; } -lean_ctor_set(x_193, 0, x_192); -lean_ctor_set(x_193, 1, x_190); -return x_193; +lean_ctor_set(x_201, 0, x_200); +lean_ctor_set(x_201, 1, x_198); +x_11 = x_201; +goto block_16; } } 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; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; uint8_t x_205; -lean_free_object(x_9); +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; uint8_t x_213; +lean_free_object(x_17); +lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -x_194 = lean_ctor_get(x_148, 0); -lean_inc(x_194); -lean_dec(x_148); -x_195 = lean_ctor_get(x_10, 0); -lean_inc(x_195); -x_196 = lean_ctor_get(x_194, 0); -lean_inc(x_196); -x_197 = lean_ctor_get(x_194, 1); -lean_inc(x_197); -x_198 = lean_ctor_get(x_194, 2); -lean_inc(x_198); -x_199 = lean_ctor_get(x_194, 3); -lean_inc(x_199); -lean_dec(x_194); -x_200 = lean_array_push(x_199, x_3); -x_201 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_201, 0, x_196); -lean_ctor_set(x_201, 1, x_197); -lean_ctor_set(x_201, 2, x_198); -lean_ctor_set(x_201, 3, x_200); -x_202 = lean_ctor_get(x_10, 2); +x_202 = lean_ctor_get(x_156, 0); lean_inc(x_202); -x_203 = lean_ctor_get(x_10, 3); +lean_dec(x_156); +x_203 = lean_ctor_get(x_18, 0); lean_inc(x_203); -x_204 = lean_ctor_get(x_10, 4); +x_204 = lean_ctor_get(x_202, 0); lean_inc(x_204); -lean_dec(x_10); -x_205 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2(x_1, x_147); -if (x_205 == 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; lean_object* x_212; lean_object* x_213; lean_object* x_214; uint8_t x_215; -x_206 = lean_unsigned_to_nat(1u); -x_207 = lean_nat_add(x_132, x_206); -lean_dec(x_132); -x_208 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_208, 0, x_1); -lean_ctor_set(x_208, 1, x_201); -lean_ctor_set(x_208, 2, x_147); -x_209 = lean_array_uset(x_133, x_146, x_208); -x_210 = lean_unsigned_to_nat(4u); -x_211 = lean_nat_mul(x_207, x_210); -x_212 = lean_unsigned_to_nat(3u); -x_213 = lean_nat_div(x_211, x_212); -lean_dec(x_211); -x_214 = lean_array_get_size(x_209); -x_215 = lean_nat_dec_le(x_213, x_214); -lean_dec(x_214); -lean_dec(x_213); -if (x_215 == 0) -{ -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; -x_216 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__3(x_209); -x_217 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_217, 0, x_207); -lean_ctor_set(x_217, 1, x_216); -x_218 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_218, 0, x_195); -lean_ctor_set(x_218, 1, x_217); -lean_ctor_set(x_218, 2, x_202); -lean_ctor_set(x_218, 3, x_203); -lean_ctor_set(x_218, 4, x_204); -x_219 = lean_st_ref_set(x_7, x_218, x_13); -x_220 = lean_ctor_get(x_219, 1); -lean_inc(x_220); -if (lean_is_exclusive(x_219)) { - lean_ctor_release(x_219, 0); - lean_ctor_release(x_219, 1); - x_221 = x_219; -} else { - lean_dec_ref(x_219); - x_221 = lean_box(0); -} -x_222 = lean_box(0); -if (lean_is_scalar(x_221)) { - x_223 = lean_alloc_ctor(0, 2, 0); -} else { - x_223 = x_221; -} -lean_ctor_set(x_223, 0, x_222); -lean_ctor_set(x_223, 1, x_220); -return x_223; -} -else +x_205 = lean_ctor_get(x_202, 1); +lean_inc(x_205); +x_206 = lean_ctor_get(x_202, 2); +lean_inc(x_206); +x_207 = lean_ctor_get(x_202, 3); +lean_inc(x_207); +lean_dec(x_202); +x_208 = lean_array_push(x_207, x_4); +x_209 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_209, 0, x_204); +lean_ctor_set(x_209, 1, x_205); +lean_ctor_set(x_209, 2, x_206); +lean_ctor_set(x_209, 3, x_208); +x_210 = lean_ctor_get(x_18, 2); +lean_inc(x_210); +x_211 = lean_ctor_get(x_18, 3); +lean_inc(x_211); +x_212 = lean_ctor_get(x_18, 4); +lean_inc(x_212); +lean_dec(x_18); +x_213 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2(x_2, x_155); +if (x_213 == 0) +{ +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; uint8_t x_223; +x_214 = lean_unsigned_to_nat(1u); +x_215 = lean_nat_add(x_140, x_214); +lean_dec(x_140); +x_216 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_216, 0, x_2); +lean_ctor_set(x_216, 1, x_209); +lean_ctor_set(x_216, 2, x_155); +x_217 = lean_array_uset(x_141, x_154, x_216); +x_218 = lean_unsigned_to_nat(4u); +x_219 = lean_nat_mul(x_215, x_218); +x_220 = lean_unsigned_to_nat(3u); +x_221 = lean_nat_div(x_219, x_220); +lean_dec(x_219); +x_222 = lean_array_get_size(x_217); +x_223 = lean_nat_dec_le(x_221, x_222); +lean_dec(x_222); +lean_dec(x_221); +if (x_223 == 0) { -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; -x_224 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_224, 0, x_207); -lean_ctor_set(x_224, 1, x_209); -x_225 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_225, 0, x_195); +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; +x_224 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__3(x_217); +x_225 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_225, 0, x_215); lean_ctor_set(x_225, 1, x_224); -lean_ctor_set(x_225, 2, x_202); -lean_ctor_set(x_225, 3, x_203); -lean_ctor_set(x_225, 4, x_204); -x_226 = lean_st_ref_set(x_7, x_225, x_13); -x_227 = lean_ctor_get(x_226, 1); -lean_inc(x_227); -if (lean_is_exclusive(x_226)) { - lean_ctor_release(x_226, 0); - lean_ctor_release(x_226, 1); - x_228 = x_226; +x_226 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_226, 0, x_203); +lean_ctor_set(x_226, 1, x_225); +lean_ctor_set(x_226, 2, x_210); +lean_ctor_set(x_226, 3, x_211); +lean_ctor_set(x_226, 4, x_212); +x_227 = lean_st_ref_set(x_9, x_226, x_21); +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_226); - x_228 = lean_box(0); + lean_dec_ref(x_227); + x_229 = lean_box(0); } -x_229 = lean_box(0); -if (lean_is_scalar(x_228)) { - x_230 = lean_alloc_ctor(0, 2, 0); +x_230 = lean_box(0); +if (lean_is_scalar(x_229)) { + x_231 = lean_alloc_ctor(0, 2, 0); } else { - x_230 = x_228; -} -lean_ctor_set(x_230, 0, x_229); -lean_ctor_set(x_230, 1, x_227); -return x_230; -} + x_231 = x_229; +} +lean_ctor_set(x_231, 0, x_230); +lean_ctor_set(x_231, 1, x_228); +x_11 = x_231; +goto block_16; +} +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_alloc_ctor(0, 2, 0); +lean_ctor_set(x_232, 0, x_215); +lean_ctor_set(x_232, 1, x_217); +x_233 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_233, 0, x_203); +lean_ctor_set(x_233, 1, x_232); +lean_ctor_set(x_233, 2, x_210); +lean_ctor_set(x_233, 3, x_211); +lean_ctor_set(x_233, 4, x_212); +x_234 = lean_st_ref_set(x_9, x_233, x_21); +x_235 = lean_ctor_get(x_234, 1); +lean_inc(x_235); +if (lean_is_exclusive(x_234)) { + lean_ctor_release(x_234, 0); + lean_ctor_release(x_234, 1); + x_236 = x_234; +} else { + lean_dec_ref(x_234); + x_236 = lean_box(0); } -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; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; -x_231 = lean_box(0); -x_232 = lean_array_uset(x_133, x_146, x_231); -x_233 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(x_1, x_201, x_147); -x_234 = lean_array_uset(x_232, x_146, x_233); -x_235 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_235, 0, x_132); -lean_ctor_set(x_235, 1, x_234); -x_236 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_236, 0, x_195); -lean_ctor_set(x_236, 1, x_235); -lean_ctor_set(x_236, 2, x_202); -lean_ctor_set(x_236, 3, x_203); -lean_ctor_set(x_236, 4, x_204); -x_237 = lean_st_ref_set(x_7, x_236, x_13); -x_238 = lean_ctor_get(x_237, 1); -lean_inc(x_238); -if (lean_is_exclusive(x_237)) { - lean_ctor_release(x_237, 0); - lean_ctor_release(x_237, 1); - x_239 = x_237; +x_237 = lean_box(0); +if (lean_is_scalar(x_236)) { + x_238 = lean_alloc_ctor(0, 2, 0); +} else { + x_238 = x_236; +} +lean_ctor_set(x_238, 0, x_237); +lean_ctor_set(x_238, 1, x_235); +x_11 = x_238; +goto block_16; +} +} +else +{ +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; +x_239 = lean_box(0); +x_240 = lean_array_uset(x_141, x_154, x_239); +x_241 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(x_2, x_209, x_155); +x_242 = lean_array_uset(x_240, x_154, x_241); +x_243 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_243, 0, x_140); +lean_ctor_set(x_243, 1, x_242); +x_244 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_244, 0, x_203); +lean_ctor_set(x_244, 1, x_243); +lean_ctor_set(x_244, 2, x_210); +lean_ctor_set(x_244, 3, x_211); +lean_ctor_set(x_244, 4, x_212); +x_245 = lean_st_ref_set(x_9, x_244, x_21); +x_246 = lean_ctor_get(x_245, 1); +lean_inc(x_246); +if (lean_is_exclusive(x_245)) { + lean_ctor_release(x_245, 0); + lean_ctor_release(x_245, 1); + x_247 = x_245; } else { - lean_dec_ref(x_237); - x_239 = lean_box(0); + lean_dec_ref(x_245); + x_247 = lean_box(0); } -x_240 = lean_box(0); -if (lean_is_scalar(x_239)) { - x_241 = lean_alloc_ctor(0, 2, 0); +x_248 = lean_box(0); +if (lean_is_scalar(x_247)) { + x_249 = lean_alloc_ctor(0, 2, 0); } else { - x_241 = x_239; + x_249 = x_247; } -lean_ctor_set(x_241, 0, x_240); -lean_ctor_set(x_241, 1, x_238); -return x_241; +lean_ctor_set(x_249, 0, x_248); +lean_ctor_set(x_249, 1, x_246); +x_11 = x_249; +goto block_16; } } } } else { -lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; uint64_t x_247; uint64_t x_248; uint64_t x_249; uint64_t x_250; uint64_t x_251; uint64_t x_252; uint64_t x_253; size_t x_254; size_t x_255; size_t x_256; size_t x_257; size_t x_258; lean_object* x_259; lean_object* x_260; -x_242 = lean_ctor_get(x_9, 1); -lean_inc(x_242); -lean_dec(x_9); -x_243 = lean_ctor_get(x_11, 0); -lean_inc(x_243); -x_244 = lean_ctor_get(x_11, 1); -lean_inc(x_244); -if (lean_is_exclusive(x_11)) { - lean_ctor_release(x_11, 0); - lean_ctor_release(x_11, 1); - x_245 = x_11; +lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; uint64_t x_255; uint64_t x_256; uint64_t x_257; uint64_t x_258; uint64_t x_259; uint64_t x_260; uint64_t x_261; size_t x_262; size_t x_263; size_t x_264; size_t x_265; size_t x_266; lean_object* x_267; lean_object* x_268; +x_250 = lean_ctor_get(x_17, 1); +lean_inc(x_250); +lean_dec(x_17); +x_251 = lean_ctor_get(x_19, 0); +lean_inc(x_251); +x_252 = lean_ctor_get(x_19, 1); +lean_inc(x_252); +if (lean_is_exclusive(x_19)) { + lean_ctor_release(x_19, 0); + lean_ctor_release(x_19, 1); + x_253 = x_19; } else { - lean_dec_ref(x_11); - x_245 = lean_box(0); -} -x_246 = lean_array_get_size(x_244); -x_247 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_1); -x_248 = 32; -x_249 = lean_uint64_shift_right(x_247, x_248); -x_250 = lean_uint64_xor(x_247, x_249); -x_251 = 16; -x_252 = lean_uint64_shift_right(x_250, x_251); -x_253 = lean_uint64_xor(x_250, x_252); -x_254 = lean_uint64_to_usize(x_253); -x_255 = lean_usize_of_nat(x_246); -lean_dec(x_246); -x_256 = 1; -x_257 = lean_usize_sub(x_255, x_256); -x_258 = lean_usize_land(x_254, x_257); -x_259 = lean_array_uget(x_244, x_258); -x_260 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences___spec__1(x_1, x_259); -if (lean_obj_tag(x_260) == 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; lean_object* x_267; lean_object* x_268; lean_object* x_269; uint8_t x_270; -x_261 = lean_ctor_get(x_10, 0); -lean_inc(x_261); -x_262 = l_Lean_LocalDecl_userName(x_2); -x_263 = lean_box(0); -x_264 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_264, 0, x_3); -lean_ctor_set(x_264, 1, x_263); -x_265 = lean_array_mk(x_264); -x_266 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_266, 0, x_262); -lean_ctor_set(x_266, 1, x_4); -lean_ctor_set(x_266, 2, x_5); -lean_ctor_set(x_266, 3, x_265); -x_267 = lean_ctor_get(x_10, 2); -lean_inc(x_267); -x_268 = lean_ctor_get(x_10, 3); -lean_inc(x_268); -x_269 = lean_ctor_get(x_10, 4); + lean_dec_ref(x_19); + x_253 = lean_box(0); +} +x_254 = lean_array_get_size(x_252); +x_255 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_2); +x_256 = 32; +x_257 = lean_uint64_shift_right(x_255, x_256); +x_258 = lean_uint64_xor(x_255, x_257); +x_259 = 16; +x_260 = lean_uint64_shift_right(x_258, x_259); +x_261 = lean_uint64_xor(x_258, x_260); +x_262 = lean_uint64_to_usize(x_261); +x_263 = lean_usize_of_nat(x_254); +lean_dec(x_254); +x_264 = 1; +x_265 = lean_usize_sub(x_263, x_264); +x_266 = lean_usize_land(x_262, x_265); +x_267 = lean_array_uget(x_252, x_266); +x_268 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__1(x_2, x_267); +if (lean_obj_tag(x_268) == 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; lean_object* x_277; uint8_t x_278; +x_269 = lean_ctor_get(x_18, 0); lean_inc(x_269); -lean_dec(x_10); -x_270 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2(x_1, x_259); -if (x_270 == 0) +x_270 = l_Lean_LocalDecl_userName(x_3); +x_271 = lean_box(0); +x_272 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_272, 0, x_4); +lean_ctor_set(x_272, 1, x_271); +x_273 = lean_array_mk(x_272); +x_274 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_274, 0, x_270); +lean_ctor_set(x_274, 1, x_5); +lean_ctor_set(x_274, 2, x_6); +lean_ctor_set(x_274, 3, x_273); +x_275 = lean_ctor_get(x_18, 2); +lean_inc(x_275); +x_276 = lean_ctor_get(x_18, 3); +lean_inc(x_276); +x_277 = lean_ctor_get(x_18, 4); +lean_inc(x_277); +lean_dec(x_18); +x_278 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2(x_2, x_267); +if (x_278 == 0) +{ +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; +x_279 = lean_unsigned_to_nat(1u); +x_280 = lean_nat_add(x_251, x_279); +lean_dec(x_251); +x_281 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_281, 0, x_2); +lean_ctor_set(x_281, 1, x_274); +lean_ctor_set(x_281, 2, x_267); +x_282 = lean_array_uset(x_252, x_266, x_281); +x_283 = lean_unsigned_to_nat(4u); +x_284 = lean_nat_mul(x_280, x_283); +x_285 = lean_unsigned_to_nat(3u); +x_286 = lean_nat_div(x_284, x_285); +lean_dec(x_284); +x_287 = lean_array_get_size(x_282); +x_288 = lean_nat_dec_le(x_286, x_287); +lean_dec(x_287); +lean_dec(x_286); +if (x_288 == 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; lean_object* x_278; lean_object* x_279; uint8_t x_280; -x_271 = lean_unsigned_to_nat(1u); -x_272 = lean_nat_add(x_243, x_271); -lean_dec(x_243); -x_273 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_273, 0, x_1); -lean_ctor_set(x_273, 1, x_266); -lean_ctor_set(x_273, 2, x_259); -x_274 = lean_array_uset(x_244, x_258, x_273); -x_275 = lean_unsigned_to_nat(4u); -x_276 = lean_nat_mul(x_272, x_275); -x_277 = lean_unsigned_to_nat(3u); -x_278 = lean_nat_div(x_276, x_277); -lean_dec(x_276); -x_279 = lean_array_get_size(x_274); -x_280 = lean_nat_dec_le(x_278, x_279); -lean_dec(x_279); -lean_dec(x_278); -if (x_280 == 0) -{ -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; -x_281 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__3(x_274); -if (lean_is_scalar(x_245)) { - x_282 = lean_alloc_ctor(0, 2, 0); +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; +x_289 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__3(x_282); +if (lean_is_scalar(x_253)) { + x_290 = lean_alloc_ctor(0, 2, 0); } else { - x_282 = x_245; -} -lean_ctor_set(x_282, 0, x_272); -lean_ctor_set(x_282, 1, x_281); -x_283 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_283, 0, x_261); -lean_ctor_set(x_283, 1, x_282); -lean_ctor_set(x_283, 2, x_267); -lean_ctor_set(x_283, 3, x_268); -lean_ctor_set(x_283, 4, x_269); -x_284 = lean_st_ref_set(x_7, x_283, x_242); -x_285 = lean_ctor_get(x_284, 1); -lean_inc(x_285); -if (lean_is_exclusive(x_284)) { - lean_ctor_release(x_284, 0); - lean_ctor_release(x_284, 1); - x_286 = x_284; + x_290 = x_253; +} +lean_ctor_set(x_290, 0, x_280); +lean_ctor_set(x_290, 1, x_289); +x_291 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_291, 0, x_269); +lean_ctor_set(x_291, 1, x_290); +lean_ctor_set(x_291, 2, x_275); +lean_ctor_set(x_291, 3, x_276); +lean_ctor_set(x_291, 4, x_277); +x_292 = lean_st_ref_set(x_9, x_291, x_250); +x_293 = lean_ctor_get(x_292, 1); +lean_inc(x_293); +if (lean_is_exclusive(x_292)) { + lean_ctor_release(x_292, 0); + lean_ctor_release(x_292, 1); + x_294 = x_292; } else { - lean_dec_ref(x_284); - x_286 = lean_box(0); + lean_dec_ref(x_292); + x_294 = lean_box(0); } -x_287 = lean_box(0); -if (lean_is_scalar(x_286)) { - x_288 = lean_alloc_ctor(0, 2, 0); +x_295 = lean_box(0); +if (lean_is_scalar(x_294)) { + x_296 = lean_alloc_ctor(0, 2, 0); } else { - x_288 = x_286; + x_296 = x_294; } -lean_ctor_set(x_288, 0, x_287); -lean_ctor_set(x_288, 1, x_285); -return x_288; +lean_ctor_set(x_296, 0, x_295); +lean_ctor_set(x_296, 1, x_293); +x_11 = x_296; +goto block_16; } else { -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; -if (lean_is_scalar(x_245)) { - x_289 = lean_alloc_ctor(0, 2, 0); +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; +if (lean_is_scalar(x_253)) { + x_297 = lean_alloc_ctor(0, 2, 0); } else { - x_289 = x_245; -} -lean_ctor_set(x_289, 0, x_272); -lean_ctor_set(x_289, 1, x_274); -x_290 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_290, 0, x_261); -lean_ctor_set(x_290, 1, x_289); -lean_ctor_set(x_290, 2, x_267); -lean_ctor_set(x_290, 3, x_268); -lean_ctor_set(x_290, 4, x_269); -x_291 = lean_st_ref_set(x_7, x_290, x_242); -x_292 = lean_ctor_get(x_291, 1); -lean_inc(x_292); -if (lean_is_exclusive(x_291)) { - lean_ctor_release(x_291, 0); - lean_ctor_release(x_291, 1); - x_293 = x_291; + x_297 = x_253; +} +lean_ctor_set(x_297, 0, x_280); +lean_ctor_set(x_297, 1, x_282); +x_298 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_298, 0, x_269); +lean_ctor_set(x_298, 1, x_297); +lean_ctor_set(x_298, 2, x_275); +lean_ctor_set(x_298, 3, x_276); +lean_ctor_set(x_298, 4, x_277); +x_299 = lean_st_ref_set(x_9, x_298, x_250); +x_300 = lean_ctor_get(x_299, 1); +lean_inc(x_300); +if (lean_is_exclusive(x_299)) { + lean_ctor_release(x_299, 0); + lean_ctor_release(x_299, 1); + x_301 = x_299; } else { - lean_dec_ref(x_291); - x_293 = lean_box(0); + lean_dec_ref(x_299); + x_301 = lean_box(0); } -x_294 = lean_box(0); -if (lean_is_scalar(x_293)) { - x_295 = lean_alloc_ctor(0, 2, 0); +x_302 = lean_box(0); +if (lean_is_scalar(x_301)) { + x_303 = lean_alloc_ctor(0, 2, 0); } else { - x_295 = x_293; + x_303 = x_301; } -lean_ctor_set(x_295, 0, x_294); -lean_ctor_set(x_295, 1, x_292); -return x_295; +lean_ctor_set(x_303, 0, x_302); +lean_ctor_set(x_303, 1, x_300); +x_11 = x_303; +goto block_16; } } else { -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; -x_296 = lean_box(0); -x_297 = lean_array_uset(x_244, x_258, x_296); -x_298 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(x_1, x_266, x_259); -x_299 = lean_array_uset(x_297, x_258, x_298); -if (lean_is_scalar(x_245)) { - x_300 = lean_alloc_ctor(0, 2, 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; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; +x_304 = lean_box(0); +x_305 = lean_array_uset(x_252, x_266, x_304); +x_306 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(x_2, x_274, x_267); +x_307 = lean_array_uset(x_305, x_266, x_306); +if (lean_is_scalar(x_253)) { + x_308 = lean_alloc_ctor(0, 2, 0); } else { - x_300 = x_245; -} -lean_ctor_set(x_300, 0, x_243); -lean_ctor_set(x_300, 1, x_299); -x_301 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_301, 0, x_261); -lean_ctor_set(x_301, 1, x_300); -lean_ctor_set(x_301, 2, x_267); -lean_ctor_set(x_301, 3, x_268); -lean_ctor_set(x_301, 4, x_269); -x_302 = lean_st_ref_set(x_7, x_301, x_242); -x_303 = lean_ctor_get(x_302, 1); -lean_inc(x_303); -if (lean_is_exclusive(x_302)) { - lean_ctor_release(x_302, 0); - lean_ctor_release(x_302, 1); - x_304 = x_302; + x_308 = x_253; +} +lean_ctor_set(x_308, 0, x_251); +lean_ctor_set(x_308, 1, x_307); +x_309 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_309, 0, x_269); +lean_ctor_set(x_309, 1, x_308); +lean_ctor_set(x_309, 2, x_275); +lean_ctor_set(x_309, 3, x_276); +lean_ctor_set(x_309, 4, x_277); +x_310 = lean_st_ref_set(x_9, x_309, x_250); +x_311 = lean_ctor_get(x_310, 1); +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_302); - x_304 = lean_box(0); + lean_dec_ref(x_310); + x_312 = lean_box(0); } -x_305 = lean_box(0); -if (lean_is_scalar(x_304)) { - x_306 = lean_alloc_ctor(0, 2, 0); +x_313 = lean_box(0); +if (lean_is_scalar(x_312)) { + x_314 = lean_alloc_ctor(0, 2, 0); } else { - x_306 = x_304; + x_314 = x_312; } -lean_ctor_set(x_306, 0, x_305); -lean_ctor_set(x_306, 1, x_303); -return x_306; +lean_ctor_set(x_314, 0, x_313); +lean_ctor_set(x_314, 1, x_311); +x_11 = x_314; +goto block_16; } } else { -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; uint8_t x_318; +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; uint8_t x_326; +lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -x_307 = lean_ctor_get(x_260, 0); -lean_inc(x_307); -lean_dec(x_260); -x_308 = lean_ctor_get(x_10, 0); -lean_inc(x_308); -x_309 = lean_ctor_get(x_307, 0); -lean_inc(x_309); -x_310 = lean_ctor_get(x_307, 1); -lean_inc(x_310); -x_311 = lean_ctor_get(x_307, 2); -lean_inc(x_311); -x_312 = lean_ctor_get(x_307, 3); -lean_inc(x_312); -lean_dec(x_307); -x_313 = lean_array_push(x_312, x_3); -x_314 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_314, 0, x_309); -lean_ctor_set(x_314, 1, x_310); -lean_ctor_set(x_314, 2, x_311); -lean_ctor_set(x_314, 3, x_313); -x_315 = lean_ctor_get(x_10, 2); +x_315 = lean_ctor_get(x_268, 0); lean_inc(x_315); -x_316 = lean_ctor_get(x_10, 3); +lean_dec(x_268); +x_316 = lean_ctor_get(x_18, 0); lean_inc(x_316); -x_317 = lean_ctor_get(x_10, 4); +x_317 = lean_ctor_get(x_315, 0); lean_inc(x_317); -lean_dec(x_10); -x_318 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2(x_1, x_259); -if (x_318 == 0) +x_318 = lean_ctor_get(x_315, 1); +lean_inc(x_318); +x_319 = lean_ctor_get(x_315, 2); +lean_inc(x_319); +x_320 = lean_ctor_get(x_315, 3); +lean_inc(x_320); +lean_dec(x_315); +x_321 = lean_array_push(x_320, x_4); +x_322 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_322, 0, x_317); +lean_ctor_set(x_322, 1, x_318); +lean_ctor_set(x_322, 2, x_319); +lean_ctor_set(x_322, 3, x_321); +x_323 = lean_ctor_get(x_18, 2); +lean_inc(x_323); +x_324 = lean_ctor_get(x_18, 3); +lean_inc(x_324); +x_325 = lean_ctor_get(x_18, 4); +lean_inc(x_325); +lean_dec(x_18); +x_326 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2(x_2, x_267); +if (x_326 == 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; lean_object* x_325; lean_object* x_326; lean_object* x_327; uint8_t x_328; -x_319 = lean_unsigned_to_nat(1u); -x_320 = lean_nat_add(x_243, x_319); -lean_dec(x_243); -x_321 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_321, 0, x_1); -lean_ctor_set(x_321, 1, x_314); -lean_ctor_set(x_321, 2, x_259); -x_322 = lean_array_uset(x_244, x_258, x_321); -x_323 = lean_unsigned_to_nat(4u); -x_324 = lean_nat_mul(x_320, x_323); -x_325 = lean_unsigned_to_nat(3u); -x_326 = lean_nat_div(x_324, x_325); -lean_dec(x_324); -x_327 = lean_array_get_size(x_322); -x_328 = lean_nat_dec_le(x_326, x_327); -lean_dec(x_327); -lean_dec(x_326); -if (x_328 == 0) -{ -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; -x_329 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__3(x_322); -if (lean_is_scalar(x_245)) { - x_330 = lean_alloc_ctor(0, 2, 0); +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; uint8_t x_336; +x_327 = lean_unsigned_to_nat(1u); +x_328 = lean_nat_add(x_251, x_327); +lean_dec(x_251); +x_329 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_329, 0, x_2); +lean_ctor_set(x_329, 1, x_322); +lean_ctor_set(x_329, 2, x_267); +x_330 = lean_array_uset(x_252, x_266, x_329); +x_331 = lean_unsigned_to_nat(4u); +x_332 = lean_nat_mul(x_328, x_331); +x_333 = lean_unsigned_to_nat(3u); +x_334 = lean_nat_div(x_332, x_333); +lean_dec(x_332); +x_335 = lean_array_get_size(x_330); +x_336 = lean_nat_dec_le(x_334, x_335); +lean_dec(x_335); +lean_dec(x_334); +if (x_336 == 0) +{ +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; +x_337 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__3(x_330); +if (lean_is_scalar(x_253)) { + x_338 = lean_alloc_ctor(0, 2, 0); } else { - x_330 = x_245; -} -lean_ctor_set(x_330, 0, x_320); -lean_ctor_set(x_330, 1, x_329); -x_331 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_331, 0, x_308); -lean_ctor_set(x_331, 1, x_330); -lean_ctor_set(x_331, 2, x_315); -lean_ctor_set(x_331, 3, x_316); -lean_ctor_set(x_331, 4, x_317); -x_332 = lean_st_ref_set(x_7, x_331, x_242); -x_333 = lean_ctor_get(x_332, 1); -lean_inc(x_333); -if (lean_is_exclusive(x_332)) { - lean_ctor_release(x_332, 0); - lean_ctor_release(x_332, 1); - x_334 = x_332; + x_338 = x_253; +} +lean_ctor_set(x_338, 0, x_328); +lean_ctor_set(x_338, 1, x_337); +x_339 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_339, 0, x_316); +lean_ctor_set(x_339, 1, x_338); +lean_ctor_set(x_339, 2, x_323); +lean_ctor_set(x_339, 3, x_324); +lean_ctor_set(x_339, 4, x_325); +x_340 = lean_st_ref_set(x_9, x_339, x_250); +x_341 = lean_ctor_get(x_340, 1); +lean_inc(x_341); +if (lean_is_exclusive(x_340)) { + lean_ctor_release(x_340, 0); + lean_ctor_release(x_340, 1); + x_342 = x_340; } else { - lean_dec_ref(x_332); - x_334 = lean_box(0); + lean_dec_ref(x_340); + x_342 = lean_box(0); } -x_335 = lean_box(0); -if (lean_is_scalar(x_334)) { - x_336 = lean_alloc_ctor(0, 2, 0); +x_343 = lean_box(0); +if (lean_is_scalar(x_342)) { + x_344 = lean_alloc_ctor(0, 2, 0); } else { - x_336 = x_334; + x_344 = x_342; } -lean_ctor_set(x_336, 0, x_335); -lean_ctor_set(x_336, 1, x_333); -return x_336; +lean_ctor_set(x_344, 0, x_343); +lean_ctor_set(x_344, 1, x_341); +x_11 = x_344; +goto block_16; } else { -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; -if (lean_is_scalar(x_245)) { - x_337 = lean_alloc_ctor(0, 2, 0); +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; +if (lean_is_scalar(x_253)) { + x_345 = lean_alloc_ctor(0, 2, 0); } else { - x_337 = x_245; -} -lean_ctor_set(x_337, 0, x_320); -lean_ctor_set(x_337, 1, x_322); -x_338 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_338, 0, x_308); -lean_ctor_set(x_338, 1, x_337); -lean_ctor_set(x_338, 2, x_315); -lean_ctor_set(x_338, 3, x_316); -lean_ctor_set(x_338, 4, x_317); -x_339 = lean_st_ref_set(x_7, x_338, x_242); -x_340 = lean_ctor_get(x_339, 1); -lean_inc(x_340); -if (lean_is_exclusive(x_339)) { - lean_ctor_release(x_339, 0); - lean_ctor_release(x_339, 1); - x_341 = x_339; + x_345 = x_253; +} +lean_ctor_set(x_345, 0, x_328); +lean_ctor_set(x_345, 1, x_330); +x_346 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_346, 0, x_316); +lean_ctor_set(x_346, 1, x_345); +lean_ctor_set(x_346, 2, x_323); +lean_ctor_set(x_346, 3, x_324); +lean_ctor_set(x_346, 4, x_325); +x_347 = lean_st_ref_set(x_9, x_346, x_250); +x_348 = lean_ctor_get(x_347, 1); +lean_inc(x_348); +if (lean_is_exclusive(x_347)) { + lean_ctor_release(x_347, 0); + lean_ctor_release(x_347, 1); + x_349 = x_347; } else { - lean_dec_ref(x_339); - x_341 = lean_box(0); + lean_dec_ref(x_347); + x_349 = lean_box(0); } -x_342 = lean_box(0); -if (lean_is_scalar(x_341)) { - x_343 = lean_alloc_ctor(0, 2, 0); +x_350 = lean_box(0); +if (lean_is_scalar(x_349)) { + x_351 = lean_alloc_ctor(0, 2, 0); } else { - x_343 = x_341; + x_351 = x_349; } -lean_ctor_set(x_343, 0, x_342); -lean_ctor_set(x_343, 1, x_340); -return x_343; +lean_ctor_set(x_351, 0, x_350); +lean_ctor_set(x_351, 1, x_348); +x_11 = x_351; +goto block_16; } } else { -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; -x_344 = lean_box(0); -x_345 = lean_array_uset(x_244, x_258, x_344); -x_346 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__6(x_1, x_314, x_259); -x_347 = lean_array_uset(x_345, x_258, x_346); -if (lean_is_scalar(x_245)) { - x_348 = lean_alloc_ctor(0, 2, 0); +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; +x_352 = lean_box(0); +x_353 = lean_array_uset(x_252, x_266, x_352); +x_354 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__6(x_2, x_322, x_267); +x_355 = lean_array_uset(x_353, x_266, x_354); +if (lean_is_scalar(x_253)) { + x_356 = lean_alloc_ctor(0, 2, 0); } else { - x_348 = x_245; -} -lean_ctor_set(x_348, 0, x_243); -lean_ctor_set(x_348, 1, x_347); -x_349 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_349, 0, x_308); -lean_ctor_set(x_349, 1, x_348); -lean_ctor_set(x_349, 2, x_315); -lean_ctor_set(x_349, 3, x_316); -lean_ctor_set(x_349, 4, x_317); -x_350 = lean_st_ref_set(x_7, x_349, x_242); -x_351 = lean_ctor_get(x_350, 1); -lean_inc(x_351); -if (lean_is_exclusive(x_350)) { - lean_ctor_release(x_350, 0); - lean_ctor_release(x_350, 1); - x_352 = x_350; + x_356 = x_253; +} +lean_ctor_set(x_356, 0, x_251); +lean_ctor_set(x_356, 1, x_355); +x_357 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_357, 0, x_316); +lean_ctor_set(x_357, 1, x_356); +lean_ctor_set(x_357, 2, x_323); +lean_ctor_set(x_357, 3, x_324); +lean_ctor_set(x_357, 4, x_325); +x_358 = lean_st_ref_set(x_9, x_357, x_250); +x_359 = lean_ctor_get(x_358, 1); +lean_inc(x_359); +if (lean_is_exclusive(x_358)) { + lean_ctor_release(x_358, 0); + lean_ctor_release(x_358, 1); + x_360 = x_358; } else { - lean_dec_ref(x_350); - x_352 = lean_box(0); + lean_dec_ref(x_358); + x_360 = lean_box(0); } -x_353 = lean_box(0); -if (lean_is_scalar(x_352)) { - x_354 = lean_alloc_ctor(0, 2, 0); +x_361 = lean_box(0); +if (lean_is_scalar(x_360)) { + x_362 = lean_alloc_ctor(0, 2, 0); } else { - x_354 = x_352; + x_362 = x_360; } -lean_ctor_set(x_354, 0, x_353); -lean_ctor_set(x_354, 1, x_351); -return x_354; +lean_ctor_set(x_362, 0, x_361); +lean_ctor_set(x_362, 1, x_359); +x_11 = x_362; +goto block_16; } } } +block_16: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +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(x_8); +x_15 = lean_apply_4(x_1, x_12, x_14, x_9, x_13); +return x_15; +} } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__1() { _start: { lean_object* x_1; @@ -11715,31 +12316,31 @@ x_1 = lean_mk_string_unchecked("_", 1, 1); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__1; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__1; x_2 = lean_string_length(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__3() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__1; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__1; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__4() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__1; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__1; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__3; +x_3 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__3; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -11747,3902 +12348,5156 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___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, uint8_t x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_9; lean_object* x_10; -x_9 = l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent(x_1); -x_10 = l_Lean_Syntax_getId(x_9); -if (lean_obj_tag(x_10) == 1) +lean_object* x_11; lean_object* x_12; +x_11 = l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent(x_1); +x_12 = l_Lean_Syntax_getId(x_11); +if (lean_obj_tag(x_12) == 1) { -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; -x_11 = lean_ctor_get(x_10, 1); -lean_inc(x_11); -lean_dec(x_10); -x_12 = lean_string_utf8_byte_size(x_11); -x_13 = lean_unsigned_to_nat(0u); -lean_inc(x_11); -x_14 = lean_alloc_ctor(0, 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_12); -x_15 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__2; -x_16 = l_Substring_nextn(x_14, x_15, x_13); -lean_dec(x_14); -x_17 = lean_nat_add(x_13, x_16); +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_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_string_utf8_byte_size(x_13); +x_15 = lean_unsigned_to_nat(0u); +lean_inc(x_13); +x_16 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_16, 0, x_13); +lean_ctor_set(x_16, 1, x_15); +lean_ctor_set(x_16, 2, x_14); +x_17 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__2; +x_18 = l_Substring_nextn(x_16, x_17, x_15); lean_dec(x_16); -x_18 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_18, 0, x_11); -lean_ctor_set(x_18, 1, x_13); -lean_ctor_set(x_18, 2, x_17); -x_19 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__4; -x_20 = l_Substring_beq(x_18, x_19); -if (x_20 == 0) +x_19 = lean_nat_add(x_15, x_18); +lean_dec(x_18); +x_20 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_20, 0, x_13); +lean_ctor_set(x_20, 1, x_15); +lean_ctor_set(x_20, 2, x_19); +x_21 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__4; +x_22 = l_Substring_beq(x_20, x_21); +if (x_22 == 0) { -lean_object* x_21; lean_object* x_22; -x_21 = lean_box(0); -x_22 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__1(x_2, x_3, x_4, x_9, x_5, x_21, x_7, x_8); -return x_22; +lean_object* x_23; lean_object* x_24; +x_23 = lean_box(0); +x_24 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__3(x_2, x_3, x_4, x_5, x_11, x_6, x_23, x_8, x_9, x_10); +return x_24; } else { -lean_object* x_23; lean_object* x_24; +uint8_t x_25; lean_object* x_26; lean_object* x_27; +lean_dec(x_11); lean_dec(x_9); +lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -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_8); -return x_24; +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_10); +return x_27; } } else { -lean_object* x_25; lean_object* x_26; -lean_dec(x_10); -x_25 = lean_box(0); -x_26 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__1(x_2, x_3, x_4, x_9, x_5, x_25, x_7, x_8); -return x_26; +lean_object* x_28; lean_object* x_29; +lean_dec(x_12); +x_28 = lean_box(0); +x_29 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__3(x_2, x_3, x_4, x_5, x_11, x_6, x_28, x_8, x_9, x_10); +return x_29; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___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_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___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) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_9 = lean_ctor_get(x_1, 0); -lean_inc(x_9); +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -x_10 = lean_ctor_get(x_9, 3); -lean_inc(x_10); -lean_dec(x_9); -x_11 = l_Lean_Linter_getLinterUnusedVariables___closed__1; -x_12 = l_Lean_Linter_getLinterValue(x_11, x_10); -if (x_12 == 0) +x_12 = lean_ctor_get(x_11, 3); +lean_inc(x_12); +lean_dec(x_11); +x_13 = l_Lean_Linter_getLinterUnusedVariables___closed__1; +x_14 = l_Lean_Linter_getLinterValue(x_13, x_12); +if (x_14 == 0) { -lean_object* x_13; lean_object* x_14; -lean_dec(x_10); -lean_dec(x_5); +uint8_t x_15; lean_object* x_16; lean_object* x_17; +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -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_8); -return x_14; +x_15 = 1; +x_16 = lean_box(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_10); +return x_17; } else { -lean_object* x_15; lean_object* x_16; -x_15 = lean_box(0); -x_16 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2(x_2, x_3, x_4, x_5, x_10, x_15, x_7, x_8); -return x_16; +lean_object* x_18; lean_object* x_19; +x_18 = lean_box(0); +x_19 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4(x_2, x_3, x_4, x_5, x_6, x_12, x_18, x_8, x_9, x_10); +return x_19; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___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, uint8_t x_9, lean_object* x_10, lean_object* x_11) { _start: { -switch (lean_obj_tag(x_3)) { -case 0: +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_1, 1); +lean_inc(x_12); +lean_dec(x_1); +lean_inc(x_2); +x_13 = lean_local_ctx_find(x_12, x_2); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; -lean_dec(x_2); -x_7 = lean_ctor_get(x_3, 0); -lean_inc(x_7); +uint8_t x_14; lean_object* x_15; lean_object* x_16; +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); -x_8 = lean_st_ref_take(x_5, x_6); -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_is_exclusive(x_9); -if (x_11 == 0) +lean_dec(x_2); +x_14 = 1; +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_11); +return x_16; +} +else { -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_9, 4); -x_13 = lean_ctor_get(x_7, 3); -lean_inc(x_13); -lean_dec(x_7); -x_14 = lean_ctor_get(x_13, 7); -lean_inc(x_14); +lean_object* x_17; lean_object* x_18; uint8_t x_19; uint8_t x_20; +x_17 = lean_ctor_get(x_13, 0); +lean_inc(x_17); lean_dec(x_13); -x_15 = lean_array_push(x_12, x_14); -lean_ctor_set(x_9, 4, x_15); -x_16 = lean_st_ref_set(x_5, x_9, x_10); -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); +x_18 = lean_ctor_get(x_6, 0); +lean_inc(x_18); +x_19 = 0; +x_20 = l_String_Range_contains(x_7, x_18, x_19); lean_dec(x_18); -x_19 = lean_box(0); -lean_ctor_set(x_16, 0, x_19); -return x_16; +if (x_20 == 0) +{ +uint8_t x_21; lean_object* x_22; lean_object* x_23; +lean_dec(x_17); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_21 = 1; +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_11); +return x_23; } 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; -} +lean_object* x_24; uint8_t x_25; +x_24 = l_Lean_LocalDecl_userName(x_17); +x_25 = l_Lean_Name_hasMacroScopes(x_24); +lean_dec(x_24); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; +x_26 = lean_box(0); +x_27 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__5(x_3, x_4, x_5, x_6, x_17, x_2, x_26, x_9, x_10, x_11); +lean_dec(x_17); +return x_27; } 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; -x_23 = lean_ctor_get(x_9, 0); -x_24 = lean_ctor_get(x_9, 1); -x_25 = lean_ctor_get(x_9, 2); -x_26 = lean_ctor_get(x_9, 3); -x_27 = lean_ctor_get(x_9, 4); -lean_inc(x_27); -lean_inc(x_26); -lean_inc(x_25); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_9); -x_28 = lean_ctor_get(x_7, 3); -lean_inc(x_28); -lean_dec(x_7); -x_29 = lean_ctor_get(x_28, 7); -lean_inc(x_29); -lean_dec(x_28); -x_30 = lean_array_push(x_27, x_29); -x_31 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_31, 0, x_23); -lean_ctor_set(x_31, 1, x_24); -lean_ctor_set(x_31, 2, x_25); -lean_ctor_set(x_31, 3, x_26); -lean_ctor_set(x_31, 4, x_30); -x_32 = lean_st_ref_set(x_5, x_31, x_10); -x_33 = lean_ctor_get(x_32, 1); -lean_inc(x_33); -if (lean_is_exclusive(x_32)) { - lean_ctor_release(x_32, 0); - lean_ctor_release(x_32, 1); - x_34 = x_32; -} else { - lean_dec_ref(x_32); - x_34 = lean_box(0); +uint8_t x_28; lean_object* x_29; lean_object* x_30; +lean_dec(x_17); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_28 = 1; +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_11); +return x_30; } -x_35 = lean_box(0); -if (lean_is_scalar(x_34)) { - x_36 = lean_alloc_ctor(0, 2, 0); -} else { - x_36 = x_34; } -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_33); -return x_36; } } -case 1: +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7___closed__1() { +_start: { -lean_object* x_37; lean_object* x_38; -x_37 = lean_ctor_get(x_3, 0); -lean_inc(x_37); -x_38 = lean_ctor_get(x_37, 3); -lean_inc(x_38); -switch (lean_obj_tag(x_38)) { +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__2___boxed), 4, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7(lean_object* x_1, lean_object* x_2, uint8_t 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) { +_start: +{ +lean_object* x_10; lean_object* x_11; +x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7___closed__1; +x_11 = lean_ctor_get(x_1, 3); +lean_inc(x_11); +switch (lean_obj_tag(x_11)) { case 1: { -lean_object* x_39; lean_object* x_40; -x_39 = lean_ctor_get(x_38, 0); -lean_inc(x_39); -lean_dec(x_38); -x_40 = l_Lean_Elab_Info_range_x3f(x_3); -if (lean_obj_tag(x_40) == 0) +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +lean_dec(x_11); +x_13 = l_Lean_Elab_Info_range_x3f(x_2); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_41; lean_object* x_42; -lean_dec(x_39); -lean_dec(x_37); -lean_dec(x_3); -lean_dec(x_2); -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_6); -return x_42; +uint8_t x_14; lean_object* x_15; lean_object* x_16; +lean_dec(x_12); +lean_dec(x_8); +lean_dec(x_4); +lean_dec(x_1); +x_14 = 1; +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_9); +return x_16; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_40, 0); -lean_inc(x_43); -lean_dec(x_40); -x_44 = l_Lean_Elab_Info_stx(x_3); -lean_dec(x_3); -x_45 = l_Lean_Syntax_getHeadInfo(x_44); -if (lean_obj_tag(x_45) == 0) +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_13, 0); +lean_inc(x_17); +lean_dec(x_13); +x_18 = l_Lean_Elab_Info_stx(x_2); +x_19 = l_Lean_Syntax_getHeadInfo(x_18); +if (lean_obj_tag(x_19) == 0) { -uint8_t x_46; -lean_dec(x_45); -x_46 = lean_ctor_get_uint8(x_37, sizeof(void*)*4); -if (x_46 == 0) +uint8_t x_20; +lean_dec(x_19); +x_20 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +if (x_20 == 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; uint8_t x_55; -lean_dec(x_44); -lean_dec(x_43); -lean_dec(x_37); -lean_dec(x_2); -x_47 = lean_st_ref_take(x_5, x_6); -x_48 = lean_ctor_get(x_47, 0); -lean_inc(x_48); -x_49 = lean_ctor_get(x_48, 2); -lean_inc(x_49); -x_50 = lean_ctor_get(x_47, 1); -lean_inc(x_50); -lean_dec(x_47); -x_51 = lean_ctor_get(x_48, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_48, 1); -lean_inc(x_52); -x_53 = lean_ctor_get(x_48, 3); -lean_inc(x_53); -x_54 = lean_ctor_get(x_48, 4); -lean_inc(x_54); -lean_dec(x_48); -x_55 = !lean_is_exclusive(x_49); -if (x_55 == 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; uint8_t x_29; +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_4); +lean_dec(x_1); +x_21 = lean_st_ref_take(x_8, x_9); +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +x_23 = lean_ctor_get(x_22, 2); +lean_inc(x_23); +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_dec(x_21); +x_25 = lean_ctor_get(x_22, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_22, 1); +lean_inc(x_26); +x_27 = lean_ctor_get(x_22, 3); +lean_inc(x_27); +x_28 = lean_ctor_get(x_22, 4); +lean_inc(x_28); +lean_dec(x_22); +x_29 = !lean_is_exclusive(x_23); +if (x_29 == 0) { -lean_object* x_56; lean_object* x_57; lean_object* x_58; uint64_t 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; size_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_49, 0); -x_57 = lean_ctor_get(x_49, 1); -x_58 = lean_array_get_size(x_57); -x_59 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_39); -x_60 = 32; -x_61 = lean_uint64_shift_right(x_59, x_60); -x_62 = lean_uint64_xor(x_59, x_61); -x_63 = 16; -x_64 = lean_uint64_shift_right(x_62, x_63); -x_65 = lean_uint64_xor(x_62, x_64); -x_66 = lean_uint64_to_usize(x_65); -x_67 = lean_usize_of_nat(x_58); -lean_dec(x_58); -x_68 = 1; -x_69 = lean_usize_sub(x_67, x_68); -x_70 = lean_usize_land(x_66, x_69); -x_71 = lean_array_uget(x_57, x_70); -x_72 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_39, x_71); -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; uint8_t x_83; -x_73 = lean_unsigned_to_nat(1u); -x_74 = lean_nat_add(x_56, x_73); +lean_object* x_30; lean_object* x_31; lean_object* x_32; uint64_t x_33; uint64_t x_34; uint64_t x_35; uint64_t x_36; uint64_t x_37; uint64_t x_38; uint64_t x_39; size_t x_40; size_t x_41; size_t x_42; size_t x_43; size_t x_44; lean_object* x_45; uint8_t x_46; +x_30 = lean_ctor_get(x_23, 0); +x_31 = lean_ctor_get(x_23, 1); +x_32 = lean_array_get_size(x_31); +x_33 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_12); +x_34 = 32; +x_35 = lean_uint64_shift_right(x_33, x_34); +x_36 = lean_uint64_xor(x_33, x_35); +x_37 = 16; +x_38 = lean_uint64_shift_right(x_36, x_37); +x_39 = lean_uint64_xor(x_36, x_38); +x_40 = lean_uint64_to_usize(x_39); +x_41 = lean_usize_of_nat(x_32); +lean_dec(x_32); +x_42 = 1; +x_43 = lean_usize_sub(x_41, x_42); +x_44 = lean_usize_land(x_40, x_43); +x_45 = lean_array_uget(x_31, x_44); +x_46 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_12, x_45); +if (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; uint8_t x_57; +x_47 = lean_unsigned_to_nat(1u); +x_48 = lean_nat_add(x_30, x_47); +lean_dec(x_30); +x_49 = lean_box(0); +x_50 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_50, 0, x_12); +lean_ctor_set(x_50, 1, x_49); +lean_ctor_set(x_50, 2, x_45); +x_51 = lean_array_uset(x_31, x_44, x_50); +x_52 = lean_unsigned_to_nat(4u); +x_53 = lean_nat_mul(x_48, 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); -x_75 = lean_box(0); -x_76 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_76, 0, x_39); -lean_ctor_set(x_76, 1, x_75); -lean_ctor_set(x_76, 2, x_71); -x_77 = lean_array_uset(x_57, x_70, x_76); -x_78 = lean_unsigned_to_nat(4u); -x_79 = lean_nat_mul(x_74, x_78); -x_80 = lean_unsigned_to_nat(3u); -x_81 = lean_nat_div(x_79, x_80); -lean_dec(x_79); -x_82 = lean_array_get_size(x_77); -x_83 = lean_nat_dec_le(x_81, x_82); -lean_dec(x_82); -lean_dec(x_81); -if (x_83 == 0) +lean_dec(x_55); +if (x_57 == 0) { -lean_object* x_84; lean_object* x_85; lean_object* x_86; uint8_t x_87; -x_84 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_77); -lean_ctor_set(x_49, 1, x_84); -lean_ctor_set(x_49, 0, x_74); -x_85 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_85, 0, x_51); -lean_ctor_set(x_85, 1, x_52); -lean_ctor_set(x_85, 2, x_49); -lean_ctor_set(x_85, 3, x_53); -lean_ctor_set(x_85, 4, x_54); -x_86 = lean_st_ref_set(x_5, x_85, x_50); -x_87 = !lean_is_exclusive(x_86); -if (x_87 == 0) -{ -lean_object* x_88; -x_88 = lean_ctor_get(x_86, 0); -lean_dec(x_88); -lean_ctor_set(x_86, 0, x_75); -return x_86; +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 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_51); +lean_ctor_set(x_23, 1, x_58); +lean_ctor_set(x_23, 0, x_48); +x_59 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_59, 0, x_25); +lean_ctor_set(x_59, 1, x_26); +lean_ctor_set(x_59, 2, x_23); +lean_ctor_set(x_59, 3, x_27); +lean_ctor_set(x_59, 4, x_28); +x_60 = lean_st_ref_set(x_8, x_59, x_24); +x_61 = lean_ctor_get(x_60, 1); +lean_inc(x_61); +lean_dec(x_60); +x_62 = lean_box(x_7); +x_63 = lean_apply_4(x_10, x_49, x_62, x_8, x_61); +return x_63; } else { -lean_object* x_89; lean_object* x_90; -x_89 = lean_ctor_get(x_86, 1); -lean_inc(x_89); -lean_dec(x_86); -x_90 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_90, 0, x_75); -lean_ctor_set(x_90, 1, x_89); -return x_90; +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +lean_ctor_set(x_23, 1, x_51); +lean_ctor_set(x_23, 0, x_48); +x_64 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_64, 0, x_25); +lean_ctor_set(x_64, 1, x_26); +lean_ctor_set(x_64, 2, x_23); +lean_ctor_set(x_64, 3, x_27); +lean_ctor_set(x_64, 4, x_28); +x_65 = lean_st_ref_set(x_8, x_64, x_24); +x_66 = lean_ctor_get(x_65, 1); +lean_inc(x_66); +lean_dec(x_65); +x_67 = lean_box(x_7); +x_68 = lean_apply_4(x_10, x_49, x_67, x_8, x_66); +return x_68; } } else { -lean_object* x_91; lean_object* x_92; uint8_t x_93; -lean_ctor_set(x_49, 1, x_77); -lean_ctor_set(x_49, 0, x_74); -x_91 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_91, 0, x_51); -lean_ctor_set(x_91, 1, x_52); -lean_ctor_set(x_91, 2, x_49); -lean_ctor_set(x_91, 3, x_53); -lean_ctor_set(x_91, 4, x_54); -x_92 = lean_st_ref_set(x_5, x_91, x_50); -x_93 = !lean_is_exclusive(x_92); -if (x_93 == 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_dec(x_45); +lean_dec(x_12); +x_69 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_69, 0, x_25); +lean_ctor_set(x_69, 1, x_26); +lean_ctor_set(x_69, 2, x_23); +lean_ctor_set(x_69, 3, x_27); +lean_ctor_set(x_69, 4, x_28); +x_70 = lean_st_ref_set(x_8, x_69, x_24); +x_71 = lean_ctor_get(x_70, 1); +lean_inc(x_71); +lean_dec(x_70); +x_72 = lean_box(0); +x_73 = lean_box(x_7); +x_74 = lean_apply_4(x_10, x_72, x_73, x_8, x_71); +return x_74; +} +} +else { -lean_object* x_94; -x_94 = lean_ctor_get(x_92, 0); -lean_dec(x_94); -lean_ctor_set(x_92, 0, x_75); -return x_92; +lean_object* x_75; lean_object* x_76; lean_object* x_77; uint64_t x_78; uint64_t x_79; uint64_t x_80; uint64_t x_81; uint64_t x_82; uint64_t x_83; uint64_t x_84; size_t x_85; size_t x_86; size_t x_87; size_t x_88; size_t x_89; lean_object* x_90; uint8_t x_91; +x_75 = lean_ctor_get(x_23, 0); +x_76 = lean_ctor_get(x_23, 1); +lean_inc(x_76); +lean_inc(x_75); +lean_dec(x_23); +x_77 = lean_array_get_size(x_76); +x_78 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_12); +x_79 = 32; +x_80 = lean_uint64_shift_right(x_78, x_79); +x_81 = lean_uint64_xor(x_78, x_80); +x_82 = 16; +x_83 = lean_uint64_shift_right(x_81, x_82); +x_84 = lean_uint64_xor(x_81, x_83); +x_85 = lean_uint64_to_usize(x_84); +x_86 = lean_usize_of_nat(x_77); +lean_dec(x_77); +x_87 = 1; +x_88 = lean_usize_sub(x_86, x_87); +x_89 = lean_usize_land(x_85, x_88); +x_90 = lean_array_uget(x_76, x_89); +x_91 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_12, x_90); +if (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; uint8_t x_102; +x_92 = lean_unsigned_to_nat(1u); +x_93 = lean_nat_add(x_75, x_92); +lean_dec(x_75); +x_94 = lean_box(0); +x_95 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_95, 0, x_12); +lean_ctor_set(x_95, 1, x_94); +lean_ctor_set(x_95, 2, x_90); +x_96 = lean_array_uset(x_76, x_89, x_95); +x_97 = lean_unsigned_to_nat(4u); +x_98 = lean_nat_mul(x_93, 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; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_103 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_96); +x_104 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_104, 0, x_93); +lean_ctor_set(x_104, 1, x_103); +x_105 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_105, 0, x_25); +lean_ctor_set(x_105, 1, x_26); +lean_ctor_set(x_105, 2, x_104); +lean_ctor_set(x_105, 3, x_27); +lean_ctor_set(x_105, 4, x_28); +x_106 = lean_st_ref_set(x_8, x_105, x_24); +x_107 = lean_ctor_get(x_106, 1); +lean_inc(x_107); +lean_dec(x_106); +x_108 = lean_box(x_7); +x_109 = lean_apply_4(x_10, x_94, x_108, x_8, x_107); +return x_109; } else { -lean_object* x_95; lean_object* x_96; -x_95 = lean_ctor_get(x_92, 1); -lean_inc(x_95); -lean_dec(x_92); -x_96 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_96, 0, x_75); -lean_ctor_set(x_96, 1, x_95); -return x_96; +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_110 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_110, 0, x_93); +lean_ctor_set(x_110, 1, x_96); +x_111 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_111, 0, x_25); +lean_ctor_set(x_111, 1, x_26); +lean_ctor_set(x_111, 2, x_110); +lean_ctor_set(x_111, 3, x_27); +lean_ctor_set(x_111, 4, x_28); +x_112 = lean_st_ref_set(x_8, x_111, x_24); +x_113 = lean_ctor_get(x_112, 1); +lean_inc(x_113); +lean_dec(x_112); +x_114 = lean_box(x_7); +x_115 = lean_apply_4(x_10, x_94, x_114, x_8, 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_dec(x_90); +lean_dec(x_12); +x_116 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_116, 0, x_75); +lean_ctor_set(x_116, 1, x_76); +x_117 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_117, 0, x_25); +lean_ctor_set(x_117, 1, x_26); +lean_ctor_set(x_117, 2, x_116); +lean_ctor_set(x_117, 3, x_27); +lean_ctor_set(x_117, 4, x_28); +x_118 = lean_st_ref_set(x_8, x_117, x_24); +x_119 = lean_ctor_get(x_118, 1); +lean_inc(x_119); +lean_dec(x_118); +x_120 = lean_box(0); +x_121 = lean_box(x_7); +x_122 = lean_apply_4(x_10, x_120, x_121, x_8, x_119); +return x_122; } } } else { -lean_object* x_97; lean_object* x_98; uint8_t x_99; -lean_dec(x_71); -lean_dec(x_39); -x_97 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_97, 0, x_51); -lean_ctor_set(x_97, 1, x_52); -lean_ctor_set(x_97, 2, x_49); -lean_ctor_set(x_97, 3, x_53); -lean_ctor_set(x_97, 4, x_54); -x_98 = lean_st_ref_set(x_5, x_97, x_50); -x_99 = !lean_is_exclusive(x_98); -if (x_99 == 0) +if (x_3 == 0) { -lean_object* x_100; lean_object* x_101; -x_100 = lean_ctor_get(x_98, 0); -lean_dec(x_100); -x_101 = lean_box(0); -lean_ctor_set(x_98, 0, x_101); -return x_98; +lean_object* x_123; lean_object* x_124; +x_123 = lean_box(0); +x_124 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__6(x_1, x_12, x_4, x_18, x_10, x_17, x_5, x_123, x_7, x_8, x_9); +return x_124; } else { -lean_object* x_102; lean_object* x_103; lean_object* x_104; -x_102 = lean_ctor_get(x_98, 1); -lean_inc(x_102); -lean_dec(x_98); -x_103 = lean_box(0); -x_104 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_104, 0, x_103); -lean_ctor_set(x_104, 1, x_102); -return x_104; +uint8_t x_125; lean_object* x_126; lean_object* x_127; +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_12); +lean_dec(x_8); +lean_dec(x_4); +lean_dec(x_1); +x_125 = 1; +x_126 = lean_box(x_125); +x_127 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_127, 0, x_126); +lean_ctor_set(x_127, 1, x_9); +return x_127; } } } else { -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; -x_105 = lean_ctor_get(x_49, 0); -x_106 = lean_ctor_get(x_49, 1); -lean_inc(x_106); -lean_inc(x_105); -lean_dec(x_49); -x_107 = lean_array_get_size(x_106); -x_108 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_39); -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_106, x_119); -x_121 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_39, x_120); -if (x_121 == 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; lean_object* x_129; lean_object* x_130; lean_object* x_131; uint8_t x_132; -x_122 = lean_unsigned_to_nat(1u); -x_123 = lean_nat_add(x_105, x_122); -lean_dec(x_105); -x_124 = lean_box(0); -x_125 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_125, 0, x_39); -lean_ctor_set(x_125, 1, x_124); -lean_ctor_set(x_125, 2, x_120); -x_126 = lean_array_uset(x_106, x_119, x_125); -x_127 = lean_unsigned_to_nat(4u); -x_128 = lean_nat_mul(x_123, x_127); -x_129 = lean_unsigned_to_nat(3u); -x_130 = lean_nat_div(x_128, x_129); -lean_dec(x_128); -x_131 = lean_array_get_size(x_126); -x_132 = lean_nat_dec_le(x_130, x_131); -lean_dec(x_131); -lean_dec(x_130); -if (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; -x_133 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_126); -x_134 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_134, 0, x_123); -lean_ctor_set(x_134, 1, x_133); -x_135 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_135, 0, x_51); -lean_ctor_set(x_135, 1, x_52); -lean_ctor_set(x_135, 2, x_134); -lean_ctor_set(x_135, 3, x_53); -lean_ctor_set(x_135, 4, x_54); -x_136 = lean_st_ref_set(x_5, x_135, x_50); -x_137 = lean_ctor_get(x_136, 1); -lean_inc(x_137); -if (lean_is_exclusive(x_136)) { - lean_ctor_release(x_136, 0); - lean_ctor_release(x_136, 1); - x_138 = x_136; -} else { - lean_dec_ref(x_136); - x_138 = lean_box(0); -} -if (lean_is_scalar(x_138)) { - x_139 = lean_alloc_ctor(0, 2, 0); -} else { - x_139 = x_138; -} -lean_ctor_set(x_139, 0, x_124); -lean_ctor_set(x_139, 1, x_137); -return x_139; -} -else -{ -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_alloc_ctor(0, 2, 0); -lean_ctor_set(x_140, 0, x_123); -lean_ctor_set(x_140, 1, x_126); -x_141 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_141, 0, x_51); -lean_ctor_set(x_141, 1, x_52); -lean_ctor_set(x_141, 2, x_140); -lean_ctor_set(x_141, 3, x_53); -lean_ctor_set(x_141, 4, x_54); -x_142 = lean_st_ref_set(x_5, x_141, x_50); -x_143 = lean_ctor_get(x_142, 1); -lean_inc(x_143); -if (lean_is_exclusive(x_142)) { - lean_ctor_release(x_142, 0); - lean_ctor_release(x_142, 1); - x_144 = x_142; -} else { - lean_dec_ref(x_142); - x_144 = lean_box(0); +uint8_t x_128; lean_object* x_129; lean_object* x_130; +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_12); +lean_dec(x_8); +lean_dec(x_4); +lean_dec(x_1); +x_128 = 1; +x_129 = lean_box(x_128); +x_130 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_130, 0, x_129); +lean_ctor_set(x_130, 1, x_9); +return x_130; } -if (lean_is_scalar(x_144)) { - x_145 = lean_alloc_ctor(0, 2, 0); -} else { - x_145 = x_144; } -lean_ctor_set(x_145, 0, x_124); -lean_ctor_set(x_145, 1, x_143); -return x_145; } +case 4: +{ +uint8_t x_131; +lean_dec(x_11); +lean_dec(x_4); +x_131 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +lean_dec(x_1); +if (x_131 == 0) +{ +lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_132 = lean_box(0); +x_133 = lean_box(x_7); +x_134 = lean_apply_4(x_10, x_132, x_133, x_8, x_9); +return x_134; } 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; -lean_dec(x_120); -lean_dec(x_39); -x_146 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_146, 0, x_105); -lean_ctor_set(x_146, 1, x_106); -x_147 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_147, 0, x_51); -lean_ctor_set(x_147, 1, x_52); -lean_ctor_set(x_147, 2, x_146); -lean_ctor_set(x_147, 3, x_53); -lean_ctor_set(x_147, 4, x_54); -x_148 = lean_st_ref_set(x_5, x_147, x_50); -x_149 = lean_ctor_get(x_148, 1); +lean_object* x_135; +x_135 = l_Lean_Elab_Info_range_x3f(x_2); +if (lean_obj_tag(x_135) == 0) +{ +uint8_t x_136; lean_object* x_137; lean_object* x_138; +lean_dec(x_8); +x_136 = 1; +x_137 = lean_box(x_136); +x_138 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_138, 0, x_137); +lean_ctor_set(x_138, 1, x_9); +return x_138; +} +else +{ +lean_object* x_139; lean_object* x_140; lean_object* x_141; +x_139 = lean_ctor_get(x_135, 0); +lean_inc(x_139); +lean_dec(x_135); +x_140 = l_Lean_Elab_Info_stx(x_2); +x_141 = l_Lean_Syntax_getHeadInfo(x_140); +lean_dec(x_140); +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; lean_object* x_147; lean_object* x_148; lean_object* x_149; uint8_t x_150; +lean_dec(x_141); +x_142 = lean_st_ref_take(x_8, x_9); +x_143 = lean_ctor_get(x_142, 0); +lean_inc(x_143); +x_144 = lean_ctor_get(x_143, 0); +lean_inc(x_144); +x_145 = lean_ctor_get(x_142, 1); +lean_inc(x_145); +lean_dec(x_142); +x_146 = lean_ctor_get(x_143, 1); +lean_inc(x_146); +x_147 = lean_ctor_get(x_143, 2); +lean_inc(x_147); +x_148 = lean_ctor_get(x_143, 3); +lean_inc(x_148); +x_149 = lean_ctor_get(x_143, 4); lean_inc(x_149); -if (lean_is_exclusive(x_148)) { - lean_ctor_release(x_148, 0); - lean_ctor_release(x_148, 1); - x_150 = x_148; -} else { - lean_dec_ref(x_148); - x_150 = lean_box(0); -} -x_151 = lean_box(0); -if (lean_is_scalar(x_150)) { - x_152 = lean_alloc_ctor(0, 2, 0); -} else { - x_152 = x_150; -} -lean_ctor_set(x_152, 0, x_151); -lean_ctor_set(x_152, 1, x_149); -return x_152; -} +lean_dec(x_143); +x_150 = !lean_is_exclusive(x_144); +if (x_150 == 0) +{ +lean_object* x_151; lean_object* x_152; lean_object* x_153; uint64_t 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; size_t x_161; size_t x_162; size_t x_163; size_t x_164; size_t x_165; lean_object* x_166; uint8_t x_167; +x_151 = lean_ctor_get(x_144, 0); +x_152 = lean_ctor_get(x_144, 1); +x_153 = lean_array_get_size(x_152); +x_154 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_139); +x_155 = 32; +x_156 = lean_uint64_shift_right(x_154, x_155); +x_157 = lean_uint64_xor(x_154, x_156); +x_158 = 16; +x_159 = lean_uint64_shift_right(x_157, x_158); +x_160 = lean_uint64_xor(x_157, x_159); +x_161 = lean_uint64_to_usize(x_160); +x_162 = lean_usize_of_nat(x_153); +lean_dec(x_153); +x_163 = 1; +x_164 = lean_usize_sub(x_162, x_163); +x_165 = lean_usize_land(x_161, x_164); +x_166 = lean_array_uget(x_152, x_165); +x_167 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__7(x_139, x_166); +if (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; lean_object* x_175; lean_object* x_176; lean_object* x_177; uint8_t x_178; +x_168 = lean_unsigned_to_nat(1u); +x_169 = lean_nat_add(x_151, x_168); +lean_dec(x_151); +x_170 = lean_box(0); +x_171 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_171, 0, x_139); +lean_ctor_set(x_171, 1, x_170); +lean_ctor_set(x_171, 2, x_166); +x_172 = lean_array_uset(x_152, x_165, x_171); +x_173 = lean_unsigned_to_nat(4u); +x_174 = lean_nat_mul(x_169, x_173); +x_175 = lean_unsigned_to_nat(3u); +x_176 = lean_nat_div(x_174, x_175); +lean_dec(x_174); +x_177 = lean_array_get_size(x_172); +x_178 = lean_nat_dec_le(x_176, x_177); +lean_dec(x_177); +lean_dec(x_176); +if (x_178 == 0) +{ +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 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__8(x_172); +lean_ctor_set(x_144, 1, x_179); +lean_ctor_set(x_144, 0, x_169); +x_180 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_180, 0, x_144); +lean_ctor_set(x_180, 1, x_146); +lean_ctor_set(x_180, 2, x_147); +lean_ctor_set(x_180, 3, x_148); +lean_ctor_set(x_180, 4, x_149); +x_181 = lean_st_ref_set(x_8, x_180, x_145); +x_182 = lean_ctor_get(x_181, 1); +lean_inc(x_182); +lean_dec(x_181); +x_183 = lean_box(x_7); +x_184 = lean_apply_4(x_10, x_170, x_183, x_8, x_182); +return x_184; +} +else +{ +lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; +lean_ctor_set(x_144, 1, x_172); +lean_ctor_set(x_144, 0, x_169); +x_185 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_185, 0, x_144); +lean_ctor_set(x_185, 1, x_146); +lean_ctor_set(x_185, 2, x_147); +lean_ctor_set(x_185, 3, x_148); +lean_ctor_set(x_185, 4, x_149); +x_186 = lean_st_ref_set(x_8, x_185, x_145); +x_187 = lean_ctor_get(x_186, 1); +lean_inc(x_187); +lean_dec(x_186); +x_188 = lean_box(x_7); +x_189 = lean_apply_4(x_10, x_170, x_188, x_8, x_187); +return x_189; } } else { -lean_object* x_153; lean_object* x_154; -x_153 = lean_ctor_get(x_37, 1); -lean_inc(x_153); -lean_dec(x_37); -lean_inc(x_39); -x_154 = lean_local_ctx_find(x_153, x_39); -if (lean_obj_tag(x_154) == 0) -{ -lean_object* x_155; lean_object* x_156; -lean_dec(x_44); -lean_dec(x_43); -lean_dec(x_39); -lean_dec(x_2); -x_155 = lean_box(0); -x_156 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_156, 0, x_155); -lean_ctor_set(x_156, 1, x_6); -return x_156; +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_166); +lean_dec(x_139); +x_190 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_190, 0, x_144); +lean_ctor_set(x_190, 1, x_146); +lean_ctor_set(x_190, 2, x_147); +lean_ctor_set(x_190, 3, x_148); +lean_ctor_set(x_190, 4, x_149); +x_191 = lean_st_ref_set(x_8, x_190, x_145); +x_192 = lean_ctor_get(x_191, 1); +lean_inc(x_192); +lean_dec(x_191); +x_193 = lean_box(0); +x_194 = lean_box(x_7); +x_195 = lean_apply_4(x_10, x_193, x_194, x_8, x_192); +return x_195; +} } else { -lean_object* x_157; lean_object* x_158; uint8_t x_159; uint8_t x_160; -x_157 = lean_ctor_get(x_154, 0); -lean_inc(x_157); -lean_dec(x_154); -x_158 = lean_ctor_get(x_43, 0); -lean_inc(x_158); -x_159 = 0; -x_160 = l_String_Range_contains(x_1, x_158, x_159); -lean_dec(x_158); -if (x_160 == 0) +lean_object* x_196; lean_object* x_197; lean_object* x_198; uint64_t x_199; uint64_t x_200; uint64_t x_201; uint64_t x_202; uint64_t x_203; uint64_t x_204; uint64_t x_205; size_t x_206; size_t x_207; size_t x_208; size_t x_209; size_t x_210; lean_object* x_211; uint8_t x_212; +x_196 = lean_ctor_get(x_144, 0); +x_197 = lean_ctor_get(x_144, 1); +lean_inc(x_197); +lean_inc(x_196); +lean_dec(x_144); +x_198 = lean_array_get_size(x_197); +x_199 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_139); +x_200 = 32; +x_201 = lean_uint64_shift_right(x_199, x_200); +x_202 = lean_uint64_xor(x_199, x_201); +x_203 = 16; +x_204 = lean_uint64_shift_right(x_202, x_203); +x_205 = lean_uint64_xor(x_202, x_204); +x_206 = lean_uint64_to_usize(x_205); +x_207 = lean_usize_of_nat(x_198); +lean_dec(x_198); +x_208 = 1; +x_209 = lean_usize_sub(x_207, x_208); +x_210 = lean_usize_land(x_206, x_209); +x_211 = lean_array_uget(x_197, x_210); +x_212 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__7(x_139, x_211); +if (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; lean_object* x_220; lean_object* x_221; lean_object* x_222; uint8_t x_223; +x_213 = lean_unsigned_to_nat(1u); +x_214 = lean_nat_add(x_196, x_213); +lean_dec(x_196); +x_215 = lean_box(0); +x_216 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_216, 0, x_139); +lean_ctor_set(x_216, 1, x_215); +lean_ctor_set(x_216, 2, x_211); +x_217 = lean_array_uset(x_197, x_210, x_216); +x_218 = lean_unsigned_to_nat(4u); +x_219 = lean_nat_mul(x_214, x_218); +x_220 = lean_unsigned_to_nat(3u); +x_221 = lean_nat_div(x_219, x_220); +lean_dec(x_219); +x_222 = lean_array_get_size(x_217); +x_223 = lean_nat_dec_le(x_221, x_222); +lean_dec(x_222); +lean_dec(x_221); +if (x_223 == 0) { -lean_object* x_161; lean_object* x_162; -lean_dec(x_157); -lean_dec(x_44); -lean_dec(x_43); -lean_dec(x_39); -lean_dec(x_2); -x_161 = lean_box(0); -x_162 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_162, 0, x_161); -lean_ctor_set(x_162, 1, x_6); -return x_162; +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; +x_224 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__8(x_217); +x_225 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_225, 0, x_214); +lean_ctor_set(x_225, 1, x_224); +x_226 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_226, 0, x_225); +lean_ctor_set(x_226, 1, x_146); +lean_ctor_set(x_226, 2, x_147); +lean_ctor_set(x_226, 3, x_148); +lean_ctor_set(x_226, 4, x_149); +x_227 = lean_st_ref_set(x_8, x_226, x_145); +x_228 = lean_ctor_get(x_227, 1); +lean_inc(x_228); +lean_dec(x_227); +x_229 = lean_box(x_7); +x_230 = lean_apply_4(x_10, x_215, x_229, x_8, x_228); +return x_230; } else { -lean_object* x_163; uint8_t x_164; -x_163 = l_Lean_LocalDecl_userName(x_157); -x_164 = l_Lean_Name_hasMacroScopes(x_163); -lean_dec(x_163); -if (x_164 == 0) -{ -lean_object* x_165; lean_object* x_166; -x_165 = lean_box(0); -x_166 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__3(x_2, x_44, x_43, x_157, x_39, x_165, x_5, x_6); -lean_dec(x_157); -return x_166; +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_alloc_ctor(0, 2, 0); +lean_ctor_set(x_231, 0, x_214); +lean_ctor_set(x_231, 1, x_217); +x_232 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_232, 0, x_231); +lean_ctor_set(x_232, 1, x_146); +lean_ctor_set(x_232, 2, x_147); +lean_ctor_set(x_232, 3, x_148); +lean_ctor_set(x_232, 4, x_149); +x_233 = lean_st_ref_set(x_8, x_232, x_145); +x_234 = lean_ctor_get(x_233, 1); +lean_inc(x_234); +lean_dec(x_233); +x_235 = lean_box(x_7); +x_236 = lean_apply_4(x_10, x_215, x_235, x_8, x_234); +return x_236; +} } else { -lean_object* x_167; lean_object* x_168; -lean_dec(x_157); -lean_dec(x_44); -lean_dec(x_43); -lean_dec(x_39); -lean_dec(x_2); -x_167 = lean_box(0); -x_168 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_168, 0, x_167); -lean_ctor_set(x_168, 1, x_6); -return x_168; +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_dec(x_211); +lean_dec(x_139); +x_237 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_237, 0, x_196); +lean_ctor_set(x_237, 1, x_197); +x_238 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_238, 0, x_237); +lean_ctor_set(x_238, 1, x_146); +lean_ctor_set(x_238, 2, x_147); +lean_ctor_set(x_238, 3, x_148); +lean_ctor_set(x_238, 4, x_149); +x_239 = lean_st_ref_set(x_8, x_238, x_145); +x_240 = lean_ctor_get(x_239, 1); +lean_inc(x_240); +lean_dec(x_239); +x_241 = lean_box(0); +x_242 = lean_box(x_7); +x_243 = lean_apply_4(x_10, x_241, x_242, x_8, x_240); +return x_243; +} +} +} +else +{ +uint8_t x_244; lean_object* x_245; lean_object* x_246; +lean_dec(x_141); +lean_dec(x_139); +lean_dec(x_8); +x_244 = 1; +x_245 = lean_box(x_244); +x_246 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_246, 0, x_245); +lean_ctor_set(x_246, 1, x_9); +return x_246; +} +} +} +} +default: +{ +lean_object* x_247; lean_object* x_248; lean_object* x_249; +lean_dec(x_11); +lean_dec(x_4); +lean_dec(x_1); +x_247 = lean_box(0); +x_248 = lean_box(x_7); +x_249 = lean_apply_4(x_10, x_247, x_248, x_8, x_9); +return x_249; } } } } +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__8(uint8_t 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) { +_start: +{ +if (x_1 == 0) +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_box(0); +x_11 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7(x_2, x_3, x_1, x_4, x_5, x_10, x_7, x_8, x_9); +return x_11; } else { -lean_object* x_169; lean_object* x_170; -lean_dec(x_45); -lean_dec(x_44); -lean_dec(x_43); -lean_dec(x_39); -lean_dec(x_37); +uint8_t x_12; lean_object* x_13; lean_object* x_14; +lean_dec(x_8); +lean_dec(x_4); lean_dec(x_2); -x_169 = lean_box(0); -x_170 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_170, 0, x_169); -lean_ctor_set(x_170, 1, x_6); -return x_170; +x_12 = 1; +x_13 = lean_box(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_9); +return x_14; } } } -case 4: +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__9(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5) { +_start: { -uint8_t x_171; -lean_dec(x_38); -lean_dec(x_2); -x_171 = lean_ctor_get_uint8(x_37, sizeof(void*)*4); -lean_dec(x_37); -if (x_171 == 0) +lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_6 = lean_st_ref_take(x_4, x_5); +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_is_exclusive(x_7); +if (x_9 == 0) { -lean_object* x_172; lean_object* x_173; -lean_dec(x_3); -x_172 = lean_box(0); -x_173 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_173, 0, x_172); -lean_ctor_set(x_173, 1, x_6); -return x_173; -} -else +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_10 = lean_ctor_get(x_7, 3); +x_11 = lean_ctor_get(x_1, 2); +lean_inc(x_11); +x_12 = l_Lean_Linter_UnusedVariables_followAliases(x_10, x_11); +x_13 = lean_ctor_get(x_1, 1); +lean_inc(x_13); +lean_dec(x_1); +x_14 = !lean_is_exclusive(x_10); +if (x_14 == 0) { -lean_object* x_174; -x_174 = l_Lean_Elab_Info_range_x3f(x_3); -if (lean_obj_tag(x_174) == 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; 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_15 = lean_ctor_get(x_10, 0); +x_16 = lean_ctor_get(x_10, 1); +x_17 = lean_array_get_size(x_16); +x_18 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_13); +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_17); +lean_dec(x_17); +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_16, x_29); +x_31 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15(x_13, x_30); +if (x_31 == 0) { -lean_object* x_175; lean_object* x_176; -lean_dec(x_3); -x_175 = lean_box(0); -x_176 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_176, 0, x_175); -lean_ctor_set(x_176, 1, x_6); -return x_176; -} -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; lean_object* x_40; uint8_t x_41; +x_32 = lean_unsigned_to_nat(1u); +x_33 = lean_nat_add(x_15, x_32); +lean_dec(x_15); +x_34 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_34, 0, x_13); +lean_ctor_set(x_34, 1, x_12); +lean_ctor_set(x_34, 2, x_30); +x_35 = lean_array_uset(x_16, x_29, 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); +lean_dec(x_39); +if (x_41 == 0) { -lean_object* x_177; lean_object* x_178; lean_object* x_179; -x_177 = lean_ctor_get(x_174, 0); -lean_inc(x_177); -lean_dec(x_174); -x_178 = l_Lean_Elab_Info_stx(x_3); -lean_dec(x_3); -x_179 = l_Lean_Syntax_getHeadInfo(x_178); -lean_dec(x_178); -if (lean_obj_tag(x_179) == 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; lean_object* x_186; lean_object* x_187; uint8_t x_188; -lean_dec(x_179); -x_180 = lean_st_ref_take(x_5, x_6); -x_181 = lean_ctor_get(x_180, 0); -lean_inc(x_181); -x_182 = lean_ctor_get(x_181, 0); -lean_inc(x_182); -x_183 = lean_ctor_get(x_180, 1); -lean_inc(x_183); -lean_dec(x_180); -x_184 = lean_ctor_get(x_181, 1); -lean_inc(x_184); -x_185 = lean_ctor_get(x_181, 2); -lean_inc(x_185); -x_186 = lean_ctor_get(x_181, 3); -lean_inc(x_186); -x_187 = lean_ctor_get(x_181, 4); -lean_inc(x_187); -lean_dec(x_181); -x_188 = !lean_is_exclusive(x_182); -if (x_188 == 0) -{ -lean_object* x_189; lean_object* x_190; lean_object* x_191; uint64_t x_192; uint64_t x_193; uint64_t x_194; uint64_t x_195; uint64_t x_196; uint64_t x_197; uint64_t x_198; size_t x_199; size_t x_200; size_t x_201; size_t x_202; size_t x_203; lean_object* x_204; uint8_t x_205; -x_189 = lean_ctor_get(x_182, 0); -x_190 = lean_ctor_get(x_182, 1); -x_191 = lean_array_get_size(x_190); -x_192 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_177); -x_193 = 32; -x_194 = lean_uint64_shift_right(x_192, x_193); -x_195 = lean_uint64_xor(x_192, x_194); -x_196 = 16; -x_197 = lean_uint64_shift_right(x_195, x_196); -x_198 = lean_uint64_xor(x_195, x_197); -x_199 = lean_uint64_to_usize(x_198); -x_200 = lean_usize_of_nat(x_191); -lean_dec(x_191); -x_201 = 1; -x_202 = lean_usize_sub(x_200, x_201); -x_203 = lean_usize_land(x_199, x_202); -x_204 = lean_array_uget(x_190, x_203); -x_205 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__7(x_177, x_204); -if (x_205 == 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; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; uint8_t x_216; -x_206 = lean_unsigned_to_nat(1u); -x_207 = lean_nat_add(x_189, x_206); -lean_dec(x_189); -x_208 = lean_box(0); -x_209 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_209, 0, x_177); -lean_ctor_set(x_209, 1, x_208); -lean_ctor_set(x_209, 2, x_204); -x_210 = lean_array_uset(x_190, x_203, x_209); -x_211 = lean_unsigned_to_nat(4u); -x_212 = lean_nat_mul(x_207, x_211); -x_213 = lean_unsigned_to_nat(3u); -x_214 = lean_nat_div(x_212, x_213); -lean_dec(x_212); -x_215 = lean_array_get_size(x_210); -x_216 = lean_nat_dec_le(x_214, x_215); -lean_dec(x_215); -lean_dec(x_214); -if (x_216 == 0) +lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_42 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__16(x_35); +lean_ctor_set(x_10, 1, x_42); +lean_ctor_set(x_10, 0, x_33); +x_43 = lean_st_ref_set(x_4, x_7, x_8); +x_44 = !lean_is_exclusive(x_43); +if (x_44 == 0) { -lean_object* x_217; lean_object* x_218; lean_object* x_219; uint8_t x_220; -x_217 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__8(x_210); -lean_ctor_set(x_182, 1, x_217); -lean_ctor_set(x_182, 0, x_207); -x_218 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_218, 0, x_182); -lean_ctor_set(x_218, 1, x_184); -lean_ctor_set(x_218, 2, x_185); -lean_ctor_set(x_218, 3, x_186); -lean_ctor_set(x_218, 4, x_187); -x_219 = lean_st_ref_set(x_5, x_218, x_183); -x_220 = !lean_is_exclusive(x_219); -if (x_220 == 0) -{ -lean_object* x_221; -x_221 = lean_ctor_get(x_219, 0); -lean_dec(x_221); -lean_ctor_set(x_219, 0, x_208); -return x_219; +lean_object* x_45; uint8_t x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_43, 0); +lean_dec(x_45); +x_46 = 1; +x_47 = lean_box(x_46); +lean_ctor_set(x_43, 0, x_47); +return x_43; } else { -lean_object* x_222; lean_object* x_223; -x_222 = lean_ctor_get(x_219, 1); -lean_inc(x_222); -lean_dec(x_219); -x_223 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_223, 0, x_208); -lean_ctor_set(x_223, 1, x_222); -return x_223; +lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; +x_48 = lean_ctor_get(x_43, 1); +lean_inc(x_48); +lean_dec(x_43); +x_49 = 1; +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; } } else { -lean_object* x_224; lean_object* x_225; uint8_t x_226; -lean_ctor_set(x_182, 1, x_210); -lean_ctor_set(x_182, 0, x_207); -x_224 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_224, 0, x_182); -lean_ctor_set(x_224, 1, x_184); -lean_ctor_set(x_224, 2, x_185); -lean_ctor_set(x_224, 3, x_186); -lean_ctor_set(x_224, 4, x_187); -x_225 = lean_st_ref_set(x_5, x_224, x_183); -x_226 = !lean_is_exclusive(x_225); -if (x_226 == 0) +lean_object* x_52; uint8_t x_53; +lean_ctor_set(x_10, 1, x_35); +lean_ctor_set(x_10, 0, x_33); +x_52 = lean_st_ref_set(x_4, x_7, x_8); +x_53 = !lean_is_exclusive(x_52); +if (x_53 == 0) { -lean_object* x_227; -x_227 = lean_ctor_get(x_225, 0); -lean_dec(x_227); -lean_ctor_set(x_225, 0, x_208); -return x_225; +lean_object* x_54; uint8_t x_55; lean_object* x_56; +x_54 = lean_ctor_get(x_52, 0); +lean_dec(x_54); +x_55 = 1; +x_56 = lean_box(x_55); +lean_ctor_set(x_52, 0, x_56); +return x_52; } else { -lean_object* x_228; lean_object* x_229; -x_228 = lean_ctor_get(x_225, 1); -lean_inc(x_228); -lean_dec(x_225); -x_229 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_229, 0, x_208); -lean_ctor_set(x_229, 1, x_228); -return x_229; +lean_object* x_57; uint8_t x_58; lean_object* x_59; lean_object* x_60; +x_57 = lean_ctor_get(x_52, 1); +lean_inc(x_57); +lean_dec(x_52); +x_58 = 1; +x_59 = lean_box(x_58); +x_60 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_60, 0, x_59); +lean_ctor_set(x_60, 1, x_57); +return x_60; } } } else { -lean_object* x_230; lean_object* x_231; uint8_t x_232; -lean_dec(x_204); -lean_dec(x_177); -x_230 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_230, 0, x_182); -lean_ctor_set(x_230, 1, x_184); -lean_ctor_set(x_230, 2, x_185); -lean_ctor_set(x_230, 3, x_186); -lean_ctor_set(x_230, 4, x_187); -x_231 = lean_st_ref_set(x_5, x_230, x_183); -x_232 = !lean_is_exclusive(x_231); -if (x_232 == 0) -{ -lean_object* x_233; lean_object* x_234; -x_233 = lean_ctor_get(x_231, 0); -lean_dec(x_233); -x_234 = lean_box(0); -lean_ctor_set(x_231, 0, x_234); -return x_231; +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_box(0); +x_62 = lean_array_uset(x_16, x_29, x_61); +x_63 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(x_13, x_12, x_30); +x_64 = lean_array_uset(x_62, x_29, x_63); +lean_ctor_set(x_10, 1, x_64); +x_65 = lean_st_ref_set(x_4, x_7, x_8); +x_66 = !lean_is_exclusive(x_65); +if (x_66 == 0) +{ +lean_object* x_67; uint8_t x_68; lean_object* x_69; +x_67 = lean_ctor_get(x_65, 0); +lean_dec(x_67); +x_68 = 1; +x_69 = lean_box(x_68); +lean_ctor_set(x_65, 0, x_69); +return x_65; } else { -lean_object* x_235; lean_object* x_236; lean_object* x_237; -x_235 = lean_ctor_get(x_231, 1); -lean_inc(x_235); -lean_dec(x_231); -x_236 = lean_box(0); -x_237 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_237, 0, x_236); -lean_ctor_set(x_237, 1, x_235); -return x_237; +lean_object* x_70; uint8_t x_71; lean_object* x_72; lean_object* x_73; +x_70 = lean_ctor_get(x_65, 1); +lean_inc(x_70); +lean_dec(x_65); +x_71 = 1; +x_72 = lean_box(x_71); +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_238; lean_object* x_239; lean_object* x_240; uint64_t x_241; uint64_t x_242; uint64_t x_243; uint64_t x_244; uint64_t x_245; uint64_t x_246; uint64_t x_247; size_t x_248; size_t x_249; size_t x_250; size_t x_251; size_t x_252; lean_object* x_253; uint8_t x_254; -x_238 = lean_ctor_get(x_182, 0); -x_239 = lean_ctor_get(x_182, 1); -lean_inc(x_239); -lean_inc(x_238); -lean_dec(x_182); -x_240 = lean_array_get_size(x_239); -x_241 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_177); -x_242 = 32; -x_243 = lean_uint64_shift_right(x_241, x_242); -x_244 = lean_uint64_xor(x_241, x_243); -x_245 = 16; -x_246 = lean_uint64_shift_right(x_244, x_245); -x_247 = lean_uint64_xor(x_244, x_246); -x_248 = lean_uint64_to_usize(x_247); -x_249 = lean_usize_of_nat(x_240); -lean_dec(x_240); -x_250 = 1; -x_251 = lean_usize_sub(x_249, x_250); -x_252 = lean_usize_land(x_248, x_251); -x_253 = lean_array_uget(x_239, x_252); -x_254 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__7(x_177, x_253); -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_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; uint8_t x_265; -x_255 = lean_unsigned_to_nat(1u); -x_256 = lean_nat_add(x_238, x_255); -lean_dec(x_238); -x_257 = lean_box(0); -x_258 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_258, 0, x_177); -lean_ctor_set(x_258, 1, x_257); -lean_ctor_set(x_258, 2, x_253); -x_259 = lean_array_uset(x_239, x_252, x_258); -x_260 = lean_unsigned_to_nat(4u); -x_261 = lean_nat_mul(x_256, x_260); -x_262 = lean_unsigned_to_nat(3u); -x_263 = lean_nat_div(x_261, x_262); -lean_dec(x_261); -x_264 = lean_array_get_size(x_259); -x_265 = lean_nat_dec_le(x_263, x_264); -lean_dec(x_264); -lean_dec(x_263); -if (x_265 == 0) -{ -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_266 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__8(x_259); -x_267 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_267, 0, x_256); -lean_ctor_set(x_267, 1, x_266); -x_268 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_268, 0, x_267); -lean_ctor_set(x_268, 1, x_184); -lean_ctor_set(x_268, 2, x_185); -lean_ctor_set(x_268, 3, x_186); -lean_ctor_set(x_268, 4, x_187); -x_269 = lean_st_ref_set(x_5, x_268, x_183); -x_270 = lean_ctor_get(x_269, 1); -lean_inc(x_270); -if (lean_is_exclusive(x_269)) { - lean_ctor_release(x_269, 0); - lean_ctor_release(x_269, 1); - x_271 = x_269; +lean_object* x_74; lean_object* x_75; lean_object* x_76; uint64_t x_77; uint64_t x_78; uint64_t x_79; uint64_t x_80; uint64_t x_81; uint64_t x_82; uint64_t x_83; size_t x_84; size_t x_85; size_t x_86; size_t x_87; size_t x_88; lean_object* x_89; uint8_t x_90; +x_74 = lean_ctor_get(x_10, 0); +x_75 = lean_ctor_get(x_10, 1); +lean_inc(x_75); +lean_inc(x_74); +lean_dec(x_10); +x_76 = lean_array_get_size(x_75); +x_77 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_13); +x_78 = 32; +x_79 = lean_uint64_shift_right(x_77, x_78); +x_80 = lean_uint64_xor(x_77, x_79); +x_81 = 16; +x_82 = lean_uint64_shift_right(x_80, x_81); +x_83 = lean_uint64_xor(x_80, x_82); +x_84 = lean_uint64_to_usize(x_83); +x_85 = lean_usize_of_nat(x_76); +lean_dec(x_76); +x_86 = 1; +x_87 = lean_usize_sub(x_85, x_86); +x_88 = lean_usize_land(x_84, x_87); +x_89 = lean_array_uget(x_75, x_88); +x_90 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15(x_13, x_89); +if (x_90 == 0) +{ +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; uint8_t x_100; +x_91 = lean_unsigned_to_nat(1u); +x_92 = lean_nat_add(x_74, x_91); +lean_dec(x_74); +x_93 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_93, 0, x_13); +lean_ctor_set(x_93, 1, x_12); +lean_ctor_set(x_93, 2, x_89); +x_94 = lean_array_uset(x_75, x_88, x_93); +x_95 = lean_unsigned_to_nat(4u); +x_96 = lean_nat_mul(x_92, x_95); +x_97 = lean_unsigned_to_nat(3u); +x_98 = lean_nat_div(x_96, x_97); +lean_dec(x_96); +x_99 = lean_array_get_size(x_94); +x_100 = lean_nat_dec_le(x_98, x_99); +lean_dec(x_99); +lean_dec(x_98); +if (x_100 == 0) +{ +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; +x_101 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__16(x_94); +x_102 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_102, 0, x_92); +lean_ctor_set(x_102, 1, x_101); +lean_ctor_set(x_7, 3, x_102); +x_103 = lean_st_ref_set(x_4, x_7, x_8); +x_104 = lean_ctor_get(x_103, 1); +lean_inc(x_104); +if (lean_is_exclusive(x_103)) { + lean_ctor_release(x_103, 0); + lean_ctor_release(x_103, 1); + x_105 = x_103; } else { - lean_dec_ref(x_269); - x_271 = lean_box(0); + lean_dec_ref(x_103); + x_105 = lean_box(0); } -if (lean_is_scalar(x_271)) { - x_272 = lean_alloc_ctor(0, 2, 0); +x_106 = 1; +x_107 = lean_box(x_106); +if (lean_is_scalar(x_105)) { + x_108 = lean_alloc_ctor(0, 2, 0); } else { - x_272 = x_271; -} -lean_ctor_set(x_272, 0, x_257); -lean_ctor_set(x_272, 1, x_270); -return x_272; -} -else -{ -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_alloc_ctor(0, 2, 0); -lean_ctor_set(x_273, 0, x_256); -lean_ctor_set(x_273, 1, x_259); -x_274 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_274, 0, x_273); -lean_ctor_set(x_274, 1, x_184); -lean_ctor_set(x_274, 2, x_185); -lean_ctor_set(x_274, 3, x_186); -lean_ctor_set(x_274, 4, x_187); -x_275 = lean_st_ref_set(x_5, x_274, x_183); -x_276 = lean_ctor_get(x_275, 1); -lean_inc(x_276); -if (lean_is_exclusive(x_275)) { - lean_ctor_release(x_275, 0); - lean_ctor_release(x_275, 1); - x_277 = x_275; + x_108 = x_105; +} +lean_ctor_set(x_108, 0, x_107); +lean_ctor_set(x_108, 1, x_104); +return x_108; +} +else +{ +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; uint8_t x_113; lean_object* x_114; lean_object* x_115; +x_109 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_109, 0, x_92); +lean_ctor_set(x_109, 1, x_94); +lean_ctor_set(x_7, 3, x_109); +x_110 = lean_st_ref_set(x_4, x_7, x_8); +x_111 = lean_ctor_get(x_110, 1); +lean_inc(x_111); +if (lean_is_exclusive(x_110)) { + lean_ctor_release(x_110, 0); + lean_ctor_release(x_110, 1); + x_112 = x_110; } else { - lean_dec_ref(x_275); - x_277 = lean_box(0); + lean_dec_ref(x_110); + x_112 = lean_box(0); } -if (lean_is_scalar(x_277)) { - x_278 = lean_alloc_ctor(0, 2, 0); +x_113 = 1; +x_114 = lean_box(x_113); +if (lean_is_scalar(x_112)) { + x_115 = lean_alloc_ctor(0, 2, 0); } else { - x_278 = x_277; + x_115 = x_112; } -lean_ctor_set(x_278, 0, x_257); -lean_ctor_set(x_278, 1, x_276); -return x_278; +lean_ctor_set(x_115, 0, x_114); +lean_ctor_set(x_115, 1, x_111); +return x_115; } } 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; -lean_dec(x_253); -lean_dec(x_177); -x_279 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_279, 0, x_238); -lean_ctor_set(x_279, 1, x_239); -x_280 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_280, 0, x_279); -lean_ctor_set(x_280, 1, x_184); -lean_ctor_set(x_280, 2, x_185); -lean_ctor_set(x_280, 3, x_186); -lean_ctor_set(x_280, 4, x_187); -x_281 = lean_st_ref_set(x_5, x_280, x_183); -x_282 = lean_ctor_get(x_281, 1); -lean_inc(x_282); -if (lean_is_exclusive(x_281)) { - lean_ctor_release(x_281, 0); - lean_ctor_release(x_281, 1); - x_283 = x_281; +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; +x_116 = lean_box(0); +x_117 = lean_array_uset(x_75, x_88, x_116); +x_118 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(x_13, x_12, x_89); +x_119 = lean_array_uset(x_117, x_88, x_118); +x_120 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_120, 0, x_74); +lean_ctor_set(x_120, 1, x_119); +lean_ctor_set(x_7, 3, x_120); +x_121 = lean_st_ref_set(x_4, x_7, x_8); +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_281); - x_283 = lean_box(0); + lean_dec_ref(x_121); + x_123 = lean_box(0); } -x_284 = lean_box(0); -if (lean_is_scalar(x_283)) { - x_285 = lean_alloc_ctor(0, 2, 0); +x_124 = 1; +x_125 = lean_box(x_124); +if (lean_is_scalar(x_123)) { + x_126 = lean_alloc_ctor(0, 2, 0); } else { - x_285 = x_283; -} -lean_ctor_set(x_285, 0, x_284); -lean_ctor_set(x_285, 1, x_282); -return x_285; -} -} -} -else -{ -lean_object* x_286; lean_object* x_287; -lean_dec(x_179); -lean_dec(x_177); -x_286 = lean_box(0); -x_287 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_287, 0, x_286); -lean_ctor_set(x_287, 1, x_6); -return x_287; -} -} -} -} -default: -{ -lean_object* x_288; lean_object* x_289; -lean_dec(x_38); -lean_dec(x_37); -lean_dec(x_3); -lean_dec(x_2); -x_288 = lean_box(0); -x_289 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_289, 0, x_288); -lean_ctor_set(x_289, 1, x_6); -return x_289; -} -} -} -case 9: -{ -lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; uint8_t x_294; -lean_dec(x_2); -x_290 = lean_ctor_get(x_3, 0); -lean_inc(x_290); -lean_dec(x_3); -x_291 = lean_st_ref_take(x_5, x_6); -x_292 = lean_ctor_get(x_291, 0); -lean_inc(x_292); -x_293 = lean_ctor_get(x_291, 1); -lean_inc(x_293); -lean_dec(x_291); -x_294 = !lean_is_exclusive(x_292); -if (x_294 == 0) -{ -lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; uint8_t x_299; -x_295 = lean_ctor_get(x_292, 3); -x_296 = lean_ctor_get(x_290, 2); -lean_inc(x_296); -x_297 = l_Lean_Linter_UnusedVariables_followAliases(x_295, x_296); -x_298 = lean_ctor_get(x_290, 1); -lean_inc(x_298); -lean_dec(x_290); -x_299 = !lean_is_exclusive(x_295); -if (x_299 == 0) -{ -lean_object* x_300; lean_object* x_301; lean_object* x_302; uint64_t x_303; uint64_t x_304; uint64_t x_305; uint64_t x_306; uint64_t x_307; uint64_t x_308; uint64_t x_309; size_t x_310; size_t x_311; size_t x_312; size_t x_313; size_t x_314; lean_object* x_315; uint8_t x_316; -x_300 = lean_ctor_get(x_295, 0); -x_301 = lean_ctor_get(x_295, 1); -x_302 = lean_array_get_size(x_301); -x_303 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_298); -x_304 = 32; -x_305 = lean_uint64_shift_right(x_303, x_304); -x_306 = lean_uint64_xor(x_303, x_305); -x_307 = 16; -x_308 = lean_uint64_shift_right(x_306, x_307); -x_309 = lean_uint64_xor(x_306, x_308); -x_310 = lean_uint64_to_usize(x_309); -x_311 = lean_usize_of_nat(x_302); -lean_dec(x_302); -x_312 = 1; -x_313 = lean_usize_sub(x_311, x_312); -x_314 = lean_usize_land(x_310, x_313); -x_315 = lean_array_uget(x_301, x_314); -x_316 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11(x_298, x_315); -if (x_316 == 0) -{ -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; uint8_t x_326; -x_317 = lean_unsigned_to_nat(1u); -x_318 = lean_nat_add(x_300, x_317); -lean_dec(x_300); -x_319 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_319, 0, x_298); -lean_ctor_set(x_319, 1, x_297); -lean_ctor_set(x_319, 2, x_315); -x_320 = lean_array_uset(x_301, x_314, x_319); -x_321 = lean_unsigned_to_nat(4u); -x_322 = lean_nat_mul(x_318, x_321); -x_323 = lean_unsigned_to_nat(3u); -x_324 = lean_nat_div(x_322, x_323); -lean_dec(x_322); -x_325 = lean_array_get_size(x_320); -x_326 = lean_nat_dec_le(x_324, x_325); -lean_dec(x_325); -lean_dec(x_324); -if (x_326 == 0) -{ -lean_object* x_327; lean_object* x_328; uint8_t x_329; -x_327 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__12(x_320); -lean_ctor_set(x_295, 1, x_327); -lean_ctor_set(x_295, 0, x_318); -x_328 = lean_st_ref_set(x_5, x_292, x_293); -x_329 = !lean_is_exclusive(x_328); -if (x_329 == 0) -{ -lean_object* x_330; lean_object* x_331; -x_330 = lean_ctor_get(x_328, 0); -lean_dec(x_330); -x_331 = lean_box(0); -lean_ctor_set(x_328, 0, x_331); -return x_328; -} -else -{ -lean_object* x_332; lean_object* x_333; lean_object* x_334; -x_332 = lean_ctor_get(x_328, 1); -lean_inc(x_332); -lean_dec(x_328); -x_333 = lean_box(0); -x_334 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_334, 0, x_333); -lean_ctor_set(x_334, 1, x_332); -return x_334; -} -} -else -{ -lean_object* x_335; uint8_t x_336; -lean_ctor_set(x_295, 1, x_320); -lean_ctor_set(x_295, 0, x_318); -x_335 = lean_st_ref_set(x_5, x_292, x_293); -x_336 = !lean_is_exclusive(x_335); -if (x_336 == 0) -{ -lean_object* x_337; lean_object* x_338; -x_337 = lean_ctor_get(x_335, 0); -lean_dec(x_337); -x_338 = lean_box(0); -lean_ctor_set(x_335, 0, x_338); -return x_335; -} -else -{ -lean_object* x_339; lean_object* x_340; lean_object* x_341; -x_339 = lean_ctor_get(x_335, 1); -lean_inc(x_339); -lean_dec(x_335); -x_340 = lean_box(0); -x_341 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_341, 0, x_340); -lean_ctor_set(x_341, 1, x_339); -return x_341; + x_126 = x_123; } +lean_ctor_set(x_126, 0, x_125); +lean_ctor_set(x_126, 1, x_122); +return x_126; } } -else -{ -lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; uint8_t x_347; -x_342 = lean_box(0); -x_343 = lean_array_uset(x_301, x_314, x_342); -x_344 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(x_298, x_297, x_315); -x_345 = lean_array_uset(x_343, x_314, x_344); -lean_ctor_set(x_295, 1, x_345); -x_346 = lean_st_ref_set(x_5, x_292, x_293); -x_347 = !lean_is_exclusive(x_346); -if (x_347 == 0) -{ -lean_object* x_348; lean_object* x_349; -x_348 = lean_ctor_get(x_346, 0); -lean_dec(x_348); -x_349 = lean_box(0); -lean_ctor_set(x_346, 0, x_349); -return x_346; } else { -lean_object* x_350; lean_object* x_351; lean_object* x_352; -x_350 = lean_ctor_get(x_346, 1); -lean_inc(x_350); -lean_dec(x_346); -x_351 = lean_box(0); -x_352 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_352, 0, x_351); -lean_ctor_set(x_352, 1, x_350); -return x_352; -} -} -} -else -{ -lean_object* x_353; lean_object* x_354; lean_object* x_355; uint64_t x_356; uint64_t x_357; uint64_t x_358; uint64_t x_359; uint64_t x_360; uint64_t x_361; uint64_t x_362; size_t x_363; size_t x_364; size_t x_365; size_t x_366; size_t x_367; lean_object* x_368; uint8_t x_369; -x_353 = lean_ctor_get(x_295, 0); -x_354 = lean_ctor_get(x_295, 1); -lean_inc(x_354); -lean_inc(x_353); -lean_dec(x_295); -x_355 = lean_array_get_size(x_354); -x_356 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_298); -x_357 = 32; -x_358 = lean_uint64_shift_right(x_356, x_357); -x_359 = lean_uint64_xor(x_356, x_358); -x_360 = 16; -x_361 = lean_uint64_shift_right(x_359, x_360); -x_362 = lean_uint64_xor(x_359, x_361); -x_363 = lean_uint64_to_usize(x_362); -x_364 = lean_usize_of_nat(x_355); -lean_dec(x_355); -x_365 = 1; -x_366 = lean_usize_sub(x_364, x_365); -x_367 = lean_usize_land(x_363, x_366); -x_368 = lean_array_uget(x_354, x_367); -x_369 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11(x_298, x_368); -if (x_369 == 0) -{ -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; uint8_t x_379; -x_370 = lean_unsigned_to_nat(1u); -x_371 = lean_nat_add(x_353, x_370); -lean_dec(x_353); -x_372 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_372, 0, x_298); -lean_ctor_set(x_372, 1, x_297); -lean_ctor_set(x_372, 2, x_368); -x_373 = lean_array_uset(x_354, x_367, x_372); -x_374 = lean_unsigned_to_nat(4u); -x_375 = lean_nat_mul(x_371, x_374); -x_376 = lean_unsigned_to_nat(3u); -x_377 = lean_nat_div(x_375, x_376); -lean_dec(x_375); -x_378 = lean_array_get_size(x_373); -x_379 = lean_nat_dec_le(x_377, x_378); -lean_dec(x_378); -lean_dec(x_377); -if (x_379 == 0) -{ -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; -x_380 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__12(x_373); -x_381 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_381, 0, x_371); -lean_ctor_set(x_381, 1, x_380); -lean_ctor_set(x_292, 3, x_381); -x_382 = lean_st_ref_set(x_5, x_292, x_293); -x_383 = lean_ctor_get(x_382, 1); -lean_inc(x_383); -if (lean_is_exclusive(x_382)) { - lean_ctor_release(x_382, 0); - lean_ctor_release(x_382, 1); - x_384 = x_382; -} else { - lean_dec_ref(x_382); - x_384 = lean_box(0); -} -x_385 = lean_box(0); -if (lean_is_scalar(x_384)) { - x_386 = lean_alloc_ctor(0, 2, 0); -} else { - x_386 = x_384; -} -lean_ctor_set(x_386, 0, x_385); -lean_ctor_set(x_386, 1, x_383); -return x_386; -} -else -{ -lean_object* x_387; lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; lean_object* x_392; -x_387 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_387, 0, x_371); -lean_ctor_set(x_387, 1, x_373); -lean_ctor_set(x_292, 3, x_387); -x_388 = lean_st_ref_set(x_5, x_292, x_293); -x_389 = lean_ctor_get(x_388, 1); -lean_inc(x_389); -if (lean_is_exclusive(x_388)) { - lean_ctor_release(x_388, 0); - lean_ctor_release(x_388, 1); - x_390 = x_388; -} else { - lean_dec_ref(x_388); - x_390 = lean_box(0); -} -x_391 = lean_box(0); -if (lean_is_scalar(x_390)) { - x_392 = lean_alloc_ctor(0, 2, 0); -} else { - x_392 = x_390; -} -lean_ctor_set(x_392, 0, x_391); -lean_ctor_set(x_392, 1, x_389); -return x_392; -} -} -else -{ -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; -x_393 = lean_box(0); -x_394 = lean_array_uset(x_354, x_367, x_393); -x_395 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(x_298, x_297, x_368); -x_396 = lean_array_uset(x_394, x_367, x_395); -x_397 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_397, 0, x_353); -lean_ctor_set(x_397, 1, x_396); -lean_ctor_set(x_292, 3, x_397); -x_398 = lean_st_ref_set(x_5, x_292, x_293); -x_399 = lean_ctor_get(x_398, 1); -lean_inc(x_399); -if (lean_is_exclusive(x_398)) { - lean_ctor_release(x_398, 0); - lean_ctor_release(x_398, 1); - x_400 = x_398; -} else { - lean_dec_ref(x_398); - x_400 = lean_box(0); -} -x_401 = lean_box(0); -if (lean_is_scalar(x_400)) { - x_402 = lean_alloc_ctor(0, 2, 0); -} else { - x_402 = x_400; -} -lean_ctor_set(x_402, 0, x_401); -lean_ctor_set(x_402, 1, x_399); -return x_402; -} -} -} -else -{ -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; uint64_t x_415; uint64_t x_416; uint64_t x_417; uint64_t x_418; uint64_t x_419; uint64_t x_420; uint64_t x_421; size_t x_422; size_t x_423; size_t x_424; size_t x_425; size_t x_426; lean_object* x_427; uint8_t x_428; -x_403 = lean_ctor_get(x_292, 0); -x_404 = lean_ctor_get(x_292, 1); -x_405 = lean_ctor_get(x_292, 2); -x_406 = lean_ctor_get(x_292, 3); -x_407 = lean_ctor_get(x_292, 4); -lean_inc(x_407); -lean_inc(x_406); -lean_inc(x_405); -lean_inc(x_404); -lean_inc(x_403); -lean_dec(x_292); -x_408 = lean_ctor_get(x_290, 2); -lean_inc(x_408); -x_409 = l_Lean_Linter_UnusedVariables_followAliases(x_406, x_408); -x_410 = lean_ctor_get(x_290, 1); -lean_inc(x_410); -lean_dec(x_290); -x_411 = lean_ctor_get(x_406, 0); -lean_inc(x_411); -x_412 = lean_ctor_get(x_406, 1); -lean_inc(x_412); -if (lean_is_exclusive(x_406)) { - lean_ctor_release(x_406, 0); - lean_ctor_release(x_406, 1); - x_413 = x_406; +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; uint64_t x_139; uint64_t x_140; uint64_t x_141; uint64_t x_142; uint64_t x_143; uint64_t x_144; uint64_t x_145; size_t x_146; size_t x_147; size_t x_148; size_t x_149; size_t x_150; lean_object* x_151; uint8_t x_152; +x_127 = lean_ctor_get(x_7, 0); +x_128 = lean_ctor_get(x_7, 1); +x_129 = lean_ctor_get(x_7, 2); +x_130 = lean_ctor_get(x_7, 3); +x_131 = lean_ctor_get(x_7, 4); +lean_inc(x_131); +lean_inc(x_130); +lean_inc(x_129); +lean_inc(x_128); +lean_inc(x_127); +lean_dec(x_7); +x_132 = lean_ctor_get(x_1, 2); +lean_inc(x_132); +x_133 = l_Lean_Linter_UnusedVariables_followAliases(x_130, x_132); +x_134 = lean_ctor_get(x_1, 1); +lean_inc(x_134); +lean_dec(x_1); +x_135 = lean_ctor_get(x_130, 0); +lean_inc(x_135); +x_136 = lean_ctor_get(x_130, 1); +lean_inc(x_136); +if (lean_is_exclusive(x_130)) { + lean_ctor_release(x_130, 0); + lean_ctor_release(x_130, 1); + x_137 = x_130; } else { - lean_dec_ref(x_406); - x_413 = lean_box(0); -} -x_414 = lean_array_get_size(x_412); -x_415 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_410); -x_416 = 32; -x_417 = lean_uint64_shift_right(x_415, x_416); -x_418 = lean_uint64_xor(x_415, x_417); -x_419 = 16; -x_420 = lean_uint64_shift_right(x_418, x_419); -x_421 = lean_uint64_xor(x_418, x_420); -x_422 = lean_uint64_to_usize(x_421); -x_423 = lean_usize_of_nat(x_414); -lean_dec(x_414); -x_424 = 1; -x_425 = lean_usize_sub(x_423, x_424); -x_426 = lean_usize_land(x_422, x_425); -x_427 = lean_array_uget(x_412, x_426); -x_428 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11(x_410, x_427); -if (x_428 == 0) -{ -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; uint8_t x_438; -x_429 = lean_unsigned_to_nat(1u); -x_430 = lean_nat_add(x_411, x_429); -lean_dec(x_411); -x_431 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_431, 0, x_410); -lean_ctor_set(x_431, 1, x_409); -lean_ctor_set(x_431, 2, x_427); -x_432 = lean_array_uset(x_412, x_426, x_431); -x_433 = lean_unsigned_to_nat(4u); -x_434 = lean_nat_mul(x_430, x_433); -x_435 = lean_unsigned_to_nat(3u); -x_436 = lean_nat_div(x_434, x_435); -lean_dec(x_434); -x_437 = lean_array_get_size(x_432); -x_438 = lean_nat_dec_le(x_436, x_437); -lean_dec(x_437); -lean_dec(x_436); -if (x_438 == 0) -{ -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; -x_439 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__12(x_432); -if (lean_is_scalar(x_413)) { - x_440 = lean_alloc_ctor(0, 2, 0); + lean_dec_ref(x_130); + x_137 = lean_box(0); +} +x_138 = lean_array_get_size(x_136); +x_139 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_134); +x_140 = 32; +x_141 = lean_uint64_shift_right(x_139, x_140); +x_142 = lean_uint64_xor(x_139, x_141); +x_143 = 16; +x_144 = lean_uint64_shift_right(x_142, x_143); +x_145 = lean_uint64_xor(x_142, x_144); +x_146 = lean_uint64_to_usize(x_145); +x_147 = lean_usize_of_nat(x_138); +lean_dec(x_138); +x_148 = 1; +x_149 = lean_usize_sub(x_147, x_148); +x_150 = lean_usize_land(x_146, x_149); +x_151 = lean_array_uget(x_136, x_150); +x_152 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15(x_134, x_151); +if (x_152 == 0) +{ +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; uint8_t x_162; +x_153 = lean_unsigned_to_nat(1u); +x_154 = lean_nat_add(x_135, x_153); +lean_dec(x_135); +x_155 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_155, 0, x_134); +lean_ctor_set(x_155, 1, x_133); +lean_ctor_set(x_155, 2, x_151); +x_156 = lean_array_uset(x_136, x_150, x_155); +x_157 = lean_unsigned_to_nat(4u); +x_158 = lean_nat_mul(x_154, x_157); +x_159 = lean_unsigned_to_nat(3u); +x_160 = lean_nat_div(x_158, x_159); +lean_dec(x_158); +x_161 = lean_array_get_size(x_156); +x_162 = lean_nat_dec_le(x_160, x_161); +lean_dec(x_161); +lean_dec(x_160); +if (x_162 == 0) +{ +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_object* x_170; lean_object* x_171; +x_163 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__16(x_156); +if (lean_is_scalar(x_137)) { + x_164 = lean_alloc_ctor(0, 2, 0); } else { - x_440 = x_413; -} -lean_ctor_set(x_440, 0, x_430); -lean_ctor_set(x_440, 1, x_439); -x_441 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_441, 0, x_403); -lean_ctor_set(x_441, 1, x_404); -lean_ctor_set(x_441, 2, x_405); -lean_ctor_set(x_441, 3, x_440); -lean_ctor_set(x_441, 4, x_407); -x_442 = lean_st_ref_set(x_5, x_441, x_293); -x_443 = lean_ctor_get(x_442, 1); -lean_inc(x_443); -if (lean_is_exclusive(x_442)) { - lean_ctor_release(x_442, 0); - lean_ctor_release(x_442, 1); - x_444 = x_442; + x_164 = x_137; +} +lean_ctor_set(x_164, 0, x_154); +lean_ctor_set(x_164, 1, x_163); +x_165 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_165, 0, x_127); +lean_ctor_set(x_165, 1, x_128); +lean_ctor_set(x_165, 2, x_129); +lean_ctor_set(x_165, 3, x_164); +lean_ctor_set(x_165, 4, x_131); +x_166 = lean_st_ref_set(x_4, x_165, x_8); +x_167 = lean_ctor_get(x_166, 1); +lean_inc(x_167); +if (lean_is_exclusive(x_166)) { + lean_ctor_release(x_166, 0); + lean_ctor_release(x_166, 1); + x_168 = x_166; } else { - lean_dec_ref(x_442); - x_444 = lean_box(0); + lean_dec_ref(x_166); + x_168 = lean_box(0); } -x_445 = lean_box(0); -if (lean_is_scalar(x_444)) { - x_446 = lean_alloc_ctor(0, 2, 0); +x_169 = 1; +x_170 = lean_box(x_169); +if (lean_is_scalar(x_168)) { + x_171 = lean_alloc_ctor(0, 2, 0); } else { - x_446 = x_444; + x_171 = x_168; } -lean_ctor_set(x_446, 0, x_445); -lean_ctor_set(x_446, 1, x_443); -return x_446; +lean_ctor_set(x_171, 0, x_170); +lean_ctor_set(x_171, 1, x_167); +return x_171; } else { -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; -if (lean_is_scalar(x_413)) { - x_447 = lean_alloc_ctor(0, 2, 0); +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; uint8_t x_177; lean_object* x_178; lean_object* x_179; +if (lean_is_scalar(x_137)) { + x_172 = lean_alloc_ctor(0, 2, 0); } else { - x_447 = x_413; -} -lean_ctor_set(x_447, 0, x_430); -lean_ctor_set(x_447, 1, x_432); -x_448 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_448, 0, x_403); -lean_ctor_set(x_448, 1, x_404); -lean_ctor_set(x_448, 2, x_405); -lean_ctor_set(x_448, 3, x_447); -lean_ctor_set(x_448, 4, x_407); -x_449 = lean_st_ref_set(x_5, x_448, x_293); -x_450 = lean_ctor_get(x_449, 1); -lean_inc(x_450); -if (lean_is_exclusive(x_449)) { - lean_ctor_release(x_449, 0); - lean_ctor_release(x_449, 1); - x_451 = x_449; + x_172 = x_137; +} +lean_ctor_set(x_172, 0, x_154); +lean_ctor_set(x_172, 1, x_156); +x_173 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_173, 0, x_127); +lean_ctor_set(x_173, 1, x_128); +lean_ctor_set(x_173, 2, x_129); +lean_ctor_set(x_173, 3, x_172); +lean_ctor_set(x_173, 4, x_131); +x_174 = lean_st_ref_set(x_4, x_173, x_8); +x_175 = lean_ctor_get(x_174, 1); +lean_inc(x_175); +if (lean_is_exclusive(x_174)) { + lean_ctor_release(x_174, 0); + lean_ctor_release(x_174, 1); + x_176 = x_174; } else { - lean_dec_ref(x_449); - x_451 = lean_box(0); + lean_dec_ref(x_174); + x_176 = lean_box(0); } -x_452 = lean_box(0); -if (lean_is_scalar(x_451)) { - x_453 = lean_alloc_ctor(0, 2, 0); +x_177 = 1; +x_178 = lean_box(x_177); +if (lean_is_scalar(x_176)) { + x_179 = lean_alloc_ctor(0, 2, 0); } else { - x_453 = x_451; + x_179 = x_176; } -lean_ctor_set(x_453, 0, x_452); -lean_ctor_set(x_453, 1, x_450); -return x_453; +lean_ctor_set(x_179, 0, x_178); +lean_ctor_set(x_179, 1, x_175); +return x_179; } } else { -lean_object* x_454; lean_object* x_455; 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; lean_object* x_463; lean_object* x_464; -x_454 = lean_box(0); -x_455 = lean_array_uset(x_412, x_426, x_454); -x_456 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(x_410, x_409, x_427); -x_457 = lean_array_uset(x_455, x_426, x_456); -if (lean_is_scalar(x_413)) { - x_458 = lean_alloc_ctor(0, 2, 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; lean_object* x_186; lean_object* x_187; lean_object* x_188; uint8_t x_189; lean_object* x_190; lean_object* x_191; +x_180 = lean_box(0); +x_181 = lean_array_uset(x_136, x_150, x_180); +x_182 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(x_134, x_133, x_151); +x_183 = lean_array_uset(x_181, x_150, x_182); +if (lean_is_scalar(x_137)) { + x_184 = lean_alloc_ctor(0, 2, 0); } else { - x_458 = x_413; -} -lean_ctor_set(x_458, 0, x_411); -lean_ctor_set(x_458, 1, x_457); -x_459 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_459, 0, x_403); -lean_ctor_set(x_459, 1, x_404); -lean_ctor_set(x_459, 2, x_405); -lean_ctor_set(x_459, 3, x_458); -lean_ctor_set(x_459, 4, x_407); -x_460 = lean_st_ref_set(x_5, x_459, x_293); -x_461 = lean_ctor_get(x_460, 1); -lean_inc(x_461); -if (lean_is_exclusive(x_460)) { - lean_ctor_release(x_460, 0); - lean_ctor_release(x_460, 1); - x_462 = x_460; + x_184 = x_137; +} +lean_ctor_set(x_184, 0, x_135); +lean_ctor_set(x_184, 1, x_183); +x_185 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_185, 0, x_127); +lean_ctor_set(x_185, 1, x_128); +lean_ctor_set(x_185, 2, x_129); +lean_ctor_set(x_185, 3, x_184); +lean_ctor_set(x_185, 4, x_131); +x_186 = lean_st_ref_set(x_4, x_185, x_8); +x_187 = lean_ctor_get(x_186, 1); +lean_inc(x_187); +if (lean_is_exclusive(x_186)) { + lean_ctor_release(x_186, 0); + lean_ctor_release(x_186, 1); + x_188 = x_186; } else { - lean_dec_ref(x_460); - x_462 = lean_box(0); + lean_dec_ref(x_186); + x_188 = lean_box(0); } -x_463 = lean_box(0); -if (lean_is_scalar(x_462)) { - x_464 = lean_alloc_ctor(0, 2, 0); +x_189 = 1; +x_190 = lean_box(x_189); +if (lean_is_scalar(x_188)) { + x_191 = lean_alloc_ctor(0, 2, 0); } else { - x_464 = x_462; + x_191 = x_188; } -lean_ctor_set(x_464, 0, x_463); -lean_ctor_set(x_464, 1, x_461); -return x_464; +lean_ctor_set(x_191, 0, x_190); +lean_ctor_set(x_191, 1, x_187); +return x_191; } } } -default: +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__1() { +_start: { -lean_object* x_465; lean_object* x_466; -lean_dec(x_3); -lean_dec(x_2); -x_465 = lean_box(0); -x_466 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_466, 0, x_465); -lean_ctor_set(x_466, 1, x_6); -return x_466; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("MutualDef", 9, 9); +return x_1; } } +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("body", 4, 4); +return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__3() { _start: { -lean_object* x_6; lean_object* x_7; -x_6 = lean_box(0); -x_7 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_5); -return x_7; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__1; +x_2 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__4() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__5___boxed), 5, 0); +x_1 = l_Lean_Linter_linter_unusedVariables_analyzeTactics; return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21(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) { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__5() { _start: { -uint8_t x_8; -x_8 = lean_usize_dec_lt(x_4, x_3); -if (x_8 == 0) -{ -lean_object* x_9; -lean_dec(x_6); -lean_dec(x_1); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_5); -lean_ctor_set(x_9, 1, x_7); -return x_9; +lean_object* x_1; +x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); +return x_1; } -else +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__6() { +_start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -lean_dec(x_5); -x_10 = lean_array_uget(x_2, x_4); -lean_inc(x_1); -x_11 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__4___boxed), 6, 1); -lean_closure_set(x_11, 0, x_1); -x_12 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___closed__1; -lean_inc(x_6); -x_13 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences___spec__16(x_11, x_12, x_10, x_6, x_7); -if (lean_obj_tag(x_13) == 0) -{ -lean_object* x_14; size_t x_15; size_t x_16; lean_object* x_17; -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -lean_dec(x_13); -x_15 = 1; -x_16 = lean_usize_add(x_4, x_15); -x_17 = lean_box(0); -x_4 = x_16; -x_5 = x_17; -x_7 = x_14; -goto _start; +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__5; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; } -else +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10(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) { +_start: { -uint8_t x_19; -lean_dec(x_6); +switch (lean_obj_tag(x_3)) { +case 0: +{ +lean_dec(x_2); lean_dec(x_1); -x_19 = !lean_is_exclusive(x_13); -if (x_19 == 0) +if (x_5 == 0) { -return x_13; +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_box(0); +x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__1(x_8, x_9, x_5, x_6, x_7); +lean_dec(x_6); +return x_10; } 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; -} -} +uint8_t x_11; lean_object* x_12; lean_object* x_13; +lean_dec(x_6); +lean_dec(x_3); +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_7); +return x_13; } } +case 1: +{ +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_3, 0); +lean_inc(x_14); +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); +x_17 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__3; +x_18 = lean_name_eq(x_16, x_17); +lean_dec(x_16); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +x_19 = lean_box(0); +x_20 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__8(x_5, x_14, x_3, x_2, x_1, x_19, x_5, x_6, x_7); +lean_dec(x_1); +lean_dec(x_3); +return x_20; } -LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +else { -size_t x_5; size_t x_6; lean_object* x_7; lean_object* x_8; -x_5 = lean_array_size(x_1); -x_6 = 0; -x_7 = lean_box(0); -x_8 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21(x_2, x_1, x_5, x_6, x_7, x_3, x_4); -if (lean_obj_tag(x_8) == 0) +lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_21 = lean_ctor_get(x_2, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_21, 3); +lean_inc(x_22); +x_23 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__4; +x_24 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_22, x_23); +lean_dec(x_22); +if (x_24 == 0) { -uint8_t x_9; -x_9 = !lean_is_exclusive(x_8); -if (x_9 == 0) +uint8_t x_25; +x_25 = !lean_is_exclusive(x_3); +if (x_25 == 0) { -lean_object* x_10; -x_10 = lean_ctor_get(x_8, 0); -lean_dec(x_10); -lean_ctor_set(x_8, 0, x_7); -return x_8; +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; uint8_t x_34; +x_26 = lean_ctor_get(x_3, 0); +lean_dec(x_26); +x_27 = lean_ctor_get(x_21, 2); +lean_inc(x_27); +lean_dec(x_21); +x_28 = lean_ctor_get(x_14, 3); +lean_inc(x_28); +lean_dec(x_14); +x_29 = l_Lean_instantiateMVarsCore(x_27, x_28); +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +lean_dec(x_29); +x_31 = lean_st_ref_take(x_6, x_7); +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_is_exclusive(x_32); +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; uint8_t x_42; lean_object* x_43; +x_35 = lean_ctor_get(x_32, 4); +x_36 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__6; +x_37 = lean_box(0); +x_38 = l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(x_36, x_37, x_30); +x_39 = lean_array_push(x_35, x_38); +lean_ctor_set(x_32, 4, x_39); +x_40 = lean_st_ref_set(x_6, x_32, x_33); +x_41 = lean_ctor_get(x_40, 1); +lean_inc(x_41); +lean_dec(x_40); +x_42 = l_Lean_PersistentArray_anyM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__11(x_4); +x_43 = l_Lean_PersistentArray_toArray___rarg(x_4); +lean_ctor_set(x_3, 0, x_2); +if (x_5 == 0) +{ +lean_object* x_44; +x_44 = l_Lean_Linter_UnusedVariables_collectReferences_go(x_1, x_43, x_3, x_42, x_6, x_41); +lean_dec(x_43); +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; +x_46 = lean_ctor_get(x_44, 0); +lean_dec(x_46); +x_47 = 0; +x_48 = lean_box(x_47); +lean_ctor_set(x_44, 0, x_48); +return x_44; } else { -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_8, 1); -lean_inc(x_11); -lean_dec(x_8); -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_7); -lean_ctor_set(x_12, 1, x_11); -return x_12; +lean_object* x_49; uint8_t x_50; lean_object* x_51; lean_object* x_52; +x_49 = lean_ctor_get(x_44, 1); +lean_inc(x_49); +lean_dec(x_44); +x_50 = 0; +x_51 = lean_box(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_49); +return x_52; } } else { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_8); -if (x_13 == 0) +uint8_t x_53; +x_53 = !lean_is_exclusive(x_44); +if (x_53 == 0) { -return x_8; +return x_44; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_8, 0); -x_15 = lean_ctor_get(x_8, 1); -lean_inc(x_15); -lean_inc(x_14); -lean_dec(x_8); -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_object* x_54; lean_object* x_55; lean_object* x_56; +x_54 = lean_ctor_get(x_44, 0); +x_55 = lean_ctor_get(x_44, 1); +lean_inc(x_55); +lean_inc(x_54); +lean_dec(x_44); +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 +{ +uint8_t x_57; lean_object* x_58; +x_57 = 1; +x_58 = l_Lean_Linter_UnusedVariables_collectReferences_go(x_1, x_43, x_3, x_57, x_6, x_41); +lean_dec(x_43); +if (lean_obj_tag(x_58) == 0) +{ +uint8_t x_59; +x_59 = !lean_is_exclusive(x_58); +if (x_59 == 0) +{ +lean_object* x_60; uint8_t x_61; lean_object* x_62; +x_60 = lean_ctor_get(x_58, 0); +lean_dec(x_60); +x_61 = 0; +x_62 = lean_box(x_61); +lean_ctor_set(x_58, 0, x_62); +return x_58; } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences___spec__1___boxed(lean_object* x_1, lean_object* x_2) { -_start: +else { -lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences___spec__1(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -return x_3; +lean_object* x_63; uint8_t x_64; lean_object* x_65; lean_object* x_66; +x_63 = lean_ctor_get(x_58, 1); +lean_inc(x_63); +lean_dec(x_58); +x_64 = 0; +x_65 = lean_box(x_64); +x_66 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_66, 0, x_65); +lean_ctor_set(x_66, 1, x_63); +return x_66; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2___boxed(lean_object* x_1, lean_object* x_2) { -_start: +else { -uint8_t x_3; lean_object* x_4; -x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__2(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; -} +uint8_t x_67; +x_67 = !lean_is_exclusive(x_58); +if (x_67 == 0) +{ +return x_58; } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__7___boxed(lean_object* x_1, lean_object* x_2) { -_start: +else { -uint8_t x_3; lean_object* x_4; -x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__7(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; +lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_68 = lean_ctor_get(x_58, 0); +x_69 = lean_ctor_get(x_58, 1); +lean_inc(x_69); +lean_inc(x_68); +lean_dec(x_58); +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_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11___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_Linter_UnusedVariables_collectReferences___spec__11(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_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences___spec__16___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: +else { -lean_object* x_8; -x_8 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences___spec__16___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_5); -return x_8; +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; lean_object* x_84; +x_71 = lean_ctor_get(x_32, 0); +x_72 = lean_ctor_get(x_32, 1); +x_73 = lean_ctor_get(x_32, 2); +x_74 = lean_ctor_get(x_32, 3); +x_75 = lean_ctor_get(x_32, 4); +lean_inc(x_75); +lean_inc(x_74); +lean_inc(x_73); +lean_inc(x_72); +lean_inc(x_71); +lean_dec(x_32); +x_76 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__6; +x_77 = lean_box(0); +x_78 = l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(x_76, x_77, x_30); +x_79 = lean_array_push(x_75, x_78); +x_80 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_80, 0, x_71); +lean_ctor_set(x_80, 1, x_72); +lean_ctor_set(x_80, 2, x_73); +lean_ctor_set(x_80, 3, x_74); +lean_ctor_set(x_80, 4, x_79); +x_81 = lean_st_ref_set(x_6, x_80, x_33); +x_82 = lean_ctor_get(x_81, 1); +lean_inc(x_82); +lean_dec(x_81); +x_83 = l_Lean_PersistentArray_anyM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__11(x_4); +x_84 = l_Lean_PersistentArray_toArray___rarg(x_4); +lean_ctor_set(x_3, 0, x_2); +if (x_5 == 0) +{ +lean_object* x_85; +x_85 = l_Lean_Linter_UnusedVariables_collectReferences_go(x_1, x_84, x_3, x_83, x_6, x_82); +lean_dec(x_84); +if (lean_obj_tag(x_85) == 0) +{ +lean_object* x_86; lean_object* x_87; uint8_t x_88; lean_object* x_89; lean_object* x_90; +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 = 0; +x_89 = lean_box(x_88); +if (lean_is_scalar(x_87)) { + x_90 = lean_alloc_ctor(0, 2, 0); +} else { + x_90 = x_87; } +lean_ctor_set(x_90, 0, x_89); +lean_ctor_set(x_90, 1, x_86); +return x_90; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___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: +else { -lean_object* x_9; -x_9 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___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_2); -return x_9; +lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_91 = lean_ctor_get(x_85, 0); +lean_inc(x_91); +x_92 = lean_ctor_get(x_85, 1); +lean_inc(x_92); +if (lean_is_exclusive(x_85)) { + lean_ctor_release(x_85, 0); + lean_ctor_release(x_85, 1); + x_93 = x_85; +} else { + lean_dec_ref(x_85); + x_93 = lean_box(0); } +if (lean_is_scalar(x_93)) { + x_94 = lean_alloc_ctor(1, 2, 0); +} else { + x_94 = x_93; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___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_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___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_3); -return x_9; +lean_ctor_set(x_94, 0, x_91); +lean_ctor_set(x_94, 1, x_92); +return x_94; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___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) { -_start: +else { -lean_object* x_9; -x_9 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__3(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_4); -return x_9; +uint8_t x_95; lean_object* x_96; +x_95 = 1; +x_96 = l_Lean_Linter_UnusedVariables_collectReferences_go(x_1, x_84, x_3, x_95, x_6, x_82); +lean_dec(x_84); +if (lean_obj_tag(x_96) == 0) +{ +lean_object* x_97; lean_object* x_98; uint8_t x_99; lean_object* x_100; lean_object* x_101; +x_97 = lean_ctor_get(x_96, 1); +lean_inc(x_97); +if (lean_is_exclusive(x_96)) { + lean_ctor_release(x_96, 0); + lean_ctor_release(x_96, 1); + x_98 = x_96; +} else { + lean_dec_ref(x_96); + x_98 = lean_box(0); } +x_99 = 0; +x_100 = lean_box(x_99); +if (lean_is_scalar(x_98)) { + x_101 = lean_alloc_ctor(0, 2, 0); +} else { + x_101 = x_98; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___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) { -_start: +lean_ctor_set(x_101, 0, x_100); +lean_ctor_set(x_101, 1, x_97); +return x_101; +} +else { -lean_object* x_7; -x_7 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -return x_7; +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_102 = lean_ctor_get(x_96, 0); +lean_inc(x_102); +x_103 = lean_ctor_get(x_96, 1); +lean_inc(x_103); +if (lean_is_exclusive(x_96)) { + lean_ctor_release(x_96, 0); + lean_ctor_release(x_96, 1); + x_104 = x_96; +} else { + lean_dec_ref(x_96); + 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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +lean_ctor_set(x_105, 0, x_102); +lean_ctor_set(x_105, 1, x_103); +return x_105; +} +} +} +} +else { -lean_object* x_6; -x_6 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__5(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); +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; uint8_t x_126; lean_object* x_127; lean_object* x_128; +lean_dec(x_3); +x_106 = lean_ctor_get(x_21, 2); +lean_inc(x_106); +lean_dec(x_21); +x_107 = lean_ctor_get(x_14, 3); +lean_inc(x_107); +lean_dec(x_14); +x_108 = l_Lean_instantiateMVarsCore(x_106, x_107); +x_109 = lean_ctor_get(x_108, 0); +lean_inc(x_109); +lean_dec(x_108); +x_110 = lean_st_ref_take(x_6, x_7); +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); +x_114 = lean_ctor_get(x_111, 1); +lean_inc(x_114); +x_115 = lean_ctor_get(x_111, 2); +lean_inc(x_115); +x_116 = lean_ctor_get(x_111, 3); +lean_inc(x_116); +x_117 = lean_ctor_get(x_111, 4); +lean_inc(x_117); +if (lean_is_exclusive(x_111)) { + lean_ctor_release(x_111, 0); + lean_ctor_release(x_111, 1); + lean_ctor_release(x_111, 2); + lean_ctor_release(x_111, 3); + lean_ctor_release(x_111, 4); + x_118 = x_111; +} else { + lean_dec_ref(x_111); + x_118 = lean_box(0); +} +x_119 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__6; +x_120 = lean_box(0); +x_121 = l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(x_119, x_120, x_109); +x_122 = lean_array_push(x_117, x_121); +if (lean_is_scalar(x_118)) { + x_123 = lean_alloc_ctor(0, 5, 0); +} else { + x_123 = x_118; +} +lean_ctor_set(x_123, 0, x_113); +lean_ctor_set(x_123, 1, x_114); +lean_ctor_set(x_123, 2, x_115); +lean_ctor_set(x_123, 3, x_116); +lean_ctor_set(x_123, 4, x_122); +x_124 = lean_st_ref_set(x_6, x_123, x_112); +x_125 = lean_ctor_get(x_124, 1); +lean_inc(x_125); +lean_dec(x_124); +x_126 = l_Lean_PersistentArray_anyM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__11(x_4); +x_127 = l_Lean_PersistentArray_toArray___rarg(x_4); +x_128 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_128, 0, x_2); +if (x_5 == 0) +{ +lean_object* x_129; +x_129 = l_Lean_Linter_UnusedVariables_collectReferences_go(x_1, x_127, x_128, x_126, x_6, x_125); +lean_dec(x_127); +if (lean_obj_tag(x_129) == 0) +{ +lean_object* x_130; lean_object* x_131; uint8_t x_132; lean_object* x_133; lean_object* x_134; +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 = 0; +x_133 = lean_box(x_132); +if (lean_is_scalar(x_131)) { + x_134 = lean_alloc_ctor(0, 2, 0); +} else { + x_134 = x_131; +} +lean_ctor_set(x_134, 0, x_133); +lean_ctor_set(x_134, 1, x_130); +return x_134; +} +else +{ +lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; +x_135 = lean_ctor_get(x_129, 0); +lean_inc(x_135); +x_136 = lean_ctor_get(x_129, 1); +lean_inc(x_136); +if (lean_is_exclusive(x_129)) { + lean_ctor_release(x_129, 0); + lean_ctor_release(x_129, 1); + x_137 = x_129; +} else { + lean_dec_ref(x_129); + x_137 = lean_box(0); +} +if (lean_is_scalar(x_137)) { + x_138 = lean_alloc_ctor(1, 2, 0); +} else { + x_138 = x_137; +} +lean_ctor_set(x_138, 0, x_135); +lean_ctor_set(x_138, 1, x_136); +return x_138; +} +} +else +{ +uint8_t x_139; lean_object* x_140; +x_139 = 1; +x_140 = l_Lean_Linter_UnusedVariables_collectReferences_go(x_1, x_127, x_128, x_139, x_6, x_125); +lean_dec(x_127); +if (lean_obj_tag(x_140) == 0) +{ +lean_object* x_141; lean_object* x_142; uint8_t x_143; lean_object* x_144; lean_object* x_145; +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 = 0; +x_144 = lean_box(x_143); +if (lean_is_scalar(x_142)) { + x_145 = lean_alloc_ctor(0, 2, 0); +} else { + x_145 = x_142; +} +lean_ctor_set(x_145, 0, x_144); +lean_ctor_set(x_145, 1, x_141); +return x_145; +} +else +{ +lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; +x_146 = lean_ctor_get(x_140, 0); +lean_inc(x_146); +x_147 = lean_ctor_get(x_140, 1); +lean_inc(x_147); +if (lean_is_exclusive(x_140)) { + lean_ctor_release(x_140, 0); + lean_ctor_release(x_140, 1); + x_148 = x_140; +} else { + lean_dec_ref(x_140); + 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_dec(x_21); +x_150 = lean_box(0); +x_151 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__8(x_5, x_14, x_3, x_2, x_1, x_150, x_5, x_6, x_7); +lean_dec(x_1); lean_dec(x_3); +return x_151; +} +} +} +case 9: +{ lean_dec(x_2); lean_dec(x_1); -return x_6; +if (x_5 == 0) +{ +lean_object* x_152; lean_object* x_153; lean_object* x_154; +x_152 = lean_ctor_get(x_3, 0); +lean_inc(x_152); +lean_dec(x_3); +x_153 = lean_box(0); +x_154 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__9(x_152, x_153, x_5, x_6, x_7); +lean_dec(x_6); +return x_154; } +else +{ +uint8_t x_155; lean_object* x_156; lean_object* x_157; +lean_dec(x_6); +lean_dec(x_3); +x_155 = 1; +x_156 = lean_box(x_155); +x_157 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_157, 0, x_156); +lean_ctor_set(x_157, 1, x_7); +return x_157; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__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) { -_start: +} +default: { -size_t x_8; size_t x_9; lean_object* x_10; -x_8 = lean_unbox_usize(x_3); +uint8_t x_158; lean_object* x_159; lean_object* x_160; +lean_dec(x_6); lean_dec(x_3); -x_9 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21(x_1, x_2, x_8, x_9, x_5, x_6, x_7); lean_dec(x_2); -return x_10; +lean_dec(x_1); +x_158 = 1; +x_159 = lean_box(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_7); +return x_160; } } -LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_5; -x_5 = l_Lean_Linter_UnusedVariables_collectReferences(x_1, x_2, x_3, x_4); -lean_dec(x_1); -return x_5; +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; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___closed__1() { _start: { -if (lean_obj_tag(x_4) == 0) +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__11___boxed), 6, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, uint8_t x_7, lean_object* x_8, lean_object* x_9) { +_start: { +uint8_t x_10; +x_10 = lean_usize_dec_lt(x_5, x_4); +if (x_10 == 0) +{ +lean_object* x_11; +lean_dec(x_8); +lean_dec(x_2); lean_dec(x_1); -return x_3; +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_6); +lean_ctor_set(x_11, 1, x_9); +return x_11; } else { -uint8_t x_5; -x_5 = !lean_is_exclusive(x_4); -if (x_5 == 0) -{ -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_6 = lean_ctor_get(x_4, 0); -x_7 = lean_ctor_get(x_4, 1); -x_8 = lean_ctor_get(x_4, 2); -x_9 = lean_ctor_get(x_2, 3); -x_10 = l_Lean_Linter_UnusedVariables_followAliases(x_9, x_7); -x_11 = !lean_is_exclusive(x_3); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; uint64_t 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; size_t x_22; size_t x_23; size_t x_24; size_t x_25; size_t x_26; lean_object* x_27; uint8_t x_28; -x_12 = lean_ctor_get(x_3, 0); -x_13 = lean_ctor_get(x_3, 1); -x_14 = lean_array_get_size(x_13); -x_15 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_6); -x_16 = 32; -x_17 = lean_uint64_shift_right(x_15, x_16); -x_18 = lean_uint64_xor(x_15, x_17); -x_19 = 16; -x_20 = lean_uint64_shift_right(x_18, x_19); -x_21 = lean_uint64_xor(x_18, x_20); -x_22 = lean_uint64_to_usize(x_21); -x_23 = lean_usize_of_nat(x_14); -lean_dec(x_14); -x_24 = 1; -x_25 = lean_usize_sub(x_23, x_24); -x_26 = lean_usize_land(x_22, x_25); -x_27 = lean_array_uget(x_13, x_26); -x_28 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11(x_6, 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_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; -x_29 = lean_unsigned_to_nat(1u); -x_30 = lean_nat_add(x_12, x_29); -lean_dec(x_12); -lean_ctor_set(x_4, 2, x_27); -lean_ctor_set(x_4, 1, x_10); -x_31 = lean_array_uset(x_13, x_26, x_4); -x_32 = lean_unsigned_to_nat(4u); -x_33 = lean_nat_mul(x_30, x_32); -x_34 = lean_unsigned_to_nat(3u); -x_35 = lean_nat_div(x_33, x_34); -lean_dec(x_33); -x_36 = lean_array_get_size(x_31); -x_37 = lean_nat_dec_le(x_35, x_36); -lean_dec(x_36); -lean_dec(x_35); -if (x_37 == 0) +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_6); +x_12 = lean_array_uget(x_3, x_5); +lean_inc(x_1); +x_13 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___boxed), 7, 1); +lean_closure_set(x_13, 0, x_1); +x_14 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___closed__1; +lean_inc(x_8); +lean_inc(x_2); +x_15 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20(x_13, x_14, x_2, x_12, x_7, x_8, x_9); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_38; -x_38 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__12(x_31); -lean_ctor_set(x_3, 1, x_38); -lean_ctor_set(x_3, 0, x_30); -x_4 = x_8; +lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +lean_dec(x_15); +x_17 = 1; +x_18 = lean_usize_add(x_5, x_17); +x_19 = lean_box(0); +x_5 = x_18; +x_6 = x_19; +x_9 = x_16; goto _start; } else { -lean_ctor_set(x_3, 1, x_31); -lean_ctor_set(x_3, 0, x_30); -x_4 = x_8; -goto _start; -} +uint8_t x_21; +lean_dec(x_8); +lean_dec(x_2); +lean_dec(x_1); +x_21 = !lean_is_exclusive(x_15); +if (x_21 == 0) +{ +return x_15; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -lean_free_object(x_4); -lean_inc(x_1); -x_41 = lean_array_uset(x_13, x_26, x_1); -x_42 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(x_6, x_10, x_27); -x_43 = lean_array_uset(x_41, x_26, x_42); -lean_ctor_set(x_3, 1, x_43); -x_4 = x_8; -goto _start; +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_15, 0); +x_23 = lean_ctor_get(x_15, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_15); +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_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6) { +_start: { -lean_object* x_45; lean_object* x_46; lean_object* x_47; uint64_t x_48; uint64_t x_49; uint64_t x_50; uint64_t x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; size_t x_55; size_t x_56; size_t x_57; size_t x_58; size_t x_59; lean_object* x_60; uint8_t x_61; -x_45 = lean_ctor_get(x_3, 0); -x_46 = lean_ctor_get(x_3, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_3); -x_47 = lean_array_get_size(x_46); -x_48 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_6); -x_49 = 32; -x_50 = lean_uint64_shift_right(x_48, x_49); -x_51 = lean_uint64_xor(x_48, x_50); -x_52 = 16; -x_53 = lean_uint64_shift_right(x_51, x_52); -x_54 = lean_uint64_xor(x_51, x_53); -x_55 = lean_uint64_to_usize(x_54); -x_56 = lean_usize_of_nat(x_47); -lean_dec(x_47); -x_57 = 1; -x_58 = lean_usize_sub(x_56, x_57); -x_59 = lean_usize_land(x_55, x_58); -x_60 = lean_array_uget(x_46, x_59); -x_61 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11(x_6, x_60); -if (x_61 == 0) +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_array_size(x_2); +x_8 = 0; +x_9 = lean_box(0); +x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24(x_1, x_3, x_2, x_7, x_8, x_9, x_4, x_5, x_6); +if (lean_obj_tag(x_10) == 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; uint8_t x_70; -x_62 = lean_unsigned_to_nat(1u); -x_63 = lean_nat_add(x_45, x_62); -lean_dec(x_45); -lean_ctor_set(x_4, 2, x_60); -lean_ctor_set(x_4, 1, x_10); -x_64 = lean_array_uset(x_46, x_59, x_4); -x_65 = lean_unsigned_to_nat(4u); -x_66 = lean_nat_mul(x_63, 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) +uint8_t x_11; +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) { -lean_object* x_71; lean_object* x_72; -x_71 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__12(x_64); -x_72 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_72, 0, x_63); -lean_ctor_set(x_72, 1, x_71); -x_3 = x_72; -x_4 = x_8; -goto _start; +lean_object* x_12; +x_12 = lean_ctor_get(x_10, 0); +lean_dec(x_12); +lean_ctor_set(x_10, 0, x_9); +return x_10; } else { -lean_object* x_74; -x_74 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_74, 0, x_63); -lean_ctor_set(x_74, 1, x_64); -x_3 = x_74; -x_4 = x_8; -goto _start; +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_10, 1); +lean_inc(x_13); +lean_dec(x_10); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_9); +lean_ctor_set(x_14, 1, x_13); +return x_14; } } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; -lean_free_object(x_4); -lean_inc(x_1); -x_76 = lean_array_uset(x_46, x_59, x_1); -x_77 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(x_6, x_10, 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_45); -lean_ctor_set(x_79, 1, x_78); -x_3 = x_79; -x_4 = x_8; -goto _start; -} -} +uint8_t x_15; +x_15 = !lean_is_exclusive(x_10); +if (x_15 == 0) +{ +return x_10; } 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; uint64_t x_90; uint64_t x_91; uint64_t x_92; uint64_t x_93; uint64_t x_94; uint64_t x_95; uint64_t x_96; size_t x_97; size_t x_98; size_t x_99; size_t x_100; size_t x_101; lean_object* x_102; uint8_t x_103; -x_81 = lean_ctor_get(x_4, 0); -x_82 = lean_ctor_get(x_4, 1); -x_83 = lean_ctor_get(x_4, 2); -lean_inc(x_83); -lean_inc(x_82); -lean_inc(x_81); -lean_dec(x_4); -x_84 = lean_ctor_get(x_2, 3); -x_85 = l_Lean_Linter_UnusedVariables_followAliases(x_84, x_82); -x_86 = lean_ctor_get(x_3, 0); -lean_inc(x_86); -x_87 = lean_ctor_get(x_3, 1); -lean_inc(x_87); -if (lean_is_exclusive(x_3)) { - lean_ctor_release(x_3, 0); - lean_ctor_release(x_3, 1); - x_88 = x_3; -} else { - lean_dec_ref(x_3); - x_88 = lean_box(0); +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; } -x_89 = lean_array_get_size(x_87); -x_90 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_81); -x_91 = 32; -x_92 = lean_uint64_shift_right(x_90, x_91); -x_93 = lean_uint64_xor(x_90, x_92); -x_94 = 16; -x_95 = lean_uint64_shift_right(x_93, x_94); -x_96 = lean_uint64_xor(x_93, x_95); -x_97 = lean_uint64_to_usize(x_96); -x_98 = lean_usize_of_nat(x_89); -lean_dec(x_89); -x_99 = 1; -x_100 = lean_usize_sub(x_98, x_99); -x_101 = lean_usize_land(x_97, x_100); -x_102 = lean_array_uget(x_87, x_101); -x_103 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__11(x_81, x_102); -if (x_103 == 0) +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: { -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; uint8_t x_113; -x_104 = lean_unsigned_to_nat(1u); -x_105 = lean_nat_add(x_86, x_104); -lean_dec(x_86); -x_106 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_106, 0, x_81); -lean_ctor_set(x_106, 1, x_85); -lean_ctor_set(x_106, 2, x_102); -x_107 = lean_array_uset(x_87, x_101, x_106); -x_108 = lean_unsigned_to_nat(4u); -x_109 = lean_nat_mul(x_105, x_108); -x_110 = lean_unsigned_to_nat(3u); -x_111 = lean_nat_div(x_109, x_110); -lean_dec(x_109); -x_112 = lean_array_get_size(x_107); -x_113 = lean_nat_dec_le(x_111, x_112); -lean_dec(x_112); -lean_dec(x_111); -if (x_113 == 0) +lean_object* x_3; +x_3 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__1(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_Linter_UnusedVariables_collectReferences_go___spec__2___boxed(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_114; lean_object* x_115; -x_114 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences___spec__12(x_107); -if (lean_is_scalar(x_88)) { - x_115 = lean_alloc_ctor(0, 2, 0); -} else { - x_115 = x_88; +uint8_t x_3; lean_object* x_4; +x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__2(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; } -lean_ctor_set(x_115, 0, x_105); -lean_ctor_set(x_115, 1, x_114); -x_3 = x_115; -x_4 = x_83; -goto _start; } -else +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__7___boxed(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_117; -if (lean_is_scalar(x_88)) { - x_117 = lean_alloc_ctor(0, 2, 0); -} else { - x_117 = x_88; +uint8_t x_3; lean_object* x_4; +x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__7(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; } -lean_ctor_set(x_117, 0, x_105); -lean_ctor_set(x_117, 1, x_107); -x_3 = x_117; -x_4 = x_83; -goto _start; +} +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; uint8_t x_6; lean_object* x_7; +x_4 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_5 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_6 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__13(x_1, x_4, x_5); +lean_dec(x_1); +x_7 = lean_box(x_6); +return x_7; } } -else +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___lambda__1___boxed(lean_object* x_1) { +_start: { -lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; -lean_inc(x_1); -x_119 = lean_array_uset(x_87, x_101, x_1); -x_120 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences___spec__15(x_81, x_85, x_102); -x_121 = lean_array_uset(x_119, x_101, x_120); -if (lean_is_scalar(x_88)) { - x_122 = lean_alloc_ctor(0, 2, 0); -} else { - x_122 = x_88; +uint8_t x_2; lean_object* x_3; +x_2 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___lambda__1(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; } -lean_ctor_set(x_122, 0, x_86); -lean_ctor_set(x_122, 1, x_121); -x_3 = x_122; -x_4 = x_83; -goto _start; } +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; uint8_t x_6; lean_object* x_7; +x_4 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_5 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_6 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14(x_1, x_4, x_5); +lean_dec(x_1); +x_7 = lean_box(x_6); +return x_7; } } +LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__12___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l_Lean_PersistentArray_anyMAux___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__12(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__11___boxed(lean_object* x_1) { _start: { -if (lean_obj_tag(x_2) == 0) +uint8_t x_2; lean_object* x_3; +x_2 = l_Lean_PersistentArray_anyM___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__11(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15___boxed(lean_object* x_1, lean_object* x_2) { +_start: { -return x_1; +uint8_t x_3; lean_object* x_4; +x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15(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_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -uint8_t x_3; -x_3 = !lean_is_exclusive(x_2); -if (x_3 == 0) +uint8_t x_5; lean_object* x_6; +x_5 = lean_unbox(x_2); +lean_dec(x_2); +x_6 = l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22(x_1, x_5, x_3, x_4); +return x_6; +} +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__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) { +_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; 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_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_ctor_get(x_1, 0); -lean_inc(x_7); -x_8 = lean_ctor_get(x_1, 1); -lean_inc(x_8); -x_9 = lean_array_get_size(x_8); -x_10 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_4); -x_11 = 32; -x_12 = lean_uint64_shift_right(x_10, x_11); -x_13 = lean_uint64_xor(x_10, x_12); -x_14 = 16; -x_15 = lean_uint64_shift_right(x_13, x_14); -x_16 = lean_uint64_xor(x_13, x_15); -x_17 = lean_uint64_to_usize(x_16); -x_18 = lean_usize_of_nat(x_9); -lean_dec(x_9); -x_19 = 1; -x_20 = lean_usize_sub(x_18, x_19); -x_21 = lean_usize_land(x_17, x_20); -x_22 = lean_array_uget(x_8, x_21); -x_23 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_4, x_22); -lean_dec(x_22); -lean_dec(x_4); -if (x_23 == 0) +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_6); +lean_dec(x_6); +x_10 = l_List_mapM_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__23(x_1, x_2, x_3, x_4, x_5, x_9, x_7, x_8); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__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) { +_start: { -lean_dec(x_8); -lean_dec(x_7); -lean_free_object(x_2); +uint8_t x_8; lean_object* x_9; +x_8 = lean_unbox(x_5); lean_dec(x_5); -x_2 = x_6; -goto _start; +x_9 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21(x_1, x_2, x_3, x_4, x_8, x_6, x_7); +return x_9; } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20___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: { -uint8_t x_25; -x_25 = !lean_is_exclusive(x_1); -if (x_25 == 0) +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_6); +lean_dec(x_6); +x_10 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20___lambda__1(x_1, x_2, x_3, x_4, x_5, x_9, x_7, x_8); +lean_dec(x_5); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__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) { +_start: { -lean_object* x_26; lean_object* x_27; uint64_t x_28; uint64_t x_29; uint64_t x_30; uint64_t x_31; uint64_t x_32; size_t x_33; size_t x_34; lean_object* x_35; uint8_t x_36; -x_26 = lean_ctor_get(x_1, 1); -lean_dec(x_26); -x_27 = lean_ctor_get(x_1, 0); -lean_dec(x_27); -x_28 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_5); -x_29 = lean_uint64_shift_right(x_28, x_11); -x_30 = lean_uint64_xor(x_28, x_29); -x_31 = lean_uint64_shift_right(x_30, x_14); -x_32 = lean_uint64_xor(x_30, x_31); -x_33 = lean_uint64_to_usize(x_32); -x_34 = lean_usize_land(x_33, x_20); -x_35 = lean_array_uget(x_8, x_34); -x_36 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_5, x_35); -if (x_36 == 0) +uint8_t x_8; lean_object* x_9; +x_8 = lean_unbox(x_5); +lean_dec(x_5); +x_9 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__20(x_1, x_2, x_3, x_4, x_8, x_6, x_7); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___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_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; -x_37 = lean_unsigned_to_nat(1u); -x_38 = lean_nat_add(x_7, x_37); +uint8_t x_6; lean_object* x_7; +x_6 = lean_unbox(x_3); +lean_dec(x_3); +x_7 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__1(x_1, x_2, x_6, x_4, x_5); +lean_dec(x_4); +lean_dec(x_2); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; lean_object* x_6; +x_5 = lean_unbox(x_2); +lean_dec(x_2); +x_6 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__2(x_1, x_5, x_3, x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___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: +{ +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_8); +lean_dec(x_8); +x_12 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_11, x_9, x_10); lean_dec(x_7); -x_39 = lean_box(0); -lean_ctor_set(x_2, 2, x_35); -lean_ctor_set(x_2, 1, x_39); -lean_ctor_set(x_2, 0, x_5); -x_40 = lean_array_uset(x_8, x_34, x_2); -x_41 = lean_unsigned_to_nat(4u); -x_42 = lean_nat_mul(x_38, x_41); -x_43 = lean_unsigned_to_nat(3u); -x_44 = lean_nat_div(x_42, x_43); -lean_dec(x_42); -x_45 = lean_array_get_size(x_40); -x_46 = lean_nat_dec_le(x_44, x_45); -lean_dec(x_45); -lean_dec(x_44); -if (x_46 == 0) +lean_dec(x_3); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___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) { +_start: { -lean_object* x_47; -x_47 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_40); -lean_ctor_set(x_1, 1, x_47); -lean_ctor_set(x_1, 0, x_38); -x_2 = x_6; -goto _start; +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_8); +lean_dec(x_8); +x_12 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_11, x_9, x_10); +lean_dec(x_7); +lean_dec(x_4); +return x_12; } -else +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___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) { +_start: { -lean_ctor_set(x_1, 1, x_40); -lean_ctor_set(x_1, 0, x_38); -x_2 = x_6; -goto _start; +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_8); +lean_dec(x_8); +x_12 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_11, x_9, x_10); +lean_dec(x_7); +lean_dec(x_5); +return x_12; } } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___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_dec(x_35); -lean_free_object(x_2); +uint8_t x_12; lean_object* x_13; +x_12 = lean_unbox(x_9); +lean_dec(x_9); +x_13 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_12, x_10, x_11); +lean_dec(x_8); +lean_dec(x_7); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___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) { +_start: +{ +uint8_t x_10; uint8_t x_11; lean_object* x_12; +x_10 = lean_unbox(x_3); +lean_dec(x_3); +x_11 = lean_unbox(x_7); +lean_dec(x_7); +x_12 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7(x_1, x_2, x_10, x_4, x_5, x_6, x_11, x_8, x_9); +lean_dec(x_6); lean_dec(x_5); -x_2 = x_6; -goto _start; +lean_dec(x_2); +return x_12; } } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___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) { +_start: { -uint64_t x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; uint64_t x_55; size_t x_56; size_t x_57; lean_object* x_58; uint8_t x_59; +uint8_t x_10; uint8_t x_11; lean_object* x_12; +x_10 = lean_unbox(x_1); lean_dec(x_1); -x_51 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_5); -x_52 = lean_uint64_shift_right(x_51, x_11); -x_53 = lean_uint64_xor(x_51, x_52); -x_54 = lean_uint64_shift_right(x_53, x_14); -x_55 = lean_uint64_xor(x_53, x_54); -x_56 = lean_uint64_to_usize(x_55); -x_57 = lean_usize_land(x_56, x_20); -x_58 = lean_array_uget(x_8, x_57); -x_59 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_5, x_58); -if (x_59 == 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; lean_object* x_68; uint8_t x_69; -x_60 = lean_unsigned_to_nat(1u); -x_61 = lean_nat_add(x_7, x_60); +x_11 = lean_unbox(x_7); lean_dec(x_7); -x_62 = lean_box(0); -lean_ctor_set(x_2, 2, x_58); -lean_ctor_set(x_2, 1, x_62); -lean_ctor_set(x_2, 0, x_5); -x_63 = lean_array_uset(x_8, x_57, x_2); -x_64 = lean_unsigned_to_nat(4u); -x_65 = lean_nat_mul(x_61, x_64); -x_66 = lean_unsigned_to_nat(3u); -x_67 = lean_nat_div(x_65, x_66); -lean_dec(x_65); -x_68 = lean_array_get_size(x_63); -x_69 = lean_nat_dec_le(x_67, x_68); -lean_dec(x_68); -lean_dec(x_67); -if (x_69 == 0) +x_12 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__8(x_10, x_2, x_3, x_4, x_5, x_6, x_11, x_8, x_9); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__9___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_70; lean_object* x_71; -x_70 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_63); -x_71 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_71, 0, x_61); -lean_ctor_set(x_71, 1, x_70); -x_1 = x_71; -x_2 = x_6; -goto _start; +uint8_t x_6; lean_object* x_7; +x_6 = lean_unbox(x_3); +lean_dec(x_3); +x_7 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__9(x_1, x_2, x_6, x_4, x_5); +lean_dec(x_4); +lean_dec(x_2); +return x_7; } -else +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___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) { +_start: { -lean_object* x_73; -x_73 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_73, 0, x_61); -lean_ctor_set(x_73, 1, x_63); -x_1 = x_73; -x_2 = x_6; -goto _start; +uint8_t x_8; lean_object* x_9; +x_8 = lean_unbox(x_5); +lean_dec(x_5); +x_9 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10(x_1, x_2, x_3, x_4, x_8, x_6, x_7); +lean_dec(x_4); +return x_9; } } -else +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___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) { +_start: { -lean_object* x_75; -lean_dec(x_58); -lean_free_object(x_2); +uint8_t x_7; lean_object* x_8; +x_7 = lean_unbox(x_4); +lean_dec(x_4); +x_8 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__11(x_1, x_2, x_3, x_7, x_5, x_6); lean_dec(x_5); -x_75 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_75, 0, x_7); -lean_ctor_set(x_75, 1, x_8); -x_1 = x_75; -x_2 = x_6; -goto _start; +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_8; } } +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__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) { +_start: +{ +size_t x_10; size_t x_11; uint8_t x_12; lean_object* x_13; +x_10 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_11 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_12 = lean_unbox(x_7); +lean_dec(x_7); +x_13 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24(x_1, x_2, x_3, x_10, x_11, x_6, x_12, x_8, x_9); +lean_dec(x_3); +return x_13; } } -else +LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences_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) { +_start: { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* 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; size_t x_90; size_t x_91; size_t x_92; size_t x_93; size_t x_94; lean_object* x_95; uint8_t x_96; -x_77 = lean_ctor_get(x_2, 0); +uint8_t x_7; lean_object* x_8; +x_7 = lean_unbox(x_4); +lean_dec(x_4); +x_8 = l_Lean_Linter_UnusedVariables_collectReferences_go(x_1, x_2, x_3, x_7, x_5, x_6); +lean_dec(x_2); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; uint8_t x_6; lean_object* x_7; +x_5 = lean_box(0); +x_6 = 0; +x_7 = l_Lean_Linter_UnusedVariables_collectReferences_go(x_2, x_1, x_5, x_6, x_3, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_collectReferences___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_Linter_UnusedVariables_collectReferences(x_1, x_2, x_3, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +lean_dec(x_1); +return x_3; +} +else +{ +uint8_t x_5; +x_5 = !lean_is_exclusive(x_4); +if (x_5 == 0) +{ +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_6 = lean_ctor_get(x_4, 0); +x_7 = lean_ctor_get(x_4, 1); +x_8 = lean_ctor_get(x_4, 2); +x_9 = lean_ctor_get(x_2, 3); +x_10 = l_Lean_Linter_UnusedVariables_followAliases(x_9, x_7); +x_11 = !lean_is_exclusive(x_3); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint64_t 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; size_t x_22; size_t x_23; size_t x_24; size_t x_25; size_t x_26; lean_object* x_27; uint8_t x_28; +x_12 = lean_ctor_get(x_3, 0); +x_13 = lean_ctor_get(x_3, 1); +x_14 = lean_array_get_size(x_13); +x_15 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_6); +x_16 = 32; +x_17 = lean_uint64_shift_right(x_15, x_16); +x_18 = lean_uint64_xor(x_15, x_17); +x_19 = 16; +x_20 = lean_uint64_shift_right(x_18, x_19); +x_21 = lean_uint64_xor(x_18, x_20); +x_22 = lean_uint64_to_usize(x_21); +x_23 = lean_usize_of_nat(x_14); +lean_dec(x_14); +x_24 = 1; +x_25 = lean_usize_sub(x_23, x_24); +x_26 = lean_usize_land(x_22, x_25); +x_27 = lean_array_uget(x_13, x_26); +x_28 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15(x_6, 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_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_29 = lean_unsigned_to_nat(1u); +x_30 = lean_nat_add(x_12, x_29); +lean_dec(x_12); +lean_ctor_set(x_4, 2, x_27); +lean_ctor_set(x_4, 1, x_10); +x_31 = lean_array_uset(x_13, x_26, x_4); +x_32 = lean_unsigned_to_nat(4u); +x_33 = lean_nat_mul(x_30, x_32); +x_34 = lean_unsigned_to_nat(3u); +x_35 = lean_nat_div(x_33, x_34); +lean_dec(x_33); +x_36 = lean_array_get_size(x_31); +x_37 = lean_nat_dec_le(x_35, x_36); +lean_dec(x_36); +lean_dec(x_35); +if (x_37 == 0) +{ +lean_object* x_38; +x_38 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__16(x_31); +lean_ctor_set(x_3, 1, x_38); +lean_ctor_set(x_3, 0, x_30); +x_4 = x_8; +goto _start; +} +else +{ +lean_ctor_set(x_3, 1, x_31); +lean_ctor_set(x_3, 0, x_30); +x_4 = x_8; +goto _start; +} +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; +lean_free_object(x_4); +lean_inc(x_1); +x_41 = lean_array_uset(x_13, x_26, x_1); +x_42 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(x_6, x_10, x_27); +x_43 = lean_array_uset(x_41, x_26, x_42); +lean_ctor_set(x_3, 1, x_43); +x_4 = x_8; +goto _start; +} +} +else +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; uint64_t x_48; uint64_t x_49; uint64_t x_50; uint64_t x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; size_t x_55; size_t x_56; size_t x_57; size_t x_58; size_t x_59; lean_object* x_60; uint8_t x_61; +x_45 = lean_ctor_get(x_3, 0); +x_46 = lean_ctor_get(x_3, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_3); +x_47 = lean_array_get_size(x_46); +x_48 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_6); +x_49 = 32; +x_50 = lean_uint64_shift_right(x_48, x_49); +x_51 = lean_uint64_xor(x_48, x_50); +x_52 = 16; +x_53 = lean_uint64_shift_right(x_51, x_52); +x_54 = lean_uint64_xor(x_51, x_53); +x_55 = lean_uint64_to_usize(x_54); +x_56 = lean_usize_of_nat(x_47); +lean_dec(x_47); +x_57 = 1; +x_58 = lean_usize_sub(x_56, x_57); +x_59 = lean_usize_land(x_55, x_58); +x_60 = lean_array_uget(x_46, x_59); +x_61 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15(x_6, 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; uint8_t x_70; +x_62 = lean_unsigned_to_nat(1u); +x_63 = lean_nat_add(x_45, x_62); +lean_dec(x_45); +lean_ctor_set(x_4, 2, x_60); +lean_ctor_set(x_4, 1, x_10); +x_64 = lean_array_uset(x_46, x_59, x_4); +x_65 = lean_unsigned_to_nat(4u); +x_66 = lean_nat_mul(x_63, 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; lean_object* x_72; +x_71 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__16(x_64); +x_72 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_72, 0, x_63); +lean_ctor_set(x_72, 1, x_71); +x_3 = x_72; +x_4 = x_8; +goto _start; +} +else +{ +lean_object* x_74; +x_74 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_74, 0, x_63); +lean_ctor_set(x_74, 1, x_64); +x_3 = x_74; +x_4 = x_8; +goto _start; +} +} +else +{ +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +lean_free_object(x_4); +lean_inc(x_1); +x_76 = lean_array_uset(x_46, x_59, x_1); +x_77 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(x_6, x_10, 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_45); +lean_ctor_set(x_79, 1, x_78); +x_3 = x_79; +x_4 = x_8; +goto _start; +} +} +} +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; uint64_t x_90; uint64_t x_91; uint64_t x_92; uint64_t x_93; uint64_t x_94; uint64_t x_95; uint64_t x_96; size_t x_97; size_t x_98; size_t x_99; size_t x_100; size_t x_101; lean_object* x_102; uint8_t x_103; +x_81 = lean_ctor_get(x_4, 0); +x_82 = lean_ctor_get(x_4, 1); +x_83 = lean_ctor_get(x_4, 2); +lean_inc(x_83); +lean_inc(x_82); +lean_inc(x_81); +lean_dec(x_4); +x_84 = lean_ctor_get(x_2, 3); +x_85 = l_Lean_Linter_UnusedVariables_followAliases(x_84, x_82); +x_86 = lean_ctor_get(x_3, 0); +lean_inc(x_86); +x_87 = lean_ctor_get(x_3, 1); +lean_inc(x_87); +if (lean_is_exclusive(x_3)) { + lean_ctor_release(x_3, 0); + lean_ctor_release(x_3, 1); + x_88 = x_3; +} else { + lean_dec_ref(x_3); + x_88 = lean_box(0); +} +x_89 = lean_array_get_size(x_87); +x_90 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_81); +x_91 = 32; +x_92 = lean_uint64_shift_right(x_90, x_91); +x_93 = lean_uint64_xor(x_90, x_92); +x_94 = 16; +x_95 = lean_uint64_shift_right(x_93, x_94); +x_96 = lean_uint64_xor(x_93, x_95); +x_97 = lean_uint64_to_usize(x_96); +x_98 = lean_usize_of_nat(x_89); +lean_dec(x_89); +x_99 = 1; +x_100 = lean_usize_sub(x_98, x_99); +x_101 = lean_usize_land(x_97, x_100); +x_102 = lean_array_uget(x_87, x_101); +x_103 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__15(x_81, x_102); +if (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; lean_object* x_111; lean_object* x_112; uint8_t x_113; +x_104 = lean_unsigned_to_nat(1u); +x_105 = lean_nat_add(x_86, x_104); +lean_dec(x_86); +x_106 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_106, 0, x_81); +lean_ctor_set(x_106, 1, x_85); +lean_ctor_set(x_106, 2, x_102); +x_107 = lean_array_uset(x_87, x_101, x_106); +x_108 = lean_unsigned_to_nat(4u); +x_109 = lean_nat_mul(x_105, x_108); +x_110 = lean_unsigned_to_nat(3u); +x_111 = lean_nat_div(x_109, x_110); +lean_dec(x_109); +x_112 = lean_array_get_size(x_107); +x_113 = lean_nat_dec_le(x_111, x_112); +lean_dec(x_112); +lean_dec(x_111); +if (x_113 == 0) +{ +lean_object* x_114; lean_object* x_115; +x_114 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__16(x_107); +if (lean_is_scalar(x_88)) { + x_115 = lean_alloc_ctor(0, 2, 0); +} else { + x_115 = x_88; +} +lean_ctor_set(x_115, 0, x_105); +lean_ctor_set(x_115, 1, x_114); +x_3 = x_115; +x_4 = x_83; +goto _start; +} +else +{ +lean_object* x_117; +if (lean_is_scalar(x_88)) { + x_117 = lean_alloc_ctor(0, 2, 0); +} else { + x_117 = x_88; +} +lean_ctor_set(x_117, 0, x_105); +lean_ctor_set(x_117, 1, x_107); +x_3 = x_117; +x_4 = x_83; +goto _start; +} +} +else +{ +lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; +lean_inc(x_1); +x_119 = lean_array_uset(x_87, x_101, x_1); +x_120 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__19(x_81, x_85, x_102); +x_121 = lean_array_uset(x_119, x_101, x_120); +if (lean_is_scalar(x_88)) { + x_122 = lean_alloc_ctor(0, 2, 0); +} else { + x_122 = x_88; +} +lean_ctor_set(x_122, 0, x_86); +lean_ctor_set(x_122, 1, x_121); +x_3 = x_122; +x_4 = x_83; +goto _start; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +return x_1; +} +else +{ +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_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_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_ctor_get(x_1, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_1, 1); +lean_inc(x_8); +x_9 = lean_array_get_size(x_8); +x_10 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_4); +x_11 = 32; +x_12 = lean_uint64_shift_right(x_10, x_11); +x_13 = lean_uint64_xor(x_10, x_12); +x_14 = 16; +x_15 = lean_uint64_shift_right(x_13, x_14); +x_16 = lean_uint64_xor(x_13, x_15); +x_17 = lean_uint64_to_usize(x_16); +x_18 = lean_usize_of_nat(x_9); +lean_dec(x_9); +x_19 = 1; +x_20 = lean_usize_sub(x_18, x_19); +x_21 = lean_usize_land(x_17, x_20); +x_22 = lean_array_uget(x_8, x_21); +x_23 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_4, x_22); +lean_dec(x_22); +lean_dec(x_4); +if (x_23 == 0) +{ +lean_dec(x_8); +lean_dec(x_7); +lean_free_object(x_2); +lean_dec(x_5); +x_2 = x_6; +goto _start; +} +else +{ +uint8_t x_25; +x_25 = !lean_is_exclusive(x_1); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; uint64_t x_28; uint64_t x_29; uint64_t x_30; uint64_t x_31; uint64_t x_32; size_t x_33; size_t x_34; lean_object* x_35; uint8_t x_36; +x_26 = lean_ctor_get(x_1, 1); +lean_dec(x_26); +x_27 = lean_ctor_get(x_1, 0); +lean_dec(x_27); +x_28 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_5); +x_29 = lean_uint64_shift_right(x_28, x_11); +x_30 = lean_uint64_xor(x_28, x_29); +x_31 = lean_uint64_shift_right(x_30, x_14); +x_32 = lean_uint64_xor(x_30, x_31); +x_33 = lean_uint64_to_usize(x_32); +x_34 = lean_usize_land(x_33, x_20); +x_35 = lean_array_uget(x_8, x_34); +x_36 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_5, x_35); +if (x_36 == 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; uint8_t x_46; +x_37 = lean_unsigned_to_nat(1u); +x_38 = lean_nat_add(x_7, x_37); +lean_dec(x_7); +x_39 = lean_box(0); +lean_ctor_set(x_2, 2, x_35); +lean_ctor_set(x_2, 1, x_39); +lean_ctor_set(x_2, 0, x_5); +x_40 = lean_array_uset(x_8, x_34, x_2); +x_41 = lean_unsigned_to_nat(4u); +x_42 = lean_nat_mul(x_38, x_41); +x_43 = lean_unsigned_to_nat(3u); +x_44 = lean_nat_div(x_42, x_43); +lean_dec(x_42); +x_45 = lean_array_get_size(x_40); +x_46 = lean_nat_dec_le(x_44, x_45); +lean_dec(x_45); +lean_dec(x_44); +if (x_46 == 0) +{ +lean_object* x_47; +x_47 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_40); +lean_ctor_set(x_1, 1, x_47); +lean_ctor_set(x_1, 0, x_38); +x_2 = x_6; +goto _start; +} +else +{ +lean_ctor_set(x_1, 1, x_40); +lean_ctor_set(x_1, 0, x_38); +x_2 = x_6; +goto _start; +} +} +else +{ +lean_dec(x_35); +lean_free_object(x_2); +lean_dec(x_5); +x_2 = x_6; +goto _start; +} +} +else +{ +uint64_t x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; uint64_t x_55; size_t x_56; size_t x_57; lean_object* x_58; uint8_t x_59; +lean_dec(x_1); +x_51 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_5); +x_52 = lean_uint64_shift_right(x_51, x_11); +x_53 = lean_uint64_xor(x_51, x_52); +x_54 = lean_uint64_shift_right(x_53, x_14); +x_55 = lean_uint64_xor(x_53, x_54); +x_56 = lean_uint64_to_usize(x_55); +x_57 = lean_usize_land(x_56, x_20); +x_58 = lean_array_uget(x_8, x_57); +x_59 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_5, x_58); +if (x_59 == 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; lean_object* x_68; uint8_t x_69; +x_60 = lean_unsigned_to_nat(1u); +x_61 = lean_nat_add(x_7, x_60); +lean_dec(x_7); +x_62 = lean_box(0); +lean_ctor_set(x_2, 2, x_58); +lean_ctor_set(x_2, 1, x_62); +lean_ctor_set(x_2, 0, x_5); +x_63 = lean_array_uset(x_8, x_57, x_2); +x_64 = lean_unsigned_to_nat(4u); +x_65 = lean_nat_mul(x_61, x_64); +x_66 = lean_unsigned_to_nat(3u); +x_67 = lean_nat_div(x_65, x_66); +lean_dec(x_65); +x_68 = lean_array_get_size(x_63); +x_69 = lean_nat_dec_le(x_67, x_68); +lean_dec(x_68); +lean_dec(x_67); +if (x_69 == 0) +{ +lean_object* x_70; lean_object* x_71; +x_70 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_63); +x_71 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_71, 0, x_61); +lean_ctor_set(x_71, 1, x_70); +x_1 = x_71; +x_2 = x_6; +goto _start; +} +else +{ +lean_object* x_73; +x_73 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_73, 0, x_61); +lean_ctor_set(x_73, 1, x_63); +x_1 = x_73; +x_2 = x_6; +goto _start; +} +} +else +{ +lean_object* x_75; +lean_dec(x_58); +lean_free_object(x_2); +lean_dec(x_5); +x_75 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_75, 0, x_7); +lean_ctor_set(x_75, 1, x_8); +x_1 = x_75; +x_2 = x_6; +goto _start; +} +} +} +} +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; 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; size_t x_90; size_t x_91; size_t x_92; size_t x_93; size_t x_94; lean_object* x_95; uint8_t x_96; +x_77 = lean_ctor_get(x_2, 0); x_78 = lean_ctor_get(x_2, 1); x_79 = lean_ctor_get(x_2, 2); lean_inc(x_79); lean_inc(x_78); lean_inc(x_77); lean_dec(x_2); -x_80 = lean_ctor_get(x_1, 0); -lean_inc(x_80); -x_81 = lean_ctor_get(x_1, 1); -lean_inc(x_81); -x_82 = lean_array_get_size(x_81); -x_83 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_77); -x_84 = 32; -x_85 = lean_uint64_shift_right(x_83, x_84); -x_86 = lean_uint64_xor(x_83, x_85); -x_87 = 16; -x_88 = lean_uint64_shift_right(x_86, x_87); -x_89 = lean_uint64_xor(x_86, x_88); -x_90 = lean_uint64_to_usize(x_89); -x_91 = lean_usize_of_nat(x_82); -lean_dec(x_82); -x_92 = 1; -x_93 = lean_usize_sub(x_91, x_92); -x_94 = lean_usize_land(x_90, x_93); -x_95 = lean_array_uget(x_81, x_94); -x_96 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_77, x_95); -lean_dec(x_95); -lean_dec(x_77); -if (x_96 == 0) +x_80 = lean_ctor_get(x_1, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_1, 1); +lean_inc(x_81); +x_82 = lean_array_get_size(x_81); +x_83 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_77); +x_84 = 32; +x_85 = lean_uint64_shift_right(x_83, x_84); +x_86 = lean_uint64_xor(x_83, x_85); +x_87 = 16; +x_88 = lean_uint64_shift_right(x_86, x_87); +x_89 = lean_uint64_xor(x_86, x_88); +x_90 = lean_uint64_to_usize(x_89); +x_91 = lean_usize_of_nat(x_82); +lean_dec(x_82); +x_92 = 1; +x_93 = lean_usize_sub(x_91, x_92); +x_94 = lean_usize_land(x_90, x_93); +x_95 = lean_array_uget(x_81, x_94); +x_96 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_77, x_95); +lean_dec(x_95); +lean_dec(x_77); +if (x_96 == 0) +{ +lean_dec(x_81); +lean_dec(x_80); +lean_dec(x_78); +x_2 = x_79; +goto _start; +} +else +{ +lean_object* x_98; uint64_t x_99; uint64_t x_100; uint64_t x_101; uint64_t x_102; uint64_t x_103; size_t x_104; size_t x_105; lean_object* x_106; uint8_t x_107; +if (lean_is_exclusive(x_1)) { + lean_ctor_release(x_1, 0); + lean_ctor_release(x_1, 1); + x_98 = x_1; +} else { + lean_dec_ref(x_1); + x_98 = lean_box(0); +} +x_99 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_78); +x_100 = lean_uint64_shift_right(x_99, x_84); +x_101 = lean_uint64_xor(x_99, x_100); +x_102 = lean_uint64_shift_right(x_101, x_87); +x_103 = lean_uint64_xor(x_101, x_102); +x_104 = lean_uint64_to_usize(x_103); +x_105 = lean_usize_land(x_104, x_93); +x_106 = lean_array_uget(x_81, x_105); +x_107 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_78, x_106); +if (x_107 == 0) +{ +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; uint8_t x_118; +x_108 = lean_unsigned_to_nat(1u); +x_109 = lean_nat_add(x_80, x_108); +lean_dec(x_80); +x_110 = lean_box(0); +x_111 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_111, 0, x_78); +lean_ctor_set(x_111, 1, x_110); +lean_ctor_set(x_111, 2, x_106); +x_112 = lean_array_uset(x_81, x_105, x_111); +x_113 = lean_unsigned_to_nat(4u); +x_114 = lean_nat_mul(x_109, x_113); +x_115 = lean_unsigned_to_nat(3u); +x_116 = lean_nat_div(x_114, x_115); +lean_dec(x_114); +x_117 = lean_array_get_size(x_112); +x_118 = lean_nat_dec_le(x_116, x_117); +lean_dec(x_117); +lean_dec(x_116); +if (x_118 == 0) +{ +lean_object* x_119; lean_object* x_120; +x_119 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_112); +if (lean_is_scalar(x_98)) { + x_120 = lean_alloc_ctor(0, 2, 0); +} else { + x_120 = x_98; +} +lean_ctor_set(x_120, 0, x_109); +lean_ctor_set(x_120, 1, x_119); +x_1 = x_120; +x_2 = x_79; +goto _start; +} +else +{ +lean_object* x_122; +if (lean_is_scalar(x_98)) { + x_122 = lean_alloc_ctor(0, 2, 0); +} else { + x_122 = x_98; +} +lean_ctor_set(x_122, 0, x_109); +lean_ctor_set(x_122, 1, x_112); +x_1 = x_122; +x_2 = x_79; +goto _start; +} +} +else +{ +lean_object* x_124; +lean_dec(x_106); +lean_dec(x_78); +if (lean_is_scalar(x_98)) { + x_124 = lean_alloc_ctor(0, 2, 0); +} else { + x_124 = x_98; +} +lean_ctor_set(x_124, 0, x_80); +lean_ctor_set(x_124, 1, x_81); +x_1 = x_124; +x_2 = x_79; +goto _start; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_inc(x_2); +return x_2; +} +else +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; +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_name_eq(x_4, x_1); +if (x_7 == 0) +{ +x_3 = x_6; +goto _start; +} +else +{ +lean_inc(x_5); +return x_5; +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4(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; lean_object* x_6; lean_object* x_7; +x_3 = lean_ctor_get(x_2, 0); +x_4 = lean_ctor_get(x_2, 1); +x_5 = lean_ctor_get(x_2, 2); +lean_inc(x_4); +lean_inc(x_3); +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_3); +lean_ctor_set(x_6, 1, x_4); +x_7 = lean_array_push(x_1, x_6); +x_1 = x_7; +x_2 = x_5; +goto _start; +} +} +} +static lean_object* _init_l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8___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_Command_instMonadCommandElabM; +x_3 = l_instInhabitedOfMonad___rarg(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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; +x_5 = l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8___closed__1; +x_6 = lean_panic_fn(x_5, x_1); +x_7 = lean_apply_3(x_6, x_2, x_3, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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, lean_object* x_8) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_9; lean_object* x_10; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_9 = l_List_reverse___rarg(x_5); +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_11; +x_11 = !lean_is_exclusive(x_4); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_4, 0); +x_13 = lean_ctor_get(x_4, 1); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__7(x_1, x_2, x_3, x_12, x_6, x_7, x_8); +if (lean_obj_tag(x_14) == 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_4, 1, x_5); +lean_ctor_set(x_4, 0, x_15); +{ +lean_object* _tmp_3 = x_13; +lean_object* _tmp_4 = x_4; +lean_object* _tmp_7 = x_16; +x_4 = _tmp_3; +x_5 = _tmp_4; +x_8 = _tmp_7; +} +goto _start; +} +else +{ +uint8_t x_18; +lean_free_object(x_4); +lean_dec(x_13); +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_18 = !lean_is_exclusive(x_14); +if (x_18 == 0) { -lean_dec(x_81); -lean_dec(x_80); -lean_dec(x_78); -x_2 = x_79; +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_4, 0); +x_23 = lean_ctor_get(x_4, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_4); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_24 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__7(x_1, x_2, x_3, x_22, 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); +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_5); +x_4 = x_23; +x_5 = x_27; +x_8 = x_26; goto _start; } else { -lean_object* x_98; uint64_t x_99; uint64_t x_100; uint64_t x_101; uint64_t x_102; uint64_t x_103; size_t x_104; size_t x_105; lean_object* x_106; uint8_t x_107; -if (lean_is_exclusive(x_1)) { - lean_ctor_release(x_1, 0); - lean_ctor_release(x_1, 1); - x_98 = x_1; +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_3); +lean_dec(x_2); +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_1); - x_98 = lean_box(0); + lean_dec_ref(x_24); + x_31 = lean_box(0); } -x_99 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_78); -x_100 = lean_uint64_shift_right(x_99, x_84); -x_101 = lean_uint64_xor(x_99, x_100); -x_102 = lean_uint64_shift_right(x_101, x_87); -x_103 = lean_uint64_xor(x_101, x_102); -x_104 = lean_uint64_to_usize(x_103); -x_105 = lean_usize_land(x_104, x_93); -x_106 = lean_array_uget(x_81, x_105); -x_107 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_78, x_106); -if (x_107 == 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; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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) { +_start: { -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; uint8_t x_118; -x_108 = lean_unsigned_to_nat(1u); -x_109 = lean_nat_add(x_80, x_108); -lean_dec(x_80); -x_110 = lean_box(0); -x_111 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_111, 0, x_78); -lean_ctor_set(x_111, 1, x_110); -lean_ctor_set(x_111, 2, x_106); -x_112 = lean_array_uset(x_81, x_105, x_111); -x_113 = lean_unsigned_to_nat(4u); -x_114 = lean_nat_mul(x_109, x_113); -x_115 = lean_unsigned_to_nat(3u); -x_116 = lean_nat_div(x_114, x_115); -lean_dec(x_114); -x_117 = lean_array_get_size(x_112); -x_118 = lean_nat_dec_le(x_116, x_117); -lean_dec(x_117); -lean_dec(x_116); -if (x_118 == 0) +if (lean_obj_tag(x_3) == 0) { -lean_object* x_119; lean_object* x_120; -x_119 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_112); -if (lean_is_scalar(x_98)) { - x_120 = lean_alloc_ctor(0, 2, 0); -} else { - x_120 = x_98; +switch (lean_obj_tag(x_4)) { +case 0: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_ctor_get(x_4, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_4, 1); +lean_inc(x_9); +lean_dec(x_4); +x_10 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_8, x_3); +x_3 = x_10; +x_4 = x_9; +goto _start; +} +case 1: +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__4; +x_13 = l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8(x_12, x_5, x_6, x_7); +return x_13; +} +default: +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +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_7); +return x_15; +} +} +} +else +{ +switch (lean_obj_tag(x_4)) { +case 0: +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_4, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_4, 1); +lean_inc(x_17); +lean_dec(x_4); +x_18 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_16, x_3); +x_3 = x_18; +x_4 = x_17; +goto _start; +} +case 1: +{ +uint8_t x_20; +x_20 = !lean_is_exclusive(x_3); +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_3, 0); +x_22 = lean_ctor_get(x_4, 0); +lean_inc(x_22); +x_23 = lean_ctor_get(x_4, 1); +lean_inc(x_23); +lean_dec(x_4); +lean_inc(x_1); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_23); +lean_inc(x_22); +lean_inc(x_21); +x_24 = lean_apply_6(x_1, x_21, x_22, x_23, x_5, x_6, x_7); +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) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_dec(x_1); +x_27 = lean_ctor_get(x_24, 1); +lean_inc(x_27); +lean_dec(x_24); +x_28 = lean_box(0); +x_29 = lean_apply_7(x_2, x_21, x_22, x_23, x_28, x_5, x_6, x_27); +if (lean_obj_tag(x_29) == 0) +{ +uint8_t x_30; +x_30 = !lean_is_exclusive(x_29); +if (x_30 == 0) +{ +lean_object* x_31; +x_31 = lean_ctor_get(x_29, 0); +lean_ctor_set(x_3, 0, x_31); +lean_ctor_set(x_29, 0, x_3); +return x_29; +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_29, 0); +x_33 = lean_ctor_get(x_29, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_29); +lean_ctor_set(x_3, 0, x_32); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_3); +lean_ctor_set(x_34, 1, x_33); +return x_34; } -lean_ctor_set(x_120, 0, x_109); -lean_ctor_set(x_120, 1, x_119); -x_1 = x_120; -x_2 = x_79; -goto _start; } else { -lean_object* x_122; -if (lean_is_scalar(x_98)) { - x_122 = lean_alloc_ctor(0, 2, 0); -} else { - x_122 = x_98; +uint8_t x_35; +lean_free_object(x_3); +x_35 = !lean_is_exclusive(x_29); +if (x_35 == 0) +{ +return x_29; +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_29, 0); +x_37 = lean_ctor_get(x_29, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_29); +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_ctor_set(x_122, 0, x_109); -lean_ctor_set(x_122, 1, x_112); -x_1 = x_122; -x_2 = x_79; -goto _start; } } else { -lean_object* x_124; -lean_dec(x_106); -lean_dec(x_78); -if (lean_is_scalar(x_98)) { - x_124 = lean_alloc_ctor(0, 2, 0); -} else { - x_124 = x_98; +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_24, 1); +lean_inc(x_39); +lean_dec(x_24); +lean_inc(x_21); +x_40 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_22); +x_41 = l_Lean_PersistentArray_toList___rarg(x_23); +x_42 = lean_box(0); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_2); +x_43 = l_List_mapM_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__9(x_1, x_2, x_40, x_41, x_42, x_5, x_6, x_39); +if (lean_obj_tag(x_43) == 0) +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; +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_apply_7(x_2, x_21, x_22, x_23, x_44, x_5, x_6, x_45); +if (lean_obj_tag(x_46) == 0) +{ +uint8_t x_47; +x_47 = !lean_is_exclusive(x_46); +if (x_47 == 0) +{ +lean_object* x_48; lean_object* x_49; +x_48 = lean_ctor_get(x_46, 0); +x_49 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_46, 0, x_49); +return x_46; } -lean_ctor_set(x_124, 0, x_80); -lean_ctor_set(x_124, 1, x_81); -x_1 = x_124; -x_2 = x_79; -goto _start; +else +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +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, 1, 0); +lean_ctor_set(x_52, 0, x_50); +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 +{ +uint8_t x_54; +x_54 = !lean_is_exclusive(x_46); +if (x_54 == 0) +{ +return x_46; } +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_46, 0); +x_56 = lean_ctor_get(x_46, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_46); +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_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(lean_object* x_1, lean_object* x_2) { -_start: +else { -if (lean_obj_tag(x_2) == 0) +uint8_t x_58; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_58 = !lean_is_exclusive(x_43); +if (x_58 == 0) { -return x_1; +return x_43; } else { -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_2, 0); -x_4 = lean_ctor_get(x_2, 1); -x_5 = lean_ctor_get(x_2, 2); -lean_inc(x_4); -lean_inc(x_3); -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_3); -lean_ctor_set(x_6, 1, x_4); -x_7 = lean_array_push(x_1, x_6); -x_1 = x_7; -x_2 = x_5; -goto _start; +lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_43, 0); +x_60 = lean_ctor_get(x_43, 1); +lean_inc(x_60); +lean_inc(x_59); +lean_dec(x_43); +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; } } } -static lean_object* _init_l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8___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_Command_instMonadCommandElabM; -x_3 = l_instInhabitedOfMonad___rarg(x_2, x_1); -return x_3; } +else +{ +uint8_t x_62; +lean_dec(x_23); +lean_dec(x_22); +lean_free_object(x_3); +lean_dec(x_21); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +x_62 = !lean_is_exclusive(x_24); +if (x_62 == 0) +{ +return x_24; } -LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +else { -lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_5 = l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8___closed__1; -x_6 = lean_panic_fn(x_5, x_1); -x_7 = lean_apply_3(x_6, x_2, x_3, x_4); -return x_7; +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_24, 0); +x_64 = lean_ctor_get(x_24, 1); +lean_inc(x_64); +lean_inc(x_63); +lean_dec(x_24); +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_List_mapM_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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, lean_object* x_8) { -_start: -{ -if (lean_obj_tag(x_4) == 0) +} +else { -lean_object* x_9; lean_object* x_10; -lean_dec(x_7); -lean_dec(x_6); +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_66 = lean_ctor_get(x_3, 0); +lean_inc(x_66); lean_dec(x_3); -lean_dec(x_2); +x_67 = lean_ctor_get(x_4, 0); +lean_inc(x_67); +x_68 = lean_ctor_get(x_4, 1); +lean_inc(x_68); +lean_dec(x_4); +lean_inc(x_1); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_68); +lean_inc(x_67); +lean_inc(x_66); +x_69 = lean_apply_6(x_1, x_66, x_67, x_68, x_5, x_6, x_7); +if (lean_obj_tag(x_69) == 0) +{ +lean_object* x_70; uint8_t x_71; +x_70 = lean_ctor_get(x_69, 0); +lean_inc(x_70); +x_71 = lean_unbox(x_70); +lean_dec(x_70); +if (x_71 == 0) +{ +lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_dec(x_1); -x_9 = l_List_reverse___rarg(x_5); -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; +x_72 = lean_ctor_get(x_69, 1); +lean_inc(x_72); +lean_dec(x_69); +x_73 = lean_box(0); +x_74 = lean_apply_7(x_2, x_66, x_67, x_68, x_73, x_5, x_6, x_72); +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_74); + x_77 = lean_box(0); +} +x_78 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_78, 0, x_75); +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 { -uint8_t x_11; -x_11 = !lean_is_exclusive(x_4); -if (x_11 == 0) +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_80 = lean_ctor_get(x_74, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_74, 1); +lean_inc(x_81); +if (lean_is_exclusive(x_74)) { + lean_ctor_release(x_74, 0); + lean_ctor_release(x_74, 1); + x_82 = x_74; +} else { + lean_dec_ref(x_74); + 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_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_4, 0); -x_13 = lean_ctor_get(x_4, 1); -lean_inc(x_7); +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_69, 1); +lean_inc(x_84); +lean_dec(x_69); +lean_inc(x_66); +x_85 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_85, 0, x_66); +x_86 = l_Lean_Elab_Info_updateContext_x3f(x_85, x_67); +x_87 = l_Lean_PersistentArray_toList___rarg(x_68); +x_88 = lean_box(0); lean_inc(x_6); -lean_inc(x_3); +lean_inc(x_5); lean_inc(x_2); -lean_inc(x_1); -x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__7(x_1, x_2, x_3, x_12, x_6, x_7, x_8); -if (lean_obj_tag(x_14) == 0) +x_89 = l_List_mapM_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__9(x_1, x_2, x_86, x_87, x_88, x_5, x_6, x_84); +if (lean_obj_tag(x_89) == 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_4, 1, x_5); -lean_ctor_set(x_4, 0, x_15); +lean_object* x_90; lean_object* x_91; lean_object* x_92; +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_7(x_2, x_66, x_67, x_68, x_90, x_5, x_6, x_91); +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_92); + x_95 = lean_box(0); +} +x_96 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_96, 0, x_93); +if (lean_is_scalar(x_95)) { + x_97 = lean_alloc_ctor(0, 2, 0); +} else { + x_97 = x_95; +} +lean_ctor_set(x_97, 0, x_96); +lean_ctor_set(x_97, 1, x_94); +return x_97; +} +else { -lean_object* _tmp_3 = x_13; -lean_object* _tmp_4 = x_4; -lean_object* _tmp_7 = x_16; -x_4 = _tmp_3; -x_5 = _tmp_4; -x_8 = _tmp_7; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; +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_92); + 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; } -goto _start; } else { -uint8_t x_18; -lean_free_object(x_4); -lean_dec(x_13); -lean_dec(x_7); +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +lean_dec(x_68); +lean_dec(x_67); +lean_dec(x_66); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_18 = !lean_is_exclusive(x_14); -if (x_18 == 0) -{ -return x_14; +x_102 = lean_ctor_get(x_89, 0); +lean_inc(x_102); +x_103 = lean_ctor_get(x_89, 1); +lean_inc(x_103); +if (lean_is_exclusive(x_89)) { + lean_ctor_release(x_89, 0); + lean_ctor_release(x_89, 1); + x_104 = x_89; +} else { + lean_dec_ref(x_89); + x_104 = lean_box(0); } -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; +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_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_4, 0); -x_23 = lean_ctor_get(x_4, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_4); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_1); -x_24 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__7(x_1, x_2, x_3, x_22, 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); -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_5); -x_4 = x_23; -x_5 = 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_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; +lean_dec(x_68); +lean_dec(x_67); +lean_dec(x_66); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_3); lean_dec(x_2); 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; +x_106 = lean_ctor_get(x_69, 0); +lean_inc(x_106); +x_107 = lean_ctor_get(x_69, 1); +lean_inc(x_107); +if (lean_is_exclusive(x_69)) { + lean_ctor_release(x_69, 0); + lean_ctor_release(x_69, 1); + x_108 = x_69; } else { - lean_dec_ref(x_24); - x_31 = lean_box(0); + lean_dec_ref(x_69); + x_108 = lean_box(0); } -if (lean_is_scalar(x_31)) { - x_32 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_108)) { + x_109 = 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; -} -} -} + x_109 = x_108; } +lean_ctor_set(x_109, 0, x_106); +lean_ctor_set(x_109, 1, x_107); +return x_109; } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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) { -_start: -{ -if (lean_obj_tag(x_3) == 0) -{ -switch (lean_obj_tag(x_4)) { -case 0: -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_8 = lean_ctor_get(x_4, 0); -lean_inc(x_8); -x_9 = lean_ctor_get(x_4, 1); -lean_inc(x_9); -lean_dec(x_4); -x_10 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_8, x_3); -x_3 = x_10; -x_4 = x_9; -goto _start; } -case 1: -{ -lean_object* x_12; lean_object* x_13; -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__4; -x_13 = l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8(x_12, x_5, x_6, x_7); -return x_13; } default: { -lean_object* x_14; lean_object* x_15; +lean_object* x_110; lean_object* x_111; 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_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; +x_110 = lean_box(0); +x_111 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_111, 0, x_110); +lean_ctor_set(x_111, 1, x_7); +return x_111; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___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: +{ +uint8_t x_7; lean_object* x_8; lean_object* x_9; +x_7 = 1; +x_8 = lean_box(x_7); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_6); +return x_9; +} +} +static lean_object* _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2___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_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___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; lean_object* x_11; lean_object* x_12; +x_9 = lean_box(0); +x_10 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; +x_11 = l_List_filterMapTR_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__1(x_5, x_10); +x_12 = l_List_filterMapTR_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__2(x_11, x_10); +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_13; uint8_t x_14; uint8_t x_15; +x_13 = lean_ctor_get(x_1, 0); +x_14 = 0; +x_15 = l_Lean_Elab_Info_contains(x_3, x_13, x_14); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +lean_dec(x_3); +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_8); +return x_17; } +else +{ +lean_object* x_18; uint8_t x_19; uint8_t x_20; +x_18 = lean_ctor_get(x_1, 1); +x_19 = 1; +x_20 = l_Lean_Elab_Info_contains(x_3, x_18, x_19); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; +lean_dec(x_3); +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_8); +return x_22; } else { -switch (lean_obj_tag(x_4)) { -case 0: +if (lean_obj_tag(x_3) == 3) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_4, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_4, 1); -lean_inc(x_17); -lean_dec(x_4); -x_18 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_16, x_3); -x_3 = x_18; -x_4 = x_17; -goto _start; +uint8_t x_23; +x_23 = !lean_is_exclusive(x_3); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_3, 0); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_9); +lean_ctor_set_tag(x_3, 1); +lean_ctor_set(x_3, 0, x_25); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_3); +lean_ctor_set(x_26, 1, x_8); +return x_26; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_27 = lean_ctor_get(x_3, 0); +lean_inc(x_27); +lean_dec(x_3); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_9); +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_8); +return x_30; } -case 1: -{ -uint8_t x_20; -x_20 = !lean_is_exclusive(x_3); -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_3, 0); -x_22 = lean_ctor_get(x_4, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_4, 1); -lean_inc(x_23); -lean_dec(x_4); -lean_inc(x_1); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_23); -lean_inc(x_22); -lean_inc(x_21); -x_24 = lean_apply_6(x_1, x_21, x_22, x_23, x_5, x_6, x_7); -if (lean_obj_tag(x_24) == 0) +} +else { -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, 1); -lean_inc(x_25); -lean_dec(x_24); -lean_inc(x_21); -x_26 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_22); -x_27 = l_Lean_PersistentArray_toList___rarg(x_23); -x_28 = lean_box(0); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_2); -x_29 = l_List_mapM_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__9(x_1, x_2, x_26, x_27, x_28, x_5, x_6, x_25); -if (lean_obj_tag(x_29) == 0) +lean_object* x_31; lean_object* x_32; +lean_dec(x_3); +x_31 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2___closed__1; +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_8); +return x_32; +} +} +} +} +else { -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 = lean_apply_7(x_2, x_21, x_22, x_23, x_30, x_5, x_6, x_31); -if (lean_obj_tag(x_32) == 0) +switch (lean_obj_tag(x_3)) { +case 1: { uint8_t x_33; -x_33 = !lean_is_exclusive(x_32); +x_33 = !lean_is_exclusive(x_3); if (x_33 == 0) { -lean_object* x_34; lean_object* x_35; -x_34 = lean_ctor_get(x_32, 0); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_32, 0, x_35); -return x_32; +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_3, 0); +lean_dec(x_34); +x_35 = lean_ctor_get(x_12, 0); +lean_inc(x_35); +lean_dec(x_12); +lean_ctor_set(x_3, 0, x_35); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_3); +lean_ctor_set(x_36, 1, x_8); +return x_36; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_36 = lean_ctor_get(x_32, 0); -x_37 = lean_ctor_get(x_32, 1); +lean_object* x_37; lean_object* x_38; lean_object* x_39; +lean_dec(x_3); +x_37 = lean_ctor_get(x_12, 0); lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_32); +lean_dec(x_12); x_38 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 0, x_37); x_39 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_37); +lean_ctor_set(x_39, 1, x_8); return x_39; } } -else +case 3: { uint8_t x_40; -x_40 = !lean_is_exclusive(x_32); +x_40 = !lean_is_exclusive(x_12); if (x_40 == 0) { -return x_32; +lean_object* x_41; lean_object* x_42; uint8_t x_43; +x_41 = lean_ctor_get(x_12, 0); +x_42 = lean_ctor_get(x_12, 1); +lean_dec(x_42); +x_43 = !lean_is_exclusive(x_3); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; +x_44 = lean_ctor_get(x_3, 0); +lean_ctor_set(x_12, 1, x_41); +lean_ctor_set(x_12, 0, x_44); +lean_ctor_set_tag(x_3, 1); +lean_ctor_set(x_3, 0, x_12); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_3); +lean_ctor_set(x_45, 1, x_8); +return x_45; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_32, 0); -x_42 = lean_ctor_get(x_32, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_32); -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_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_3, 0); +lean_inc(x_46); +lean_dec(x_3); +lean_ctor_set(x_12, 1, x_41); +lean_ctor_set(x_12, 0, x_46); +x_47 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_47, 0, x_12); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_8); +return x_48; } } else { -uint8_t x_44; -lean_dec(x_23); -lean_dec(x_22); -lean_dec(x_21); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_2); -x_44 = !lean_is_exclusive(x_29); -if (x_44 == 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; +x_49 = lean_ctor_get(x_12, 0); +lean_inc(x_49); +lean_dec(x_12); +x_50 = lean_ctor_get(x_3, 0); +lean_inc(x_50); +if (lean_is_exclusive(x_3)) { + lean_ctor_release(x_3, 0); + x_51 = x_3; +} else { + lean_dec_ref(x_3); + 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_49); +if (lean_is_scalar(x_51)) { + x_53 = lean_alloc_ctor(1, 1, 0); +} else { + x_53 = x_51; + lean_ctor_set_tag(x_53, 1); +} +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_8); +return x_54; +} +} +default: { -return x_29; +uint8_t x_55; +x_55 = !lean_is_exclusive(x_3); +if (x_55 == 0) +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_56 = lean_ctor_get(x_3, 0); +lean_dec(x_56); +x_57 = lean_ctor_get(x_12, 0); +lean_inc(x_57); +lean_dec(x_12); +lean_ctor_set_tag(x_3, 1); +lean_ctor_set(x_3, 0, x_57); +x_58 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_58, 0, x_3); +lean_ctor_set(x_58, 1, x_8); +return x_58; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_29, 0); -x_46 = lean_ctor_get(x_29, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_29); -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_59; lean_object* x_60; lean_object* x_61; +lean_dec(x_3); +x_59 = lean_ctor_get(x_12, 0); +lean_inc(x_59); +lean_dec(x_12); +x_60 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_60, 0, x_59); +x_61 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_61, 0, x_60); +lean_ctor_set(x_61, 1, x_8); +return x_61; +} +} +} +} +} +} +static lean_object* _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__1___boxed), 6, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6(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; +x_6 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2___boxed), 8, 1); +lean_closure_set(x_6, 0, x_1); +x_7 = lean_box(0); +x_8 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___closed__1; +x_9 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__7(x_8, x_6, x_7, x_2, x_3, x_4, x_5); +return x_9; } } +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5(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_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6(x_1, x_2, x_3, x_4, x_5); +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_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_6, 0); +lean_dec(x_9); +x_10 = lean_box(0); +lean_ctor_set(x_6, 0, x_10); +return x_6; } else { -uint8_t x_48; -lean_dec(x_23); -lean_dec(x_22); -lean_free_object(x_3); -lean_dec(x_21); +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); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_48 = !lean_is_exclusive(x_24); -if (x_48 == 0) +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 { -return x_24; +lean_object* x_14; +x_14 = lean_ctor_get(x_7, 0); +lean_inc(x_14); +lean_dec(x_7); +if (lean_obj_tag(x_14) == 0) +{ +uint8_t x_15; +x_15 = !lean_is_exclusive(x_6); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_6, 0); +lean_dec(x_16); +x_17 = lean_box(0); +lean_ctor_set(x_6, 0, x_17); +return x_6; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_24, 0); -x_50 = lean_ctor_get(x_24, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_24); -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_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_6, 1); +lean_inc(x_18); +lean_dec(x_6); +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_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_52 = lean_ctor_get(x_3, 0); -lean_inc(x_52); -lean_dec(x_3); -x_53 = lean_ctor_get(x_4, 0); -lean_inc(x_53); -x_54 = lean_ctor_get(x_4, 1); -lean_inc(x_54); -lean_dec(x_4); -lean_inc(x_1); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_54); -lean_inc(x_53); -lean_inc(x_52); -x_55 = lean_apply_6(x_1, x_52, x_53, x_54, x_5, x_6, x_7); -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; lean_object* x_61; -x_56 = lean_ctor_get(x_55, 1); -lean_inc(x_56); -lean_dec(x_55); -lean_inc(x_52); -x_57 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_57, 0, x_52); -x_58 = l_Lean_Elab_Info_updateContext_x3f(x_57, x_53); -x_59 = l_Lean_PersistentArray_toList___rarg(x_54); -x_60 = lean_box(0); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_2); -x_61 = l_List_mapM_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__9(x_1, x_2, x_58, x_59, x_60, x_5, x_6, x_56); -if (lean_obj_tag(x_61) == 0) +uint8_t x_21; +x_21 = !lean_is_exclusive(x_6); +if (x_21 == 0) { -lean_object* x_62; lean_object* x_63; lean_object* x_64; -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_apply_7(x_2, x_52, x_53, x_54, x_62, x_5, x_6, x_63); -if (lean_obj_tag(x_64) == 0) +lean_object* x_22; uint8_t x_23; +x_22 = lean_ctor_get(x_6, 0); +lean_dec(x_22); +x_23 = !lean_is_exclusive(x_14); +if (x_23 == 0) { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -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); -} -x_68 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_68, 0, x_65); -if (lean_is_scalar(x_67)) { - x_69 = lean_alloc_ctor(0, 2, 0); -} else { - x_69 = x_67; -} -lean_ctor_set(x_69, 0, x_68); -lean_ctor_set(x_69, 1, x_66); -return x_69; +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_14, 0); +x_25 = l_List_reverse___rarg(x_24); +lean_ctor_set(x_14, 0, x_25); +lean_ctor_set(x_6, 0, x_14); +return x_6; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_70 = lean_ctor_get(x_64, 0); -lean_inc(x_70); -x_71 = lean_ctor_get(x_64, 1); -lean_inc(x_71); -if (lean_is_exclusive(x_64)) { - lean_ctor_release(x_64, 0); - lean_ctor_release(x_64, 1); - x_72 = x_64; -} else { - lean_dec_ref(x_64); - x_72 = lean_box(0); -} -if (lean_is_scalar(x_72)) { - x_73 = lean_alloc_ctor(1, 2, 0); -} else { - x_73 = x_72; -} -lean_ctor_set(x_73, 0, x_70); -lean_ctor_set(x_73, 1, x_71); -return x_73; +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_14, 0); +lean_inc(x_26); +lean_dec(x_14); +x_27 = l_List_reverse___rarg(x_26); +x_28 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_6, 0, x_28); +return x_6; } } else { -lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -lean_dec(x_54); -lean_dec(x_53); -lean_dec(x_52); +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_6, 1); +lean_inc(x_29); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_2); -x_74 = lean_ctor_get(x_61, 0); -lean_inc(x_74); -x_75 = lean_ctor_get(x_61, 1); -lean_inc(x_75); -if (lean_is_exclusive(x_61)) { - lean_ctor_release(x_61, 0); - lean_ctor_release(x_61, 1); - x_76 = x_61; +x_30 = lean_ctor_get(x_14, 0); +lean_inc(x_30); +if (lean_is_exclusive(x_14)) { + lean_ctor_release(x_14, 0); + x_31 = x_14; } else { - lean_dec_ref(x_61); - x_76 = lean_box(0); + lean_dec_ref(x_14); + x_31 = lean_box(0); } -if (lean_is_scalar(x_76)) { - x_77 = lean_alloc_ctor(1, 2, 0); +x_32 = l_List_reverse___rarg(x_30); +if (lean_is_scalar(x_31)) { + x_33 = lean_alloc_ctor(1, 1, 0); } else { - x_77 = x_76; -} -lean_ctor_set(x_77, 0, x_74); -lean_ctor_set(x_77, 1, x_75); -return x_77; -} + x_33 = x_31; } -else -{ -lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -lean_dec(x_54); -lean_dec(x_53); -lean_dec(x_52); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_78 = lean_ctor_get(x_55, 0); -lean_inc(x_78); -x_79 = lean_ctor_get(x_55, 1); -lean_inc(x_79); -if (lean_is_exclusive(x_55)) { - lean_ctor_release(x_55, 0); - lean_ctor_release(x_55, 1); - x_80 = x_55; -} else { - lean_dec_ref(x_55); - x_80 = lean_box(0); +lean_ctor_set(x_33, 0, 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_29); +return x_34; } -if (lean_is_scalar(x_80)) { - x_81 = lean_alloc_ctor(1, 2, 0); -} else { - x_81 = x_80; } -lean_ctor_set(x_81, 0, x_78); -lean_ctor_set(x_81, 1, x_79); -return x_81; } } +else +{ +uint8_t x_35; +x_35 = !lean_is_exclusive(x_6); +if (x_35 == 0) +{ +return x_6; } -default: +else { -lean_object* x_82; lean_object* x_83; +lean_object* x_36; lean_object* x_37; lean_object* x_38; +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); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_82 = lean_box(0); -x_83 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_83, 0, x_82); -lean_ctor_set(x_83, 1, x_7); -return x_83; -} +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_Lean_Elab_InfoTree_visitM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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) { _start: { -lean_object* x_7; lean_object* x_8; -x_7 = lean_box(0); -x_8 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__7(x_1, x_2, x_7, x_3, x_4, x_5, x_6); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___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: +uint8_t x_7; +x_7 = lean_usize_dec_eq(x_5, x_6); +if (x_7 == 0) { -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_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2___closed__1() { -_start: +lean_object* x_8; lean_object* x_9; uint8_t x_10; +x_8 = lean_array_uget(x_4, x_5); +lean_inc(x_2); +lean_inc(x_3); +lean_inc(x_1); +x_9 = lean_apply_3(x_8, x_1, x_3, x_2); +x_10 = lean_unbox(x_9); +lean_dec(x_9); +if (x_10 == 0) { -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; -} +size_t x_11; size_t x_12; +x_11 = 1; +x_12 = lean_usize_add(x_5, x_11); +x_5 = x_12; +goto _start; } -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___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; lean_object* x_11; lean_object* x_12; -x_9 = lean_box(0); -x_10 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1; -x_11 = l_List_filterMapTR_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__1(x_5, x_10); -x_12 = l_List_filterMapTR_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__2(x_11, x_10); -if (lean_obj_tag(x_12) == 0) -{ -lean_object* x_13; uint8_t x_14; uint8_t x_15; -x_13 = lean_ctor_get(x_1, 0); -x_14 = 0; -x_15 = l_Lean_Elab_Info_contains(x_3, x_13, x_14); -if (x_15 == 0) +else { -lean_object* x_16; lean_object* x_17; +uint8_t x_14; lean_dec(x_3); -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_8); -return x_17; +lean_dec(x_2); +lean_dec(x_1); +x_14 = 1; +return x_14; +} } else { -lean_object* x_18; uint8_t x_19; uint8_t x_20; -x_18 = lean_ctor_get(x_1, 1); -x_19 = 1; -x_20 = l_Lean_Elab_Info_contains(x_3, x_18, x_19); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; +uint8_t x_15; lean_dec(x_3); -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_8); -return x_22; +lean_dec(x_2); +lean_dec(x_1); +x_15 = 0; +return x_15; } -else +} +} +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(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_3) == 3) +uint8_t x_7; +x_7 = lean_usize_dec_eq(x_5, x_6); +if (x_7 == 0) { -uint8_t x_23; -x_23 = !lean_is_exclusive(x_3); -if (x_23 == 0) +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_25; lean_object* x_26; uint64_t x_27; uint64_t x_28; uint64_t x_29; uint64_t x_30; uint64_t x_31; size_t x_32; size_t x_33; size_t x_34; size_t x_35; lean_object* x_36; uint8_t x_37; +x_8 = lean_array_uget(x_4, x_5); +x_9 = lean_ctor_get(x_2, 1); +x_10 = lean_array_get_size(x_9); +x_11 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_8); +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_10); +lean_dec(x_10); +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_9, x_22); +x_24 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(x_8, x_8, x_23); +lean_dec(x_23); +lean_dec(x_8); +x_25 = lean_ctor_get(x_3, 1); +x_26 = lean_array_get_size(x_25); +x_27 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_24); +x_28 = lean_uint64_shift_right(x_27, x_12); +x_29 = lean_uint64_xor(x_27, x_28); +x_30 = lean_uint64_shift_right(x_29, x_15); +x_31 = lean_uint64_xor(x_29, x_30); +x_32 = lean_uint64_to_usize(x_31); +x_33 = lean_usize_of_nat(x_26); +lean_dec(x_26); +x_34 = lean_usize_sub(x_33, x_20); +x_35 = lean_usize_land(x_32, x_34); +x_36 = lean_array_uget(x_25, x_35); +x_37 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_24, x_36); +lean_dec(x_36); +lean_dec(x_24); +if (x_37 == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_3, 0); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_9); -lean_ctor_set_tag(x_3, 1); -lean_ctor_set(x_3, 0, x_25); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_3); -lean_ctor_set(x_26, 1, x_8); -return x_26; +size_t x_38; +x_38 = lean_usize_add(x_5, x_20); +x_5 = x_38; +goto _start; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_27 = lean_ctor_get(x_3, 0); -lean_inc(x_27); -lean_dec(x_3); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_9); -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_8); -return x_30; +uint8_t x_40; +x_40 = 1; +return x_40; } } else { -lean_object* x_31; lean_object* x_32; -lean_dec(x_3); -x_31 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2___closed__1; -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_8); -return x_32; -} +uint8_t x_41; +x_41 = 0; +return x_41; } } } -else -{ -switch (lean_obj_tag(x_3)) { -case 1: +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__12(lean_object* x_1, lean_object* x_2) { +_start: { -uint8_t x_33; -x_33 = !lean_is_exclusive(x_3); -if (x_33 == 0) +if (lean_obj_tag(x_2) == 0) { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_3, 0); -lean_dec(x_34); -x_35 = lean_ctor_get(x_12, 0); -lean_inc(x_35); -lean_dec(x_12); -lean_ctor_set(x_3, 0, x_35); -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_3); -lean_ctor_set(x_36, 1, x_8); -return x_36; +return x_1; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -lean_dec(x_3); -x_37 = lean_ctor_get(x_12, 0); -lean_inc(x_37); -lean_dec(x_12); -x_38 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_38, 0, x_37); -x_39 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_8); -return x_39; +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, 2); +lean_inc(x_4); +lean_dec(x_2); +x_5 = lean_array_push(x_1, x_3); +x_1 = x_5; +x_2 = x_4; +goto _start; } } -case 3: -{ -uint8_t x_40; -x_40 = !lean_is_exclusive(x_12); -if (x_40 == 0) +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: { -lean_object* x_41; lean_object* x_42; uint8_t x_43; -x_41 = lean_ctor_get(x_12, 0); -x_42 = lean_ctor_get(x_12, 1); -lean_dec(x_42); -x_43 = !lean_is_exclusive(x_3); -if (x_43 == 0) +if (lean_obj_tag(x_3) == 0) { -lean_object* x_44; lean_object* x_45; -x_44 = lean_ctor_get(x_3, 0); -lean_ctor_set(x_12, 1, x_41); -lean_ctor_set(x_12, 0, x_44); -lean_ctor_set_tag(x_3, 1); -lean_ctor_set(x_3, 0, x_12); -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_3); -lean_ctor_set(x_45, 1, x_8); -return x_45; +lean_object* x_4; +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(0); +return x_4; } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_46 = lean_ctor_get(x_3, 0); -lean_inc(x_46); -lean_dec(x_3); -lean_ctor_set(x_12, 1, x_41); -lean_ctor_set(x_12, 0, x_46); -x_47 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_47, 0, x_12); -x_48 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_48, 0, x_47); -lean_ctor_set(x_48, 1, x_8); -return x_48; -} +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_name_eq(x_6, x_1); +if (x_9 == 0) +{ +lean_object* x_10; +x_10 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_1, x_2, x_8); +lean_ctor_set(x_3, 2, x_10); +return x_3; } 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; -x_49 = lean_ctor_get(x_12, 0); -lean_inc(x_49); -lean_dec(x_12); -x_50 = lean_ctor_get(x_3, 0); -lean_inc(x_50); -if (lean_is_exclusive(x_3)) { - lean_ctor_release(x_3, 0); - x_51 = x_3; -} else { - lean_dec_ref(x_3); - 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_49); -if (lean_is_scalar(x_51)) { - x_53 = lean_alloc_ctor(1, 1, 0); -} else { - x_53 = x_51; - lean_ctor_set_tag(x_53, 1); -} -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_8); -return x_54; +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; } } -default: +else { -uint8_t x_55; -x_55 = !lean_is_exclusive(x_3); -if (x_55 == 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 = lean_name_eq(x_11, x_1); +if (x_14 == 0) { -lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_56 = lean_ctor_get(x_3, 0); -lean_dec(x_56); -x_57 = lean_ctor_get(x_12, 0); -lean_inc(x_57); -lean_dec(x_12); -lean_ctor_set_tag(x_3, 1); -lean_ctor_set(x_3, 0, x_57); -x_58 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_58, 0, x_3); -lean_ctor_set(x_58, 1, x_8); -return x_58; +lean_object* x_15; lean_object* x_16; +x_15 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(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_59; lean_object* x_60; lean_object* x_61; -lean_dec(x_3); -x_59 = lean_ctor_get(x_12, 0); -lean_inc(x_59); +lean_object* x_17; lean_dec(x_12); -x_60 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_60, 0, x_59); -x_61 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_61, 0, x_60); -lean_ctor_set(x_61, 1, x_8); -return x_61; -} +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; } } } } } -static lean_object* _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___closed__1() { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__1___boxed), 6, 0); -return x_1; +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; lean_object* x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; size_t 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_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_ctor_get(x_1, 1); +x_12 = lean_array_get_size(x_11); +x_13 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_6); +x_14 = 32; +x_15 = lean_uint64_shift_right(x_13, x_14); +x_16 = lean_uint64_xor(x_13, x_15); +x_17 = 16; +x_18 = lean_uint64_shift_right(x_16, x_17); +x_19 = lean_uint64_xor(x_16, x_18); +x_20 = lean_uint64_to_usize(x_19); +x_21 = lean_usize_of_nat(x_12); +lean_dec(x_12); +x_22 = lean_usize_sub(x_21, x_9); +x_23 = lean_usize_land(x_20, x_22); +x_24 = lean_array_uget(x_11, x_23); +x_25 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(x_6, x_6, x_24); +lean_dec(x_24); +lean_dec(x_6); +x_26 = lean_array_uset(x_8, x_3, x_25); +x_3 = x_10; +x_4 = x_26; +goto _start; } -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5(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; -x_6 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2___boxed), 8, 1); -lean_closure_set(x_6, 0, x_1); -x_7 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___closed__1; -x_8 = l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6(x_7, x_6, x_2, x_3, x_4, x_5); -return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4(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_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { _start: { -lean_object* x_6; -x_6 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5(x_1, x_2, x_3, x_4, x_5); -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_8; -x_8 = !lean_is_exclusive(x_6); -if (x_8 == 0) +uint8_t x_7; +x_7 = lean_usize_dec_lt(x_5, x_4); +if (x_7 == 0) { -lean_object* x_9; lean_object* x_10; -x_9 = lean_ctor_get(x_6, 0); -lean_dec(x_9); -x_10 = lean_box(0); -lean_ctor_set(x_6, 0, x_10); +lean_dec(x_1); return x_6; } else { -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 = 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_8; uint8_t x_9; +x_8 = lean_array_uget(x_3, x_5); +x_9 = !lean_is_exclusive(x_6); +if (x_9 == 0) { -lean_object* x_14; -x_14 = lean_ctor_get(x_7, 0); -lean_inc(x_14); -lean_dec(x_7); -if (lean_obj_tag(x_14) == 0) +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; size_t x_20; size_t x_21; size_t x_22; size_t x_23; size_t x_24; lean_object* x_25; uint8_t x_26; +x_10 = lean_ctor_get(x_6, 0); +x_11 = lean_ctor_get(x_6, 1); +x_12 = lean_array_get_size(x_11); +x_13 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_8); +x_14 = 32; +x_15 = lean_uint64_shift_right(x_13, x_14); +x_16 = lean_uint64_xor(x_13, x_15); +x_17 = 16; +x_18 = lean_uint64_shift_right(x_16, x_17); +x_19 = lean_uint64_xor(x_16, x_18); +x_20 = lean_uint64_to_usize(x_19); +x_21 = lean_usize_of_nat(x_12); +lean_dec(x_12); +x_22 = 1; +x_23 = lean_usize_sub(x_21, x_22); +x_24 = lean_usize_land(x_20, x_23); +x_25 = lean_array_uget(x_11, x_24); +x_26 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_8, x_25); +if (x_26 == 0) { -uint8_t x_15; -x_15 = !lean_is_exclusive(x_6); -if (x_15 == 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; uint8_t x_37; +x_27 = lean_unsigned_to_nat(1u); +x_28 = lean_nat_add(x_10, x_27); +lean_dec(x_10); +x_29 = lean_box(0); +x_30 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_30, 0, x_8); +lean_ctor_set(x_30, 1, x_29); +lean_ctor_set(x_30, 2, x_25); +x_31 = lean_array_uset(x_11, x_24, x_30); +x_32 = lean_unsigned_to_nat(4u); +x_33 = lean_nat_mul(x_28, x_32); +x_34 = lean_unsigned_to_nat(3u); +x_35 = lean_nat_div(x_33, x_34); +lean_dec(x_33); +x_36 = lean_array_get_size(x_31); +x_37 = lean_nat_dec_le(x_35, x_36); +lean_dec(x_36); +lean_dec(x_35); +if (x_37 == 0) { -lean_object* x_16; lean_object* x_17; -x_16 = lean_ctor_get(x_6, 0); -lean_dec(x_16); -x_17 = lean_box(0); -lean_ctor_set(x_6, 0, x_17); -return x_6; +lean_object* x_38; size_t x_39; +x_38 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_31); +lean_ctor_set(x_6, 1, x_38); +lean_ctor_set(x_6, 0, x_28); +x_39 = lean_usize_add(x_5, x_22); +x_5 = x_39; +goto _start; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_6, 1); -lean_inc(x_18); -lean_dec(x_6); -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; +size_t x_41; +lean_ctor_set(x_6, 1, x_31); +lean_ctor_set(x_6, 0, x_28); +x_41 = lean_usize_add(x_5, x_22); +x_5 = x_41; +goto _start; } } else { -uint8_t x_21; -x_21 = !lean_is_exclusive(x_6); -if (x_21 == 0) +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; size_t x_47; +lean_inc(x_1); +x_43 = lean_array_uset(x_11, x_24, x_1); +x_44 = lean_box(0); +x_45 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_8, x_44, x_25); +x_46 = lean_array_uset(x_43, x_24, x_45); +lean_ctor_set(x_6, 1, x_46); +x_47 = lean_usize_add(x_5, x_22); +x_5 = x_47; +goto _start; +} +} +else { -lean_object* x_22; uint8_t x_23; -x_22 = lean_ctor_get(x_6, 0); -lean_dec(x_22); -x_23 = !lean_is_exclusive(x_14); -if (x_23 == 0) +lean_object* x_49; lean_object* x_50; lean_object* x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; uint64_t x_55; uint64_t x_56; uint64_t x_57; uint64_t x_58; size_t x_59; size_t x_60; size_t x_61; size_t x_62; size_t x_63; lean_object* x_64; uint8_t x_65; +x_49 = lean_ctor_get(x_6, 0); +x_50 = lean_ctor_get(x_6, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_6); +x_51 = lean_array_get_size(x_50); +x_52 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_8); +x_53 = 32; +x_54 = lean_uint64_shift_right(x_52, x_53); +x_55 = lean_uint64_xor(x_52, x_54); +x_56 = 16; +x_57 = lean_uint64_shift_right(x_55, x_56); +x_58 = lean_uint64_xor(x_55, x_57); +x_59 = lean_uint64_to_usize(x_58); +x_60 = lean_usize_of_nat(x_51); +lean_dec(x_51); +x_61 = 1; +x_62 = lean_usize_sub(x_60, x_61); +x_63 = lean_usize_land(x_59, x_62); +x_64 = lean_array_uget(x_50, x_63); +x_65 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_8, 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; lean_object* x_74; lean_object* x_75; uint8_t x_76; +x_66 = lean_unsigned_to_nat(1u); +x_67 = lean_nat_add(x_49, x_66); +lean_dec(x_49); +x_68 = lean_box(0); +x_69 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_69, 0, x_8); +lean_ctor_set(x_69, 1, x_68); +lean_ctor_set(x_69, 2, x_64); +x_70 = lean_array_uset(x_50, x_63, x_69); +x_71 = lean_unsigned_to_nat(4u); +x_72 = lean_nat_mul(x_67, x_71); +x_73 = lean_unsigned_to_nat(3u); +x_74 = lean_nat_div(x_72, x_73); +lean_dec(x_72); +x_75 = lean_array_get_size(x_70); +x_76 = lean_nat_dec_le(x_74, x_75); +lean_dec(x_75); +lean_dec(x_74); +if (x_76 == 0) { -lean_object* x_24; lean_object* x_25; -x_24 = lean_ctor_get(x_14, 0); -x_25 = l_List_reverse___rarg(x_24); -lean_ctor_set(x_14, 0, x_25); -lean_ctor_set(x_6, 0, x_14); -return x_6; +lean_object* x_77; lean_object* x_78; size_t x_79; +x_77 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_70); +x_78 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_78, 0, x_67); +lean_ctor_set(x_78, 1, x_77); +x_79 = lean_usize_add(x_5, x_61); +x_5 = x_79; +x_6 = x_78; +goto _start; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_14, 0); -lean_inc(x_26); -lean_dec(x_14); -x_27 = l_List_reverse___rarg(x_26); -x_28 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_6, 0, x_28); -return x_6; +lean_object* x_81; size_t x_82; +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_67); +lean_ctor_set(x_81, 1, x_70); +x_82 = lean_usize_add(x_5, x_61); +x_5 = x_82; +x_6 = x_81; +goto _start; } } 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_6, 1); -lean_inc(x_29); -lean_dec(x_6); -x_30 = lean_ctor_get(x_14, 0); -lean_inc(x_30); -if (lean_is_exclusive(x_14)) { - lean_ctor_release(x_14, 0); - x_31 = x_14; -} else { - lean_dec_ref(x_14); - x_31 = lean_box(0); -} -x_32 = l_List_reverse___rarg(x_30); -if (lean_is_scalar(x_31)) { - x_33 = lean_alloc_ctor(1, 1, 0); -} else { - x_33 = x_31; +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; size_t x_89; +lean_inc(x_1); +x_84 = lean_array_uset(x_50, x_63, x_1); +x_85 = lean_box(0); +x_86 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_8, x_85, x_64); +x_87 = lean_array_uset(x_84, x_63, x_86); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_49); +lean_ctor_set(x_88, 1, x_87); +x_89 = lean_usize_add(x_5, x_61); +x_5 = x_89; +x_6 = x_88; +goto _start; } -lean_ctor_set(x_33, 0, 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_29); -return x_34; } } } } -else +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: { -uint8_t x_35; -x_35 = !lean_is_exclusive(x_6); -if (x_35 == 0) +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) { -return x_6; +return x_4; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -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_object* 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; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; size_t 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_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_ctor_get(x_1, 1); +x_12 = lean_array_get_size(x_11); +x_13 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_6); +x_14 = 32; +x_15 = lean_uint64_shift_right(x_13, x_14); +x_16 = lean_uint64_xor(x_13, x_15); +x_17 = 16; +x_18 = lean_uint64_shift_right(x_16, x_17); +x_19 = lean_uint64_xor(x_16, x_18); +x_20 = lean_uint64_to_usize(x_19); +x_21 = lean_usize_of_nat(x_12); +lean_dec(x_12); +x_22 = lean_usize_sub(x_21, x_9); +x_23 = lean_usize_land(x_20, x_22); +x_24 = lean_array_uget(x_11, x_23); +x_25 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(x_6, x_6, x_24); +lean_dec(x_24); lean_dec(x_6); -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; -} +x_26 = lean_array_uset(x_8, x_3, x_25); +x_3 = x_10; +x_4 = x_26; +goto _start; } } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { _start: { uint8_t x_7; -x_7 = lean_usize_dec_eq(x_5, x_6); +x_7 = lean_usize_dec_lt(x_5, x_4); if (x_7 == 0) { -lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_8 = lean_array_uget(x_4, x_5); -lean_inc(x_2); -lean_inc(x_3); -lean_inc(x_1); -x_9 = lean_apply_3(x_8, x_1, x_3, x_2); -x_10 = lean_unbox(x_9); -lean_dec(x_9); -if (x_10 == 0) +lean_dec(x_1); +return x_6; +} +else +{ +lean_object* x_8; uint8_t x_9; +x_8 = lean_array_uget(x_3, x_5); +x_9 = !lean_is_exclusive(x_6); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; size_t x_20; size_t x_21; size_t x_22; size_t x_23; size_t x_24; lean_object* x_25; uint8_t x_26; +x_10 = lean_ctor_get(x_6, 0); +x_11 = lean_ctor_get(x_6, 1); +x_12 = lean_array_get_size(x_11); +x_13 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_8); +x_14 = 32; +x_15 = lean_uint64_shift_right(x_13, x_14); +x_16 = lean_uint64_xor(x_13, x_15); +x_17 = 16; +x_18 = lean_uint64_shift_right(x_16, x_17); +x_19 = lean_uint64_xor(x_16, x_18); +x_20 = lean_uint64_to_usize(x_19); +x_21 = lean_usize_of_nat(x_12); +lean_dec(x_12); +x_22 = 1; +x_23 = lean_usize_sub(x_21, x_22); +x_24 = lean_usize_land(x_20, x_23); +x_25 = lean_array_uget(x_11, x_24); +x_26 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_8, 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; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_27 = lean_unsigned_to_nat(1u); +x_28 = lean_nat_add(x_10, x_27); +lean_dec(x_10); +x_29 = lean_box(0); +x_30 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_30, 0, x_8); +lean_ctor_set(x_30, 1, x_29); +lean_ctor_set(x_30, 2, x_25); +x_31 = lean_array_uset(x_11, x_24, x_30); +x_32 = lean_unsigned_to_nat(4u); +x_33 = lean_nat_mul(x_28, x_32); +x_34 = lean_unsigned_to_nat(3u); +x_35 = lean_nat_div(x_33, x_34); +lean_dec(x_33); +x_36 = lean_array_get_size(x_31); +x_37 = lean_nat_dec_le(x_35, x_36); +lean_dec(x_36); +lean_dec(x_35); +if (x_37 == 0) { -size_t x_11; size_t x_12; -x_11 = 1; -x_12 = lean_usize_add(x_5, x_11); -x_5 = x_12; +lean_object* x_38; size_t x_39; +x_38 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_31); +lean_ctor_set(x_6, 1, x_38); +lean_ctor_set(x_6, 0, x_28); +x_39 = lean_usize_add(x_5, x_22); +x_5 = x_39; goto _start; } else { -uint8_t x_14; -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_14 = 1; -return x_14; +size_t x_41; +lean_ctor_set(x_6, 1, x_31); +lean_ctor_set(x_6, 0, x_28); +x_41 = lean_usize_add(x_5, x_22); +x_5 = x_41; +goto _start; } } else { -uint8_t x_15; -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_15 = 0; -return x_15; -} +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; size_t x_47; +lean_inc(x_1); +x_43 = lean_array_uset(x_11, x_24, x_1); +x_44 = lean_box(0); +x_45 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_8, x_44, x_25); +x_46 = lean_array_uset(x_43, x_24, x_45); +lean_ctor_set(x_6, 1, x_46); +x_47 = lean_usize_add(x_5, x_22); +x_5 = x_47; +goto _start; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -if (lean_obj_tag(x_3) == 0) +lean_object* x_49; lean_object* x_50; lean_object* x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; uint64_t x_55; uint64_t x_56; uint64_t x_57; uint64_t x_58; size_t x_59; size_t x_60; size_t x_61; size_t x_62; size_t x_63; lean_object* x_64; uint8_t x_65; +x_49 = lean_ctor_get(x_6, 0); +x_50 = lean_ctor_get(x_6, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_6); +x_51 = lean_array_get_size(x_50); +x_52 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_8); +x_53 = 32; +x_54 = lean_uint64_shift_right(x_52, x_53); +x_55 = lean_uint64_xor(x_52, x_54); +x_56 = 16; +x_57 = lean_uint64_shift_right(x_55, x_56); +x_58 = lean_uint64_xor(x_55, x_57); +x_59 = lean_uint64_to_usize(x_58); +x_60 = lean_usize_of_nat(x_51); +lean_dec(x_51); +x_61 = 1; +x_62 = lean_usize_sub(x_60, x_61); +x_63 = lean_usize_land(x_59, x_62); +x_64 = lean_array_uget(x_50, x_63); +x_65 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_8, 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; lean_object* x_74; lean_object* x_75; uint8_t x_76; +x_66 = lean_unsigned_to_nat(1u); +x_67 = lean_nat_add(x_49, x_66); +lean_dec(x_49); +x_68 = lean_box(0); +x_69 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_69, 0, x_8); +lean_ctor_set(x_69, 1, x_68); +lean_ctor_set(x_69, 2, x_64); +x_70 = lean_array_uset(x_50, x_63, x_69); +x_71 = lean_unsigned_to_nat(4u); +x_72 = lean_nat_mul(x_67, x_71); +x_73 = lean_unsigned_to_nat(3u); +x_74 = lean_nat_div(x_72, x_73); +lean_dec(x_72); +x_75 = lean_array_get_size(x_70); +x_76 = lean_nat_dec_le(x_74, x_75); +lean_dec(x_75); +lean_dec(x_74); +if (x_76 == 0) { -lean_inc(x_2); -return x_2; +lean_object* x_77; lean_object* x_78; size_t x_79; +x_77 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_70); +x_78 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_78, 0, x_67); +lean_ctor_set(x_78, 1, x_77); +x_79 = lean_usize_add(x_5, x_61); +x_5 = x_79; +x_6 = x_78; +goto _start; } else { -lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; -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_name_eq(x_4, x_1); -if (x_7 == 0) -{ -x_3 = x_6; +lean_object* x_81; size_t x_82; +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_67); +lean_ctor_set(x_81, 1, x_70); +x_82 = lean_usize_add(x_5, x_61); +x_5 = x_82; +x_6 = x_81; goto _start; } +} else { -lean_inc(x_5); -return x_5; +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; size_t x_89; +lean_inc(x_1); +x_84 = lean_array_uset(x_50, x_63, x_1); +x_85 = lean_box(0); +x_86 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_8, x_85, x_64); +x_87 = lean_array_uset(x_84, x_63, x_86); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_49); +lean_ctor_set(x_88, 1, x_87); +x_89 = lean_usize_add(x_5, x_61); +x_5 = x_89; +x_6 = x_88; +goto _start; } } } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { -uint8_t x_7; -x_7 = lean_usize_dec_eq(x_5, x_6); -if (x_7 == 0) -{ -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_25; lean_object* x_26; uint64_t x_27; uint64_t x_28; uint64_t x_29; uint64_t x_30; uint64_t x_31; size_t x_32; size_t x_33; size_t x_34; size_t x_35; lean_object* x_36; uint8_t x_37; -x_8 = lean_array_uget(x_4, x_5); -x_9 = lean_ctor_get(x_2, 1); -x_10 = lean_array_get_size(x_9); -x_11 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_8); -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_10); -lean_dec(x_10); -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_9, x_22); -x_24 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(x_8, x_8, x_23); -lean_dec(x_23); -lean_dec(x_8); -x_25 = lean_ctor_get(x_3, 1); -x_26 = lean_array_get_size(x_25); -x_27 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_24); -x_28 = lean_uint64_shift_right(x_27, x_12); -x_29 = lean_uint64_xor(x_27, x_28); -x_30 = lean_uint64_shift_right(x_29, x_15); -x_31 = lean_uint64_xor(x_29, x_30); -x_32 = lean_uint64_to_usize(x_31); -x_33 = lean_usize_of_nat(x_26); -lean_dec(x_26); -x_34 = lean_usize_sub(x_33, x_20); -x_35 = lean_usize_land(x_32, x_34); -x_36 = lean_array_uget(x_25, x_35); -x_37 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_24, x_36); -lean_dec(x_36); -lean_dec(x_24); -if (x_37 == 0) +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_2, x_3); +if (x_5 == 0) { -size_t x_38; -x_38 = lean_usize_add(x_5, x_20); -x_5 = x_38; +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_Linter_UnusedVariables_unusedVariables___elambda__1___spec__12(x_4, 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 { -uint8_t x_40; -x_40 = 1; -return x_40; -} -} -else -{ -uint8_t x_41; -x_41 = 0; -return x_41; +return x_4; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(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_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { -if (lean_obj_tag(x_4) == 0) -{ -return x_3; -} -else -{ uint8_t x_5; -x_5 = !lean_is_exclusive(x_4); +x_5 = lean_usize_dec_lt(x_3, 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; 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; uint8_t x_25; -x_6 = lean_ctor_get(x_4, 0); -x_7 = lean_ctor_get(x_4, 2); -x_8 = lean_ctor_get(x_4, 1); -lean_dec(x_8); -x_9 = lean_ctor_get(x_2, 1); -x_10 = lean_array_get_size(x_9); -x_11 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_6); -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_10); -lean_dec(x_10); -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_9, x_22); -x_24 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(x_6, x_6, x_23); -lean_dec(x_23); -lean_dec(x_6); -x_25 = !lean_is_exclusive(x_3); -if (x_25 == 0) -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; uint64_t x_29; uint64_t x_30; uint64_t x_31; uint64_t x_32; uint64_t x_33; size_t x_34; size_t x_35; size_t x_36; size_t x_37; lean_object* x_38; uint8_t x_39; -x_26 = lean_ctor_get(x_3, 0); -x_27 = lean_ctor_get(x_3, 1); -x_28 = lean_array_get_size(x_27); -x_29 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_24); -x_30 = lean_uint64_shift_right(x_29, x_12); -x_31 = lean_uint64_xor(x_29, x_30); -x_32 = lean_uint64_shift_right(x_31, x_15); -x_33 = lean_uint64_xor(x_31, x_32); -x_34 = lean_uint64_to_usize(x_33); -x_35 = lean_usize_of_nat(x_28); -lean_dec(x_28); -x_36 = lean_usize_sub(x_35, x_20); -x_37 = lean_usize_land(x_34, x_36); -x_38 = lean_array_uget(x_27, x_37); -x_39 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_24, 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; -x_40 = lean_unsigned_to_nat(1u); -x_41 = lean_nat_add(x_26, x_40); -lean_dec(x_26); -x_42 = lean_box(0); -lean_ctor_set(x_4, 2, x_38); -lean_ctor_set(x_4, 1, x_42); -lean_ctor_set(x_4, 0, x_24); -x_43 = lean_array_uset(x_27, x_37, x_4); -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___at_Lean_MVarId_getNondepPropHyps___spec__7(x_43); -lean_ctor_set(x_3, 1, x_50); -lean_ctor_set(x_3, 0, x_41); -x_4 = x_7; -goto _start; +return x_4; } else { -lean_ctor_set(x_3, 1, x_43); -lean_ctor_set(x_3, 0, x_41); -x_4 = x_7; +lean_object* 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; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; size_t 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_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_ctor_get(x_1, 1); +x_12 = lean_array_get_size(x_11); +x_13 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_6); +x_14 = 32; +x_15 = lean_uint64_shift_right(x_13, x_14); +x_16 = lean_uint64_xor(x_13, x_15); +x_17 = 16; +x_18 = lean_uint64_shift_right(x_16, x_17); +x_19 = lean_uint64_xor(x_16, x_18); +x_20 = lean_uint64_to_usize(x_19); +x_21 = lean_usize_of_nat(x_12); +lean_dec(x_12); +x_22 = lean_usize_sub(x_21, x_9); +x_23 = lean_usize_land(x_20, x_22); +x_24 = lean_array_uget(x_11, x_23); +x_25 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(x_6, x_6, x_24); +lean_dec(x_24); +lean_dec(x_6); +x_26 = lean_array_uset(x_8, x_3, x_25); +x_3 = x_10; +x_4 = x_26; goto _start; } } -else -{ -lean_dec(x_38); -lean_dec(x_24); -lean_free_object(x_4); -x_4 = x_7; -goto _start; } +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; +x_7 = lean_usize_dec_lt(x_5, x_4); +if (x_7 == 0) +{ +lean_dec(x_1); +return x_6; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; uint64_t x_57; uint64_t x_58; uint64_t x_59; uint64_t x_60; uint64_t x_61; size_t x_62; size_t x_63; size_t x_64; size_t x_65; lean_object* x_66; uint8_t x_67; -x_54 = lean_ctor_get(x_3, 0); -x_55 = lean_ctor_get(x_3, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_3); -x_56 = lean_array_get_size(x_55); -x_57 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_24); -x_58 = lean_uint64_shift_right(x_57, x_12); -x_59 = lean_uint64_xor(x_57, x_58); -x_60 = lean_uint64_shift_right(x_59, x_15); -x_61 = lean_uint64_xor(x_59, x_60); -x_62 = lean_uint64_to_usize(x_61); -x_63 = lean_usize_of_nat(x_56); -lean_dec(x_56); -x_64 = lean_usize_sub(x_63, x_20); -x_65 = lean_usize_land(x_62, x_64); -x_66 = lean_array_uget(x_55, x_65); -x_67 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_24, x_66); -if (x_67 == 0) +lean_object* x_8; uint8_t x_9; +x_8 = lean_array_uget(x_3, x_5); +x_9 = !lean_is_exclusive(x_6); +if (x_9 == 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_54, x_68); -lean_dec(x_54); -x_70 = lean_box(0); -lean_ctor_set(x_4, 2, x_66); -lean_ctor_set(x_4, 1, x_70); -lean_ctor_set(x_4, 0, x_24); -x_71 = lean_array_uset(x_55, x_65, x_4); -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_10; lean_object* x_11; lean_object* x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; size_t x_20; size_t x_21; size_t x_22; size_t x_23; size_t x_24; lean_object* x_25; uint8_t x_26; +x_10 = lean_ctor_get(x_6, 0); +x_11 = lean_ctor_get(x_6, 1); +x_12 = lean_array_get_size(x_11); +x_13 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_8); +x_14 = 32; +x_15 = lean_uint64_shift_right(x_13, x_14); +x_16 = lean_uint64_xor(x_13, x_15); +x_17 = 16; +x_18 = lean_uint64_shift_right(x_16, x_17); +x_19 = lean_uint64_xor(x_16, x_18); +x_20 = lean_uint64_to_usize(x_19); +x_21 = lean_usize_of_nat(x_12); +lean_dec(x_12); +x_22 = 1; +x_23 = lean_usize_sub(x_21, x_22); +x_24 = lean_usize_land(x_20, x_23); +x_25 = lean_array_uget(x_11, x_24); +x_26 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_8, 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; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_27 = lean_unsigned_to_nat(1u); +x_28 = lean_nat_add(x_10, x_27); +lean_dec(x_10); +x_29 = lean_box(0); +x_30 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_30, 0, x_8); +lean_ctor_set(x_30, 1, x_29); +lean_ctor_set(x_30, 2, x_25); +x_31 = lean_array_uset(x_11, x_24, x_30); +x_32 = lean_unsigned_to_nat(4u); +x_33 = lean_nat_mul(x_28, x_32); +x_34 = lean_unsigned_to_nat(3u); +x_35 = lean_nat_div(x_33, x_34); +lean_dec(x_33); +x_36 = lean_array_get_size(x_31); +x_37 = lean_nat_dec_le(x_35, x_36); +lean_dec(x_36); +lean_dec(x_35); +if (x_37 == 0) { -lean_object* x_78; lean_object* x_79; -x_78 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_71); -x_79 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_79, 0, x_69); -lean_ctor_set(x_79, 1, x_78); -x_3 = x_79; -x_4 = x_7; +lean_object* x_38; size_t x_39; +x_38 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_31); +lean_ctor_set(x_6, 1, x_38); +lean_ctor_set(x_6, 0, x_28); +x_39 = lean_usize_add(x_5, x_22); +x_5 = x_39; goto _start; } else { -lean_object* x_81; -x_81 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_81, 0, x_69); -lean_ctor_set(x_81, 1, x_71); -x_3 = x_81; -x_4 = x_7; +size_t x_41; +lean_ctor_set(x_6, 1, x_31); +lean_ctor_set(x_6, 0, x_28); +x_41 = lean_usize_add(x_5, x_22); +x_5 = x_41; goto _start; } } else { -lean_object* x_83; -lean_dec(x_66); -lean_dec(x_24); -lean_free_object(x_4); -x_83 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_83, 0, x_54); -lean_ctor_set(x_83, 1, x_55); -x_3 = x_83; -x_4 = x_7; +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; size_t x_47; +lean_inc(x_1); +x_43 = lean_array_uset(x_11, x_24, x_1); +x_44 = lean_box(0); +x_45 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_8, x_44, x_25); +x_46 = lean_array_uset(x_43, x_24, x_45); +lean_ctor_set(x_6, 1, x_46); +x_47 = lean_usize_add(x_5, x_22); +x_5 = x_47; goto _start; } } -} else { -lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint64_t x_89; uint64_t x_90; uint64_t x_91; uint64_t x_92; uint64_t x_93; uint64_t x_94; uint64_t x_95; size_t x_96; size_t x_97; size_t x_98; size_t x_99; size_t 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; uint64_t x_107; uint64_t x_108; uint64_t x_109; uint64_t x_110; uint64_t x_111; size_t x_112; size_t x_113; size_t x_114; size_t x_115; lean_object* x_116; uint8_t x_117; -x_85 = lean_ctor_get(x_4, 0); -x_86 = lean_ctor_get(x_4, 2); -lean_inc(x_86); -lean_inc(x_85); -lean_dec(x_4); -x_87 = lean_ctor_get(x_2, 1); -x_88 = lean_array_get_size(x_87); -x_89 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_85); -x_90 = 32; -x_91 = lean_uint64_shift_right(x_89, x_90); -x_92 = lean_uint64_xor(x_89, x_91); -x_93 = 16; -x_94 = lean_uint64_shift_right(x_92, x_93); -x_95 = lean_uint64_xor(x_92, x_94); -x_96 = lean_uint64_to_usize(x_95); -x_97 = lean_usize_of_nat(x_88); -lean_dec(x_88); -x_98 = 1; -x_99 = lean_usize_sub(x_97, x_98); -x_100 = lean_usize_land(x_96, x_99); -x_101 = lean_array_uget(x_87, x_100); -x_102 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(x_85, x_85, x_101); -lean_dec(x_101); -lean_dec(x_85); -x_103 = lean_ctor_get(x_3, 0); -lean_inc(x_103); -x_104 = lean_ctor_get(x_3, 1); -lean_inc(x_104); -if (lean_is_exclusive(x_3)) { - lean_ctor_release(x_3, 0); - lean_ctor_release(x_3, 1); - x_105 = x_3; -} else { - lean_dec_ref(x_3); - x_105 = lean_box(0); -} -x_106 = lean_array_get_size(x_104); -x_107 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_102); -x_108 = lean_uint64_shift_right(x_107, x_90); -x_109 = lean_uint64_xor(x_107, x_108); -x_110 = lean_uint64_shift_right(x_109, x_93); -x_111 = lean_uint64_xor(x_109, x_110); -x_112 = lean_uint64_to_usize(x_111); -x_113 = lean_usize_of_nat(x_106); -lean_dec(x_106); -x_114 = lean_usize_sub(x_113, x_98); -x_115 = lean_usize_land(x_112, x_114); -x_116 = lean_array_uget(x_104, x_115); -x_117 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_102, x_116); -if (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; lean_object* x_125; lean_object* x_126; lean_object* x_127; uint8_t x_128; -x_118 = lean_unsigned_to_nat(1u); -x_119 = lean_nat_add(x_103, x_118); -lean_dec(x_103); -x_120 = lean_box(0); -x_121 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_121, 0, x_102); -lean_ctor_set(x_121, 1, x_120); -lean_ctor_set(x_121, 2, x_116); -x_122 = lean_array_uset(x_104, x_115, x_121); -x_123 = lean_unsigned_to_nat(4u); -x_124 = lean_nat_mul(x_119, x_123); -x_125 = lean_unsigned_to_nat(3u); -x_126 = lean_nat_div(x_124, x_125); -lean_dec(x_124); -x_127 = lean_array_get_size(x_122); -x_128 = lean_nat_dec_le(x_126, x_127); -lean_dec(x_127); -lean_dec(x_126); -if (x_128 == 0) +lean_object* x_49; lean_object* x_50; lean_object* x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; uint64_t x_55; uint64_t x_56; uint64_t x_57; uint64_t x_58; size_t x_59; size_t x_60; size_t x_61; size_t x_62; size_t x_63; lean_object* x_64; uint8_t x_65; +x_49 = lean_ctor_get(x_6, 0); +x_50 = lean_ctor_get(x_6, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_6); +x_51 = lean_array_get_size(x_50); +x_52 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1724_(x_8); +x_53 = 32; +x_54 = lean_uint64_shift_right(x_52, x_53); +x_55 = lean_uint64_xor(x_52, x_54); +x_56 = 16; +x_57 = lean_uint64_shift_right(x_55, x_56); +x_58 = lean_uint64_xor(x_55, x_57); +x_59 = lean_uint64_to_usize(x_58); +x_60 = lean_usize_of_nat(x_51); +lean_dec(x_51); +x_61 = 1; +x_62 = lean_usize_sub(x_60, x_61); +x_63 = lean_usize_land(x_59, x_62); +x_64 = lean_array_uget(x_50, x_63); +x_65 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_8, 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; lean_object* x_74; lean_object* x_75; uint8_t x_76; +x_66 = lean_unsigned_to_nat(1u); +x_67 = lean_nat_add(x_49, x_66); +lean_dec(x_49); +x_68 = lean_box(0); +x_69 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_69, 0, x_8); +lean_ctor_set(x_69, 1, x_68); +lean_ctor_set(x_69, 2, x_64); +x_70 = lean_array_uset(x_50, x_63, x_69); +x_71 = lean_unsigned_to_nat(4u); +x_72 = lean_nat_mul(x_67, x_71); +x_73 = lean_unsigned_to_nat(3u); +x_74 = lean_nat_div(x_72, x_73); +lean_dec(x_72); +x_75 = lean_array_get_size(x_70); +x_76 = lean_nat_dec_le(x_74, x_75); +lean_dec(x_75); +lean_dec(x_74); +if (x_76 == 0) { -lean_object* x_129; lean_object* x_130; -x_129 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_122); -if (lean_is_scalar(x_105)) { - x_130 = lean_alloc_ctor(0, 2, 0); -} else { - x_130 = x_105; -} -lean_ctor_set(x_130, 0, x_119); -lean_ctor_set(x_130, 1, x_129); -x_3 = x_130; -x_4 = x_86; +lean_object* x_77; lean_object* x_78; size_t x_79; +x_77 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_70); +x_78 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_78, 0, x_67); +lean_ctor_set(x_78, 1, x_77); +x_79 = lean_usize_add(x_5, x_61); +x_5 = x_79; +x_6 = x_78; goto _start; } else { -lean_object* x_132; -if (lean_is_scalar(x_105)) { - x_132 = lean_alloc_ctor(0, 2, 0); -} else { - x_132 = x_105; -} -lean_ctor_set(x_132, 0, x_119); -lean_ctor_set(x_132, 1, x_122); -x_3 = x_132; -x_4 = x_86; +lean_object* x_81; size_t x_82; +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_67); +lean_ctor_set(x_81, 1, x_70); +x_82 = lean_usize_add(x_5, x_61); +x_5 = x_82; +x_6 = x_81; goto _start; } } else { -lean_object* x_134; -lean_dec(x_116); -lean_dec(x_102); -if (lean_is_scalar(x_105)) { - x_134 = lean_alloc_ctor(0, 2, 0); -} else { - x_134 = x_105; -} -lean_ctor_set(x_134, 0, x_103); -lean_ctor_set(x_134, 1, x_104); -x_3 = x_134; -x_4 = x_86; +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; size_t x_89; +lean_inc(x_1); +x_84 = lean_array_uset(x_50, x_63, x_1); +x_85 = lean_box(0); +x_86 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_8, x_85, x_64); +x_87 = lean_array_uset(x_84, x_63, x_86); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_49); +lean_ctor_set(x_88, 1, x_87); +x_89 = lean_usize_add(x_5, x_61); +x_5 = x_89; +x_6 = x_88; goto _start; } } } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { -_start: -{ -uint8_t x_7; -x_7 = lean_usize_dec_eq(x_4, x_5); -if (x_7 == 0) -{ -lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; -x_8 = lean_array_uget(x_3, x_4); -x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_1, x_2, x_6, x_8); -x_10 = 1; -x_11 = lean_usize_add(x_4, x_10); -x_4 = x_11; -x_6 = x_9; -goto _start; -} -else -{ -return x_6; -} -} -} -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; @@ -15677,14 +17532,14 @@ return x_9; } } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___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_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___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; lean_object* x_9; x_7 = lean_ctor_get(x_6, 2); lean_inc(x_7); lean_dec(x_6); -x_8 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__1___boxed), 2, 1); +x_8 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__1___boxed), 2, 1); lean_closure_set(x_8, 0, x_1); x_9 = l_Lean_Syntax_findStack_x3f(x_7, x_2, x_8); if (lean_obj_tag(x_9) == 0) @@ -15741,7 +17596,7 @@ return x_20; } } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15(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_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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, size_t x_7, size_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { uint8_t x_12; @@ -15753,7 +17608,7 @@ x_13 = lean_array_uget(x_6, x_7); lean_inc(x_10); lean_inc(x_9); lean_inc(x_2); -x_14 = l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4(x_2, x_13, x_9, x_10, x_11); +x_14 = l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5(x_2, x_13, x_9, x_10, x_11); if (lean_obj_tag(x_14) == 0) { lean_object* x_15; @@ -15789,7 +17644,7 @@ lean_inc(x_3); lean_inc(x_1); lean_inc(x_5); lean_inc(x_2); -x_24 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__2___boxed), 6, 5); +x_24 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__2___boxed), 6, 5); lean_closure_set(x_24, 0, x_2); lean_closure_set(x_24, 1, x_5); lean_closure_set(x_24, 2, x_1); @@ -15836,7 +17691,7 @@ lean_inc(x_3); lean_inc(x_1); lean_inc(x_5); lean_inc(x_2); -x_33 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__2___boxed), 6, 5); +x_33 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__2___boxed), 6, 5); lean_closure_set(x_33, 0, x_2); lean_closure_set(x_33, 1, x_5); lean_closure_set(x_33, 2, x_1); @@ -15921,7 +17776,7 @@ return x_47; } } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; @@ -15945,12 +17800,12 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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, size_t x_7, size_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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, size_t x_7, size_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; uint8_t x_13; lean_inc(x_1); -x_12 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___lambda__1___boxed), 2, 1); +x_12 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___lambda__1___boxed), 2, 1); lean_closure_set(x_12, 0, x_1); x_13 = lean_usize_dec_eq(x_7, x_8); if (x_13 == 0) @@ -15960,7 +17815,7 @@ x_14 = lean_array_uget(x_6, x_7); lean_inc(x_10); lean_inc(x_9); lean_inc(x_3); -x_15 = l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4(x_3, x_14, x_9, x_10, x_11); +x_15 = l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5(x_3, x_14, x_9, x_10, x_11); if (lean_obj_tag(x_15) == 0) { lean_object* x_16; @@ -15996,7 +17851,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); lean_inc(x_3); -x_25 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__2___boxed), 6, 5); +x_25 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__2___boxed), 6, 5); lean_closure_set(x_25, 0, x_3); lean_closure_set(x_25, 1, x_12); lean_closure_set(x_25, 2, x_2); @@ -16042,7 +17897,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); lean_inc(x_3); -x_34 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__2___boxed), 6, 5); +x_34 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__2___boxed), 6, 5); lean_closure_set(x_34, 0, x_3); lean_closure_set(x_34, 1, x_12); lean_closure_set(x_34, 2, x_2); @@ -16129,7 +17984,7 @@ return x_48; } } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(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_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(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: { uint8_t x_7; @@ -16173,7 +18028,7 @@ return x_15; } } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18(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_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24(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: { uint8_t x_7; @@ -16198,7 +18053,7 @@ 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_9, x_22); -x_24 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(x_8, x_8, x_23); +x_24 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(x_8, x_8, x_23); lean_dec(x_23); lean_dec(x_8); x_25 = lean_ctor_get(x_3, 1); @@ -16239,7 +18094,7 @@ return x_41; } } } -LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__1(lean_object* x_1) { +LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__1(lean_object* x_1) { _start: { uint8_t x_2; @@ -16258,7 +18113,7 @@ return x_4; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2(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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2(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_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; @@ -16278,218 +18133,251 @@ lean_ctor_set(x_14, 1, x_8); return x_14; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___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, uint8_t x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +static size_t _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3___closed__1() { _start: { -if (x_10 == 0) +lean_object* x_1; size_t x_2; +x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; +x_2 = lean_array_size(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___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, uint8_t 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_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; -x_16 = lean_box(0); -x_17 = lean_mk_array(x_3, x_16); -x_18 = lean_unsigned_to_nat(0u); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_17); -x_20 = lean_st_mk_ref(x_19, x_15); -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -if (lean_is_exclusive(x_20)) { - lean_ctor_release(x_20, 0); - lean_ctor_release(x_20, 1); - x_23 = x_20; +if (x_12 == 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_25; lean_object* x_26; lean_object* x_27; +x_18 = lean_box(0); +x_19 = lean_mk_array(x_3, x_18); +x_20 = lean_unsigned_to_nat(0u); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_19); +x_22 = lean_st_mk_ref(x_21, x_17); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_22)) { + lean_ctor_release(x_22, 0); + lean_ctor_release(x_22, 1); + x_25 = x_22; } else { - lean_dec_ref(x_20); - x_23 = lean_box(0); + lean_dec_ref(x_22); + x_25 = lean_box(0); } -x_24 = lean_ctor_get(x_4, 4); +x_26 = lean_ctor_get(x_4, 4); lean_inc(x_5); -x_25 = l_Lean_Linter_UnusedVariables_visitAssignments(x_21, x_5, x_24, x_22); -lean_dec(x_21); -if (lean_obj_tag(x_25) == 0) +x_27 = l_Lean_Linter_UnusedVariables_visitAssignments(x_23, x_5, x_26, x_24); +lean_dec(x_23); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_26; lean_object* x_27; 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_26 = lean_ctor_get(x_25, 1); -lean_inc(x_26); -lean_dec(x_25); -x_66 = lean_st_ref_take(x_5, x_26); -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_object* x_28; lean_object* x_29; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; size_t x_74; +x_28 = lean_ctor_get(x_27, 1); +lean_inc(x_28); +lean_dec(x_27); +x_68 = lean_st_ref_take(x_5, x_28); +x_69 = lean_ctor_get(x_68, 0); lean_inc(x_69); -lean_dec(x_67); -x_70 = lean_array_get_size(x_69); -x_71 = lean_nat_dec_lt(x_18, x_70); -if (x_71 == 0) -{ -lean_object* x_72; lean_object* x_73; -lean_dec(x_70); +x_70 = lean_ctor_get(x_68, 1); +lean_inc(x_70); +lean_dec(x_68); +x_71 = lean_ctor_get(x_69, 1); +lean_inc(x_71); lean_dec(x_69); -x_72 = lean_st_ref_set(x_5, x_9, x_68); -x_73 = lean_ctor_get(x_72, 1); -lean_inc(x_73); +x_72 = lean_array_get_size(x_71); +x_73 = lean_nat_dec_lt(x_20, x_72); +x_74 = 0; +if (x_73 == 0) +{ +size_t x_75; lean_object* x_76; lean_object* x_77; size_t x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_dec(x_72); -x_27 = x_73; -goto block_65; +lean_dec(x_71); +x_75 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3___closed__1; +x_76 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; +x_77 = l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14(x_9, x_75, x_74, x_76); +x_78 = lean_array_size(x_77); +lean_inc(x_11); +x_79 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15(x_10, x_11, x_77, x_78, x_74, x_11); +lean_dec(x_77); +lean_dec(x_11); +x_80 = lean_st_ref_set(x_5, x_79, x_70); +x_81 = lean_ctor_get(x_80, 1); +lean_inc(x_81); +lean_dec(x_80); +x_29 = x_81; +goto block_67; } else { -uint8_t x_74; -x_74 = lean_nat_dec_le(x_70, x_70); -if (x_74 == 0) +uint8_t x_82; +x_82 = lean_nat_dec_le(x_72, x_72); +if (x_82 == 0) { -lean_object* x_75; lean_object* x_76; -lean_dec(x_70); -lean_dec(x_69); -x_75 = lean_st_ref_set(x_5, x_9, x_68); -x_76 = lean_ctor_get(x_75, 1); -lean_inc(x_76); -lean_dec(x_75); -x_27 = x_76; -goto block_65; +size_t x_83; lean_object* x_84; lean_object* x_85; size_t x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +lean_dec(x_72); +lean_dec(x_71); +x_83 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3___closed__1; +x_84 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; +x_85 = l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16(x_9, x_83, x_74, x_84); +x_86 = lean_array_size(x_85); +lean_inc(x_11); +x_87 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(x_10, x_11, x_85, x_86, x_74, x_11); +lean_dec(x_85); +lean_dec(x_11); +x_88 = lean_st_ref_set(x_5, x_87, x_70); +x_89 = lean_ctor_get(x_88, 1); +lean_inc(x_89); +lean_dec(x_88); +x_29 = x_89; +goto block_67; } else { -size_t x_77; size_t x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_77 = 0; -x_78 = lean_usize_of_nat(x_70); -lean_dec(x_70); -x_79 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14(x_7, x_8, x_69, x_77, x_78, x_9); -lean_dec(x_69); -x_80 = lean_st_ref_set(x_5, x_79, x_68); -x_81 = lean_ctor_get(x_80, 1); -lean_inc(x_81); -lean_dec(x_80); -x_27 = x_81; -goto block_65; +size_t x_90; lean_object* x_91; lean_object* x_92; size_t x_93; lean_object* x_94; size_t x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +x_90 = lean_usize_of_nat(x_72); +lean_dec(x_72); +x_91 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; +x_92 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18(x_71, x_74, x_90, x_91); +lean_dec(x_71); +x_93 = lean_array_size(x_92); +x_94 = l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19(x_9, x_93, x_74, x_92); +x_95 = lean_array_size(x_94); +lean_inc(x_11); +x_96 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(x_10, x_11, x_94, x_95, x_74, x_11); +lean_dec(x_94); +lean_dec(x_11); +x_97 = lean_st_ref_set(x_5, x_96, x_70); +x_98 = lean_ctor_get(x_97, 1); +lean_inc(x_98); +lean_dec(x_97); +x_29 = x_98; +goto block_67; } } -block_65: +block_67: { -lean_object* x_28; uint8_t x_29; -x_28 = lean_st_ref_get(x_5, x_27); +lean_object* x_30; uint8_t x_31; +x_30 = lean_st_ref_get(x_5, x_29); lean_dec(x_5); -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) +x_31 = !lean_is_exclusive(x_30); +if (x_31 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; -x_30 = lean_ctor_get(x_28, 0); -x_31 = lean_ctor_get(x_28, 1); -x_32 = lean_array_get_size(x_6); -x_33 = lean_nat_dec_lt(x_18, x_32); -if (x_33 == 0) +lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; +x_32 = lean_ctor_get(x_30, 0); +x_33 = lean_ctor_get(x_30, 1); +x_34 = lean_array_get_size(x_6); +x_35 = lean_nat_dec_lt(x_20, x_34); +if (x_35 == 0) { -uint8_t x_34; lean_object* x_35; lean_object* x_36; +uint8_t x_36; lean_object* x_37; lean_object* x_38; +lean_dec(x_34); +lean_free_object(x_30); lean_dec(x_32); -lean_free_object(x_28); -lean_dec(x_30); -lean_dec(x_23); -x_34 = 1; -x_35 = lean_box(0); -x_36 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2(x_1, x_2, x_34, x_11, x_35, x_13, x_14, x_31); -return x_36; +lean_dec(x_25); +x_36 = 1; +x_37 = lean_box(0); +x_38 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2(x_1, x_2, x_36, x_13, x_37, x_15, x_16, x_33); +return x_38; } else { -size_t x_37; size_t x_38; uint8_t x_39; -x_37 = 0; -x_38 = lean_usize_of_nat(x_32); +size_t x_39; size_t x_40; uint8_t x_41; +x_39 = 0; +x_40 = lean_usize_of_nat(x_34); +lean_dec(x_34); +x_41 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(x_7, x_8, x_32, x_6, x_39, x_40); lean_dec(x_32); -x_39 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__12(x_7, x_8, x_30, x_6, x_37, x_38); -lean_dec(x_30); -if (x_39 == 0) +if (x_41 == 0) { -uint8_t x_40; lean_object* x_41; lean_object* x_42; -lean_free_object(x_28); -lean_dec(x_23); -x_40 = 1; -x_41 = lean_box(0); -x_42 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2(x_1, x_2, x_40, x_11, x_41, x_13, x_14, x_31); -return x_42; +uint8_t x_42; lean_object* x_43; lean_object* x_44; +lean_free_object(x_30); +lean_dec(x_25); +x_42 = 1; +x_43 = lean_box(0); +x_44 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2(x_1, x_2, x_42, x_13, x_43, x_15, x_16, x_33); +return x_44; } else { -uint8_t x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +uint8_t x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_dec(x_2); lean_dec(x_1); -x_43 = 1; -x_44 = lean_box(x_43); -if (lean_is_scalar(x_23)) { - x_45 = lean_alloc_ctor(0, 2, 0); +x_45 = 1; +x_46 = lean_box(x_45); +if (lean_is_scalar(x_25)) { + x_47 = lean_alloc_ctor(0, 2, 0); } else { - x_45 = x_23; + x_47 = x_25; } -lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_11); -x_46 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_28, 0, x_46); -return x_28; +lean_ctor_set(x_47, 0, x_46); +lean_ctor_set(x_47, 1, x_13); +x_48 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_30, 0, x_48); +return x_30; } } } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; -x_47 = lean_ctor_get(x_28, 0); -x_48 = lean_ctor_get(x_28, 1); -lean_inc(x_48); -lean_inc(x_47); -lean_dec(x_28); -x_49 = lean_array_get_size(x_6); -x_50 = lean_nat_dec_lt(x_18, x_49); -if (x_50 == 0) +lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; +x_49 = lean_ctor_get(x_30, 0); +x_50 = lean_ctor_get(x_30, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_30); +x_51 = lean_array_get_size(x_6); +x_52 = lean_nat_dec_lt(x_20, x_51); +if (x_52 == 0) { -uint8_t x_51; lean_object* x_52; lean_object* x_53; +uint8_t x_53; lean_object* x_54; lean_object* x_55; +lean_dec(x_51); lean_dec(x_49); -lean_dec(x_47); -lean_dec(x_23); -x_51 = 1; -x_52 = lean_box(0); -x_53 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2(x_1, x_2, x_51, x_11, x_52, x_13, x_14, x_48); -return x_53; +lean_dec(x_25); +x_53 = 1; +x_54 = lean_box(0); +x_55 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2(x_1, x_2, x_53, x_13, x_54, x_15, x_16, x_50); +return x_55; } else { -size_t x_54; size_t x_55; uint8_t x_56; -x_54 = 0; -x_55 = lean_usize_of_nat(x_49); +size_t x_56; size_t x_57; uint8_t x_58; +x_56 = 0; +x_57 = lean_usize_of_nat(x_51); +lean_dec(x_51); +x_58 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(x_7, x_8, x_49, x_6, x_56, x_57); lean_dec(x_49); -x_56 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__12(x_7, x_8, x_47, x_6, x_54, x_55); -lean_dec(x_47); -if (x_56 == 0) +if (x_58 == 0) { -uint8_t x_57; lean_object* x_58; lean_object* x_59; -lean_dec(x_23); -x_57 = 1; -x_58 = lean_box(0); -x_59 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2(x_1, x_2, x_57, x_11, x_58, x_13, x_14, x_48); -return x_59; +uint8_t x_59; lean_object* x_60; lean_object* x_61; +lean_dec(x_25); +x_59 = 1; +x_60 = lean_box(0); +x_61 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2(x_1, x_2, x_59, x_13, x_60, x_15, x_16, x_50); +return x_61; } else { -uint8_t x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +uint8_t x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_dec(x_2); lean_dec(x_1); -x_60 = 1; -x_61 = lean_box(x_60); -if (lean_is_scalar(x_23)) { - x_62 = lean_alloc_ctor(0, 2, 0); +x_62 = 1; +x_63 = lean_box(x_62); +if (lean_is_scalar(x_25)) { + x_64 = lean_alloc_ctor(0, 2, 0); } else { - x_62 = x_23; + x_64 = x_25; } -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_11); -x_63 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_63, 0, x_62); -x_64 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_64, 0, x_63); -lean_ctor_set(x_64, 1, x_48); -return x_64; +lean_ctor_set(x_64, 1, x_13); +x_65 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_65, 0, x_64); +x_66 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_66, 0, x_65); +lean_ctor_set(x_66, 1, x_50); +return x_66; } } } @@ -16497,417 +18385,425 @@ return x_64; } else { -uint8_t x_82; +uint8_t x_99; +lean_dec(x_13); lean_dec(x_11); -lean_dec(x_9); +lean_dec(x_10); lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); -x_82 = !lean_is_exclusive(x_25); -if (x_82 == 0) +x_99 = !lean_is_exclusive(x_27); +if (x_99 == 0) { -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_ctor_get(x_25, 0); -x_84 = lean_ctor_get(x_13, 6); -x_85 = lean_io_error_to_string(x_83); -x_86 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_86, 0, x_85); -x_87 = l_Lean_MessageData_ofFormat(x_86); -lean_inc(x_84); -if (lean_is_scalar(x_23)) { - x_88 = lean_alloc_ctor(0, 2, 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; +x_100 = lean_ctor_get(x_27, 0); +x_101 = lean_ctor_get(x_15, 6); +x_102 = lean_io_error_to_string(x_100); +x_103 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_103, 0, x_102); +x_104 = l_Lean_MessageData_ofFormat(x_103); +lean_inc(x_101); +if (lean_is_scalar(x_25)) { + x_105 = lean_alloc_ctor(0, 2, 0); } else { - x_88 = x_23; + x_105 = x_25; } -lean_ctor_set(x_88, 0, x_84); -lean_ctor_set(x_88, 1, x_87); -lean_ctor_set(x_25, 0, x_88); -return x_25; +lean_ctor_set(x_105, 0, x_101); +lean_ctor_set(x_105, 1, x_104); +lean_ctor_set(x_27, 0, x_105); +return x_27; } 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; -x_89 = lean_ctor_get(x_25, 0); -x_90 = lean_ctor_get(x_25, 1); -lean_inc(x_90); -lean_inc(x_89); -lean_dec(x_25); -x_91 = lean_ctor_get(x_13, 6); -x_92 = lean_io_error_to_string(x_89); -x_93 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_93, 0, x_92); -x_94 = l_Lean_MessageData_ofFormat(x_93); -lean_inc(x_91); -if (lean_is_scalar(x_23)) { - x_95 = lean_alloc_ctor(0, 2, 0); +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; +x_106 = lean_ctor_get(x_27, 0); +x_107 = lean_ctor_get(x_27, 1); +lean_inc(x_107); +lean_inc(x_106); +lean_dec(x_27); +x_108 = lean_ctor_get(x_15, 6); +x_109 = lean_io_error_to_string(x_106); +x_110 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_110, 0, x_109); +x_111 = l_Lean_MessageData_ofFormat(x_110); +lean_inc(x_108); +if (lean_is_scalar(x_25)) { + x_112 = lean_alloc_ctor(0, 2, 0); } else { - x_95 = x_23; + x_112 = x_25; } -lean_ctor_set(x_95, 0, x_91); -lean_ctor_set(x_95, 1, x_94); -x_96 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_96, 0, x_95); -lean_ctor_set(x_96, 1, x_90); -return x_96; +lean_ctor_set(x_112, 0, x_108); +lean_ctor_set(x_112, 1, x_111); +x_113 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_113, 0, x_112); +lean_ctor_set(x_113, 1, x_107); +return x_113; } } } else { -lean_object* x_97; lean_object* x_98; -lean_dec(x_9); +lean_object* x_114; lean_object* x_115; +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_5); lean_dec(x_3); -x_97 = lean_box(0); -x_98 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2(x_1, x_2, x_10, x_11, x_97, x_13, x_14, x_15); -return x_98; +x_114 = lean_box(0); +x_115 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2(x_1, x_2, x_12, x_13, x_114, x_15, x_16, x_17); +return x_115; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___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, uint8_t x_10, 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, lean_object* x_19, lean_object* x_20, lean_object* x_21) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___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, uint8_t 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) { _start: { -uint8_t x_22; lean_object* x_23; -if (x_10 == 0) +uint8_t x_24; lean_object* x_25; +if (x_12 == 0) { -uint8_t x_31; +uint8_t x_33; +lean_dec(x_16); +lean_dec(x_15); lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -x_31 = 0; -x_22 = x_31; -x_23 = x_21; -goto block_30; +x_33 = 0; +x_24 = x_33; +x_25 = x_23; +goto block_32; } else { -size_t x_32; size_t x_33; lean_object* x_34; -x_32 = 0; -x_33 = lean_usize_of_nat(x_11); -lean_inc(x_20); -lean_inc(x_19); +size_t x_34; size_t x_35; lean_object* x_36; +x_34 = 0; +x_35 = lean_usize_of_nat(x_13); +lean_inc(x_22); +lean_inc(x_21); lean_inc(x_1); -lean_inc(x_12); -x_34 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16(x_12, x_13, x_12, x_1, x_14, x_15, x_32, x_33, x_19, x_20, x_21); -if (lean_obj_tag(x_34) == 0) +lean_inc(x_14); +x_36 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22(x_14, x_15, x_14, x_1, x_16, x_17, x_34, x_35, x_21, x_22, x_23); +if (lean_obj_tag(x_36) == 0) { -lean_object* x_35; lean_object* x_36; uint8_t x_37; -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_unbox(x_35); -lean_dec(x_35); -x_22 = x_37; -x_23 = x_36; -goto block_30; +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 = lean_unbox(x_37); +lean_dec(x_37); +x_24 = x_39; +x_25 = x_38; +goto block_32; } else { -uint8_t x_38; -lean_dec(x_20); +uint8_t x_40; +lean_dec(x_22); +lean_dec(x_21); lean_dec(x_19); -lean_dec(x_17); -lean_dec(x_9); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_38 = !lean_is_exclusive(x_34); -if (x_38 == 0) +x_40 = !lean_is_exclusive(x_36); +if (x_40 == 0) { -return x_34; +return x_36; } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_34, 0); -x_40 = lean_ctor_get(x_34, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_34); -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_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; } } } -block_30: +block_32: { -if (x_22 == 0) +if (x_24 == 0) { -lean_object* x_24; lean_object* x_25; -x_24 = lean_box(0); -x_25 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_16, x_17, x_24, x_19, x_20, x_23); -lean_dec(x_20); -lean_dec(x_19); -return x_25; +lean_object* x_26; lean_object* x_27; +x_26 = lean_box(0); +x_27 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___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_18, x_19, x_26, x_21, x_22, x_25); +lean_dec(x_22); +lean_dec(x_21); +return x_27; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -lean_dec(x_20); -lean_dec(x_19); -lean_dec(x_9); +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_26 = lean_box(x_16); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_17); -x_28 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_28, 0, x_27); +x_28 = lean_box(x_18); x_29 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_23); -return x_29; +lean_ctor_set(x_29, 1, x_19); +x_30 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_30, 0, 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_25); +return x_31; } } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__1___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__1___boxed), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___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, uint8_t 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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___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, lean_object* x_13, uint8_t 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, lean_object* x_22, lean_object* x_23, lean_object* x_24) { _start: { -lean_object* x_23; lean_object* x_24; lean_object* x_25; +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_inc(x_1); -x_23 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___lambda__1___boxed), 2, 1); -lean_closure_set(x_23, 0, x_1); -x_24 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5___closed__1; -x_25 = l_Lean_Syntax_findStack_x3f(x_2, x_23, x_24); -if (lean_obj_tag(x_25) == 0) +x_25 = lean_alloc_closure((void*)(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___lambda__1___boxed), 2, 1); +lean_closure_set(x_25, 0, x_1); +x_26 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5___closed__1; +x_27 = l_Lean_Syntax_findStack_x3f(x_2, x_25, x_26); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_26 = lean_box(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_18); -x_28 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_28, 0, x_27); +x_28 = lean_box(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_22); -return x_29; +lean_ctor_set(x_29, 1, x_20); +x_30 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_30, 0, 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 { -uint8_t x_30; -x_30 = !lean_is_exclusive(x_25); -if (x_30 == 0) +uint8_t x_32; +x_32 = !lean_is_exclusive(x_27); +if (x_32 == 0) { -lean_object* x_31; -x_31 = lean_ctor_get(x_25, 0); -if (lean_obj_tag(x_31) == 0) +lean_object* x_33; +x_33 = lean_ctor_get(x_27, 0); +if (lean_obj_tag(x_33) == 0) { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_34; lean_object* x_35; lean_object* x_36; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_32 = lean_box(x_17); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_18); -lean_ctor_set(x_25, 0, x_33); -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_25); -lean_ctor_set(x_34, 1, x_22); -return x_34; +x_34 = lean_box(x_19); +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_20); +lean_ctor_set(x_27, 0, x_35); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_27); +lean_ctor_set(x_36, 1, x_24); +return x_36; } else { -uint8_t x_35; -x_35 = !lean_is_exclusive(x_31); -if (x_35 == 0) -{ -lean_object* x_36; uint8_t x_37; -x_36 = lean_ctor_get(x_31, 0); -x_37 = !lean_is_exclusive(x_36); +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_40; uint8_t x_41; -x_38 = lean_ctor_get(x_31, 1); -x_39 = lean_ctor_get(x_36, 0); -x_40 = lean_ctor_get(x_36, 1); -lean_dec(x_40); -x_41 = l_Lean_Syntax_isIdent(x_39); -lean_dec(x_39); -if (x_41 == 0) +lean_object* x_38; uint8_t x_39; +x_38 = lean_ctor_get(x_33, 0); +x_39 = !lean_is_exclusive(x_38); +if (x_39 == 0) { -lean_object* x_42; lean_object* x_43; -lean_free_object(x_36); -lean_free_object(x_31); -lean_dec(x_38); -lean_free_object(x_25); -x_42 = lean_box(0); -x_43 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_42, x_20, x_21, x_22); -return x_43; +lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; +x_40 = lean_ctor_get(x_33, 1); +x_41 = lean_ctor_get(x_38, 0); +x_42 = lean_ctor_get(x_38, 1); +lean_dec(x_42); +x_43 = l_Lean_Syntax_isIdent(x_41); +lean_dec(x_41); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; +lean_free_object(x_38); +lean_free_object(x_33); +lean_dec(x_40); +lean_free_object(x_27); +x_44 = lean_box(0); +x_45 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(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_1, x_16, x_17, x_18, x_19, x_20, x_44, x_22, x_23, x_24); +return x_45; } else { -lean_object* x_44; lean_object* x_45; uint8_t x_46; -x_44 = lean_array_get_size(x_14); -x_45 = lean_unsigned_to_nat(0u); -x_46 = lean_nat_dec_lt(x_45, x_44); -if (x_46 == 0) +lean_object* x_46; lean_object* x_47; uint8_t x_48; +x_46 = lean_array_get_size(x_16); +x_47 = lean_unsigned_to_nat(0u); +x_48 = lean_nat_dec_lt(x_47, x_46); +if (x_48 == 0) { -lean_object* x_47; lean_object* x_48; -lean_dec(x_44); -lean_free_object(x_36); -lean_free_object(x_31); -lean_dec(x_38); -lean_free_object(x_25); -x_47 = lean_box(0); -x_48 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_47, x_20, x_21, x_22); -return x_48; +lean_object* x_49; lean_object* x_50; +lean_dec(x_46); +lean_free_object(x_38); +lean_free_object(x_33); +lean_dec(x_40); +lean_free_object(x_27); +x_49 = lean_box(0); +x_50 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(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_1, x_16, x_17, x_18, x_19, x_20, x_49, x_22, x_23, x_24); +return x_50; } else { -size_t x_49; size_t x_50; uint8_t x_51; -x_49 = 0; -x_50 = lean_usize_of_nat(x_44); -lean_dec(x_44); -lean_inc(x_15); +size_t x_51; size_t x_52; uint8_t x_53; +x_51 = 0; +x_52 = lean_usize_of_nat(x_46); +lean_dec(x_46); +lean_inc(x_17); lean_inc(x_3); -x_51 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(x_3, x_15, x_38, x_14, x_49, x_50); -if (x_51 == 0) -{ -lean_object* x_52; lean_object* x_53; -lean_free_object(x_36); -lean_free_object(x_31); -lean_free_object(x_25); -x_52 = lean_box(0); -x_53 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_52, x_20, x_21, x_22); -return x_53; +x_53 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(x_3, x_17, x_40, x_16, x_51, x_52); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; +lean_free_object(x_38); +lean_free_object(x_33); +lean_free_object(x_27); +x_54 = lean_box(0); +x_55 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(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_1, x_16, x_17, x_18, x_19, x_20, x_54, x_22, x_23, x_24); +return x_55; } else { -lean_object* x_54; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_56; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_54 = lean_box(x_17); -lean_ctor_set(x_36, 1, x_18); -lean_ctor_set(x_36, 0, x_54); -lean_ctor_set(x_25, 0, x_36); -lean_ctor_set_tag(x_31, 0); -lean_ctor_set(x_31, 1, x_22); -lean_ctor_set(x_31, 0, x_25); -return x_31; +x_56 = lean_box(x_19); +lean_ctor_set(x_38, 1, x_20); +lean_ctor_set(x_38, 0, x_56); +lean_ctor_set(x_27, 0, x_38); +lean_ctor_set_tag(x_33, 0); +lean_ctor_set(x_33, 1, x_24); +lean_ctor_set(x_33, 0, x_27); +return x_33; } } } } else { -lean_object* x_55; lean_object* x_56; uint8_t x_57; -x_55 = lean_ctor_get(x_31, 1); -x_56 = lean_ctor_get(x_36, 0); -lean_inc(x_56); -lean_dec(x_36); -x_57 = l_Lean_Syntax_isIdent(x_56); -lean_dec(x_56); -if (x_57 == 0) +lean_object* x_57; lean_object* x_58; uint8_t x_59; +x_57 = lean_ctor_get(x_33, 1); +x_58 = lean_ctor_get(x_38, 0); +lean_inc(x_58); +lean_dec(x_38); +x_59 = l_Lean_Syntax_isIdent(x_58); +lean_dec(x_58); +if (x_59 == 0) { -lean_object* x_58; lean_object* x_59; -lean_free_object(x_31); -lean_dec(x_55); -lean_free_object(x_25); -x_58 = lean_box(0); -x_59 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_58, x_20, x_21, x_22); -return x_59; +lean_object* x_60; lean_object* x_61; +lean_free_object(x_33); +lean_dec(x_57); +lean_free_object(x_27); +x_60 = lean_box(0); +x_61 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(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_1, x_16, x_17, x_18, x_19, x_20, x_60, x_22, x_23, x_24); +return x_61; } else { -lean_object* x_60; lean_object* x_61; uint8_t x_62; -x_60 = lean_array_get_size(x_14); -x_61 = lean_unsigned_to_nat(0u); -x_62 = lean_nat_dec_lt(x_61, x_60); -if (x_62 == 0) +lean_object* x_62; lean_object* x_63; uint8_t x_64; +x_62 = lean_array_get_size(x_16); +x_63 = lean_unsigned_to_nat(0u); +x_64 = lean_nat_dec_lt(x_63, x_62); +if (x_64 == 0) { -lean_object* x_63; lean_object* x_64; -lean_dec(x_60); -lean_free_object(x_31); -lean_dec(x_55); -lean_free_object(x_25); -x_63 = lean_box(0); -x_64 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_63, x_20, x_21, x_22); -return x_64; +lean_object* x_65; lean_object* x_66; +lean_dec(x_62); +lean_free_object(x_33); +lean_dec(x_57); +lean_free_object(x_27); +x_65 = lean_box(0); +x_66 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(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_1, x_16, x_17, x_18, x_19, x_20, x_65, x_22, x_23, x_24); +return x_66; } else { -size_t x_65; size_t x_66; uint8_t x_67; -x_65 = 0; -x_66 = lean_usize_of_nat(x_60); -lean_dec(x_60); -lean_inc(x_15); +size_t x_67; size_t x_68; uint8_t x_69; +x_67 = 0; +x_68 = lean_usize_of_nat(x_62); +lean_dec(x_62); +lean_inc(x_17); lean_inc(x_3); -x_67 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(x_3, x_15, x_55, x_14, x_65, x_66); -if (x_67 == 0) +x_69 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(x_3, x_17, x_57, x_16, x_67, x_68); +if (x_69 == 0) { -lean_object* x_68; lean_object* x_69; -lean_free_object(x_31); -lean_free_object(x_25); -x_68 = lean_box(0); -x_69 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_68, x_20, x_21, x_22); -return x_69; +lean_object* x_70; lean_object* x_71; +lean_free_object(x_33); +lean_free_object(x_27); +x_70 = lean_box(0); +x_71 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(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_1, x_16, x_17, x_18, x_19, x_20, x_70, x_22, x_23, x_24); +return x_71; } else { -lean_object* x_70; lean_object* x_71; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_72; lean_object* x_73; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_70 = lean_box(x_17); -x_71 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_71, 0, x_70); -lean_ctor_set(x_71, 1, x_18); -lean_ctor_set(x_25, 0, x_71); -lean_ctor_set_tag(x_31, 0); -lean_ctor_set(x_31, 1, x_22); -lean_ctor_set(x_31, 0, x_25); -return x_31; +x_72 = lean_box(x_19); +x_73 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_73, 0, x_72); +lean_ctor_set(x_73, 1, x_20); +lean_ctor_set(x_27, 0, x_73); +lean_ctor_set_tag(x_33, 0); +lean_ctor_set(x_33, 1, x_24); +lean_ctor_set(x_33, 0, x_27); +return x_33; } } } @@ -16915,95 +18811,96 @@ return x_31; } 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_31, 0); -x_73 = lean_ctor_get(x_31, 1); -lean_inc(x_73); -lean_inc(x_72); -lean_dec(x_31); -x_74 = lean_ctor_get(x_72, 0); +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_33, 0); +x_75 = lean_ctor_get(x_33, 1); +lean_inc(x_75); 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_dec(x_33); +x_76 = lean_ctor_get(x_74, 0); +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_72); - x_75 = lean_box(0); + lean_dec_ref(x_74); + x_77 = lean_box(0); } -x_76 = l_Lean_Syntax_isIdent(x_74); -lean_dec(x_74); -if (x_76 == 0) +x_78 = l_Lean_Syntax_isIdent(x_76); +lean_dec(x_76); +if (x_78 == 0) { -lean_object* x_77; lean_object* x_78; +lean_object* x_79; lean_object* x_80; +lean_dec(x_77); lean_dec(x_75); -lean_dec(x_73); -lean_free_object(x_25); -x_77 = lean_box(0); -x_78 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_77, x_20, x_21, x_22); -return x_78; +lean_free_object(x_27); +x_79 = lean_box(0); +x_80 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(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_1, x_16, x_17, x_18, x_19, x_20, x_79, x_22, x_23, x_24); +return x_80; } else { -lean_object* x_79; lean_object* x_80; uint8_t x_81; -x_79 = lean_array_get_size(x_14); -x_80 = lean_unsigned_to_nat(0u); -x_81 = lean_nat_dec_lt(x_80, x_79); -if (x_81 == 0) +lean_object* x_81; lean_object* x_82; uint8_t x_83; +x_81 = lean_array_get_size(x_16); +x_82 = lean_unsigned_to_nat(0u); +x_83 = lean_nat_dec_lt(x_82, x_81); +if (x_83 == 0) { -lean_object* x_82; lean_object* x_83; -lean_dec(x_79); +lean_object* x_84; lean_object* x_85; +lean_dec(x_81); +lean_dec(x_77); lean_dec(x_75); -lean_dec(x_73); -lean_free_object(x_25); -x_82 = lean_box(0); -x_83 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_82, x_20, x_21, x_22); -return x_83; +lean_free_object(x_27); +x_84 = lean_box(0); +x_85 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(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_1, x_16, x_17, x_18, x_19, x_20, x_84, x_22, x_23, x_24); +return x_85; } else { -size_t x_84; size_t x_85; uint8_t x_86; -x_84 = 0; -x_85 = lean_usize_of_nat(x_79); -lean_dec(x_79); -lean_inc(x_15); +size_t x_86; size_t x_87; uint8_t x_88; +x_86 = 0; +x_87 = lean_usize_of_nat(x_81); +lean_dec(x_81); +lean_inc(x_17); lean_inc(x_3); -x_86 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(x_3, x_15, x_73, x_14, x_84, x_85); -if (x_86 == 0) +x_88 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(x_3, x_17, x_75, x_16, x_86, x_87); +if (x_88 == 0) { -lean_object* x_87; lean_object* x_88; -lean_dec(x_75); -lean_free_object(x_25); -x_87 = lean_box(0); -x_88 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_87, x_20, x_21, x_22); -return x_88; +lean_object* x_89; lean_object* x_90; +lean_dec(x_77); +lean_free_object(x_27); +x_89 = lean_box(0); +x_90 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(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_1, x_16, x_17, x_18, x_19, x_20, x_89, x_22, x_23, x_24); +return x_90; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_91; lean_object* x_92; lean_object* x_93; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_89 = lean_box(x_17); -if (lean_is_scalar(x_75)) { - x_90 = lean_alloc_ctor(0, 2, 0); +x_91 = lean_box(x_19); +if (lean_is_scalar(x_77)) { + x_92 = lean_alloc_ctor(0, 2, 0); } else { - x_90 = x_75; + x_92 = x_77; } -lean_ctor_set(x_90, 0, x_89); -lean_ctor_set(x_90, 1, x_18); -lean_ctor_set(x_25, 0, x_90); -x_91 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_91, 0, x_25); -lean_ctor_set(x_91, 1, x_22); -return x_91; +lean_ctor_set(x_92, 0, x_91); +lean_ctor_set(x_92, 1, x_20); +lean_ctor_set(x_27, 0, x_92); +x_93 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_93, 0, x_27); +lean_ctor_set(x_93, 1, x_24); +return x_93; } } } @@ -17012,139 +18909,140 @@ return x_91; } else { -lean_object* x_92; -x_92 = lean_ctor_get(x_25, 0); -lean_inc(x_92); -lean_dec(x_25); -if (lean_obj_tag(x_92) == 0) +lean_object* x_94; +x_94 = lean_ctor_get(x_27, 0); +lean_inc(x_94); +lean_dec(x_27); +if (lean_obj_tag(x_94) == 0) { -lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_93 = lean_box(x_17); -x_94 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_94, 0, x_93); -lean_ctor_set(x_94, 1, x_18); -x_95 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_95, 0, x_94); +x_95 = lean_box(x_19); x_96 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_96, 0, x_95); -lean_ctor_set(x_96, 1, x_22); -return x_96; +lean_ctor_set(x_96, 1, x_20); +x_97 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_97, 0, x_96); +x_98 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_98, 0, x_97); +lean_ctor_set(x_98, 1, x_24); +return x_98; } else { -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_97 = lean_ctor_get(x_92, 0); -lean_inc(x_97); -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_92); - x_99 = lean_box(0); -} -x_100 = lean_ctor_get(x_97, 0); +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_94, 0); +lean_inc(x_99); +x_100 = lean_ctor_get(x_94, 1); lean_inc(x_100); -if (lean_is_exclusive(x_97)) { - lean_ctor_release(x_97, 0); - lean_ctor_release(x_97, 1); - x_101 = x_97; +if (lean_is_exclusive(x_94)) { + lean_ctor_release(x_94, 0); + lean_ctor_release(x_94, 1); + x_101 = x_94; } else { - lean_dec_ref(x_97); + lean_dec_ref(x_94); x_101 = lean_box(0); } -x_102 = l_Lean_Syntax_isIdent(x_100); -lean_dec(x_100); -if (x_102 == 0) +x_102 = lean_ctor_get(x_99, 0); +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 = l_Lean_Syntax_isIdent(x_102); +lean_dec(x_102); +if (x_104 == 0) { -lean_object* x_103; lean_object* x_104; +lean_object* x_105; lean_object* x_106; +lean_dec(x_103); lean_dec(x_101); -lean_dec(x_99); -lean_dec(x_98); -x_103 = lean_box(0); -x_104 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_103, x_20, x_21, x_22); -return x_104; +lean_dec(x_100); +x_105 = lean_box(0); +x_106 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(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_1, x_16, x_17, x_18, x_19, x_20, x_105, x_22, x_23, x_24); +return x_106; } else { -lean_object* x_105; lean_object* x_106; uint8_t x_107; -x_105 = lean_array_get_size(x_14); -x_106 = lean_unsigned_to_nat(0u); -x_107 = lean_nat_dec_lt(x_106, x_105); -if (x_107 == 0) +lean_object* x_107; lean_object* x_108; uint8_t x_109; +x_107 = lean_array_get_size(x_16); +x_108 = lean_unsigned_to_nat(0u); +x_109 = lean_nat_dec_lt(x_108, x_107); +if (x_109 == 0) { -lean_object* x_108; lean_object* x_109; -lean_dec(x_105); +lean_object* x_110; lean_object* x_111; +lean_dec(x_107); +lean_dec(x_103); lean_dec(x_101); -lean_dec(x_99); -lean_dec(x_98); -x_108 = lean_box(0); -x_109 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_108, x_20, x_21, x_22); -return x_109; +lean_dec(x_100); +x_110 = lean_box(0); +x_111 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(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_1, x_16, x_17, x_18, x_19, x_20, x_110, x_22, x_23, x_24); +return x_111; } else { -size_t x_110; size_t x_111; uint8_t x_112; -x_110 = 0; -x_111 = lean_usize_of_nat(x_105); -lean_dec(x_105); -lean_inc(x_15); +size_t x_112; size_t x_113; uint8_t x_114; +x_112 = 0; +x_113 = lean_usize_of_nat(x_107); +lean_dec(x_107); +lean_inc(x_17); lean_inc(x_3); -x_112 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(x_3, x_15, x_98, x_14, x_110, x_111); -if (x_112 == 0) +x_114 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(x_3, x_17, x_100, x_16, x_112, x_113); +if (x_114 == 0) { -lean_object* x_113; lean_object* x_114; +lean_object* x_115; lean_object* x_116; +lean_dec(x_103); lean_dec(x_101); -lean_dec(x_99); -x_113 = lean_box(0); -x_114 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_1, x_14, x_15, x_16, x_17, x_18, x_113, x_20, x_21, x_22); -return x_114; +x_115 = lean_box(0); +x_116 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4(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_1, x_16, x_17, x_18, x_19, x_20, x_115, x_22, x_23, x_24); +return x_116; } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_115 = lean_box(x_17); -if (lean_is_scalar(x_101)) { - x_116 = lean_alloc_ctor(0, 2, 0); -} else { - x_116 = x_101; -} -lean_ctor_set(x_116, 0, x_115); -lean_ctor_set(x_116, 1, x_18); -x_117 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_117, 0, x_116); -if (lean_is_scalar(x_99)) { +x_117 = lean_box(x_19); +if (lean_is_scalar(x_103)) { x_118 = lean_alloc_ctor(0, 2, 0); } else { - x_118 = x_99; - lean_ctor_set_tag(x_118, 0); + x_118 = x_103; } lean_ctor_set(x_118, 0, x_117); -lean_ctor_set(x_118, 1, x_22); -return x_118; +lean_ctor_set(x_118, 1, x_20); +x_119 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_119, 0, x_118); +if (lean_is_scalar(x_101)) { + x_120 = lean_alloc_ctor(0, 2, 0); +} else { + x_120 = x_101; + lean_ctor_set_tag(x_120, 0); } +lean_ctor_set(x_120, 0, x_119); +lean_ctor_set(x_120, 1, x_24); +return x_120; } } } @@ -17152,54 +19050,56 @@ return x_118; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___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, uint8_t 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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___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_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, uint8_t x_19, lean_object* x_20, lean_object* x_21, lean_object* x_22, lean_object* x_23, lean_object* x_24) { _start: { -lean_object* x_23; uint8_t x_24; -x_23 = lean_ctor_get(x_6, 0); -lean_inc(x_23); -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_6, 0); +lean_inc(x_25); +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; uint64_t x_28; uint64_t x_29; uint64_t x_30; uint64_t x_31; uint64_t x_32; uint64_t x_33; uint64_t x_34; size_t x_35; size_t x_36; size_t x_37; size_t x_38; size_t x_39; lean_object* x_40; uint8_t x_41; -x_25 = lean_ctor_get(x_23, 1); -x_26 = lean_ctor_get(x_23, 0); -lean_dec(x_26); -x_27 = lean_array_get_size(x_25); -x_28 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_1); -x_29 = 32; -x_30 = lean_uint64_shift_right(x_28, x_29); -x_31 = lean_uint64_xor(x_28, x_30); -x_32 = 16; -x_33 = lean_uint64_shift_right(x_31, x_32); -x_34 = lean_uint64_xor(x_31, x_33); -x_35 = lean_uint64_to_usize(x_34); -x_36 = lean_usize_of_nat(x_27); +lean_object* x_27; lean_object* x_28; lean_object* x_29; uint64_t x_30; uint64_t x_31; uint64_t x_32; uint64_t x_33; uint64_t x_34; uint64_t x_35; uint64_t x_36; size_t x_37; size_t x_38; size_t x_39; size_t x_40; size_t x_41; lean_object* x_42; uint8_t x_43; +x_27 = lean_ctor_get(x_25, 1); +x_28 = lean_ctor_get(x_25, 0); +lean_dec(x_28); +x_29 = lean_array_get_size(x_27); +x_30 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_1); +x_31 = 32; +x_32 = lean_uint64_shift_right(x_30, x_31); +x_33 = lean_uint64_xor(x_30, x_32); +x_34 = 16; +x_35 = lean_uint64_shift_right(x_33, x_34); +x_36 = lean_uint64_xor(x_33, x_35); +x_37 = lean_uint64_to_usize(x_36); +x_38 = lean_usize_of_nat(x_29); +lean_dec(x_29); +x_39 = 1; +x_40 = lean_usize_sub(x_38, x_39); +x_41 = lean_usize_land(x_37, x_40); +x_42 = lean_array_uget(x_27, x_41); lean_dec(x_27); -x_37 = 1; -x_38 = lean_usize_sub(x_36, x_37); -x_39 = lean_usize_land(x_35, x_38); -x_40 = lean_array_uget(x_25, x_39); -lean_dec(x_25); -x_41 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__7(x_1, x_40); -lean_dec(x_40); -if (x_41 == 0) +x_43 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__7(x_1, x_42); +lean_dec(x_42); +if (x_43 == 0) { -lean_object* x_42; lean_object* x_43; -lean_free_object(x_23); -x_42 = lean_box(0); -x_43 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__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, x_14, x_15, x_16, x_17, x_18, x_42, x_20, x_21, x_22); +lean_object* x_44; lean_object* x_45; +lean_free_object(x_25); +x_44 = lean_box(0); +x_45 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__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, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_44, x_22, x_23, x_24); lean_dec(x_6); -return x_43; +return x_45; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_46; lean_object* x_47; lean_object* x_48; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -17207,57 +19107,58 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_44 = lean_box(x_17); -lean_ctor_set(x_23, 1, x_18); -lean_ctor_set(x_23, 0, x_44); -x_45 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_45, 0, x_23); -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_22); -return x_46; +x_46 = lean_box(x_19); +lean_ctor_set(x_25, 1, x_20); +lean_ctor_set(x_25, 0, x_46); +x_47 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_47, 0, x_25); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_24); +return x_48; } } else { -lean_object* x_47; lean_object* x_48; uint64_t x_49; uint64_t x_50; uint64_t x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; uint64_t x_55; size_t x_56; size_t x_57; size_t x_58; size_t x_59; size_t x_60; lean_object* x_61; uint8_t x_62; -x_47 = lean_ctor_get(x_23, 1); -lean_inc(x_47); -lean_dec(x_23); -x_48 = lean_array_get_size(x_47); -x_49 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_1); -x_50 = 32; -x_51 = lean_uint64_shift_right(x_49, x_50); -x_52 = lean_uint64_xor(x_49, x_51); -x_53 = 16; -x_54 = lean_uint64_shift_right(x_52, x_53); -x_55 = lean_uint64_xor(x_52, x_54); -x_56 = lean_uint64_to_usize(x_55); -x_57 = lean_usize_of_nat(x_48); -lean_dec(x_48); -x_58 = 1; -x_59 = lean_usize_sub(x_57, x_58); -x_60 = lean_usize_land(x_56, x_59); -x_61 = lean_array_uget(x_47, x_60); -lean_dec(x_47); -x_62 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences___spec__7(x_1, x_61); -lean_dec(x_61); -if (x_62 == 0) +lean_object* x_49; lean_object* x_50; uint64_t x_51; uint64_t x_52; uint64_t x_53; uint64_t x_54; uint64_t x_55; uint64_t x_56; uint64_t x_57; size_t x_58; size_t x_59; size_t x_60; size_t x_61; size_t x_62; lean_object* x_63; uint8_t x_64; +x_49 = lean_ctor_get(x_25, 1); +lean_inc(x_49); +lean_dec(x_25); +x_50 = lean_array_get_size(x_49); +x_51 = l___private_Lean_Syntax_0__String_hashRange____x40_Lean_Syntax___hyg_169_(x_1); +x_52 = 32; +x_53 = lean_uint64_shift_right(x_51, x_52); +x_54 = lean_uint64_xor(x_51, x_53); +x_55 = 16; +x_56 = lean_uint64_shift_right(x_54, x_55); +x_57 = lean_uint64_xor(x_54, x_56); +x_58 = lean_uint64_to_usize(x_57); +x_59 = lean_usize_of_nat(x_50); +lean_dec(x_50); +x_60 = 1; +x_61 = lean_usize_sub(x_59, x_60); +x_62 = lean_usize_land(x_58, x_61); +x_63 = lean_array_uget(x_49, x_62); +lean_dec(x_49); +x_64 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__7(x_1, x_63); +lean_dec(x_63); +if (x_64 == 0) { -lean_object* x_63; lean_object* x_64; -x_63 = lean_box(0); -x_64 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__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, x_14, x_15, x_16, x_17, x_18, x_63, x_20, x_21, x_22); +lean_object* x_65; lean_object* x_66; +x_65 = lean_box(0); +x_66 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__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, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_65, x_22, x_23, x_24); lean_dec(x_6); -return x_64; +return x_66; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); +lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -17265,567 +19166,580 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_65 = lean_box(x_17); -x_66 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_66, 0, x_65); -lean_ctor_set(x_66, 1, x_18); -x_67 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_67, 0, x_66); +x_67 = lean_box(x_19); x_68 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_68, 0, x_67); -lean_ctor_set(x_68, 1, x_22); -return x_68; +lean_ctor_set(x_68, 1, x_20); +x_69 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_69, 0, x_68); +x_70 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_70, 0, x_69); +lean_ctor_set(x_70, 1, x_24); +return x_70; } } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19(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, size_t x_13, size_t x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25(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, size_t x_16, size_t x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20, lean_object* x_21) { _start: { -uint8_t x_19; -x_19 = lean_usize_dec_lt(x_14, x_13); -if (x_19 == 0) +uint8_t x_22; +x_22 = lean_usize_dec_lt(x_17, x_16); +if (x_22 == 0) { -lean_object* x_20; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); +lean_object* x_23; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_15); -lean_ctor_set(x_20, 1, x_18); -return x_20; +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_18); +lean_ctor_set(x_23, 1, x_21); +return x_23; } 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_array_uget(x_12, x_14); -x_22 = lean_ctor_get(x_21, 1); -lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 0); -lean_inc(x_23); -lean_dec(x_21); -x_24 = lean_ctor_get(x_22, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_22, 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; lean_object* x_30; uint8_t x_31; +x_24 = lean_array_uget(x_15, x_17); +x_25 = lean_ctor_get(x_24, 1); lean_inc(x_25); -x_26 = lean_ctor_get(x_22, 2); +x_26 = lean_ctor_get(x_24, 0); lean_inc(x_26); -x_27 = lean_ctor_get(x_22, 3); +lean_dec(x_24); +x_27 = lean_ctor_get(x_25, 0); lean_inc(x_27); -lean_dec(x_22); -x_28 = !lean_is_exclusive(x_15); -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; uint8_t x_36; -x_29 = lean_ctor_get(x_15, 0); -x_30 = lean_ctor_get(x_15, 1); -x_31 = lean_st_ref_get(x_10, x_18); -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_27); -x_35 = lean_unsigned_to_nat(0u); -x_36 = lean_nat_dec_lt(x_35, x_34); -if (x_36 == 0) +x_28 = lean_ctor_get(x_25, 1); +lean_inc(x_28); +x_29 = lean_ctor_get(x_25, 2); +lean_inc(x_29); +x_30 = lean_ctor_get(x_25, 3); +lean_inc(x_30); +lean_dec(x_25); +x_31 = !lean_is_exclusive(x_18); +if (x_31 == 0) { -lean_object* x_37; uint8_t x_38; lean_object* x_39; +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_32 = lean_ctor_get(x_18, 0); +x_33 = lean_ctor_get(x_18, 1); +x_34 = lean_st_ref_get(x_13, x_21); +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_array_get_size(x_30); +x_38 = lean_unsigned_to_nat(0u); +x_39 = lean_nat_dec_lt(x_38, x_37); +if (x_39 == 0) +{ +lean_object* x_40; uint8_t x_41; lean_object* x_42; +lean_dec(x_37); +lean_dec(x_35); +lean_free_object(x_18); +x_40 = lean_box(0); +x_41 = lean_unbox(x_32); lean_dec(x_32); -lean_free_object(x_15); -x_37 = lean_box(0); -x_38 = lean_unbox(x_29); -lean_dec(x_29); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_11); -lean_inc(x_6); -lean_inc(x_10); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_14); lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_13); +lean_inc(x_9); lean_inc(x_5); lean_inc(x_1); -x_39 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__6(x_23, x_1, x_25, x_24, x_5, x_7, x_10, x_27, x_8, x_9, x_6, x_4, x_3, x_11, x_26, x_2, x_38, x_30, x_37, x_16, x_17, x_33); -lean_dec(x_27); -if (lean_obj_tag(x_39) == 0) +x_42 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__6(x_26, x_1, x_28, x_27, x_5, x_9, x_13, x_30, x_11, x_12, x_10, x_6, x_7, x_4, x_3, x_14, x_29, x_2, x_41, x_33, x_40, x_19, x_20, x_36); +lean_dec(x_30); +if (lean_obj_tag(x_42) == 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_43; +x_43 = lean_ctor_get(x_42, 0); +lean_inc(x_43); +if (lean_obj_tag(x_43) == 0) { -uint8_t x_41; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); +uint8_t x_44; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_41 = !lean_is_exclusive(x_39); -if (x_41 == 0) +x_44 = !lean_is_exclusive(x_42); +if (x_44 == 0) { -lean_object* x_42; lean_object* x_43; -x_42 = lean_ctor_get(x_39, 0); -lean_dec(x_42); -x_43 = lean_ctor_get(x_40, 0); -lean_inc(x_43); -lean_dec(x_40); -lean_ctor_set(x_39, 0, x_43); -return x_39; +lean_object* x_45; lean_object* x_46; +x_45 = lean_ctor_get(x_42, 0); +lean_dec(x_45); +x_46 = lean_ctor_get(x_43, 0); +lean_inc(x_46); +lean_dec(x_43); +lean_ctor_set(x_42, 0, x_46); +return x_42; } 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_ctor_get(x_40, 0); -lean_inc(x_45); -lean_dec(x_40); -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_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_42, 1); +lean_inc(x_47); +lean_dec(x_42); +x_48 = lean_ctor_get(x_43, 0); +lean_inc(x_48); +lean_dec(x_43); +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_47; lean_object* x_48; size_t x_49; size_t x_50; -x_47 = lean_ctor_get(x_39, 1); -lean_inc(x_47); -lean_dec(x_39); -x_48 = lean_ctor_get(x_40, 0); -lean_inc(x_48); -lean_dec(x_40); -x_49 = 1; -x_50 = lean_usize_add(x_14, x_49); -x_14 = x_50; -x_15 = x_48; -x_18 = x_47; +lean_object* x_50; lean_object* x_51; size_t x_52; size_t x_53; +x_50 = lean_ctor_get(x_42, 1); +lean_inc(x_50); +lean_dec(x_42); +x_51 = lean_ctor_get(x_43, 0); +lean_inc(x_51); +lean_dec(x_43); +x_52 = 1; +x_53 = lean_usize_add(x_17, x_52); +x_17 = x_53; +x_18 = x_51; +x_21 = x_50; goto _start; } } else { -uint8_t x_52; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); +uint8_t x_55; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_52 = !lean_is_exclusive(x_39); -if (x_52 == 0) +x_55 = !lean_is_exclusive(x_42); +if (x_55 == 0) { -return x_39; +return x_42; } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; -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_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_42, 0); +x_57 = lean_ctor_get(x_42, 1); +lean_inc(x_57); +lean_inc(x_56); +lean_dec(x_42); +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 { -size_t x_56; size_t x_57; uint8_t x_58; -x_56 = 0; -x_57 = lean_usize_of_nat(x_34); -lean_dec(x_34); -x_58 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18(x_8, x_9, x_32, x_27, x_56, x_57); -lean_dec(x_32); -if (x_58 == 0) +size_t x_59; size_t x_60; uint8_t x_61; +x_59 = 0; +x_60 = lean_usize_of_nat(x_37); +lean_dec(x_37); +x_61 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24(x_11, x_12, x_35, x_30, x_59, x_60); +lean_dec(x_35); +if (x_61 == 0) { -lean_object* x_59; uint8_t x_60; lean_object* x_61; -lean_free_object(x_15); -x_59 = lean_box(0); -x_60 = lean_unbox(x_29); -lean_dec(x_29); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_11); -lean_inc(x_6); -lean_inc(x_10); +lean_object* x_62; uint8_t x_63; lean_object* x_64; +lean_free_object(x_18); +x_62 = lean_box(0); +x_63 = lean_unbox(x_32); +lean_dec(x_32); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_14); lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_13); +lean_inc(x_9); lean_inc(x_5); lean_inc(x_1); -x_61 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__6(x_23, x_1, x_25, x_24, x_5, x_7, x_10, x_27, x_8, x_9, x_6, x_4, x_3, x_11, x_26, x_2, x_60, x_30, x_59, x_16, x_17, x_33); -lean_dec(x_27); -if (lean_obj_tag(x_61) == 0) +x_64 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__6(x_26, x_1, x_28, x_27, x_5, x_9, x_13, x_30, x_11, x_12, x_10, x_6, x_7, x_4, x_3, x_14, x_29, x_2, x_63, x_33, x_62, x_19, x_20, x_36); +lean_dec(x_30); +if (lean_obj_tag(x_64) == 0) { -lean_object* x_62; -x_62 = lean_ctor_get(x_61, 0); -lean_inc(x_62); -if (lean_obj_tag(x_62) == 0) +lean_object* x_65; +x_65 = lean_ctor_get(x_64, 0); +lean_inc(x_65); +if (lean_obj_tag(x_65) == 0) { -uint8_t x_63; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); +uint8_t x_66; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_63 = !lean_is_exclusive(x_61); -if (x_63 == 0) +x_66 = !lean_is_exclusive(x_64); +if (x_66 == 0) { -lean_object* x_64; lean_object* x_65; -x_64 = lean_ctor_get(x_61, 0); -lean_dec(x_64); -x_65 = lean_ctor_get(x_62, 0); -lean_inc(x_65); -lean_dec(x_62); -lean_ctor_set(x_61, 0, x_65); -return x_61; +lean_object* x_67; lean_object* x_68; +x_67 = lean_ctor_get(x_64, 0); +lean_dec(x_67); +x_68 = lean_ctor_get(x_65, 0); +lean_inc(x_68); +lean_dec(x_65); +lean_ctor_set(x_64, 0, x_68); +return x_64; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_61, 1); -lean_inc(x_66); -lean_dec(x_61); -x_67 = lean_ctor_get(x_62, 0); -lean_inc(x_67); -lean_dec(x_62); -x_68 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_68, 0, x_67); -lean_ctor_set(x_68, 1, x_66); -return x_68; +lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_64, 1); +lean_inc(x_69); +lean_dec(x_64); +x_70 = lean_ctor_get(x_65, 0); +lean_inc(x_70); +lean_dec(x_65); +x_71 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_71, 0, x_70); +lean_ctor_set(x_71, 1, x_69); +return x_71; } } else { -lean_object* x_69; lean_object* x_70; size_t x_71; size_t x_72; -x_69 = lean_ctor_get(x_61, 1); -lean_inc(x_69); -lean_dec(x_61); -x_70 = lean_ctor_get(x_62, 0); -lean_inc(x_70); -lean_dec(x_62); -x_71 = 1; -x_72 = lean_usize_add(x_14, x_71); -x_14 = x_72; -x_15 = x_70; -x_18 = x_69; +lean_object* x_72; lean_object* x_73; size_t x_74; size_t x_75; +x_72 = lean_ctor_get(x_64, 1); +lean_inc(x_72); +lean_dec(x_64); +x_73 = lean_ctor_get(x_65, 0); +lean_inc(x_73); +lean_dec(x_65); +x_74 = 1; +x_75 = lean_usize_add(x_17, x_74); +x_17 = x_75; +x_18 = x_73; +x_21 = x_72; goto _start; } } else { -uint8_t x_74; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); +uint8_t x_77; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_74 = !lean_is_exclusive(x_61); -if (x_74 == 0) +x_77 = !lean_is_exclusive(x_64); +if (x_77 == 0) { -return x_61; +return x_64; } else { -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_61, 0); -x_76 = lean_ctor_get(x_61, 1); -lean_inc(x_76); -lean_inc(x_75); -lean_dec(x_61); -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_78; lean_object* x_79; lean_object* x_80; +x_78 = lean_ctor_get(x_64, 0); +x_79 = lean_ctor_get(x_64, 1); +lean_inc(x_79); +lean_inc(x_78); +lean_dec(x_64); +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 { -size_t x_78; size_t x_79; +size_t x_81; size_t x_82; +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); -x_78 = 1; -x_79 = lean_usize_add(x_14, x_78); -x_14 = x_79; -x_18 = x_33; +x_81 = 1; +x_82 = lean_usize_add(x_17, x_81); +x_17 = x_82; +x_21 = x_36; goto _start; } } } 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; uint8_t x_88; -x_81 = lean_ctor_get(x_15, 0); -x_82 = lean_ctor_get(x_15, 1); -lean_inc(x_82); -lean_inc(x_81); -lean_dec(x_15); -x_83 = lean_st_ref_get(x_10, x_18); -x_84 = lean_ctor_get(x_83, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_83, 1); +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_18, 0); +x_85 = lean_ctor_get(x_18, 1); lean_inc(x_85); -lean_dec(x_83); -x_86 = lean_array_get_size(x_27); -x_87 = lean_unsigned_to_nat(0u); -x_88 = lean_nat_dec_lt(x_87, x_86); -if (x_88 == 0) -{ -lean_object* x_89; uint8_t x_90; lean_object* x_91; +lean_inc(x_84); +lean_dec(x_18); +x_86 = lean_st_ref_get(x_13, x_21); +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_array_get_size(x_30); +x_90 = lean_unsigned_to_nat(0u); +x_91 = lean_nat_dec_lt(x_90, x_89); +if (x_91 == 0) +{ +lean_object* x_92; uint8_t x_93; lean_object* x_94; +lean_dec(x_89); +lean_dec(x_87); +x_92 = lean_box(0); +x_93 = lean_unbox(x_84); lean_dec(x_84); -x_89 = lean_box(0); -x_90 = lean_unbox(x_81); -lean_dec(x_81); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_11); -lean_inc(x_6); -lean_inc(x_10); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_14); lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_13); +lean_inc(x_9); lean_inc(x_5); lean_inc(x_1); -x_91 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__6(x_23, x_1, x_25, x_24, x_5, x_7, x_10, x_27, x_8, x_9, x_6, x_4, x_3, x_11, x_26, x_2, x_90, x_82, x_89, x_16, x_17, x_85); -lean_dec(x_27); -if (lean_obj_tag(x_91) == 0) +x_94 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__6(x_26, x_1, x_28, x_27, x_5, x_9, x_13, x_30, x_11, x_12, x_10, x_6, x_7, x_4, x_3, x_14, x_29, x_2, x_93, x_85, x_92, x_19, x_20, x_88); +lean_dec(x_30); +if (lean_obj_tag(x_94) == 0) { -lean_object* x_92; -x_92 = lean_ctor_get(x_91, 0); -lean_inc(x_92); -if (lean_obj_tag(x_92) == 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_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); +lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -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; +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_91); - x_94 = lean_box(0); + lean_dec_ref(x_94); + x_97 = lean_box(0); } -x_95 = lean_ctor_get(x_92, 0); -lean_inc(x_95); -lean_dec(x_92); -if (lean_is_scalar(x_94)) { - x_96 = lean_alloc_ctor(0, 2, 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_96 = x_94; + x_99 = x_97; } -lean_ctor_set(x_96, 0, x_95); -lean_ctor_set(x_96, 1, x_93); -return x_96; +lean_ctor_set(x_99, 0, x_98); +lean_ctor_set(x_99, 1, x_96); +return x_99; } else { -lean_object* x_97; lean_object* x_98; size_t x_99; size_t x_100; -x_97 = lean_ctor_get(x_91, 1); -lean_inc(x_97); -lean_dec(x_91); -x_98 = lean_ctor_get(x_92, 0); -lean_inc(x_98); -lean_dec(x_92); -x_99 = 1; -x_100 = lean_usize_add(x_14, x_99); -x_14 = x_100; -x_15 = x_98; -x_18 = x_97; +lean_object* x_100; lean_object* x_101; size_t x_102; size_t x_103; +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_102 = 1; +x_103 = lean_usize_add(x_17, x_102); +x_17 = x_103; +x_18 = x_101; +x_21 = x_100; goto _start; } } else { -lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); +lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_102 = lean_ctor_get(x_91, 0); -lean_inc(x_102); -x_103 = lean_ctor_get(x_91, 1); -lean_inc(x_103); -if (lean_is_exclusive(x_91)) { - lean_ctor_release(x_91, 0); - lean_ctor_release(x_91, 1); - x_104 = x_91; +x_105 = lean_ctor_get(x_94, 0); +lean_inc(x_105); +x_106 = lean_ctor_get(x_94, 1); +lean_inc(x_106); +if (lean_is_exclusive(x_94)) { + lean_ctor_release(x_94, 0); + lean_ctor_release(x_94, 1); + x_107 = x_94; } else { - lean_dec_ref(x_91); - x_104 = lean_box(0); + lean_dec_ref(x_94); + x_107 = lean_box(0); } -if (lean_is_scalar(x_104)) { - x_105 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_107)) { + x_108 = lean_alloc_ctor(1, 2, 0); } else { - x_105 = x_104; + x_108 = x_107; } -lean_ctor_set(x_105, 0, x_102); -lean_ctor_set(x_105, 1, x_103); -return x_105; +lean_ctor_set(x_108, 0, x_105); +lean_ctor_set(x_108, 1, x_106); +return x_108; } } else { -size_t x_106; size_t x_107; uint8_t x_108; -x_106 = 0; -x_107 = lean_usize_of_nat(x_86); -lean_dec(x_86); -x_108 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18(x_8, x_9, x_84, x_27, x_106, x_107); -lean_dec(x_84); -if (x_108 == 0) +size_t x_109; size_t x_110; uint8_t x_111; +x_109 = 0; +x_110 = lean_usize_of_nat(x_89); +lean_dec(x_89); +x_111 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24(x_11, x_12, x_87, x_30, x_109, x_110); +lean_dec(x_87); +if (x_111 == 0) { -lean_object* x_109; uint8_t x_110; lean_object* x_111; -x_109 = lean_box(0); -x_110 = lean_unbox(x_81); -lean_dec(x_81); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_11); -lean_inc(x_6); -lean_inc(x_10); +lean_object* x_112; uint8_t x_113; lean_object* x_114; +x_112 = lean_box(0); +x_113 = lean_unbox(x_84); +lean_dec(x_84); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_14); lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_13); +lean_inc(x_9); lean_inc(x_5); lean_inc(x_1); -x_111 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__6(x_23, x_1, x_25, x_24, x_5, x_7, x_10, x_27, x_8, x_9, x_6, x_4, x_3, x_11, x_26, x_2, x_110, x_82, x_109, x_16, x_17, x_85); -lean_dec(x_27); -if (lean_obj_tag(x_111) == 0) +x_114 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__6(x_26, x_1, x_28, x_27, x_5, x_9, x_13, x_30, x_11, x_12, x_10, x_6, x_7, x_4, x_3, x_14, x_29, x_2, x_113, x_85, x_112, x_19, x_20, x_88); +lean_dec(x_30); +if (lean_obj_tag(x_114) == 0) { -lean_object* x_112; -x_112 = lean_ctor_get(x_111, 0); -lean_inc(x_112); -if (lean_obj_tag(x_112) == 0) +lean_object* x_115; +x_115 = lean_ctor_get(x_114, 0); +lean_inc(x_115); +if (lean_obj_tag(x_115) == 0) { -lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); +lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_113 = lean_ctor_get(x_111, 1); -lean_inc(x_113); -if (lean_is_exclusive(x_111)) { - lean_ctor_release(x_111, 0); - lean_ctor_release(x_111, 1); - x_114 = x_111; +x_116 = lean_ctor_get(x_114, 1); +lean_inc(x_116); +if (lean_is_exclusive(x_114)) { + lean_ctor_release(x_114, 0); + lean_ctor_release(x_114, 1); + x_117 = x_114; } else { - lean_dec_ref(x_111); - x_114 = lean_box(0); + lean_dec_ref(x_114); + x_117 = lean_box(0); } -x_115 = lean_ctor_get(x_112, 0); -lean_inc(x_115); -lean_dec(x_112); -if (lean_is_scalar(x_114)) { - x_116 = lean_alloc_ctor(0, 2, 0); +x_118 = lean_ctor_get(x_115, 0); +lean_inc(x_118); +lean_dec(x_115); +if (lean_is_scalar(x_117)) { + x_119 = lean_alloc_ctor(0, 2, 0); } else { - x_116 = x_114; + x_119 = x_117; } -lean_ctor_set(x_116, 0, x_115); -lean_ctor_set(x_116, 1, x_113); -return x_116; +lean_ctor_set(x_119, 0, x_118); +lean_ctor_set(x_119, 1, x_116); +return x_119; } else { -lean_object* x_117; lean_object* x_118; size_t x_119; size_t x_120; -x_117 = lean_ctor_get(x_111, 1); -lean_inc(x_117); -lean_dec(x_111); -x_118 = lean_ctor_get(x_112, 0); -lean_inc(x_118); -lean_dec(x_112); -x_119 = 1; -x_120 = lean_usize_add(x_14, x_119); -x_14 = x_120; -x_15 = x_118; -x_18 = x_117; +lean_object* x_120; lean_object* x_121; size_t x_122; size_t x_123; +x_120 = lean_ctor_get(x_114, 1); +lean_inc(x_120); +lean_dec(x_114); +x_121 = lean_ctor_get(x_115, 0); +lean_inc(x_121); +lean_dec(x_115); +x_122 = 1; +x_123 = lean_usize_add(x_17, x_122); +x_17 = x_123; +x_18 = x_121; +x_21 = x_120; goto _start; } } else { -lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_11); -lean_dec(x_10); +lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_122 = lean_ctor_get(x_111, 0); -lean_inc(x_122); -x_123 = lean_ctor_get(x_111, 1); -lean_inc(x_123); -if (lean_is_exclusive(x_111)) { - lean_ctor_release(x_111, 0); - lean_ctor_release(x_111, 1); - x_124 = x_111; +x_125 = lean_ctor_get(x_114, 0); +lean_inc(x_125); +x_126 = lean_ctor_get(x_114, 1); +lean_inc(x_126); +if (lean_is_exclusive(x_114)) { + lean_ctor_release(x_114, 0); + lean_ctor_release(x_114, 1); + x_127 = x_114; } else { - lean_dec_ref(x_111); - x_124 = lean_box(0); + lean_dec_ref(x_114); + x_127 = lean_box(0); } -if (lean_is_scalar(x_124)) { - x_125 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_127)) { + x_128 = lean_alloc_ctor(1, 2, 0); } else { - x_125 = x_124; + x_128 = x_127; } -lean_ctor_set(x_125, 0, x_122); -lean_ctor_set(x_125, 1, x_123); -return x_125; +lean_ctor_set(x_128, 0, x_125); +lean_ctor_set(x_128, 1, x_126); +return x_128; } } else { -lean_object* x_126; size_t x_127; size_t x_128; +lean_object* x_129; size_t x_130; size_t x_131; +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); -x_126 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_126, 0, x_81); -lean_ctor_set(x_126, 1, x_82); -x_127 = 1; -x_128 = lean_usize_add(x_14, x_127); -x_14 = x_128; -x_15 = x_126; -x_18 = x_85; +x_129 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_129, 0, x_84); +lean_ctor_set(x_129, 1, x_85); +x_130 = 1; +x_131 = lean_usize_add(x_17, x_130); +x_17 = x_131; +x_18 = x_129; +x_21 = x_88; goto _start; } } @@ -17833,7 +19747,7 @@ goto _start; } } } -static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__1() { +static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__1() { _start: { lean_object* x_1; @@ -17841,7 +19755,7 @@ x_1 = lean_mk_string_unchecked("Init.Data.Option.BasicAux", 25, 25); return x_1; } } -static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__2() { +static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__2() { _start: { lean_object* x_1; @@ -17849,7 +19763,7 @@ x_1 = lean_mk_string_unchecked("Option.get!", 11, 11); return x_1; } } -static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__3() { +static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__3() { _start: { lean_object* x_1; @@ -17857,20 +19771,20 @@ x_1 = lean_mk_string_unchecked("value is none", 13, 13); return x_1; } } -static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__4() { +static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___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; -x_1 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__1; -x_2 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__2; +x_1 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__1; +x_2 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__2; x_3 = lean_unsigned_to_nat(16u); x_4 = lean_unsigned_to_nat(14u); -x_5 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__3; +x_5 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___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 uint8_t l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; @@ -17882,7 +19796,7 @@ x_7 = l_Lean_Syntax_getPos_x3f(x_6, x_4); if (lean_obj_tag(x_5) == 0) { lean_object* x_8; lean_object* x_9; -x_8 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__4; +x_8 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__4; x_9 = l_panic___at_Lean_Parser_ParserState_mkUnexpectedTokenErrors___spec__1(x_8); if (lean_obj_tag(x_7) == 0) { @@ -17913,7 +19827,7 @@ lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; x_14 = lean_ctor_get(x_5, 0); lean_inc(x_14); lean_dec(x_5); -x_15 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__4; +x_15 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__4; x_16 = l_panic___at_Lean_Parser_ParserState_mkUnexpectedTokenErrors___spec__1(x_15); x_17 = lean_nat_dec_lt(x_14, x_16); lean_dec(x_16); @@ -17937,15 +19851,15 @@ return x_20; } } } -static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___closed__1() { +static lean_object* _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___boxed), 2, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -17958,7 +19872,7 @@ return x_1; else { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_5 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___closed__1; +x_5 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___closed__1; lean_inc(x_2); x_6 = l_Array_qpartition___rarg(x_1, x_5, x_2, x_3); x_7 = lean_ctor_get(x_6, 0); @@ -17970,7 +19884,7 @@ x_9 = lean_nat_dec_le(x_3, x_7); if (x_9 == 0) { lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(x_8, x_2, x_7); +x_10 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(x_8, x_2, x_7); x_11 = lean_unsigned_to_nat(1u); x_12 = lean_nat_add(x_7, x_11); lean_dec(x_7); @@ -17987,7 +19901,7 @@ return x_8; } } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__1() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__1() { _start: { lean_object* x_1; @@ -17995,16 +19909,16 @@ x_1 = lean_mk_string_unchecked("note: this linter can be disabled with `set_opti return x_1; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__2() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__1; +x_1 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__3() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__3() { _start: { lean_object* x_1; @@ -18012,16 +19926,16 @@ x_1 = lean_mk_string_unchecked(" false`", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__4() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__3; +x_1 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__5() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -18030,7 +19944,7 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__6() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__6() { _start: { lean_object* x_1; @@ -18038,16 +19952,16 @@ x_1 = lean_mk_string_unchecked("\n", 1, 1); return x_1; } } -static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__7() { +static lean_object* _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__6; +x_1 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__6; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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) { _start: { uint8_t x_7; @@ -18060,19 +19974,19 @@ x_9 = lean_ctor_get(x_1, 1); lean_dec(x_9); lean_inc(x_8); x_10 = l_Lean_MessageData_ofName(x_8); -x_11 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__2; +x_11 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__2; lean_ctor_set_tag(x_1, 7); lean_ctor_set(x_1, 1, x_10); lean_ctor_set(x_1, 0, x_11); -x_12 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__4; +x_12 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__4; x_13 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_13, 0, x_1); lean_ctor_set(x_13, 1, x_12); -x_14 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__5; +x_14 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__5; x_15 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_3); -x_16 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__7; +x_16 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__7; x_17 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); @@ -18097,19 +20011,19 @@ lean_inc(x_23); lean_dec(x_1); lean_inc(x_23); x_24 = l_Lean_MessageData_ofName(x_23); -x_25 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__2; +x_25 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__2; x_26 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_26, 0, x_25); lean_ctor_set(x_26, 1, x_24); -x_27 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__4; +x_27 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__4; 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_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__5; +x_29 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__5; x_30 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_30, 0, x_29); lean_ctor_set(x_30, 1, x_3); -x_31 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__7; +x_31 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___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); @@ -18128,7 +20042,7 @@ return x_37; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__1() { _start: { lean_object* x_1; @@ -18136,16 +20050,16 @@ x_1 = lean_mk_string_unchecked("unused variable `", 17, 17); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__1; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__3() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__3() { _start: { lean_object* x_1; @@ -18153,16 +20067,16 @@ x_1 = lean_mk_string_unchecked("`", 1, 1); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__4() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__3; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22(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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28(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) { _start: { uint8_t x_8; @@ -18188,17 +20102,17 @@ lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean x_12 = lean_ctor_get(x_10, 0); x_13 = lean_ctor_get(x_10, 1); x_14 = l_Lean_MessageData_ofName(x_13); -x_15 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__2; +x_15 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__2; lean_ctor_set_tag(x_10, 7); lean_ctor_set(x_10, 1, x_14); lean_ctor_set(x_10, 0, x_15); -x_16 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__4; +x_16 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__4; x_17 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_17, 0, x_10); lean_ctor_set(x_17, 1, x_16); x_18 = l_Lean_Linter_getLinterUnusedVariables___closed__1; lean_inc(x_5); -x_19 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21(x_18, x_12, x_17, x_5, x_6, x_7); +x_19 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27(x_18, x_12, x_17, x_5, x_6, x_7); lean_dec(x_12); x_20 = lean_ctor_get(x_19, 1); lean_inc(x_20); @@ -18220,17 +20134,17 @@ lean_inc(x_26); lean_inc(x_25); lean_dec(x_10); x_27 = l_Lean_MessageData_ofName(x_26); -x_28 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__2; +x_28 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__2; x_29 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_29, 0, x_28); lean_ctor_set(x_29, 1, x_27); -x_30 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__4; +x_30 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__4; x_31 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_31, 0, x_29); lean_ctor_set(x_31, 1, x_30); x_32 = l_Lean_Linter_getLinterUnusedVariables___closed__1; lean_inc(x_5); -x_33 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21(x_32, x_25, x_31, x_5, x_6, x_7); +x_33 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27(x_32, x_25, x_31, x_5, x_6, x_7); lean_dec(x_25); x_34 = lean_ctor_get(x_33, 1); lean_inc(x_34); @@ -18246,7 +20160,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(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_Linter_UnusedVariables_unusedVariables___elambda__1___spec__29(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -18255,7 +20169,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_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(x_4, x_6); +x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4(x_4, x_6); lean_dec(x_6); x_8 = 1; x_9 = lean_usize_add(x_2, x_8); @@ -18269,7 +20183,7 @@ return x_4; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24(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_Linter_UnusedVariables_unusedVariables___elambda__1___spec__30(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -18291,7 +20205,7 @@ return x_4; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25(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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__31(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { _start: { uint8_t x_7; @@ -18315,7 +20229,7 @@ return x_6; } } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(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_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__32(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; @@ -18447,9 +20361,8 @@ if (x_18 == 0) { lean_dec(x_16); lean_dec(x_15); -lean_dec(x_9); -lean_inc(x_8); -x_20 = x_8; +lean_inc(x_9); +x_20 = x_9; goto block_110; } else @@ -18460,9 +20373,8 @@ if (x_111 == 0) { lean_dec(x_16); lean_dec(x_15); -lean_dec(x_9); -lean_inc(x_8); -x_20 = x_8; +lean_inc(x_9); +x_20 = x_9; goto block_110; } else @@ -18471,8 +20383,9 @@ size_t x_112; size_t x_113; lean_object* x_114; x_112 = 0; x_113 = lean_usize_of_nat(x_16); lean_dec(x_16); +lean_inc(x_9); lean_inc(x_8); -x_114 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25(x_9, x_1, x_15, x_112, x_113, x_8); +x_114 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__31(x_8, x_1, x_15, x_112, x_113, x_9); lean_dec(x_15); x_20 = x_114; goto block_110; @@ -18525,7 +20438,7 @@ size_t x_104; size_t x_105; lean_object* x_106; lean_object* x_107; lean_object* x_104 = 0; x_105 = lean_usize_of_nat(x_22); lean_dec(x_22); -x_106 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24(x_21, x_104, x_105, x_19); +x_106 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__30(x_21, x_104, x_105, x_19); lean_dec(x_21); x_107 = lean_st_mk_ref(x_106, x_13); x_108 = lean_ctor_get(x_107, 0); @@ -18584,7 +20497,7 @@ else size_t x_60; lean_object* x_61; x_60 = lean_usize_of_nat(x_32); lean_dec(x_32); -x_61 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(x_31, x_36, x_60, x_2); +x_61 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__29(x_31, x_36, x_60, x_2); lean_dec(x_31); x_37 = x_61; goto block_58; @@ -18596,9 +20509,11 @@ size_t x_38; lean_object* x_39; x_38 = lean_array_size(x_37); lean_inc(x_12); lean_inc(x_11); -x_39 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19(x_3, x_4, x_5, x_6, x_7, x_8, x_1, x_20, x_20, x_24, x_28, x_37, x_38, x_36, x_26, x_11, x_12, x_29); +lean_inc(x_9); +x_39 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_9, x_1, x_20, x_20, x_20, x_24, x_28, x_37, x_38, x_36, x_26, x_11, x_12, x_29); lean_dec(x_37); lean_dec(x_20); +lean_dec(x_9); 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; size_t x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; @@ -18614,11 +20529,11 @@ x_43 = lean_array_get_size(x_42); x_44 = lean_unsigned_to_nat(1u); x_45 = lean_nat_sub(x_43, x_44); lean_dec(x_43); -x_46 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(x_42, x_17, x_45); +x_46 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(x_42, x_17, x_45); lean_dec(x_45); x_47 = lean_array_size(x_46); x_48 = lean_box(0); -x_49 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22(x_46, x_47, x_36, x_48, x_11, x_12, x_41); +x_49 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28(x_46, x_47, x_36, x_48, x_11, x_12, x_41); lean_dec(x_12); lean_dec(x_46); x_50 = !lean_is_exclusive(x_49); @@ -18713,7 +20628,7 @@ else size_t x_94; lean_object* x_95; x_94 = lean_usize_of_nat(x_66); lean_dec(x_66); -x_95 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(x_65, x_71, x_94, x_2); +x_95 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__29(x_65, x_71, x_94, x_2); lean_dec(x_65); x_72 = x_95; goto block_92; @@ -18725,9 +20640,11 @@ size_t x_73; lean_object* x_74; x_73 = lean_array_size(x_72); lean_inc(x_12); lean_inc(x_11); -x_74 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19(x_3, x_4, x_5, x_6, x_7, x_8, x_1, x_20, x_20, x_24, x_62, x_72, x_73, x_71, x_70, x_11, x_12, x_63); +lean_inc(x_9); +x_74 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_9, x_1, x_20, x_20, x_20, x_24, x_62, x_72, x_73, x_71, x_70, x_11, x_12, x_63); lean_dec(x_72); lean_dec(x_20); +lean_dec(x_9); 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; lean_object* x_80; lean_object* x_81; size_t x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; @@ -18743,11 +20660,11 @@ x_78 = lean_array_get_size(x_77); x_79 = lean_unsigned_to_nat(1u); x_80 = lean_nat_sub(x_78, x_79); lean_dec(x_78); -x_81 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(x_77, x_17, x_80); +x_81 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(x_77, x_17, x_80); lean_dec(x_80); x_82 = lean_array_size(x_81); x_83 = lean_box(0); -x_84 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22(x_81, x_82, x_71, x_83, x_11, x_12, x_76); +x_84 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28(x_81, x_82, x_71, x_83, x_11, x_12, x_76); lean_dec(x_12); lean_dec(x_81); x_85 = lean_ctor_get(x_84, 1); @@ -18806,7 +20723,7 @@ static lean_object* _init_l_Lean_Linter_UnusedVariables_unusedVariables___elambd { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Linter_UnusedVariables_visitAssignments___closed__3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; x_3 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_1); @@ -18858,11 +20775,11 @@ 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_free_object(x_18); -x_26 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1; +x_26 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; x_27 = l_Lean_Linter_UnusedVariables_visitAssignments___closed__1; x_28 = l_Lean_Linter_UnusedVariables_visitAssignments___closed__3; x_29 = lean_box(0); -x_30 = l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__1(x_20, x_26, x_3, x_1, x_4, x_5, x_27, x_28, x_10, x_29, x_7, x_8, x_21); +x_30 = l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__1(x_20, x_26, x_3, x_1, x_4, x_5, x_27, x_10, x_28, x_29, x_7, x_8, x_21); return x_30; } else @@ -18896,11 +20813,11 @@ lean_dec(x_35); if (x_37 == 0) { lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_38 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1; +x_38 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; x_39 = l_Lean_Linter_UnusedVariables_visitAssignments___closed__1; x_40 = l_Lean_Linter_UnusedVariables_visitAssignments___closed__3; x_41 = lean_box(0); -x_42 = l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__1(x_32, x_38, x_3, x_1, x_4, x_5, x_39, x_40, x_10, x_41, x_7, x_8, x_33); +x_42 = l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__1(x_32, x_38, x_3, x_1, x_4, x_5, x_39, x_10, x_40, x_41, x_7, x_8, x_33); return x_42; } else @@ -19007,11 +20924,11 @@ 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_dec(x_65); -x_70 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1; +x_70 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1; x_71 = l_Lean_Linter_UnusedVariables_visitAssignments___closed__1; x_72 = l_Lean_Linter_UnusedVariables_visitAssignments___closed__3; x_73 = lean_box(0); -x_74 = l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__1(x_63, x_70, x_3, x_1, x_4, x_5, x_71, x_72, x_10, x_73, x_7, x_8, x_64); +x_74 = l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__1(x_63, x_70, x_3, x_1, x_4, x_5, x_71, x_10, x_72, x_73, x_7, x_8, x_64); return x_74; } else @@ -19131,7 +21048,7 @@ else size_t x_28; size_t x_29; lean_object* x_30; x_28 = 0; x_29 = lean_usize_of_nat(x_18); -x_30 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(x_17, x_28, x_29, x_3, x_4, x_13); +x_30 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__32(x_17, x_28, x_29, x_3, x_4, x_13); if (lean_obj_tag(x_30) == 0) { lean_object* x_31; lean_object* x_32; uint8_t x_33; @@ -19371,7 +21288,7 @@ static lean_object* _init_l_Lean_Linter_UnusedVariables_unusedVariables___closed lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__7; x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__8; -x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__11; +x_3 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__11; x_4 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_8____closed__2; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; @@ -19414,20 +21331,31 @@ lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(x_1, x_2, x_3); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__3(x_1, x_2); +x_3 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__4(x_1, x_2); lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___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_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___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_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___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); @@ -19436,11 +21364,11 @@ lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___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_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___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_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___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_4); @@ -19463,18 +21391,7 @@ x_10 = lean_box(x_9); return x_10; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(x_1, x_2, x_3); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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) { _start: { size_t x_7; size_t x_8; uint8_t x_9; lean_object* x_10; @@ -19482,7 +21399,7 @@ 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_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__12(x_1, x_2, x_3, x_4, x_7, x_8); +x_9 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__11(x_1, x_2, x_3, x_4, x_7, x_8); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -19491,17 +21408,47 @@ x_10 = lean_box(x_9); return x_10; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14___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_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__13(x_1, x_2, x_3, x_4); +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_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14(x_1, x_5, x_6, x_4); lean_dec(x_1); -return x_5; +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15(x_1, x_2, x_3, x_7, x_8, x_6); +lean_dec(x_3); +lean_dec(x_2); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___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_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16(x_1, x_5, x_6, x_4); +lean_dec(x_1); +return x_7; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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: { size_t x_7; size_t x_8; lean_object* x_9; @@ -19509,35 +21456,74 @@ x_7 = lean_unbox_usize(x_4); lean_dec(x_4); x_8 = lean_unbox_usize(x_5); lean_dec(x_5); -x_9 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__14(x_1, x_2, x_3, x_7, x_8, x_6); +x_9 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(x_1, x_2, x_3, x_7, x_8, x_6); +lean_dec(x_3); +lean_dec(x_2); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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; +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_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18(x_1, x_5, x_6, x_4); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___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_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19(x_1, x_5, x_6, x_4); lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(x_1, x_2, x_3, x_7, x_8, x_6); +lean_dec(x_3); +lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__1(x_1, x_2); +x_3 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___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_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___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_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___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: { uint8_t x_7; lean_object* x_8; -x_7 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_3); x_8 = lean_box(x_7); return x_8; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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) { _start: { size_t x_12; size_t x_13; lean_object* x_14; @@ -19545,23 +21531,23 @@ x_12 = lean_unbox_usize(x_7); lean_dec(x_7); x_13 = lean_unbox_usize(x_8); lean_dec(x_8); -x_14 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15(x_1, x_2, x_3, x_4, x_5, x_6, x_12, x_13, x_9, x_10, x_11); +x_14 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21(x_1, x_2, x_3, x_4, x_5, x_6, x_12, x_13, x_9, x_10, x_11); lean_dec(x_6); return x_14; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16___lambda__1(x_1, x_2); +x_3 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___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_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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) { _start: { size_t x_12; size_t x_13; lean_object* x_14; @@ -19569,12 +21555,12 @@ x_12 = lean_unbox_usize(x_7); lean_dec(x_7); x_13 = lean_unbox_usize(x_8); lean_dec(x_8); -x_14 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__15___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__16(x_1, x_2, x_3, x_4, x_5, x_6, x_12, x_13, x_9, x_10, x_11); +x_14 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22(x_1, x_2, x_3, x_4, x_5, x_6, x_12, x_13, x_9, x_10, x_11); lean_dec(x_6); return x_14; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___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_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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) { _start: { size_t x_7; size_t x_8; uint8_t x_9; lean_object* x_10; @@ -19582,13 +21568,13 @@ 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_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__17(x_1, x_2, x_3, x_4, x_7, x_8); +x_9 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(x_1, x_2, x_3, x_4, x_7, x_8); lean_dec(x_4); x_10 = lean_box(x_9); return x_10; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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) { _start: { size_t x_7; size_t x_8; uint8_t x_9; lean_object* x_10; @@ -19596,7 +21582,7 @@ 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_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__18(x_1, x_2, x_3, x_4, x_7, x_8); +x_9 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24(x_1, x_2, x_3, x_4, x_7, x_8); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -19605,47 +21591,65 @@ x_10 = lean_box(x_9); return x_10; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__1___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__1___boxed(lean_object* x_1) { _start: { uint8_t x_2; lean_object* x_3; -x_2 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__1(x_1); +x_2 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__1(x_1); lean_dec(x_1); x_3 = lean_box(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___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: { uint8_t x_9; lean_object* x_10; x_9 = lean_unbox(x_3); lean_dec(x_3); -x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__2(x_1, x_2, x_9, x_4, x_5, x_6, x_7, x_8); +x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__2(x_1, x_2, x_9, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); return x_10; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___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_16; lean_object* x_17; -x_16 = lean_unbox(x_10); -lean_dec(x_10); -x_17 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_16, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_14); -lean_dec(x_13); +uint8_t x_18; lean_object* x_19; +x_18 = lean_unbox(x_12); lean_dec(x_12); +x_19 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___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_18, x_13, x_14, x_15, x_16, 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_6); lean_dec(x_4); -return x_17; +return x_19; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__4___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -19667,25 +21671,28 @@ 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]; _start: { -uint8_t x_22; uint8_t x_23; lean_object* x_24; -x_22 = lean_unbox(x_10); -lean_dec(x_10); -x_23 = lean_unbox(x_16); -lean_dec(x_16); -x_24 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_22, x_11, x_12, x_13, x_14, x_15, x_23, x_17, x_18, x_19, x_20, x_21); +uint8_t x_24; uint8_t x_25; lean_object* x_26; +x_24 = lean_unbox(x_12); +lean_dec(x_12); +x_25 = lean_unbox(x_18); lean_dec(x_18); -lean_dec(x_15); -lean_dec(x_11); +x_26 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___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_24, x_13, x_14, x_15, x_16, x_17, x_25, x_19, x_20, x_21, x_22, x_23); +lean_dec(x_20); +lean_dec(x_17); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -return x_24; +return x_26; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -19708,25 +21715,28 @@ 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]; _start: { -uint8_t x_23; uint8_t x_24; lean_object* x_25; -x_23 = lean_unbox(x_12); -lean_dec(x_12); -x_24 = lean_unbox(x_17); -lean_dec(x_17); -x_25 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_23, x_13, x_14, x_15, x_16, x_24, x_18, x_19, x_20, x_21, x_22); +uint8_t x_25; uint8_t x_26; lean_object* x_27; +x_25 = lean_unbox(x_14); +lean_dec(x_14); +x_26 = lean_unbox(x_19); lean_dec(x_19); -lean_dec(x_16); -lean_dec(x_13); +x_27 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__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, x_25, x_15, x_16, x_17, x_18, x_26, x_20, x_21, x_22, x_23, x_24); +lean_dec(x_21); +lean_dec(x_18); +lean_dec(x_15); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); -return x_25; +return x_27; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__6___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__6___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -19749,24 +21759,27 @@ 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]; _start: { -uint8_t x_23; uint8_t x_24; lean_object* x_25; -x_23 = lean_unbox(x_12); -lean_dec(x_12); -x_24 = lean_unbox(x_17); -lean_dec(x_17); -x_25 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_23, x_13, x_14, x_15, x_16, x_24, x_18, x_19, x_20, x_21, x_22); +uint8_t x_25; uint8_t x_26; lean_object* x_27; +x_25 = lean_unbox(x_14); +lean_dec(x_14); +x_26 = lean_unbox(x_19); lean_dec(x_19); -lean_dec(x_16); -lean_dec(x_13); +x_27 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__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_25, x_15, x_16, x_17, x_18, x_26, x_20, x_21, x_22, x_23, x_24); +lean_dec(x_21); +lean_dec(x_18); +lean_dec(x_15); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -return x_25; +return x_27; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -19785,55 +21798,60 @@ 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]; _start: { -uint8_t x_19; size_t x_20; size_t x_21; lean_object* x_22; -x_19 = lean_unbox(x_4); +uint8_t x_22; size_t x_23; size_t x_24; lean_object* x_25; +x_22 = lean_unbox(x_4); lean_dec(x_4); -x_20 = lean_unbox_usize(x_13); -lean_dec(x_13); -x_21 = lean_unbox_usize(x_14); -lean_dec(x_14); -x_22 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19(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_20, x_21, x_15, x_16, x_17, x_18); +x_23 = lean_unbox_usize(x_16); +lean_dec(x_16); +x_24 = lean_unbox_usize(x_17); +lean_dec(x_17); +x_25 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25(x_1, x_2, x_3, x_22, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_23, x_24, x_18, x_19, x_20, x_21); +lean_dec(x_15); lean_dec(x_12); -lean_dec(x_9); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_8); lean_dec(x_3); lean_dec(x_2); -return x_22; +return x_25; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___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_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1(x_1, x_2); +x_3 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___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_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20(x_1, x_2, x_3); +x_4 = l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(x_1, x_2, x_3); lean_dec(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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_EXPORT lean_object* l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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) { _start: { lean_object* x_7; -x_7 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_2); return x_7; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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) { _start: { size_t x_8; size_t x_9; lean_object* x_10; @@ -19841,13 +21859,13 @@ x_8 = lean_unbox_usize(x_2); lean_dec(x_2); x_9 = lean_unbox_usize(x_3); lean_dec(x_3); -x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22(x_1, x_8, x_9, x_4, x_5, x_6, x_7); +x_10 = l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28(x_1, x_8, x_9, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_1); return x_10; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23___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_Linter_UnusedVariables_unusedVariables___elambda__1___spec__29___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; @@ -19855,12 +21873,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_Linter_UnusedVariables_unusedVariables___elambda__1___spec__23(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__29(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24___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_Linter_UnusedVariables_unusedVariables___elambda__1___spec__30___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; @@ -19868,12 +21886,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_Linter_UnusedVariables_unusedVariables___elambda__1___spec__24(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__30(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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) { _start: { size_t x_7; size_t x_8; lean_object* x_9; @@ -19881,13 +21899,13 @@ x_7 = lean_unbox_usize(x_4); lean_dec(x_4); x_8 = lean_unbox_usize(x_5); lean_dec(x_5); -x_9 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25(x_1, x_2, x_3, x_7, x_8, x_6); +x_9 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__31(x_1, x_2, x_3, x_7, x_8, x_6); lean_dec(x_3); lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__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) { _start: { size_t x_7; size_t x_8; lean_object* x_9; @@ -19895,7 +21913,7 @@ x_7 = lean_unbox_usize(x_2); lean_dec(x_2); x_8 = lean_unbox_usize(x_3); lean_dec(x_3); -x_9 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26(x_1, x_7, x_8, x_4, x_5, x_6); +x_9 = l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__32(x_1, x_7, x_8, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); @@ -19946,7 +21964,7 @@ lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_initFn____x40_Lean_Linter_UnusedVariables___hyg_5794_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_UnusedVariables_initFn____x40_Lean_Linter_UnusedVariables___hyg_6304_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -20069,6 +22087,21 @@ if (lean_io_result_is_error(res)) return res; l_Lean_Linter_linter_unusedVariables_patternVars = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Linter_linter_unusedVariables_patternVars); lean_dec_ref(res); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125____closed__5); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_125_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +l_Lean_Linter_linter_unusedVariables_analyzeTactics = lean_io_result_get_value(res); +lean_mark_persistent(l_Lean_Linter_linter_unusedVariables_analyzeTactics); +lean_dec_ref(res); }l_Lean_Linter_getLinterUnusedVariables___closed__1 = _init_l_Lean_Linter_getLinterUnusedVariables___closed__1(); lean_mark_persistent(l_Lean_Linter_getLinterUnusedVariables___closed__1); l_Lean_Linter_mkIgnoreFnImpl___closed__1 = _init_l_Lean_Linter_mkIgnoreFnImpl___closed__1(); @@ -20085,418 +22118,418 @@ l_Lean_Linter_mkIgnoreFnImpl___closed__6 = _init_l_Lean_Linter_mkIgnoreFnImpl___ lean_mark_persistent(l_Lean_Linter_mkIgnoreFnImpl___closed__6); l_Lean_Linter_mkIgnoreFnImpl___closed__7 = _init_l_Lean_Linter_mkIgnoreFnImpl___closed__7(); lean_mark_persistent(l_Lean_Linter_mkIgnoreFnImpl___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_340_(lean_io_mk_world()); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_379_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Linter_builtinUnusedVariablesIgnoreFnsRef = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Linter_builtinUnusedVariablesIgnoreFnsRef); lean_dec_ref(res); }l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn___closed__1 = _init_l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn___closed__1(); lean_mark_persistent(l_Lean_Linter_addBuiltinUnusedVariablesIgnoreFn___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____lambda__6___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__10(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387____closed__10); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_387_(lean_io_mk_world()); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____lambda__6___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__10(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426____closed__10); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_426_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Linter_unusedVariablesIgnoreFnsExt = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Linter_unusedVariablesIgnoreFnsExt); lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__2___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__3___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__4___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____lambda__5___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__10(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__10); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__11(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__11); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__12(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__12); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__13 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__13(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__13); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__14 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__14(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__14); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__15 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__15(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__15); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__16 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__16(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__16); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__17 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__17(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__17); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__18 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__18(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__18); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__19 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__19(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__19); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__20 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__20(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__20); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__21 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__21(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__21); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__22 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__22(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__22); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__23 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__23(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__23); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__24 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__24(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601____closed__24); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_601_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__4___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__5___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__10(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__10); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__11(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__11); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__12(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__12); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__13 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__13(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__13); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__14 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__14(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__14); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__15 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__15(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__15); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__16 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__16(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__16); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__17 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__17(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__17); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__18 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__18(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__18); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__19 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__19(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__19); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__20 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__20(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__20); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__21 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__21(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__21); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__22 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__22(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__22); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__23 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__23(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__23); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__24 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__24(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____closed__24); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__10(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__10); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__11(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__11); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__12(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____lambda__1___closed__12); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_948_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__10); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__11(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__11); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__12(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____lambda__1___closed__12); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_987_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____lambda__1___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_982_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____lambda__1___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1021_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__10(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__10); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__11(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__11); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__12(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__12); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__13 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__13(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__13); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__14 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__14(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____lambda__1___closed__14); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1016_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__10); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__11(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__11); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__12(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__12); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__13 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__13(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__13); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__14 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__14(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____lambda__1___closed__14); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1055_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__10(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__10); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__11(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__11); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__12(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____lambda__1___closed__12); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1107_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__10); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__11(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__11); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__12(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____lambda__1___closed__12); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1146_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__10(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__10); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__11(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____lambda__1___closed__11); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1192_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__10); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__11(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____lambda__1___closed__11); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1231_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__1 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__1(); -lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__1); -l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__2 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__2(); -lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__2); -l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__3 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__3(); -lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__3); -l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__4 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__4(); -lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__4); -l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__5 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__5(); -lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__5); -l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__6 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__6(); -lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__6); -l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__7 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__7(); -lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____spec__3___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__3___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__4___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__10(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__10); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__11(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__11); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__12(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__12); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__13 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__13(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____lambda__5___closed__13); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1277_(lean_io_mk_world()); +}l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__1 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__1(); +lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__1); +l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__2 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__2(); +lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__2); +l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__3 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__3(); +lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__3); +l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__4 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__4(); +lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__4); +l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__5 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__5(); +lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__5); +l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__6 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__6(); +lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__6); +l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__7 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__7(); +lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____spec__3___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__3___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__4___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__10 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__10(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__10); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__11 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__11(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__11); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__12 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__12(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__12); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__13 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__13(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____lambda__5___closed__13); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_1316_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____lambda__1___closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2404_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____lambda__1___closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2443_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____lambda__1___closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2436_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____lambda__1___closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2475_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2555_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2594_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__6); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__7); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__8); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____lambda__1___closed__9); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2651_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__6 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__6); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__7 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__7); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__8 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__8); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__9 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____lambda__1___closed__9); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2690_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__2); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__3); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__4); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__1___closed__5); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____lambda__2___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703____closed__1); -if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2703_(lean_io_mk_world()); +}l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__2 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__2); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__3 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__3); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__4 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__4); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__5 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__1___closed__5); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2___closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____lambda__2___closed__1); +l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742____closed__1); +if (builtin) {res = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_2742_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Lean_Linter_getUnusedVariablesIgnoreFns___rarg___closed__1 = _init_l_Lean_Linter_getUnusedVariablesIgnoreFns___rarg___closed__1(); @@ -20511,70 +22544,89 @@ l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent___closed__1 lean_mark_persistent(l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent___closed__1); l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent___closed__2 = _init_l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent___closed__2(); lean_mark_persistent(l_Lean_Linter_UnusedVariables_collectReferences_skipDeclIdIfPresent___closed__2); -l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__1 = _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__1(); -lean_mark_persistent(l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__1); -l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__2 = _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__2(); -lean_mark_persistent(l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__2); -l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__3 = _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__3(); -lean_mark_persistent(l_panic___at_Lean_Linter_UnusedVariables_collectReferences___spec__19___closed__3); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__1(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__1); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__2(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__2); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__3(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__3); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__4(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences___spec__18___closed__4); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__1); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__2); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__3(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__3); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__4(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___lambda__2___closed__4); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences___spec__21___closed__1); +l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___closed__1 = _init_l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___closed__1(); +lean_mark_persistent(l_Array_anyMUnsafe_any___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__14___closed__1); +l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__1 = _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__1(); +lean_mark_persistent(l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__1); +l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__2 = _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__2(); +lean_mark_persistent(l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__2); +l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__3 = _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__3(); +lean_mark_persistent(l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__3); +l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__4 = _init_l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__4(); +lean_mark_persistent(l_panic___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__22___closed__4); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__1(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__1); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__2(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__2); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__3(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__3); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__4(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__21___closed__4); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__2); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__3(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__3); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__4(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__4___closed__4); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__7___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__2); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__3(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__3); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__4(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__4); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__5 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__5(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__5); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__6 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__6(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___lambda__10___closed__6); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_collectReferences_go___spec__24___closed__1); l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8___closed__1 = _init_l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8___closed__1(); lean_mark_persistent(l_panic___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__8___closed__1); -l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2___closed__1 = _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___lambda__2___closed__1); -l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___closed__1 = _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___closed__1(); -lean_mark_persistent(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__5___closed__1); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__19___lambda__5___closed__1); -l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__1 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__1(); -lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__1); -l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__2 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__2(); -lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__2); -l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__3 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__3(); -lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__3); -l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__4 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__4(); -lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___lambda__1___closed__4); -l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___closed__1 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___closed__1(); -lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__20___closed__1); -l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__1 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__1(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__1); -l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__2 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__2(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__2); -l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__3 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__3(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__3); -l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__4 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__4(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__4); -l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__5 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__5(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__5); -l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__6 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__6(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__6); -l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__7 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__7(); -lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__21___closed__7); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__1); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__2); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__3(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__3); -l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__4(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__22___closed__4); +l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2___closed__1 = _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___lambda__2___closed__1); +l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___closed__1 = _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___closed__1(); +lean_mark_persistent(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__6___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__3___closed__1(); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__25___lambda__5___closed__1); +l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__1 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__1(); +lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__1); +l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__2 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__2(); +lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__2); +l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__3 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__3(); +lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__3); +l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__4 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__4(); +lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___lambda__1___closed__4); +l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___closed__1 = _init_l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___closed__1(); +lean_mark_persistent(l_Array_qsort_sort___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__26___closed__1); +l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__1 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__1(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__1); +l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__2 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__2(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__2); +l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__3 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__3(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__3); +l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__4 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__4(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__4); +l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__5 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__5(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__5); +l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__6 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__6(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__6); +l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__7 = _init_l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__7(); +lean_mark_persistent(l_Lean_Linter_logLint___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__27___closed__7); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__2); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__3(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__3); +l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__4(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___spec__28___closed__4); l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__2___closed__1 = _init_l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Linter_UnusedVariables_unusedVariables___elambda__1___lambda__2___closed__1); l_Lean_Linter_UnusedVariables_unusedVariables___closed__1 = _init_l_Lean_Linter_UnusedVariables_unusedVariables___closed__1(); @@ -20585,7 +22637,7 @@ l_Lean_Linter_UnusedVariables_unusedVariables___closed__3 = _init_l_Lean_Linter_ lean_mark_persistent(l_Lean_Linter_UnusedVariables_unusedVariables___closed__3); l_Lean_Linter_UnusedVariables_unusedVariables = _init_l_Lean_Linter_UnusedVariables_unusedVariables(); lean_mark_persistent(l_Lean_Linter_UnusedVariables_unusedVariables); -if (builtin) {res = l_Lean_Linter_UnusedVariables_initFn____x40_Lean_Linter_UnusedVariables___hyg_5794_(lean_io_mk_world()); +if (builtin) {res = l_Lean_Linter_UnusedVariables_initFn____x40_Lean_Linter_UnusedVariables___hyg_6304_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Lean_MessageData_isUnusedVariableWarning___closed__1 = _init_l_Lean_MessageData_isUnusedVariableWarning___closed__1(); diff --git a/stage0/stdlib/Lean/Linter/Util.c b/stage0/stdlib/Lean/Linter/Util.c index af3e5c0d410e..38871709e0b5 100644 --- a/stage0/stdlib/Lean/Linter/Util.c +++ b/stage0/stdlib/Lean/Linter/Util.c @@ -13,26 +13,44 @@ #ifdef __cplusplus extern "C" { #endif +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3(lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go(lean_object*); -lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_PersistentArray_toList___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__1(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__4; LEAN_EXPORT lean_object* l_List_filterMapTR_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__2; +lean_object* l_Lean_Elab_Info_updateContext_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f___rarg___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5(lean_object*); +lean_object* l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterMapTR_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__2(lean_object*, lean_object*); lean_object* lean_array_to_list(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3(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_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__3; LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__2; +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__4(lean_object*); +lean_object* lean_panic_fn(lean_object*, lean_object*); lean_object* l_List_reverse___rarg(lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__4___rarg(lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_instInhabitedOfMonad___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Elab_Info_contains(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_List_filterMapTR_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__1(lean_object* x_1, lean_object* x_2) { _start: @@ -114,36 +132,328 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__4___rarg(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_5; lean_object* x_6; -x_5 = lean_box(0); -x_6 = l_Lean_Elab_InfoTree_visitM_go___rarg(x_1, x_2, x_3, x_5, x_4); +lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_3 = lean_box(0); +x_4 = l_instInhabitedOfMonad___rarg(x_1, x_3); +x_5 = lean_panic_fn(x_4, x_2); +return x_5; +} +} +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__4(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_panic___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__4___rarg), 2, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5___rarg___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; +x_8 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_1); +x_9 = l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5___rarg(x_2, x_3, x_4, x_5, x_6, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5___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: +{ +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = l_List_reverse___rarg(x_6); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +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_5, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_5, 1); +lean_inc(x_12); +lean_dec(x_5); +x_13 = lean_ctor_get(x_1, 1); +lean_inc(x_13); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg(x_1, x_2, x_3, x_4, x_11); +x_15 = lean_alloc_closure((void*)(l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5___rarg___lambda__1), 7, 6); +lean_closure_set(x_15, 0, x_6); +lean_closure_set(x_15, 1, x_1); +lean_closure_set(x_15, 2, x_2); +lean_closure_set(x_15, 3, x_3); +lean_closure_set(x_15, 4, x_4); +lean_closure_set(x_15, 5, x_12); +x_16 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_14, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5___rarg), 6, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__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; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +lean_dec(x_1); +x_4 = lean_ctor_get(x_3, 1); +lean_inc(x_4); +lean_dec(x_3); +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_2); +x_6 = lean_apply_2(x_4, lean_box(0), x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___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; +x_8 = lean_apply_4(x_1, x_2, x_3, x_4, x_7); +x_9 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__1), 2, 1); +lean_closure_set(x_9, 0, x_5); +x_10 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___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, uint8_t x_8) { +_start: +{ +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_dec(x_7); +x_9 = lean_box(0); +x_10 = lean_apply_4(x_1, x_2, x_3, x_4, x_9); +x_11 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__1), 2, 1); +lean_closure_set(x_11, 0, x_5); +x_12 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_10, x_11); +return x_12; +} +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; +lean_inc(x_2); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_2); +x_14 = l_Lean_Elab_Info_updateContext_x3f(x_13, x_3); +x_15 = l_Lean_PersistentArray_toList___rarg(x_4); +x_16 = lean_box(0); +lean_inc(x_1); +lean_inc(x_5); +x_17 = l_List_mapM_loop___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__5___rarg(x_5, x_7, x_1, x_14, x_15, x_16); +lean_inc(x_6); +x_18 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__2), 7, 6); +lean_closure_set(x_18, 0, x_1); +lean_closure_set(x_18, 1, x_2); +lean_closure_set(x_18, 2, x_3); +lean_closure_set(x_18, 3, x_4); +lean_closure_set(x_18, 4, x_5); +lean_closure_set(x_18, 5, x_6); +x_19 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_17, x_18); +return x_19; +} +} +} +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Server.InfoUtils", 21, 21); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Elab.InfoTree.visitM.go", 28, 28); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unexpected context-free info tree node", 38, 38); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___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_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__1; +x_2 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__2; +x_3 = lean_unsigned_to_nat(62u); +x_4 = lean_unsigned_to_nat(21u); +x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___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_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___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_4) == 0) +{ +switch (lean_obj_tag(x_5)) { +case 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_PartialContextInfo_mergeIntoOuter_x3f(x_6, x_4); +x_4 = x_8; +x_5 = x_7; +goto _start; +} +case 1: +{ +lean_object* x_10; lean_object* x_11; +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__4; +x_11 = l_panic___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__4___rarg(x_1, x_10); +return x_11; +} +default: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +lean_dec(x_1); +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_box(0); +x_15 = lean_apply_2(x_13, lean_box(0), x_14); +return x_15; +} +} +} +else +{ +switch (lean_obj_tag(x_5)) { +case 0: +{ +lean_object* x_16; lean_object* x_17; lean_object* 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 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_16, x_4); +x_4 = x_18; +x_5 = x_17; +goto _start; +} +case 1: +{ +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_4, 0); +lean_inc(x_20); +lean_dec(x_4); +x_21 = lean_ctor_get(x_5, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_5, 1); +lean_inc(x_22); +lean_dec(x_5); +x_23 = lean_ctor_get(x_1, 1); +lean_inc(x_23); +lean_inc(x_2); +lean_inc(x_22); +lean_inc(x_21); +lean_inc(x_20); +x_24 = lean_apply_3(x_2, x_20, x_21, x_22); +lean_inc(x_23); +x_25 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__3___boxed), 8, 7); +lean_closure_set(x_25, 0, x_3); +lean_closure_set(x_25, 1, x_20); +lean_closure_set(x_25, 2, x_21); +lean_closure_set(x_25, 3, x_22); +lean_closure_set(x_25, 4, x_1); +lean_closure_set(x_25, 5, x_23); +lean_closure_set(x_25, 6, x_2); +x_26 = lean_apply_4(x_23, lean_box(0), lean_box(0), x_24, x_25); +return x_26; +} +default: +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_27 = lean_ctor_get(x_1, 0); +lean_inc(x_27); +lean_dec(x_1); +x_28 = lean_ctor_get(x_27, 1); +lean_inc(x_28); +lean_dec(x_27); +x_29 = lean_box(0); +x_30 = lean_apply_2(x_28, lean_box(0), x_29); +return x_30; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg), 4, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg), 5, 0); return x_2; } } LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__1(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_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; lean_object* x_9; x_5 = lean_ctor_get(x_1, 0); lean_inc(x_5); lean_dec(x_1); x_6 = lean_ctor_get(x_5, 1); lean_inc(x_6); lean_dec(x_5); -x_7 = lean_box(0); -x_8 = lean_apply_2(x_6, lean_box(0), x_7); -return x_8; +x_7 = 1; +x_8 = lean_box(x_7); +x_9 = lean_apply_2(x_6, lean_box(0), x_8); +return x_9; } } static lean_object* _init_l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__1() { @@ -451,7 +761,7 @@ return x_83; LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg(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_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_inc(x_1); x_4 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__1___boxed), 4, 1); lean_closure_set(x_4, 0, x_1); @@ -459,8 +769,9 @@ lean_inc(x_1); x_5 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___boxed), 6, 2); lean_closure_set(x_5, 0, x_2); lean_closure_set(x_5, 1, x_1); -x_6 = l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg(x_1, x_4, x_5, x_3); -return x_6; +x_6 = lean_box(0); +x_7 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg(x_1, x_4, x_5, x_6, x_3); +return x_7; } } LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go(lean_object* x_1) { @@ -471,6 +782,16 @@ x_2 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___r return x_2; } } +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___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) { +_start: +{ +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_8); +lean_dec(x_8); +x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9); +return x_10; +} +} LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { @@ -608,6 +929,14 @@ lean_dec_ref(res); res = initialize_Lean_Linter_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__1(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__1); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__2(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__2); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__3(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__3); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__4(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___closed__4); l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__1 = _init_l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__1); l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__2 = _init_l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__2(); diff --git a/stage0/stdlib/Lean/Message.c b/stage0/stdlib/Lean/Message.c index 5335c1dfbb1a..19f649ef27b6 100644 --- a/stage0/stdlib/Lean/Message.c +++ b/stage0/stdlib/Lean/Message.c @@ -130,6 +130,7 @@ size_t lean_usize_of_nat(lean_object*); static lean_object* l_Lean_instBEqMessageSeverity___closed__1; LEAN_EXPORT lean_object* l_Lean_stringToMessageData(lean_object*); lean_object* l_Lean_Expr_mvar___override(lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MessageData_instCoeListExpr(lean_object*); lean_object* l_Lean_instInhabitedPersistentArrayNode(lean_object*); static lean_object* l_Lean_MessageData_formatAux___lambda__1___closed__6; @@ -326,7 +327,6 @@ LEAN_EXPORT lean_object* l_Lean_MessageData_nestD(lean_object*); static lean_object* l___private_Lean_Message_0__Lean_fromJsonMessageSeverity____x40_Lean_Message___hyg_163____lambda__2___closed__1; LEAN_EXPORT lean_object* l_panic___at_Lean_MessageData_formatAux___spec__2(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_MessageLog_hasErrors___spec__3(lean_object*, size_t, size_t); -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Message_0__Lean_fromJsonMessageSeverity____x40_Lean_Message___hyg_163____lambda__3___closed__1; LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyM___at_Lean_MessageLog_hasErrors___spec__1(lean_object*); double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); @@ -5474,7 +5474,7 @@ x_42 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_42, 0, x_14); lean_ctor_set(x_42, 1, x_41); x_43 = l___private_Lean_Message_0__Lean_fromJsonMessageSeverity____x40_Lean_Message___hyg_163____closed__1; -x_44 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_42, x_43); +x_44 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_42, x_43); x_45 = l_Lean_Json_mkObj(x_44); return x_45; } @@ -5502,7 +5502,7 @@ x_53 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_53, 0, x_14); lean_ctor_set(x_53, 1, x_52); x_54 = l___private_Lean_Message_0__Lean_fromJsonMessageSeverity____x40_Lean_Message___hyg_163____closed__1; -x_55 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_53, x_54); +x_55 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_53, x_54); x_56 = l_Lean_Json_mkObj(x_55); return x_56; } @@ -7212,7 +7212,7 @@ x_45 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_45, 0, x_17); lean_ctor_set(x_45, 1, x_44); x_46 = l___private_Lean_Message_0__Lean_fromJsonMessageSeverity____x40_Lean_Message___hyg_163____closed__1; -x_47 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_45, x_46); +x_47 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_45, x_46); x_48 = l_Lean_Json_mkObj(x_47); lean_ctor_set(x_10, 0, x_48); return x_10; @@ -7241,7 +7241,7 @@ x_56 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_56, 0, x_17); lean_ctor_set(x_56, 1, x_55); x_57 = l___private_Lean_Message_0__Lean_fromJsonMessageSeverity____x40_Lean_Message___hyg_163____closed__1; -x_58 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_56, x_57); +x_58 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_56, x_57); x_59 = l_Lean_Json_mkObj(x_58); lean_ctor_set(x_10, 0, x_59); return x_10; @@ -7334,7 +7334,7 @@ x_94 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_94, 0, x_66); lean_ctor_set(x_94, 1, x_93); x_95 = l___private_Lean_Message_0__Lean_fromJsonMessageSeverity____x40_Lean_Message___hyg_163____closed__1; -x_96 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_94, x_95); +x_96 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_94, x_95); x_97 = l_Lean_Json_mkObj(x_96); x_98 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_98, 0, x_97); @@ -7365,7 +7365,7 @@ x_106 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_106, 0, x_66); lean_ctor_set(x_106, 1, x_105); x_107 = l___private_Lean_Message_0__Lean_fromJsonMessageSeverity____x40_Lean_Message___hyg_163____closed__1; -x_108 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_106, x_107); +x_108 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_106, x_107); x_109 = l_Lean_Json_mkObj(x_108); x_110 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_110, 0, x_109); diff --git a/stage0/stdlib/Lean/Meta/FunInfo.c b/stage0/stdlib/Lean/Meta/FunInfo.c index 6f792e31e3b4..dc78ec55e1a5 100644 --- a/stage0/stdlib/Lean/Meta/FunInfo.c +++ b/stage0/stdlib/Lean/Meta/FunInfo.c @@ -40,16 +40,17 @@ LEAN_EXPORT lean_object* l_Lean_Meta_FunInfo_getArity(lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1___boxed(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_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___lambda__2(lean_object*, 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*); uint8_t l_Lean_Expr_isAppOf(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___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_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1___boxed(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_Meta_FunInfo_0__Lean_Meta_collectDeps___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_whenHasVar___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); static size_t l_Lean_PersistentHashMap_findAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__2___closed__1; uint64_t l_Lean_Meta_TransparencyMode_hash(uint8_t); @@ -58,7 +59,6 @@ lean_object* lean_st_ref_take(lean_object*, lean_object*); lean_object* l_Lean_getOutParamPositions_x3f(lean_object*, lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); 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*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getFunInfo(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_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___boxed(lean_object**); LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1861,7 +1861,7 @@ lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___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_8; uint8_t x_9; @@ -1973,7 +1973,7 @@ if (x_5 == 0) lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = lean_array_get_size(x_1); x_7 = lean_mk_empty_array_with_capacity(x_6); -x_8 = l_Array_mapIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1(x_1, x_2, x_1, x_6, x_4, lean_box(0), x_7); +x_8 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1(x_1, x_2, x_1, x_6, x_4, lean_box(0), x_7); return x_8; } else @@ -1983,11 +1983,11 @@ return x_1; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___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: { lean_object* x_8; -x_8 = l_Array_mapIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); diff --git a/stage0/stdlib/Lean/Meta/IndPredBelow.c b/stage0/stdlib/Lean/Meta/IndPredBelow.c index ec602eee359b..cb50e528ffff 100644 --- a/stage0/stdlib/Lean/Meta/IndPredBelow.c +++ b/stage0/stdlib/Lean/Meta/IndPredBelow.c @@ -20,8 +20,12 @@ static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_induction___closed__1; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCtorType_mkMotiveBinder___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_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__3___closed__3; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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*); +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitForall___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__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_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___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*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7; lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit___spec__3(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_induction(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__5___lambda__2___closed__8; @@ -30,7 +34,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCt static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__16___rarg___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__9(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___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_Meta_IndPredBelow_mkBelowMatcher_newMotive___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, 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*); @@ -41,7 +44,6 @@ LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCt static lean_object* l_Lean_Meta_IndPredBelow_backwardsChaining___lambda__3___closed__3; static lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___lambda__3___closed__2; lean_object* l_Lean_commitWhen___at___private_Lean_Meta_Tactic_Contradiction_0__Lean_Meta_elimEmptyInductive___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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_EXPORT lean_object* l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___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_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__2___boxed(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*); @@ -50,18 +52,18 @@ lean_object* l_Lean_Meta_mkForallFVars___boxed(lean_object*, lean_object*, lean_ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext_addMotives(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_Meta_IndPredBelow_mkCtorType_checkCount___spec__15(lean_object*, 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_IndPredBelow_proveBrecOn_applyCtors___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_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__3; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_rebuild___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_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_getBelowIndices___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_transform_visit_visitLambda___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___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*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__2; -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5; static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__9; +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__9; static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__5___closed__10; static lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelow___spec__1___closed__1; lean_object* lean_whnf(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__16___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__5___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_transform_visit_visitLambda___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__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*); static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn___closed__3; @@ -69,9 +71,9 @@ static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelo extern lean_object* l_Lean_maxRecDepthErrorMessage; static lean_object* l_Lean_Meta_IndPredBelow_mkBelow___closed__6; uint8_t l_Lean_Exception_isInterrupt(lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__8; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__5___closed__6; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkContext___spec__7(size_t, size_t, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___closed__2; lean_object* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -92,6 +94,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_rebuild(lean_object LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_backwardsChaining(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_findIdx_x3f_loop___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_sort___override(lean_object*); +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__8; lean_object* l_Lean_MessageData_ofList(lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__4(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__7___boxed(lean_object*, lean_object*); @@ -106,7 +109,6 @@ static lean_object* l_Lean_getConstInfoInduct___at_Lean_Meta_IndPredBelow_mkCont lean_object* lean_mk_array(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__7(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_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___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_ST_Prim_Ref_get___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Match_mkMatcher(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___lambda__2___closed__1; @@ -121,8 +123,12 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCt LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_transformFields_loop(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_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__5___lambda__2___closed__7; lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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* l_Lean_Expr_bvar___override(lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___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_EXPORT lean_object* l___private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_belowType___boxed(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_IndPredBelow_mkCtorType_checkCount___spec__13(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*); static lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__5___lambda__2___closed__6; @@ -132,36 +138,32 @@ static lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___lambda__1__ lean_object* l_Lean_Meta_ppGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_IndPredBelow_mkContext___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkContext___spec__7___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_getBelowIndices_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_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___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_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__5___closed__4; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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* 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*); static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_applyIH___closed__3; static lean_object* l_Lean_Meta_IndPredBelow_mkBelow___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitForall___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__5___lambda__1(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_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_addBelowPattern___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_Lean_getConstInfoInduct___at_Lean_Meta_IndPredBelow_mkContext___spec__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__7___rarg(lean_object*, uint8_t, 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_Meta_IndPredBelow_mkCtorType_checkCount___closed__3; LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_belowType___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_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6; -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__7; lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___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_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelow(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__9; LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__5___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_IndPredBelow_backwardsChaining___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_mkContext_motiveType___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__12(lean_object*, lean_object*, uint8_t, uint8_t, 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* 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_withLocalDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__8(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__3___rarg___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_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_modifyBinders___lambda__2___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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*); static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_closeGoal___closed__7; lean_object* l_Lean_Exception_toMessageData(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_instInhabitedVariables; @@ -176,12 +178,13 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_IndPredBelow_p static lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkIH___closed__2; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___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* l_Lean_Meta_withLocalDecl___at_Lean_Meta_GeneralizeTelescope_generalizeTelescopeAux___spec__1___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___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* l_Lean_Meta_Match_Pattern_toExpr_visit(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getConstInfoCtor___at___private_Lean_Meta_WHNF_0__Lean_Meta_toCtorWhenStructure___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_instInhabitedNat; static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__5___closed__8; lean_object* l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__5; +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__6; LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at_Lean_Meta_IndPredBelow_mkContext___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_applyIH(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkConstructor(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -190,7 +193,6 @@ LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkBe LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); 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_Meta_withLocalDecls___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___lambda__2(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*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -204,15 +206,15 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_back static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__1; static lean_object* l_Lean_Meta_IndPredBelow_backwardsChaining___lambda__3___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext_mkHeader___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___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_throwError___at_Lean_Expr_abstractRangeM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__4; +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__4; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_findBelowIdx___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_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__1(lean_object*, size_t, size_t, 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_Array_foldrMUnsafe_fold___at_Lean_Meta_IndPredBelow_mkContext_addMotives___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLetDeclImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelow___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_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__10; static lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___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_Array_zip___rarg(lean_object*, lean_object*); @@ -220,14 +222,12 @@ static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelow LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___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_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_IndPredBelow_mkContext_addMotives___spec__2(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_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*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___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_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8; static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__3___closed__2; uint64_t lean_uint64_shift_right(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_getBelowIndices(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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_Meta_IndPredBelow_mkBrecOnDecl_mkType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7; lean_object* l_StateRefT_x27_lift___rarg___boxed(lean_object*, lean_object*); lean_object* lean_nat_div(lean_object*, lean_object*); lean_object* l_Lean_MVarId_getType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -242,6 +242,7 @@ lean_object* l_Lean_registerTraceClass(lean_object*, uint8_t, lean_object*, lean static lean_object* l_Lean_Meta_IndPredBelow_mkContext_motiveName___closed__3; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___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_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_transformFields_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_EXPORT lean_object* l_Lean_Meta_transform_visit___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___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*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLocalDeclImp___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -251,7 +252,6 @@ static lean_object* l_Lean_Meta_transform___at_Lean_Meta_IndPredBelow_mkCtorType lean_object* l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__6(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_IndPredBelow_mkContext___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3; static lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___closed__2; lean_object* l_Lean_mkCasesOn(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_getBelowIndices___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -264,6 +264,7 @@ LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_find 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_object* l_Lean_Meta_check(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_closeGoal___closed__8; +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__1; lean_object* l_Lean_Meta_isInductivePredicate(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__9___rarg(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* l_Lean_FVarId_getDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -272,9 +273,9 @@ lean_object* l_outOfBounds___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkIH___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_IndPredBelow_mkBelowDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__13; static lean_object* l_Lean_Meta_IndPredBelow_backwardsChaining___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_IndPredBelow_mkBelow___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -288,9 +289,10 @@ static lean_object* l_Lean_Meta_IndPredBelow_mkBelow___closed__1; lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__1___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_IndPredBelow_mkBelowMatcher_addBelowPattern___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_withLocalDeclsD___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__2___rarg(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*); static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn___closed__2; +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__2; +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__5; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_replaceTempVars___spec__2(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__5(lean_object*, lean_object*); @@ -298,17 +300,19 @@ LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_IndPredBelow_m lean_object* l_ST_Prim_Ref_modifyGetUnsafe___rarg___boxed(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_levelZero; static lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelow___spec__1___closed__2; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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_IndPredBelow_backwardsChaining___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_IndPredBelow_proveBrecOn_applyIH___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_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLet___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__6___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_IndPredBelow_mkCtorType_replaceTempVars(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_transform___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__8___boxed(lean_object*, lean_object*); lean_object* l_Lean_Expr_constName_x21(lean_object*); extern lean_object* l_Lean_instInhabitedExpr; -LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142_(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___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* l_Lean_MVarId_applyRules(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_constName_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkBelowMatcher_transformFields_loop___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*); @@ -316,31 +320,31 @@ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_getBelowIndices_loop(lean_obje uint64_t l_Lean_Expr_hash(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkInductiveType(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_IndPredBelow_mkContext___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__12; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__3(size_t, size_t, lean_object*); +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__3; lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_intros(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_IndPredBelow_mkCtorType_rebuild___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_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext_mkHeader___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Meta_Match_MkMatcherInput_numDiscrs(lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1; static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__5___closed__5; static lean_object* l_Lean_Meta_IndPredBelow_mkBelow___closed__7; 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_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___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_Meta_IndPredBelow_mkCtorType_checkCount___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_PrettyPrinter_Delaborator_returnsPi___spec__1___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___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_throwError___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_IndPredBelow_findBelowIdx___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_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___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_IndPredBelow_proveBrecOn_applyIH___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher___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_IndPredBelow_mkCtorType_modifyBinders___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*); LEAN_EXPORT lean_object* l_Lean_Meta_transform___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__1(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_Meta_withLocalDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___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_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___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_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_modifyBinders(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_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*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext_motiveType___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_IndPredBelow_mkCtorType_checkCount___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -360,6 +364,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkIH___lambda__2_ LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___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*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext_mkHeader(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_getConstInfoInduct___at_Lean_Meta_IndPredBelow_mkContext___spec__1___closed__2; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___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_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkContext___spec__3___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*); static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__3; @@ -367,7 +372,6 @@ lean_object* l_Lean_MessageData_ofExpr(lean_object*); lean_object* l_Lean_throwError___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_newMotive___lambda__2___closed__2; -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3; uint8_t l_Lean_Expr_binderInfo(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelow___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_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -396,12 +400,12 @@ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext_motiveName(lean_obje static lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_IndPredBelow_proveBrecOn_applyIH___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Meta_IndPredBelow_backwardsChaining___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_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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*, lean_object*, lean_object*); lean_object* l_Lean_Expr_constLevels_x21(lean_object*); lean_object* l_Lean_Expr_bindingDomain_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_IndPredBelow_0__Lean_Meta_IndPredBelow_belowType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_instInhabitedVariables___closed__1; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_addMotives(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Match_Pattern_toMessageData(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -411,7 +415,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit___at_Lean_Meta_IndPredBelow LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLet___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___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*); static lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__5___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher___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_withLocalDecls___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__8; lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); @@ -436,18 +439,16 @@ LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_IndPred static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_closeGoal___closed__2; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_backwardsChaining___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8; +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__13; static lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl___closed__1; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___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* l_Lean_indentExpr(lean_object*); static lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__5___lambda__2___closed__5; LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, 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_IR_IRType_beq___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at_Lean_Meta_IndPredBelow_mkContext___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__1; static double l_Lean_addTrace___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__6___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType___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_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4; 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*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__5___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_Array_foldrMUnsafe_fold___at_Lean_Meta_IndPredBelow_mkContext_addMotives___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -460,37 +461,36 @@ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkIH___lambda__2( LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_findBelowIdx___boxed(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_Meta_IndPredBelow_findBelowIdx(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkContext___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* l_Lean_LocalDecl_type(lean_object*); uint64_t lean_uint64_xor(uint64_t, uint64_t); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_addMotives___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_foldrMUnsafe_fold___at_Lean_Meta_IndPredBelow_mkContext_addMotives___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_Array_indexOfAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps_visit___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__5; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkContext___spec__7___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Array_insertAt_x21___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_closeGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher___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_transform_visit_visitLambda___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__4___lambda__1(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_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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_nat_mul(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__6; static lean_object* l_Lean_getConstInfoInduct___at_Lean_Meta_IndPredBelow_mkContext___spec__1___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__11(lean_object*, lean_object*, uint8_t, uint8_t, 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_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___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*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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*); static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_closeGoal___closed__6; lean_object* l_Lean_mkArrow(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit___spec__2(lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_mkBelow___closed__5; static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__16___rarg___closed__6; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___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_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_ofSubarray___rarg(lean_object*); lean_object* l_Lean_MVarId_apply(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___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*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__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_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_back___rarg(lean_object*, lean_object*); lean_object* lean_expr_instantiate_rev(lean_object*, lean_object*); @@ -498,24 +498,25 @@ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_copyVarName(lean_ob lean_object* l_List_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_backwardsChaining___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__16___rarg___closed__4; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___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_Lean_addTrace___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__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_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__1___rarg(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_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1(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_IndPredBelow_mkBelow___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_PrettyPrinter_Delaborator_returnsPi___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_introNPRec(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkContext___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_replaceTempVars___spec__1(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_closeGoal___closed__9; extern lean_object* l_Lean_instInhabitedName; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___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_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__12; lean_object* lean_array_uget(lean_object*, size_t); lean_object* l_Lean_Expr_fvar___override(lean_object*); size_t lean_array_size(lean_object*); @@ -536,36 +537,31 @@ static lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkIH___closed__3; LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___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_IndPredBelow_mkBelowMatcher_addBelowPattern(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_IndPredBelow_findBelowIdx___spec__3___lambda__5___closed__3; -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__3(lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext_motiveType___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_throwError___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__1(lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_backwardsChaining___lambda__3___closed__5; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2; -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Meta_IndPredBelow_backwardsChaining___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_IndPredBelow_mkBelowMatcher_newMotive___lambda__1___closed__2; static lean_object* l_Lean_Meta_transform___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_newMotive___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_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___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_Meta_IndPredBelow_mkCtorType_mkMotiveBinder___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_string_append(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 lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___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* l_Lean_Meta_mkFreshExprSyntheticOpaqueMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__10; LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___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_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___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_array_get_size(lean_object*); lean_object* l_Lean_LocalDecl_toExpr(lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__3___lambda__1(lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelow___spec__1___closed__3; -static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2; +static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__11; static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___spec__3___closed__1; 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*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___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_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkContext___spec__3(size_t, size_t, 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_Array_foldrMUnsafe_fold___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__4(lean_object*, size_t, size_t, lean_object*); @@ -573,9 +569,7 @@ lean_object* l_List_mapTR_loop___at_Lean_Meta_Match_Alt_toMessageData___spec__2( lean_object* l_Lean_Meta_intro1Core(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_closeGoal___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*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___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_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___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_nat_add(lean_object*, lean_object*); static lean_object* l_Lean_Meta_transform_visit___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__2___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext_addMotives___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -591,13 +585,14 @@ LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_In uint8_t l_Lean_Exception_isRuntime(lean_object*); static lean_object* l_Lean_Meta_transform___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__1___closed__3; static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_closeGoal___closed__5; -static lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__11; uint8_t l_Lean_Expr_isForall(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___lambda__3___boxed(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_Meta_IndPredBelow_mkBelowMatcher___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_addBelowPattern___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_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144_(lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_transform___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___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_Lean_Meta_Match_instInhabitedPattern; @@ -622,9 +617,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow_ static lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_IndPredBelow_mkBelow___spec__1___closed__4; static lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_transformFields_loop___closed__2; lean_object* l_Lean_Meta_withNewBinderInfos___at_Lean_Meta_withInstImplicitAsImplict___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_intros___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___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_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__7___rarg___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_Meta_IndPredBelow_mkCtorType_mkBelowBinder(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1712,7 +1705,7 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___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) { _start: { lean_object* x_12; uint8_t x_13; @@ -1943,7 +1936,7 @@ lean_dec(x_18); x_21 = lean_array_get_size(x_19); x_22 = lean_mk_empty_array_with_capacity(x_21); x_23 = lean_unsigned_to_nat(0u); -x_24 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___spec__5(x_19, x_19, x_21, x_23, lean_box(0), x_22, x_2, x_3, x_4, x_5, x_20); +x_24 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___spec__5(x_19, x_19, x_21, x_23, lean_box(0), x_22, x_2, x_3, x_4, x_5, x_20); lean_dec(x_19); x_25 = lean_ctor_get(x_24, 0); lean_inc(x_25); @@ -2161,11 +2154,11 @@ x_11 = l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkContext___spec__4(x_ return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___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) { _start: { lean_object* x_12; -x_12 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___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 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkContext___spec__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_10); lean_dec(x_9); lean_dec(x_8); @@ -10018,132 +10011,6 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__3___rarg___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_array_push(x_1, x_5); -x_12 = l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__3___rarg(x_2, x_3, x_4, x_11, x_6, x_7, x_8, x_9, x_10); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___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; uint8_t x_12; -x_10 = lean_array_get_size(x_4); -x_11 = lean_array_get_size(x_1); -x_12 = lean_nat_dec_lt(x_10, x_11); -lean_dec(x_11); -if (x_12 == 0) -{ -lean_object* x_13; -lean_dec(x_10); -lean_dec(x_3); -lean_dec(x_1); -x_13 = lean_apply_6(x_2, x_4, x_5, x_6, x_7, x_8, x_9); -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; -x_14 = lean_array_fget(x_1, x_10); -lean_dec(x_10); -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 0); -lean_inc(x_16); -lean_dec(x_14); -x_17 = lean_ctor_get(x_15, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_dec(x_15); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_19 = lean_apply_6(x_18, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; uint8_t 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 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__3___rarg___lambda__1), 10, 4); -lean_closure_set(x_22, 0, x_4); -lean_closure_set(x_22, 1, x_1); -lean_closure_set(x_22, 2, x_2); -lean_closure_set(x_22, 3, x_3); -x_23 = 0; -x_24 = lean_unbox(x_17); -lean_dec(x_17); -x_25 = l_Lean_Meta_withLocalDecl___at_Lean_Meta_GeneralizeTelescope_generalizeTelescopeAux___spec__1___rarg(x_16, x_24, x_20, x_22, x_23, x_5, x_6, x_7, x_8, x_21); -return x_25; -} -else -{ -uint8_t x_26; -lean_dec(x_17); -lean_dec(x_16); -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_19); -if (x_26 == 0) -{ -return x_19; -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_19, 0); -x_28 = lean_ctor_get(x_19, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_19); -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_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__3(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__3___rarg), 9, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___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_object* x_10; -x_9 = l_Lean_Meta_transform_visit___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__2___lambda__1___closed__1; -x_10 = l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__3___rarg(x_2, x_3, x_1, x_9, x_4, x_5, x_6, x_7, x_8); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__2(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__2___rarg), 8, 0); -return x_2; -} -} LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_addMotives___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: { @@ -10211,7 +10078,7 @@ lean_closure_set(x_16, 1, x_1); lean_closure_set(x_16, 2, x_2); lean_closure_set(x_16, 3, x_3); x_17 = l_Lean_instInhabitedExpr; -x_18 = l_Lean_Meta_withLocalDecls___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__2___rarg(x_17, x_14, x_16, x_5, x_6, x_7, x_8, x_15); +x_18 = l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg(x_17, x_14, x_16, x_5, x_6, x_7, x_8, x_15); return x_18; } } @@ -10241,7 +10108,7 @@ lean_dec(x_5); return x_12; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___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) { _start: { lean_object* x_8; @@ -10251,145 +10118,69 @@ lean_ctor_set(x_8, 1, x_7); return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___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_12; uint8_t x_13; -x_12 = lean_unsigned_to_nat(0u); -x_13 = lean_nat_dec_eq(x_3, 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; uint8_t x_19; lean_object* x_20; -x_14 = lean_unsigned_to_nat(1u); -x_15 = lean_nat_sub(x_3, x_14); -lean_dec(x_3); -x_16 = lean_array_fget(x_2, x_4); -x_17 = lean_ctor_get(x_1, 2); -x_18 = lean_array_get_size(x_17); -x_19 = lean_nat_dec_lt(x_4, x_18); -lean_dec(x_18); -x_20 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1___boxed), 7, 1); -lean_closure_set(x_20, 0, x_16); -if (x_19 == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_21 = l_Lean_instInhabitedName; -x_22 = l_outOfBounds___rarg(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); -x_24 = lean_nat_add(x_4, x_14); -lean_dec(x_4); -x_25 = lean_array_push(x_6, x_23); -x_3 = x_15; -x_4 = x_24; -x_5 = lean_box(0); -x_6 = x_25; -goto _start; -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_27 = lean_array_fget(x_17, x_4); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_20); -x_29 = lean_nat_add(x_4, x_14); -lean_dec(x_4); -x_30 = lean_array_push(x_6, x_28); -x_3 = x_15; -x_4 = x_29; -x_5 = lean_box(0); -x_6 = x_30; -goto _start; -} -} -else +lean_object* x_13; uint8_t x_14; +x_13 = lean_unsigned_to_nat(0u); +x_14 = lean_nat_dec_eq(x_4, x_13); +if (x_14 == 0) { -lean_object* x_32; +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; +x_15 = lean_unsigned_to_nat(1u); +x_16 = lean_nat_sub(x_4, x_15); lean_dec(x_4); -lean_dec(x_3); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_6); -lean_ctor_set(x_32, 1, x_11); -return x_32; -} -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___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; size_t x_8; size_t x_9; uint8_t x_10; -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 = 1; -x_9 = lean_usize_add(x_2, x_8); -x_10 = !lean_is_exclusive(x_5); -if (x_10 == 0) +x_17 = lean_array_fget(x_3, x_5); +x_18 = lean_ctor_get(x_1, 2); +x_19 = lean_array_get_size(x_18); +x_20 = lean_nat_dec_lt(x_5, x_19); +lean_dec(x_19); +x_21 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1___boxed), 7, 1); +lean_closure_set(x_21, 0, x_17); +if (x_20 == 0) { -lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = lean_ctor_get(x_5, 0); -x_12 = 0; -x_13 = lean_box(x_12); -lean_ctor_set(x_5, 0, x_13); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_11); -lean_ctor_set(x_14, 1, x_5); -x_15 = lean_array_uset(x_7, x_2, x_14); -x_2 = x_9; -x_3 = x_15; +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_22 = l_Lean_instInhabitedName; +x_23 = l_outOfBounds___rarg(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); +x_25 = lean_nat_add(x_5, x_15); +lean_dec(x_5); +x_26 = lean_array_push(x_7, x_24); +x_4 = x_16; +x_5 = x_25; +x_6 = lean_box(0); +x_7 = x_26; goto _start; } else { -lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_17 = lean_ctor_get(x_5, 0); -x_18 = lean_ctor_get(x_5, 1); -lean_inc(x_18); -lean_inc(x_17); +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_28 = lean_array_fget(x_18, x_5); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_21); +x_30 = lean_nat_add(x_5, x_15); lean_dec(x_5); -x_19 = 0; -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_18); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_17); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_array_uset(x_7, x_2, x_22); -x_2 = x_9; -x_3 = x_23; +x_31 = lean_array_push(x_7, x_29); +x_4 = x_16; +x_5 = x_30; +x_6 = lean_box(0); +x_7 = x_31; goto _start; } } -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___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: +else { -size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_array_size(x_2); -x_10 = 0; -x_11 = l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__3(x_9, x_10, x_2); -x_12 = l_Lean_Meta_withLocalDecls___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__2___rarg(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8); -return x_12; -} +lean_object* x_33; +lean_dec(x_5); +lean_dec(x_4); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_7); +lean_ctor_set(x_33, 1, x_12); +return x_33; } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__2(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__2___rarg), 8, 0); -return x_2; } } LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___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) { @@ -10441,7 +10232,7 @@ lean_inc(x_10); x_11 = lean_array_get_size(x_10); x_12 = lean_mk_empty_array_with_capacity(x_11); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1(x_1, x_10, x_11, x_13, lean_box(0), x_12, x_5, x_6, x_7, x_8, x_9); +x_14 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1(x_1, x_10, x_10, x_11, x_13, lean_box(0), x_12, x_5, x_6, x_7, x_8, x_9); lean_dec(x_10); x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); @@ -10454,15 +10245,15 @@ lean_closure_set(x_17, 1, x_1); lean_closure_set(x_17, 2, x_2); lean_closure_set(x_17, 3, x_3); x_18 = l_Lean_instInhabitedExpr; -x_19 = l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__2___rarg(x_18, x_15, x_17, x_5, x_6, x_7, x_8, x_16); +x_19 = l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(x_18, x_15, x_17, x_5, x_6, x_7, x_8, x_16); return x_19; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___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) { _start: { lean_object* x_8; -x_8 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__1___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); @@ -10471,30 +10262,19 @@ lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___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_12; -x_12 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___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_object* x_13; +x_13 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___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_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_12; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___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_6 = l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__3(x_4, x_5, x_3); -return x_6; +return x_13; } } LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType___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) { @@ -11102,89 +10882,89 @@ return x_61; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___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_12; uint8_t x_13; -x_12 = lean_unsigned_to_nat(0u); -x_13 = lean_nat_dec_eq(x_3, x_12); -if (x_13 == 0) +lean_object* x_13; uint8_t x_14; +x_13 = lean_unsigned_to_nat(0u); +x_14 = lean_nat_dec_eq(x_4, x_13); +if (x_14 == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_14 = lean_unsigned_to_nat(1u); -x_15 = lean_nat_sub(x_3, x_14); -lean_dec(x_3); -x_16 = lean_array_fget(x_2, x_4); +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_unsigned_to_nat(1u); +x_16 = lean_nat_sub(x_4, x_15); +lean_dec(x_4); +x_17 = lean_array_fget(x_3, x_5); +lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_4); +lean_inc(x_5); lean_inc(x_1); -x_17 = l_Lean_Meta_IndPredBelow_mkInductiveType(x_1, x_4, x_16, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_17) == 0) +x_18 = l_Lean_Meta_IndPredBelow_mkInductiveType(x_1, x_5, x_17, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); +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); -lean_dec(x_17); -x_20 = lean_nat_add(x_4, x_14); -lean_dec(x_4); -x_21 = lean_array_push(x_6, x_18); -x_3 = x_15; -x_4 = x_20; -x_5 = lean_box(0); -x_6 = x_21; -x_11 = x_19; +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = lean_nat_add(x_5, x_15); +lean_dec(x_5); +x_22 = lean_array_push(x_7, x_19); +x_4 = x_16; +x_5 = x_21; +x_6 = lean_box(0); +x_7 = x_22; +x_12 = x_20; goto _start; } else { -uint8_t x_23; -lean_dec(x_15); +uint8_t x_24; +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_4); +lean_dec(x_5); lean_dec(x_1); -x_23 = !lean_is_exclusive(x_17); -if (x_23 == 0) +x_24 = !lean_is_exclusive(x_18); +if (x_24 == 0) { -return x_17; +return x_18; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_17, 0); -x_25 = lean_ctor_get(x_17, 1); +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_18, 0); +x_26 = lean_ctor_get(x_18, 1); +lean_inc(x_26); lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_17); -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_dec(x_18); +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 { -lean_object* x_27; +lean_object* x_28; +lean_dec(x_11); lean_dec(x_10); 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_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_6); -lean_ctor_set(x_27, 1, x_11); -return 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_12); +return x_28; } } } @@ -11199,7 +10979,7 @@ x_9 = lean_unsigned_to_nat(0u); x_10 = lean_nat_dec_lt(x_9, x_8); x_11 = lean_mk_empty_array_with_capacity(x_8); lean_inc(x_1); -x_12 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___spec__1(x_1, x_7, x_8, x_9, lean_box(0), x_11, x_2, x_3, x_4, x_5, x_6); +x_12 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___spec__1(x_1, x_7, x_7, x_8, x_9, lean_box(0), x_11, x_2, x_3, x_4, x_5, x_6); if (x_10 == 0) { lean_dec(x_7); @@ -11406,13 +11186,14 @@ return x_72; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___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_12; -x_12 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___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_object* x_13; +x_13 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowDecl___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_3); lean_dec(x_2); -return x_12; +return x_13; } } LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_backwardsChaining___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, lean_object* x_8, lean_object* x_9) { @@ -14381,7 +14162,7 @@ lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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) { _start: { lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; lean_object* x_17; @@ -14420,155 +14201,155 @@ return x_32; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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) { _start: { -lean_object* x_15; uint8_t x_16; -x_15 = lean_unsigned_to_nat(0u); -x_16 = lean_nat_dec_eq(x_6, x_15); -if (x_16 == 0) +lean_object* x_16; uint8_t x_17; +x_16 = lean_unsigned_to_nat(0u); +x_17 = lean_nat_dec_eq(x_7, x_16); +if (x_17 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_nat_sub(x_6, x_17); -lean_dec(x_6); -x_19 = lean_array_fget(x_5, x_7); -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_18 = lean_unsigned_to_nat(1u); +x_19 = lean_nat_sub(x_7, x_18); +lean_dec(x_7); +x_20 = lean_array_fget(x_6, x_8); +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -lean_inc(x_10); -x_21 = l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(x_2, x_15, x_20, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_21) == 0) +x_22 = l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(x_2, x_16, x_21, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_22) == 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_21, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); +lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; +x_23 = lean_ctor_get(x_22, 0); lean_inc(x_23); -lean_dec(x_21); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -lean_inc(x_7); +lean_inc(x_8); lean_inc(x_1); -x_24 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___lambda__1___boxed), 12, 5); -lean_closure_set(x_24, 0, x_1); -lean_closure_set(x_24, 1, x_7); -lean_closure_set(x_24, 2, x_2); -lean_closure_set(x_24, 3, x_3); -lean_closure_set(x_24, 4, x_4); -x_25 = 0; +x_25 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___lambda__1___boxed), 12, 5); +lean_closure_set(x_25, 0, x_1); +lean_closure_set(x_25, 1, x_8); +lean_closure_set(x_25, 2, x_2); +lean_closure_set(x_25, 3, x_3); +lean_closure_set(x_25, 4, x_4); +x_26 = 0; +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -lean_inc(x_10); -x_26 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_22, x_24, x_25, x_10, x_11, x_12, x_13, x_23); -if (lean_obj_tag(x_26) == 0) +x_27 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_23, x_25, x_26, x_11, x_12, x_13, x_14, x_24); +if (lean_obj_tag(x_27) == 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_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); -lean_dec(x_26); -x_29 = lean_nat_add(x_7, x_17); -lean_dec(x_7); -x_30 = lean_array_push(x_9, x_27); -x_6 = x_18; -x_7 = x_29; -x_8 = lean_box(0); -x_9 = x_30; -x_14 = x_28; +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +x_30 = lean_nat_add(x_8, x_18); +lean_dec(x_8); +x_31 = lean_array_push(x_10, x_28); +x_7 = x_19; +x_8 = x_30; +x_9 = lean_box(0); +x_10 = x_31; +x_15 = x_29; goto _start; } else { -uint8_t x_32; -lean_dec(x_18); +uint8_t x_33; +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_7); +lean_dec(x_8); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_32 = !lean_is_exclusive(x_26); -if (x_32 == 0) +x_33 = !lean_is_exclusive(x_27); +if (x_33 == 0) { -return x_26; +return x_27; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_26, 0); -x_34 = lean_ctor_get(x_26, 1); +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_27, 0); +x_35 = lean_ctor_get(x_27, 1); +lean_inc(x_35); lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_26); -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_27); +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_36; -lean_dec(x_18); +uint8_t x_37; +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_7); +lean_dec(x_8); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_36 = !lean_is_exclusive(x_21); -if (x_36 == 0) +x_37 = !lean_is_exclusive(x_22); +if (x_37 == 0) { -return x_21; +return x_22; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_21, 0); -x_38 = lean_ctor_get(x_21, 1); +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_inc(x_37); -lean_dec(x_21); -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_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; } } } else { -lean_object* x_40; +lean_object* x_41; +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_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_40 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_40, 0, x_9); -lean_ctor_set(x_40, 1, x_14); -return x_40; +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_10); +lean_ctor_set(x_41, 1, x_15); +return x_41; } } } @@ -14612,7 +14393,7 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_20); lean_inc(x_13); -x_25 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1(x_1, x_13, x_16, x_20, x_21, x_22, x_24, lean_box(0), x_23, x_5, x_6, x_7, x_8, x_9); +x_25 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1(x_1, x_13, x_16, x_20, x_21, x_21, x_22, x_24, lean_box(0), x_23, x_5, x_6, x_7, x_8, x_9); lean_dec(x_21); if (lean_obj_tag(x_25) == 0) { @@ -14733,11 +14514,11 @@ return x_56; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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) { _start: { lean_object* x_13; -x_13 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -14749,13 +14530,14 @@ lean_dec(x_1); return x_13; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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: { -lean_object* x_15; -x_15 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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_object* x_16; +x_16 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___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); +lean_dec(x_6); lean_dec(x_5); -return x_15; +return x_16; } } LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_introNPRec(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { @@ -15120,7 +14902,7 @@ return x_25; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___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: { lean_object* x_12; uint8_t x_13; @@ -15318,14 +15100,12 @@ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors(lean_ob _start: { lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -lean_inc(x_1); x_7 = lean_array_mk(x_1); x_8 = lean_array_get_size(x_7); x_9 = lean_mk_empty_array_with_capacity(x_8); x_10 = lean_unsigned_to_nat(0u); -x_11 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__3(x_1, x_7, x_8, x_10, lean_box(0), x_9, x_2, x_3, x_4, x_5, x_6); +x_11 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__3(x_7, x_7, x_8, x_10, lean_box(0), x_9, x_2, x_3, x_4, x_5, x_6); lean_dec(x_7); -lean_dec(x_1); if (lean_obj_tag(x_11) == 0) { uint8_t x_12; @@ -15425,11 +15205,11 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___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_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___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 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___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_2); lean_dec(x_1); return x_12; @@ -16461,95 +16241,95 @@ lean_dec(x_6); return x_12; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___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: { -lean_object* x_14; uint8_t x_15; -x_14 = lean_unsigned_to_nat(0u); -x_15 = lean_nat_dec_eq(x_5, x_14); -if (x_15 == 0) +lean_object* x_15; uint8_t x_16; +x_15 = lean_unsigned_to_nat(0u); +x_16 = lean_nat_dec_eq(x_6, x_15); +if (x_16 == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_16 = lean_unsigned_to_nat(1u); -x_17 = lean_nat_sub(x_5, x_16); -lean_dec(x_5); -x_18 = lean_array_fget(x_4, x_6); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_17 = lean_unsigned_to_nat(1u); +x_18 = lean_nat_sub(x_6, x_17); +lean_dec(x_6); +x_19 = lean_array_fget(x_5, x_7); +lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_6); -lean_inc(x_2); +lean_inc(x_7); lean_inc(x_3); +lean_inc(x_4); lean_inc(x_1); -x_19 = l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkIH(x_1, x_3, x_2, x_6, x_18, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_19) == 0) +x_20 = l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkIH(x_1, x_4, x_3, x_7, x_19, x_10, x_11, x_12, x_13, x_14); +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 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); +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); -lean_dec(x_19); -x_22 = lean_nat_add(x_6, x_16); -lean_dec(x_6); -x_23 = lean_array_push(x_8, x_20); -x_5 = x_17; -x_6 = x_22; -x_7 = lean_box(0); -x_8 = x_23; -x_13 = x_21; +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_nat_add(x_7, x_17); +lean_dec(x_7); +x_24 = lean_array_push(x_9, x_21); +x_6 = x_18; +x_7 = x_23; +x_8 = lean_box(0); +x_9 = x_24; +x_14 = x_22; goto _start; } else { -uint8_t x_25; -lean_dec(x_17); +uint8_t x_26; +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_dec(x_6); +lean_dec(x_7); +lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -x_25 = !lean_is_exclusive(x_19); -if (x_25 == 0) +x_26 = !lean_is_exclusive(x_20); +if (x_26 == 0) { -return x_19; +return x_20; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_19, 0); -x_27 = lean_ctor_get(x_19, 1); +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_20, 0); +x_28 = lean_ctor_get(x_20, 1); +lean_inc(x_28); lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_19); -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_dec(x_20); +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 { -lean_object* x_29; +lean_object* x_30; +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_29 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_29, 0, x_8); -lean_ctor_set(x_29, 1, x_13); -return x_29; +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_9); +lean_ctor_set(x_30, 1, x_14); +return x_30; } } } @@ -16619,7 +16399,7 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_17); -x_22 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___spec__1(x_1, x_17, x_20, x_13, x_14, x_11, lean_box(0), x_21, x_5, x_6, x_7, x_8, x_9); +x_22 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___spec__1(x_1, x_13, x_17, x_20, x_13, x_14, x_11, lean_box(0), x_21, x_5, x_6, x_7, x_8, x_9); lean_dec(x_13); if (lean_obj_tag(x_22) == 0) { @@ -16635,7 +16415,7 @@ lean_closure_set(x_25, 1, x_17); lean_closure_set(x_25, 2, x_2); lean_closure_set(x_25, 3, x_19); x_26 = l_Lean_instInhabitedExpr; -x_27 = l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__2___rarg(x_26, x_23, x_25, x_5, x_6, x_7, x_8, x_24); +x_27 = l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(x_26, x_23, x_25, x_5, x_6, x_7, x_8, x_24); return x_27; } else @@ -16706,13 +16486,14 @@ return x_18; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___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_14; -x_14 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___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_4); -return x_14; +lean_object* x_15; +x_15 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___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_5); +lean_dec(x_2); +return x_15; } } LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBrecOnDecl_mkType___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) { @@ -20282,7 +20063,7 @@ goto _start; } } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1() { _start: { lean_object* x_1; @@ -20290,16 +20071,16 @@ x_1 = lean_mk_string_unchecked("alt ", 4, 4); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1; +x_1 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3() { _start: { lean_object* x_1; @@ -20307,16 +20088,16 @@ x_1 = lean_mk_string_unchecked(":\n", 2, 2); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3; +x_1 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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_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; lean_object* x_21; lean_object* x_22; uint8_t x_23; uint8_t x_24; uint8_t x_25; lean_object* x_26; @@ -20388,11 +20169,11 @@ x_37 = l___private_Init_Data_Repr_0__Nat_reprFast(x_7); x_38 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_38, 0, x_37); x_39 = l_Lean_MessageData_ofFormat(x_38); -x_40 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2; +x_40 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___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_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4; +x_42 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4; x_43 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_43, 0, x_41); lean_ctor_set(x_43, 1, x_42); @@ -20463,7 +20244,7 @@ return x_60; } } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1() { _start: { lean_object* x_1; @@ -20471,16 +20252,16 @@ x_1 = lean_mk_string_unchecked("xs = ", 5, 5); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1; +x_1 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3() { _start: { lean_object* x_1; @@ -20488,16 +20269,16 @@ x_1 = lean_mk_string_unchecked("; oldFVars = ", 13, 13); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3; +x_1 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5() { _start: { lean_object* x_1; @@ -20505,16 +20286,16 @@ x_1 = lean_mk_string_unchecked("; fvars = ", 10, 10); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5; +x_1 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7() { _start: { lean_object* x_1; @@ -20522,16 +20303,16 @@ x_1 = lean_mk_string_unchecked("; new = ", 8, 8); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7; +x_1 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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) { _start: { lean_object* x_12; lean_object* x_13; size_t x_14; size_t 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; lean_object* x_23; lean_object* x_24; lean_object* x_25; @@ -20603,7 +20384,7 @@ lean_object* x_33; lean_object* x_34; lean_free_object(x_24); lean_dec(x_12); x_33 = lean_box(0); -x_34 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(x_25, x_17, x_22, x_16, x_31, x_23, x_3, x_4, x_33, x_7, x_8, x_9, x_10, x_28); +x_34 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(x_25, x_17, x_22, x_16, x_31, x_23, x_3, x_4, x_33, x_7, x_8, x_9, x_10, x_28); return x_34; } else @@ -20614,11 +20395,11 @@ x_35 = lean_array_to_list(x_25); x_36 = lean_box(0); x_37 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_35, x_36); x_38 = l_Lean_MessageData_ofList(x_37); -x_39 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2; +x_39 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2; lean_ctor_set_tag(x_24, 7); lean_ctor_set(x_24, 1, x_38); lean_ctor_set(x_24, 0, x_39); -x_40 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4; +x_40 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4; x_41 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_41, 0, x_24); lean_ctor_set(x_41, 1, x_40); @@ -20630,7 +20411,7 @@ x_46 = l_Lean_MessageData_ofList(x_45); x_47 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_47, 0, x_41); lean_ctor_set(x_47, 1, x_46); -x_48 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6; +x_48 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6; x_49 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_49, 0, x_47); lean_ctor_set(x_49, 1, x_48); @@ -20641,7 +20422,7 @@ x_52 = l_Lean_MessageData_ofList(x_51); x_53 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_53, 0, x_49); lean_ctor_set(x_53, 1, x_52); -x_54 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8; +x_54 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8; x_55 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_55, 0, x_53); lean_ctor_set(x_55, 1, x_54); @@ -20686,7 +20467,7 @@ lean_inc(x_77); x_78 = lean_ctor_get(x_76, 1); lean_inc(x_78); lean_dec(x_76); -x_79 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(x_25, x_17, x_22, x_16, x_31, x_23, x_3, x_4, x_77, x_7, x_8, x_9, x_10, x_78); +x_79 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(x_25, x_17, x_22, x_16, x_31, x_23, x_3, x_4, x_77, x_7, x_8, x_9, x_10, x_78); lean_dec(x_77); return x_79; } @@ -20713,7 +20494,7 @@ if (x_85 == 0) lean_object* x_86; lean_object* x_87; lean_dec(x_12); x_86 = lean_box(0); -x_87 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(x_25, x_17, x_22, x_16, x_84, x_23, x_3, x_4, x_86, x_7, x_8, x_9, x_10, x_81); +x_87 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(x_25, x_17, x_22, x_16, x_84, x_23, x_3, x_4, x_86, x_7, x_8, x_9, x_10, x_81); return x_87; } else @@ -20724,11 +20505,11 @@ x_88 = lean_array_to_list(x_25); x_89 = lean_box(0); x_90 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_88, x_89); x_91 = l_Lean_MessageData_ofList(x_90); -x_92 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2; +x_92 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2; x_93 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_93, 0, x_92); lean_ctor_set(x_93, 1, x_91); -x_94 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4; +x_94 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4; x_95 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_95, 0, x_93); lean_ctor_set(x_95, 1, x_94); @@ -20740,7 +20521,7 @@ x_100 = l_Lean_MessageData_ofList(x_99); x_101 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_101, 0, x_95); lean_ctor_set(x_101, 1, x_100); -x_102 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6; +x_102 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6; x_103 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_103, 0, x_101); lean_ctor_set(x_103, 1, x_102); @@ -20751,7 +20532,7 @@ x_106 = l_Lean_MessageData_ofList(x_105); x_107 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_107, 0, x_103); lean_ctor_set(x_107, 1, x_106); -x_108 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8; +x_108 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8; x_109 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_109, 0, x_107); lean_ctor_set(x_109, 1, x_108); @@ -20796,7 +20577,7 @@ lean_inc(x_131); x_132 = lean_ctor_get(x_130, 1); lean_inc(x_132); lean_dec(x_130); -x_133 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(x_25, x_17, x_22, x_16, x_84, x_23, x_3, x_4, x_131, x_7, x_8, x_9, x_10, x_132); +x_133 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1(x_25, x_17, x_22, x_16, x_84, x_23, x_3, x_4, x_131, x_7, x_8, x_9, x_10, x_132); lean_dec(x_131); return x_133; } @@ -20804,117 +20585,117 @@ return x_133; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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: { -lean_object* x_14; uint8_t x_15; -x_14 = lean_unsigned_to_nat(0u); -x_15 = lean_nat_dec_eq(x_5, x_14); -if (x_15 == 0) +lean_object* x_12; uint8_t x_13; +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_nat_dec_eq(x_3, x_12); +if (x_13 == 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; 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; -x_16 = lean_unsigned_to_nat(1u); -x_17 = lean_nat_sub(x_5, x_16); -lean_dec(x_5); -x_18 = lean_array_fget(x_4, x_6); -x_19 = lean_ctor_get(x_18, 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; uint8_t x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_14 = lean_unsigned_to_nat(1u); +x_15 = lean_nat_sub(x_3, x_14); +lean_dec(x_3); +x_16 = lean_array_fget(x_2, x_4); +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, 0); lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); +x_20 = lean_ctor_get(x_17, 1); lean_inc(x_20); -lean_dec(x_18); -x_21 = lean_ctor_get(x_19, 0); +lean_dec(x_17); +x_21 = lean_ctor_get(x_19, 1); lean_inc(x_21); -x_22 = lean_ctor_get(x_19, 1); -lean_inc(x_22); lean_dec(x_19); -x_23 = lean_ctor_get(x_21, 1); -lean_inc(x_23); -lean_dec(x_21); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -lean_dec(x_22); -lean_inc(x_24); -lean_inc(x_23); -x_25 = l_List_appendTR___rarg(x_23, x_24); -lean_inc(x_20); -lean_inc(x_6); -x_26 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___boxed), 11, 4); -lean_closure_set(x_26, 0, x_23); -lean_closure_set(x_26, 1, x_24); -lean_closure_set(x_26, 2, x_6); -lean_closure_set(x_26, 3, x_20); -x_27 = 0; -x_28 = lean_box(x_27); -x_29 = lean_alloc_closure((void*)(l_Lean_Meta_lambdaTelescope___at_Lean_PrettyPrinter_Delaborator_returnsPi___spec__1___rarg___boxed), 8, 3); -lean_closure_set(x_29, 0, x_20); -lean_closure_set(x_29, 1, x_26); -lean_closure_set(x_29, 2, x_28); -lean_inc(x_12); -lean_inc(x_11); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +lean_inc(x_22); +lean_inc(x_21); +x_23 = l_List_appendTR___rarg(x_21, x_22); +lean_inc(x_18); +lean_inc(x_4); +x_24 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___boxed), 11, 4); +lean_closure_set(x_24, 0, x_21); +lean_closure_set(x_24, 1, x_22); +lean_closure_set(x_24, 2, x_4); +lean_closure_set(x_24, 3, x_18); +x_25 = 0; +x_26 = lean_box(x_25); +x_27 = lean_alloc_closure((void*)(l_Lean_Meta_lambdaTelescope___at_Lean_PrettyPrinter_Delaborator_returnsPi___spec__1___rarg___boxed), 8, 3); +lean_closure_set(x_27, 0, x_18); +lean_closure_set(x_27, 1, x_24); +lean_closure_set(x_27, 2, x_26); lean_inc(x_10); lean_inc(x_9); -x_30 = l_Lean_Meta_withExistingLocalDecls___at_Lean_Meta_Match_Alt_toMessageData___spec__4___rarg(x_25, x_29, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_30) == 0) +lean_inc(x_8); +lean_inc(x_7); +x_28 = l_Lean_Meta_withExistingLocalDecls___at_Lean_Meta_Match_Alt_toMessageData___spec__4___rarg(x_23, x_27, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_28) == 0) { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* 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 = lean_nat_add(x_6, x_16); -lean_dec(x_6); -x_34 = lean_array_push(x_8, x_31); -x_5 = x_17; -x_6 = x_33; -x_7 = lean_box(0); -x_8 = x_34; -x_13 = x_32; +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* 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 = lean_nat_add(x_4, x_14); +lean_dec(x_4); +x_32 = lean_array_push(x_6, x_29); +x_3 = x_15; +x_4 = x_31; +x_5 = lean_box(0); +x_6 = x_32; +x_11 = x_30; goto _start; } else { -uint8_t x_36; -lean_dec(x_17); -lean_dec(x_12); -lean_dec(x_11); +uint8_t x_34; +lean_dec(x_15); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); -x_36 = !lean_is_exclusive(x_30); -if (x_36 == 0) +lean_dec(x_4); +x_34 = !lean_is_exclusive(x_28); +if (x_34 == 0) { -return x_30; +return x_28; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_30, 0); -x_38 = lean_ctor_get(x_30, 1); -lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_30); -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_28, 0); +x_36 = lean_ctor_get(x_28, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_28); +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_40; -lean_dec(x_12); -lean_dec(x_11); +lean_object* x_38; lean_dec(x_10); lean_dec(x_9); -lean_dec(x_6); -lean_dec(x_5); -x_40 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_40, 0, x_8); -lean_ctor_set(x_40, 1, x_13); -return x_40; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_4); +lean_dec(x_3); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_6); +lean_ctor_set(x_38, 1, x_11); +return x_38; } } } @@ -22029,7 +21810,7 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_39 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3(x_1, x_11, x_30, x_35, x_36, x_38, lean_box(0), x_37, x_5, x_6, x_7, x_8, x_31); +x_39 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3(x_35, x_35, x_36, x_38, lean_box(0), x_37, x_5, x_6, x_7, x_8, x_31); lean_dec(x_35); if (lean_obj_tag(x_39) == 0) { @@ -22395,7 +22176,7 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_116 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3(x_1, x_11, x_107, x_112, x_113, x_115, lean_box(0), x_114, x_5, x_6, x_7, x_8, x_108); +x_116 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3(x_112, x_112, x_113, x_115, lean_box(0), x_114, x_5, x_6, x_7, x_8, x_108); lean_dec(x_112); if (lean_obj_tag(x_116) == 0) { @@ -22793,11 +22574,11 @@ x_6 = l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__ return x_6; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; -x_15 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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, x_13, x_14); +x_15 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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, x_13, x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -22806,11 +22587,11 @@ lean_dec(x_9); return x_15; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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) { _start: { lean_object* x_12; -x_12 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -22819,16 +22600,14 @@ lean_dec(x_6); return x_12; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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_14; -x_14 = l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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_4); -lean_dec(x_3); +lean_object* x_12; +x_12 = l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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_2); lean_dec(x_1); -return x_14; +return x_12; } } LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_IndPredBelow_mkBelowMatcher___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) { @@ -25557,7 +25336,7 @@ lean_dec(x_3); return x_9; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__1() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -25567,27 +25346,27 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__2() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__1; +x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__1; x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__3() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__2; +x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__2; x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__8; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__4() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__4() { _start: { lean_object* x_1; @@ -25595,17 +25374,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__5() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__3; -x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__4; +x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__3; +x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__6() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__6() { _start: { lean_object* x_1; @@ -25613,47 +25392,47 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__7() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__5; -x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__6; +x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__5; +x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__8() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__7; +x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__7; x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__9() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__8; +x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__8; x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__10() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__9; +x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__9; x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_6____closed__8; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__11() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__11() { _start: { lean_object* x_1; @@ -25661,33 +25440,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__12() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__10; -x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__11; +x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__10; +x_2 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__11; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__13() { +static lean_object* _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__12; -x_2 = lean_unsigned_to_nat(8142u); +x_1 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__12; +x_2 = lean_unsigned_to_nat(8144u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144_(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_IndPredBelow_mkBelow___closed__1; x_3 = 0; -x_4 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__13; +x_4 = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__13; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); if (lean_obj_tag(x_5) == 0) { @@ -25956,30 +25735,30 @@ l_Lean_Meta_IndPredBelow_mkBelowMatcher_newMotive___lambda__2___closed__1 = _ini lean_mark_persistent(l_Lean_Meta_IndPredBelow_mkBelowMatcher_newMotive___lambda__2___closed__1); l_Lean_Meta_IndPredBelow_mkBelowMatcher_newMotive___lambda__2___closed__2 = _init_l_Lean_Meta_IndPredBelow_mkBelowMatcher_newMotive___lambda__2___closed__2(); lean_mark_persistent(l_Lean_Meta_IndPredBelow_mkBelowMatcher_newMotive___lambda__2___closed__2); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7); -l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8 = _init_l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__1); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__2); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__3); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__1___closed__4); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__1); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__2); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__3); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__4); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__5); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__6); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7); +l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8 = _init_l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__8); l_Lean_addTrace___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__6___closed__1 = _init_l_Lean_addTrace___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__6___closed__1(); l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__2___closed__1 = _init_l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__3___lambda__2___closed__1); @@ -26029,33 +25808,33 @@ l_Lean_Meta_IndPredBelow_mkBelow___closed__6 = _init_l_Lean_Meta_IndPredBelow_mk lean_mark_persistent(l_Lean_Meta_IndPredBelow_mkBelow___closed__6); l_Lean_Meta_IndPredBelow_mkBelow___closed__7 = _init_l_Lean_Meta_IndPredBelow_mkBelow___closed__7(); lean_mark_persistent(l_Lean_Meta_IndPredBelow_mkBelow___closed__7); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__1 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__1(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__1); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__2 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__2(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__2); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__3 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__3(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__3); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__4 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__4(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__4); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__5 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__5(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__5); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__6 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__6(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__6); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__7 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__7(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__7); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__8 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__8(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__8); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__9 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__9(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__9); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__10 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__10(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__10); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__11 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__11(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__11); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__12 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__12(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__12); -l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__13 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__13(); -lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142____closed__13); -if (builtin) {res = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8142_(lean_io_mk_world()); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__1 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__1(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__1); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__2 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__2(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__2); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__3 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__3(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__3); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__4 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__4(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__4); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__5 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__5(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__5); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__6 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__6(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__6); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__7 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__7(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__7); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__8 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__8(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__8); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__9 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__9(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__9); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__10 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__10(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__10); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__11 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__11(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__11); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__12 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__12(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__12); +l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__13 = _init_l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__13(); +lean_mark_persistent(l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144____closed__13); +if (builtin) {res = l_Lean_Meta_IndPredBelow_initFn____x40_Lean_Meta_IndPredBelow___hyg_8144_(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/InferType.c b/stage0/stdlib/Lean/Meta/InferType.c index 3c3d4501331c..7b140e70405c 100644 --- a/stage0/stdlib/Lean/Meta/InferType.c +++ b/stage0/stdlib/Lean/Meta/InferType.c @@ -110,6 +110,7 @@ lean_object* l_instBEqProd___rarg(lean_object*, lean_object*, lean_object*, lean LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_withAppRevAux___at_Lean_Expr_instantiateBetaRevRange_visit___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_Lean_Meta_forallBoundedTelescope___at_Lean_Meta_arrowDomainsN___spec__6(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_throwFunctionExpected___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_arrowDomainsN___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___private_Lean_Meta_InferType_0__Lean_Meta_isArrowProp___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isBVar(lean_object*); uint8_t l_Lean_Expr_hasMVar(lean_object*); @@ -203,14 +204,17 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_isArrowTyp static lean_object* l_Lean_Meta_throwFunctionExpected___rarg___closed__1; lean_object* lean_expr_lift_loose_bvars(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_throwFunctionExpected___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_arrowDomainsN___lambda__2___closed__4; lean_object* l_Lean_MVarId_isReadOnlyOrSyntheticOpaque(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_instantiateBetaRevRange___closed__8; +LEAN_EXPORT lean_object* l_Lean_Meta_arrowDomainsN___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_throwIncorrectNumberOfLevels___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_instantiateBetaRevRange_visit___closed__8; lean_object* lean_usize_to_nat(size_t); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_InferType_0__Lean_Meta_inferAppType___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* l_Lean_Meta_instInhabitedMetaM___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalContext_mkLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t); +static lean_object* l_Lean_Meta_arrowDomainsN___lambda__2___closed__1; lean_object* l_Lean_MessageData_ofExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_instantiateBetaRevRange___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_inferFVarType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -236,6 +240,7 @@ uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_isArrowType(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_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_InferType_0__Lean_Meta_inferAppType___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_Meta_arrowDomainsN___lambda__2___closed__2; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___private_Lean_Meta_InferType_0__Lean_Meta_inferForallType___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_indentExpr(lean_object*); @@ -257,6 +262,7 @@ LEAN_EXPORT lean_object* lean_infer_type(lean_object*, lean_object*, lean_object lean_object* lean_panic_fn(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_inferConstType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_inferTypeImp_infer___closed__1; +static lean_object* l_Lean_Meta_arrowDomainsN___lambda__2___closed__5; lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at___private_Lean_Meta_InferType_0__Lean_Meta_checkInferTypeCache___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getAppFn(lean_object*); @@ -325,9 +331,11 @@ lean_object* l_Lean_PersistentHashMap_getCollisionNodeSize___rarg(lean_object*); lean_object* l_Lean_FVarId_throwUnknown___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_throwUnknownMVar___rarg___closed__1; static lean_object* l_Lean_Meta_throwFunctionExpected___rarg___closed__3; +static lean_object* l_Lean_Meta_arrowDomainsN___lambda__2___closed__3; lean_object* l_Lean_Expr_lam___override(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_checkInferTypeCache___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_instantiateBetaRevRange___closed__6; +static lean_object* l_Lean_Meta_arrowDomainsN___lambda__2___closed__6; lean_object* l_Lean_Level_normalize(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_isTypeQuick(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_InferType_0__Lean_Meta_checkInferTypeCache___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -337,6 +345,7 @@ lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); lean_object* lean_expr_instantiate1(lean_object*, lean_object*); +lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Expr_instantiateBetaRevRange_visit___spec__8(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_throwTypeExcepted___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_isProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -22830,14 +22839,14 @@ LEAN_EXPORT lean_object* l_Lean_Meta_arrowDomainsN___lambda__1(lean_object* x_1, _start: { size_t x_9; size_t x_10; lean_object* x_11; -x_9 = lean_array_size(x_2); +x_9 = lean_array_size(x_1); x_10 = 0; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_2); -x_11 = l_Array_mapMUnsafe_map___at_Lean_Meta_arrowDomainsN___spec__1(x_9, x_10, x_2, x_4, x_5, x_6, x_7, x_8); +lean_inc(x_1); +x_11 = l_Array_mapMUnsafe_map___at_Lean_Meta_arrowDomainsN___spec__1(x_9, x_10, x_1, x_4, x_5, x_6, x_7, x_8); if (lean_obj_tag(x_11) == 0) { lean_object* x_12; lean_object* x_13; size_t x_14; lean_object* x_15; lean_object* x_16; @@ -22848,12 +22857,12 @@ lean_inc(x_13); lean_dec(x_11); x_14 = lean_array_size(x_12); x_15 = lean_box(0); -x_16 = l_Array_forInUnsafe_loop___at_Lean_Meta_arrowDomainsN___spec__5(x_1, x_2, x_12, x_14, x_10, x_15, x_4, x_5, x_6, x_7, x_13); +x_16 = l_Array_forInUnsafe_loop___at_Lean_Meta_arrowDomainsN___spec__5(x_2, x_1, x_12, x_14, x_10, x_15, x_4, x_5, x_6, x_7, x_13); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_2); +lean_dec(x_1); if (lean_obj_tag(x_16) == 0) { uint8_t x_17; @@ -22932,15 +22941,133 @@ return x_28; } } } +static lean_object* _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("type ", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_arrowDomainsN___lambda__2___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" does not have ", 15, 15); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_arrowDomainsN___lambda__2___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" parameters", 11, 11); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_arrowDomainsN___lambda__2___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_arrowDomainsN___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; uint8_t x_11; +x_10 = lean_array_get_size(x_3); +x_11 = lean_nat_dec_eq(x_10, x_2); +lean_dec(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; 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_dec(x_3); +x_12 = l_Lean_MessageData_ofExpr(x_1); +x_13 = l_Lean_Meta_arrowDomainsN___lambda__2___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_Meta_arrowDomainsN___lambda__2___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 = l___private_Init_Data_Repr_0__Nat_reprFast(x_2); +x_18 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_18, 0, x_17); +x_19 = l_Lean_MessageData_ofFormat(x_18); +x_20 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_20, 0, x_16); +lean_ctor_set(x_20, 1, x_19); +x_21 = l_Lean_Meta_arrowDomainsN___lambda__2___closed__6; +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 = l_Lean_throwError___at___private_Lean_Meta_InferType_0__Lean_Meta_inferProjType___spec__1(x_22, 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); +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) +{ +return x_23; +} +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(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; +} +} +else +{ +lean_object* x_28; lean_object* x_29; +lean_dec(x_2); +x_28 = lean_box(0); +x_29 = l_Lean_Meta_arrowDomainsN___lambda__1(x_3, x_1, x_28, x_5, x_6, x_7, x_8, x_9); +return x_29; +} +} +} LEAN_EXPORT lean_object* l_Lean_Meta_arrowDomainsN(lean_object* x_1, 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; lean_object* x_11; +lean_inc(x_1); x_8 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_8, 0, x_1); lean_inc(x_2); -x_9 = lean_alloc_closure((void*)(l_Lean_Meta_arrowDomainsN___lambda__1___boxed), 8, 1); +x_9 = lean_alloc_closure((void*)(l_Lean_Meta_arrowDomainsN___lambda__2___boxed), 9, 2); lean_closure_set(x_9, 0, x_2); +lean_closure_set(x_9, 1, x_1); x_10 = 0; x_11 = l_Lean_Meta_forallBoundedTelescope___at_Lean_Meta_arrowDomainsN___spec__6___rarg(x_2, x_8, x_9, x_10, x_3, x_4, x_5, x_6, x_7); return x_11; @@ -23031,6 +23158,15 @@ lean_dec(x_3); return x_9; } } +LEAN_EXPORT lean_object* l_Lean_Meta_arrowDomainsN___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_Meta_arrowDomainsN___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_4); +return x_10; +} +} LEAN_EXPORT lean_object* l_Lean_Meta_inferArgumentTypesN(lean_object* x_1, 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: { @@ -23217,6 +23353,18 @@ l_Array_forInUnsafe_loop___at_Lean_Meta_arrowDomainsN___spec__5___closed__3 = _i lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Meta_arrowDomainsN___spec__5___closed__3); l_Array_forInUnsafe_loop___at_Lean_Meta_arrowDomainsN___spec__5___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Meta_arrowDomainsN___spec__5___closed__4(); lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Meta_arrowDomainsN___spec__5___closed__4); +l_Lean_Meta_arrowDomainsN___lambda__2___closed__1 = _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Meta_arrowDomainsN___lambda__2___closed__1); +l_Lean_Meta_arrowDomainsN___lambda__2___closed__2 = _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Meta_arrowDomainsN___lambda__2___closed__2); +l_Lean_Meta_arrowDomainsN___lambda__2___closed__3 = _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Meta_arrowDomainsN___lambda__2___closed__3); +l_Lean_Meta_arrowDomainsN___lambda__2___closed__4 = _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__4(); +lean_mark_persistent(l_Lean_Meta_arrowDomainsN___lambda__2___closed__4); +l_Lean_Meta_arrowDomainsN___lambda__2___closed__5 = _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__5(); +lean_mark_persistent(l_Lean_Meta_arrowDomainsN___lambda__2___closed__5); +l_Lean_Meta_arrowDomainsN___lambda__2___closed__6 = _init_l_Lean_Meta_arrowDomainsN___lambda__2___closed__6(); +lean_mark_persistent(l_Lean_Meta_arrowDomainsN___lambda__2___closed__6); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Meta/Match/CaseArraySizes.c b/stage0/stdlib/Lean/Meta/Match/CaseArraySizes.c index d7e869b9374d..56e33ad4b24a 100644 --- a/stage0/stdlib/Lean/Meta/Match/CaseArraySizes.c +++ b/stage0/stdlib/Lean/Meta/Match/CaseArraySizes.c @@ -22,13 +22,14 @@ lean_object* l_Lean_Meta_mkLt(lean_object*, lean_object*, lean_object*, lean_obj lean_object* l_Lean_Meta_mkEqSymm(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_object* lean_array_push(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___boxed(lean_object**); lean_object* l_Lean_MVarId_assertExt(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_Array_mapFinIdxM_map___at_Lean_Meta_caseArraySizes___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_object* l_Lean_Meta_FVarSubst_get(lean_object*, lean_object*); lean_object* l_Lean_MVarId_getTag(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_CaseArraySizes_0__Lean_Meta_introArrayLit_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*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_caseArraySizes___spec__3(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* l_Lean_stringToMessageData(lean_object*); static lean_object* l_Lean_Meta_getArrayArgType___closed__6; static lean_object* l___private_Lean_Meta_Match_CaseArraySizes_0__Lean_Meta_introArrayLit_loop___closed__1; @@ -37,6 +38,7 @@ lean_object* l_Lean_Expr_appArg_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getArrayArgType___lambda__1(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_caseArraySizes___spec__1(size_t, size_t, lean_object*); 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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Meta_getArrayArgType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_caseArraySizes___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_caseArraySizes___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*); @@ -73,13 +75,11 @@ uint8_t lean_nat_dec_eq(lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_CaseArraySizes_0__Lean_Meta_introArrayLit___closed__1; lean_object* l_Lean_mkRawNatLit(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3(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* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_caseArraySizes___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_CaseArraySizes_0__Lean_Meta_introArrayLit_loop___closed__3; lean_object* l_Lean_indentExpr(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*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___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_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getArrayArgType___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_CaseArraySizes_0__Lean_Meta_mkArrayGetLit___closed__1; @@ -1144,7 +1144,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___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_Array_mapFinIdxM_map___at_Lean_Meta_caseArraySizes___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) { _start: { lean_object* x_13; @@ -1452,7 +1452,7 @@ return x_72; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* 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_object* x_17) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_caseArraySizes___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* 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_object* x_17) { _start: { lean_object* x_18; uint8_t x_19; @@ -1622,7 +1622,7 @@ x_58 = l_Lean_Expr_fvar___override(x_26); lean_inc(x_2); lean_inc(x_3); lean_inc(x_56); -x_59 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___lambda__1), 12, 7); +x_59 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___lambda__1), 12, 7); lean_closure_set(x_59, 0, x_58); lean_closure_set(x_59, 1, x_56); lean_closure_set(x_59, 2, x_3); @@ -1929,7 +1929,7 @@ lean_dec(x_38); x_41 = lean_array_get_size(x_39); x_42 = lean_mk_empty_array_with_capacity(x_41); x_43 = lean_unsigned_to_nat(0u); -x_44 = l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3(x_5, x_7, x_8, x_28, x_33, x_36, x_39, x_39, x_41, x_43, lean_box(0), x_42, x_9, x_10, x_11, x_12, x_40); +x_44 = l_Array_mapFinIdxM_map___at_Lean_Meta_caseArraySizes___spec__3(x_5, x_7, x_8, x_28, x_33, x_36, x_39, x_39, x_41, x_43, lean_box(0), x_42, x_9, x_10, x_11, x_12, x_40); lean_dec(x_39); lean_dec(x_5); return x_44; @@ -2163,7 +2163,7 @@ lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -2186,7 +2186,7 @@ lean_object* x_17 = _args[16]; size_t x_18; lean_object* x_19; x_18 = lean_unbox_usize(x_6); lean_dec(x_6); -x_19 = l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3(x_1, x_2, x_3, x_4, x_5, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +x_19 = l_Array_mapFinIdxM_map___at_Lean_Meta_caseArraySizes___spec__3(x_1, x_2, x_3, x_4, x_5, x_18, 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_1); diff --git a/stage0/stdlib/Lean/Meta/Match/Match.c b/stage0/stdlib/Lean/Meta/Match/Match.c index 151fe1ccc3de..730d254359bd 100644 --- a/stage0/stdlib/Lean/Meta/Match/Match.c +++ b/stage0/stdlib/Lean/Meta/Match/Match.c @@ -33,6 +33,7 @@ static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwNo LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__5___closed__2; static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasArrayLitPattern___closed__1; +static lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_Match_getMkMatcherInputInContext___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_constructorApp_x27_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasArrayLitPattern___lambda__1(lean_object*); @@ -42,6 +43,7 @@ lean_object* l_Lean_MVarId_contradictionCore(lean_object*, lean_object*, lean_ob LEAN_EXPORT lean_object* l_Lean_Meta_Match_processInaccessibleAsCtor___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* l_Lean_mkNatLit(lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException___rarg___closed__15; +static lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2; lean_object* l_instBEqOfDecidableEq___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandNatValuePattern___spec__1(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_Meta_Match_Match_0__Lean_Meta_Match_process___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -160,9 +162,7 @@ LEAN_EXPORT uint8_t l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isConst lean_object* lean_mk_array(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); extern uint8_t l_instInhabitedBool; -static lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1; static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasVarPattern___closed__1; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__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*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts_loop___rarg___closed__5; static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__4___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -225,6 +225,7 @@ static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandV lean_object* l_Lean_Meta_getMatcherInfo_x3f___at_Lean_Meta_reduceMatcher_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_processInaccessibleAsCtor(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_processInaccessibleAsCtor___lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__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*); static lean_object* l_Lean_Meta_Match_withMkMatcherInput___rarg___lambda__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException(lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processLeaf___lambda__2___closed__1; @@ -261,6 +262,7 @@ lean_object* l_Lean_RBNode_findCore___at_Lean_Meta_removeUnused___spec__1(lean_o LEAN_EXPORT lean_object* l_Lean_Meta_Match_withMkMatcherInput(lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException___rarg___closed__12; static lean_object* l_List_forIn_loop___at_Lean_Meta_Match_withMkMatcherInput___spec__4___closed__2; +static lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2; static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__6___closed__5; lean_object* l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processSkipInaccessible___closed__1; @@ -288,7 +290,6 @@ lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_GeneralizeTelescope_genera static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_traceStep___closed__1; LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_collectValues___spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_solveSomeLocalFVarIdCnstr_x3f_go___closed__1; -static lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4; lean_object* l_Lean_Meta_Match_Alt_replaceFVarId(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__14(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*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_getMkMatcherInputInContext___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -334,6 +335,7 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withClea LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processLeaf___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_Meta_Match_Match_0__Lean_Meta_Match_isValueOnlyTransitionCore___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_Match_Match_0__Lean_Meta_Match_processSkipInaccessible(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__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_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isArrayLitTransition___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isArrayLitTransition___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_filterTrivialCnstrs___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -358,6 +360,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_ha LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__8___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_Match_processInaccessibleAsCtor___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___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_solveSomeLocalFVarIdCnstr_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_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___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_Lean_Meta_Match_mkMatcherAuxDefinition___lambda__4___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_Match_mkMatcherAuxDefinition(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Meta_Match_withMkMatcherInput___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -372,7 +375,6 @@ LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_ static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_process___closed__4; static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processLeaf_go___closed__1; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2; 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*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___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_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_checkNextPatternTypes___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -455,6 +457,7 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withClea LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_solveCnstrs_go___spec__4___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_solveCnstrs_go___closed__3; lean_object* l_Lean_Meta_caseArraySizes(lean_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_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1___boxed(lean_object**); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Meta_Match_mkMatcher___spec__6(lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandVarIntoArrayLit_loop___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -503,6 +506,7 @@ static lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lea LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__23(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_levelZero; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_solveSomeLocalFVarIdCnstr_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_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, 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_Match_mkMatcherAuxDefinition___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processConstructor___closed__2; static lean_object* l_List_forIn_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_checkNextPatternTypes___spec__2___closed__1; @@ -511,6 +515,7 @@ static lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lea extern lean_object* l_Lean_instInhabitedExpr; LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__15(lean_object*, 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*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException___rarg___closed__8; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, 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_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processConstructor___spec__6(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__18___boxed(lean_object**); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasCtorOrInaccessible___lambda__1___boxed(lean_object*); @@ -547,7 +552,6 @@ static lean_object* l_Lean_isTracingEnabledFor___at___private_Lean_Meta_Match_Ma LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__3(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_mkMatcherAuxDefinition___lambda__4___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Meta_Match_withMkMatcherInput___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_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___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*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isBitVecValueTransition___closed__1; LEAN_EXPORT uint8_t l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_inLocalDecls(lean_object*, lean_object*); lean_object* l_instHashableProd___rarg___boxed(lean_object*, lean_object*, lean_object*); @@ -609,6 +613,7 @@ LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_ LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasRecursiveType(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_Meta_Match_Match_0__Lean_Meta_Match_solveCnstrs_go___spec__6(lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processSkipInaccessible___spec__3___closed__3; +static lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isFinValueTransition(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandBitVecValuePattern___spec__1___closed__10; static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_solveSomeLocalFVarIdCnstr_x3f___lambda__2___closed__6; @@ -638,9 +643,9 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___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_usize_to_nat(size_t); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___boxed(lean_object**); lean_object* l_Lean_Meta_instInhabitedMetaM___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandBitVecValuePattern___spec__1___closed__2; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___boxed(lean_object**); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Match_mkMatcher___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Meta_mkSimpCongrTheorem___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -653,6 +658,7 @@ LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Me static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasAsPattern___closed__1; extern lean_object* l_Lean_inheritedTraceOptions; static lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandIntValuePattern___spec__1___closed__5; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___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* l_Lean_MessageData_ofExpr(lean_object*); static lean_object* l_Lean_Meta_Match_getMkMatcherInputInContext___lambda__3___closed__1; lean_object* l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -770,7 +776,6 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withClea LEAN_EXPORT uint8_t l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isValueTransition(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Meta_Match_withMkMatcherInput___spec__2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isNatValueTransition___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2; static lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandBitVecValuePattern___spec__1___closed__7; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Match_mkMatcher___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException___rarg___closed__2; @@ -839,7 +844,6 @@ lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_obj lean_object* l_Array_ofSubarray___rarg(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processVariable(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processLeaf___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_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, 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_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException___rarg___closed__3; LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__7(lean_object*, lean_object*, lean_object*); @@ -854,7 +858,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_ex LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts_loop___rarg___lambda__1___boxed(lean_object**); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isFirstPatternVar___boxed(lean_object*); size_t lean_usize_sub(size_t, size_t); -static lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1; lean_object* lean_array_mk(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__5___boxed(lean_object**); static lean_object* l_Lean_Meta_Match_processInaccessibleAsCtor___lambda__1___closed__3; @@ -863,7 +866,6 @@ extern lean_object* l_Lean_Meta_Match_instInhabitedAlt; static lean_object* l_Lean_Meta_Match_mkMatcherAuxDefinition___lambda__4___closed__1; static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_10875____closed__3; static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__16___closed__1; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1___boxed(lean_object**); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_process___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static size_t l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Match_mkMatcherAuxDefinition___spec__2___closed__1; LEAN_EXPORT lean_object* l_List_forM___at_Lean_Meta_Match_MkMatcherInput_collectFVars___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -882,7 +884,6 @@ static lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Meta_Match_withMkM LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Match_mkMatcherAuxDefinition___spec__6(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandVarIntoCtor_x3f___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_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Match_mkMatcherAuxDefinition___spec__1___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, 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_Match_Match_0__Lean_Meta_Match_expandVarIntoCtor_x3f___lambda__2___closed__2; extern lean_object* l_Lean_instInhabitedName; static lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandBitVecValuePattern___spec__1___closed__11; @@ -914,7 +915,6 @@ size_t lean_usize_shift_left(size_t, size_t); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_setInlineAttribute(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Match_Match___hyg_14488____closed__12; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__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* l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_10837____closed__5; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Match_mkMatcher___spec__5(lean_object*, size_t, size_t, lean_object*); @@ -927,7 +927,6 @@ lean_object* l_instDecidableEqNat___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Meta_Match_processInaccessibleAsCtor___spec__2___boxed(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*); -static lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_List_mapM_loop___at_Lean_Meta_Match_instantiateAltLHSMVars___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processAsPattern___closed__1; @@ -936,6 +935,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_ex LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___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*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException___rarg___closed__1; static lean_object* l_Lean_Meta_Match_withMkMatcherInput___rarg___lambda__1___closed__2; +static lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts_loop___rarg___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_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_Match_mkMatcher___spec__12___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_Match_getMkMatcherInputInContext___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -943,6 +943,7 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withClea uint8_t l_Lean_isAuxRecursorWithSuffix(lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_10837____closed__3; +static lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1; static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__6___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isIntValueTransition(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_int_neg(lean_object*); @@ -971,7 +972,7 @@ lean_object* lean_nat_add(lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_getCollisionNodeSize___rarg(lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processConstructor___spec__7___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isValueTransition___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___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*); +LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___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*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isConstructorTransition(lean_object*); static lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandIntValuePattern___spec__1___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandVarIntoCtor_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -984,7 +985,7 @@ static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_solveSo LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__19___boxed__const__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withEqs_go___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_checkpointDefEq___at_Lean_Meta_isLevelDefEq___spec__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Meta_Match_mkMatcher___spec__15___at_Lean_Meta_Match_mkMatcher___spec__16___at_Lean_Meta_Match_mkMatcher___spec__17(lean_object*, lean_object*); uint8_t l_Lean_Expr_isFVar(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Match_processInaccessibleAsCtor___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1014,7 +1015,6 @@ lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(lean_ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__18(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isValueOnlyTransitionCore___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_Meta_Match_Match_0__Lean_Meta_Match_expandVarIntoArrayLit_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_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___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*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processLeaf___lambda__2___closed__2; lean_object* l_Lean_Meta_Match_Alt_toMessageData(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandBitVecValuePattern___spec__1___closed__3; @@ -19268,301 +19268,301 @@ 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_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7(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, uint8_t x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___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, uint8_t 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_13, lean_object* x_14) { _start: { -if (lean_obj_tag(x_12) == 0) +if (lean_obj_tag(x_13) == 0) { -lean_object* x_14; -lean_dec(x_9); -x_14 = l_List_reverse___rarg(x_13); -return x_14; +lean_object* x_15; +lean_dec(x_10); +x_15 = l_List_reverse___rarg(x_14); +return x_15; } else { -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_12, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_15, 4); +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_13, 0); lean_inc(x_16); -if (lean_obj_tag(x_16) == 0) +x_17 = lean_ctor_get(x_16, 4); +lean_inc(x_17); +if (lean_obj_tag(x_17) == 0) { -uint8_t x_17; -lean_dec(x_15); -x_17 = !lean_is_exclusive(x_12); -if (x_17 == 0) +uint8_t x_18; +lean_dec(x_16); +x_18 = !lean_is_exclusive(x_13); +if (x_18 == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_18 = lean_ctor_get(x_12, 1); -x_19 = lean_ctor_get(x_12, 0); -lean_dec(x_19); -x_20 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2; -x_21 = l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__6(x_20); -lean_ctor_set(x_12, 1, x_13); -lean_ctor_set(x_12, 0, x_21); -{ -lean_object* _tmp_7 = lean_box(0); -lean_object* _tmp_11 = x_18; -lean_object* _tmp_12 = x_12; -x_8 = _tmp_7; -x_12 = _tmp_11; +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_19 = lean_ctor_get(x_13, 1); +x_20 = lean_ctor_get(x_13, 0); +lean_dec(x_20); +x_21 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2; +x_22 = l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__6(x_21); +lean_ctor_set(x_13, 1, x_14); +lean_ctor_set(x_13, 0, x_22); +{ +lean_object* _tmp_8 = lean_box(0); +lean_object* _tmp_12 = x_19; +lean_object* _tmp_13 = x_13; +x_9 = _tmp_8; x_13 = _tmp_12; +x_14 = _tmp_13; } goto _start; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_23 = lean_ctor_get(x_12, 1); -lean_inc(x_23); -lean_dec(x_12); -x_24 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2; -x_25 = l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__6(x_24); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_13); -x_8 = lean_box(0); -x_12 = x_23; -x_13 = x_26; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_24 = lean_ctor_get(x_13, 1); +lean_inc(x_24); +lean_dec(x_13); +x_25 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2; +x_26 = l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__6(x_25); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_14); +x_9 = lean_box(0); +x_13 = x_24; +x_14 = x_27; goto _start; } } else { -lean_object* x_28; -x_28 = lean_ctor_get(x_16, 0); -lean_inc(x_28); -switch (lean_obj_tag(x_28)) { +lean_object* x_29; +x_29 = lean_ctor_get(x_17, 0); +lean_inc(x_29); +switch (lean_obj_tag(x_29)) { case 1: { -lean_object* x_29; uint8_t x_30; -x_29 = lean_ctor_get(x_12, 1); -lean_inc(x_29); -lean_dec(x_12); -x_30 = !lean_is_exclusive(x_15); -if (x_30 == 0) +lean_object* x_30; uint8_t x_31; +x_30 = lean_ctor_get(x_13, 1); +lean_inc(x_30); +lean_dec(x_13); +x_31 = !lean_is_exclusive(x_16); +if (x_31 == 0) { -lean_object* x_31; uint8_t x_32; -x_31 = lean_ctor_get(x_15, 4); -lean_dec(x_31); -x_32 = !lean_is_exclusive(x_16); -if (x_32 == 0) +lean_object* x_32; uint8_t x_33; +x_32 = lean_ctor_get(x_16, 4); +lean_dec(x_32); +x_33 = !lean_is_exclusive(x_17); +if (x_33 == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_33 = lean_ctor_get(x_16, 1); -x_34 = lean_ctor_get(x_16, 0); -lean_dec(x_34); -x_35 = lean_ctor_get(x_28, 0); -lean_inc(x_35); -lean_dec(x_28); -lean_ctor_set(x_15, 4, x_33); -lean_inc(x_9); -x_36 = l_Lean_Meta_Match_Alt_replaceFVarId(x_35, x_9, x_15); -lean_ctor_set(x_16, 1, x_13); -lean_ctor_set(x_16, 0, x_36); -x_8 = lean_box(0); -x_12 = x_29; -x_13 = x_16; +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_34 = lean_ctor_get(x_17, 1); +x_35 = lean_ctor_get(x_17, 0); +lean_dec(x_35); +x_36 = lean_ctor_get(x_29, 0); +lean_inc(x_36); +lean_dec(x_29); +lean_ctor_set(x_16, 4, x_34); +lean_inc(x_10); +x_37 = l_Lean_Meta_Match_Alt_replaceFVarId(x_36, x_10, x_16); +lean_ctor_set(x_17, 1, x_14); +lean_ctor_set(x_17, 0, x_37); +x_9 = lean_box(0); +x_13 = x_30; +x_14 = x_17; goto _start; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_38 = lean_ctor_get(x_16, 1); -lean_inc(x_38); -lean_dec(x_16); -x_39 = lean_ctor_get(x_28, 0); +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_39 = lean_ctor_get(x_17, 1); lean_inc(x_39); -lean_dec(x_28); -lean_ctor_set(x_15, 4, x_38); -lean_inc(x_9); -x_40 = l_Lean_Meta_Match_Alt_replaceFVarId(x_39, x_9, x_15); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_13); -x_8 = lean_box(0); -x_12 = x_29; -x_13 = x_41; +lean_dec(x_17); +x_40 = lean_ctor_get(x_29, 0); +lean_inc(x_40); +lean_dec(x_29); +lean_ctor_set(x_16, 4, x_39); +lean_inc(x_10); +x_41 = l_Lean_Meta_Match_Alt_replaceFVarId(x_40, x_10, x_16); +x_42 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_14); +x_9 = lean_box(0); +x_13 = x_30; +x_14 = x_42; 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; -x_43 = lean_ctor_get(x_15, 0); -x_44 = lean_ctor_get(x_15, 1); -x_45 = lean_ctor_get(x_15, 2); -x_46 = lean_ctor_get(x_15, 3); -x_47 = lean_ctor_get(x_15, 5); +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_44 = lean_ctor_get(x_16, 0); +x_45 = lean_ctor_get(x_16, 1); +x_46 = lean_ctor_get(x_16, 2); +x_47 = lean_ctor_get(x_16, 3); +x_48 = lean_ctor_get(x_16, 5); +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_15); -x_48 = lean_ctor_get(x_16, 1); -lean_inc(x_48); -if (lean_is_exclusive(x_16)) { - lean_ctor_release(x_16, 0); - lean_ctor_release(x_16, 1); - x_49 = x_16; +lean_dec(x_16); +x_49 = lean_ctor_get(x_17, 1); +lean_inc(x_49); +if (lean_is_exclusive(x_17)) { + lean_ctor_release(x_17, 0); + lean_ctor_release(x_17, 1); + x_50 = x_17; } else { - lean_dec_ref(x_16); - x_49 = lean_box(0); + lean_dec_ref(x_17); + x_50 = lean_box(0); } -x_50 = lean_ctor_get(x_28, 0); -lean_inc(x_50); -lean_dec(x_28); -x_51 = lean_alloc_ctor(0, 6, 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_46); -lean_ctor_set(x_51, 4, x_48); -lean_ctor_set(x_51, 5, x_47); -lean_inc(x_9); -x_52 = l_Lean_Meta_Match_Alt_replaceFVarId(x_50, x_9, x_51); -if (lean_is_scalar(x_49)) { - x_53 = lean_alloc_ctor(1, 2, 0); +x_51 = lean_ctor_get(x_29, 0); +lean_inc(x_51); +lean_dec(x_29); +x_52 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_52, 0, x_44); +lean_ctor_set(x_52, 1, x_45); +lean_ctor_set(x_52, 2, x_46); +lean_ctor_set(x_52, 3, x_47); +lean_ctor_set(x_52, 4, x_49); +lean_ctor_set(x_52, 5, x_48); +lean_inc(x_10); +x_53 = l_Lean_Meta_Match_Alt_replaceFVarId(x_51, x_10, x_52); +if (lean_is_scalar(x_50)) { + x_54 = lean_alloc_ctor(1, 2, 0); } else { - x_53 = x_49; + x_54 = x_50; } -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_13); -x_8 = lean_box(0); -x_12 = x_29; -x_13 = x_53; +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_14); +x_9 = lean_box(0); +x_13 = x_30; +x_14 = x_54; goto _start; } } case 3: { -lean_object* x_55; uint8_t x_56; -lean_dec(x_28); -x_55 = lean_ctor_get(x_12, 1); -lean_inc(x_55); -lean_dec(x_12); -x_56 = !lean_is_exclusive(x_15); -if (x_56 == 0) +lean_object* x_56; uint8_t x_57; +lean_dec(x_29); +x_56 = lean_ctor_get(x_13, 1); +lean_inc(x_56); +lean_dec(x_13); +x_57 = !lean_is_exclusive(x_16); +if (x_57 == 0) { -lean_object* x_57; uint8_t x_58; -x_57 = lean_ctor_get(x_15, 4); -lean_dec(x_57); -x_58 = !lean_is_exclusive(x_16); -if (x_58 == 0) +lean_object* x_58; uint8_t x_59; +x_58 = lean_ctor_get(x_16, 4); +lean_dec(x_58); +x_59 = !lean_is_exclusive(x_17); +if (x_59 == 0) { -lean_object* x_59; lean_object* x_60; -x_59 = lean_ctor_get(x_16, 1); -x_60 = lean_ctor_get(x_16, 0); -lean_dec(x_60); -lean_ctor_set(x_15, 4, x_59); -lean_ctor_set(x_16, 1, x_13); -lean_ctor_set(x_16, 0, x_15); -x_8 = lean_box(0); -x_12 = x_55; -x_13 = x_16; +lean_object* x_60; lean_object* x_61; +x_60 = lean_ctor_get(x_17, 1); +x_61 = lean_ctor_get(x_17, 0); +lean_dec(x_61); +lean_ctor_set(x_16, 4, x_60); +lean_ctor_set(x_17, 1, x_14); +lean_ctor_set(x_17, 0, x_16); +x_9 = lean_box(0); +x_13 = x_56; +x_14 = x_17; goto _start; } else { -lean_object* x_62; lean_object* x_63; -x_62 = lean_ctor_get(x_16, 1); -lean_inc(x_62); -lean_dec(x_16); -lean_ctor_set(x_15, 4, x_62); -x_63 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_63, 0, x_15); -lean_ctor_set(x_63, 1, x_13); -x_8 = lean_box(0); -x_12 = x_55; -x_13 = x_63; +lean_object* x_63; lean_object* x_64; +x_63 = lean_ctor_get(x_17, 1); +lean_inc(x_63); +lean_dec(x_17); +lean_ctor_set(x_16, 4, x_63); +x_64 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_64, 0, x_16); +lean_ctor_set(x_64, 1, x_14); +x_9 = lean_box(0); +x_13 = x_56; +x_14 = x_64; 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_15, 0); -x_66 = lean_ctor_get(x_15, 1); -x_67 = lean_ctor_get(x_15, 2); -x_68 = lean_ctor_get(x_15, 3); -x_69 = lean_ctor_get(x_15, 5); +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_66 = lean_ctor_get(x_16, 0); +x_67 = lean_ctor_get(x_16, 1); +x_68 = lean_ctor_get(x_16, 2); +x_69 = lean_ctor_get(x_16, 3); +x_70 = lean_ctor_get(x_16, 5); +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_15); -x_70 = lean_ctor_get(x_16, 1); -lean_inc(x_70); -if (lean_is_exclusive(x_16)) { - lean_ctor_release(x_16, 0); - lean_ctor_release(x_16, 1); - x_71 = x_16; +lean_dec(x_16); +x_71 = lean_ctor_get(x_17, 1); +lean_inc(x_71); +if (lean_is_exclusive(x_17)) { + lean_ctor_release(x_17, 0); + lean_ctor_release(x_17, 1); + x_72 = x_17; } else { - lean_dec_ref(x_16); - x_71 = lean_box(0); + lean_dec_ref(x_17); + x_72 = lean_box(0); } -x_72 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_72, 0, x_65); -lean_ctor_set(x_72, 1, x_66); -lean_ctor_set(x_72, 2, x_67); -lean_ctor_set(x_72, 3, x_68); -lean_ctor_set(x_72, 4, x_70); -lean_ctor_set(x_72, 5, x_69); -if (lean_is_scalar(x_71)) { - x_73 = lean_alloc_ctor(1, 2, 0); +x_73 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_73, 0, x_66); +lean_ctor_set(x_73, 1, x_67); +lean_ctor_set(x_73, 2, x_68); +lean_ctor_set(x_73, 3, x_69); +lean_ctor_set(x_73, 4, x_71); +lean_ctor_set(x_73, 5, x_70); +if (lean_is_scalar(x_72)) { + x_74 = lean_alloc_ctor(1, 2, 0); } else { - x_73 = x_71; + x_74 = x_72; } -lean_ctor_set(x_73, 0, x_72); -lean_ctor_set(x_73, 1, x_13); -x_8 = lean_box(0); -x_12 = x_55; -x_13 = x_73; +lean_ctor_set(x_74, 0, x_73); +lean_ctor_set(x_74, 1, x_14); +x_9 = lean_box(0); +x_13 = x_56; +x_14 = x_74; goto _start; } } default: { -uint8_t x_75; -lean_dec(x_28); -lean_dec(x_15); -x_75 = !lean_is_exclusive(x_16); -if (x_75 == 0) +uint8_t x_76; +lean_dec(x_29); +lean_dec(x_16); +x_76 = !lean_is_exclusive(x_17); +if (x_76 == 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_16, 1); -lean_dec(x_76); -x_77 = lean_ctor_get(x_16, 0); +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_77 = lean_ctor_get(x_17, 1); lean_dec(x_77); -x_78 = lean_ctor_get(x_12, 1); -lean_inc(x_78); -lean_dec(x_12); -x_79 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2; -x_80 = l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__6(x_79); -lean_ctor_set(x_16, 1, x_13); -lean_ctor_set(x_16, 0, x_80); -x_8 = lean_box(0); -x_12 = x_78; -x_13 = x_16; +x_78 = lean_ctor_get(x_17, 0); +lean_dec(x_78); +x_79 = lean_ctor_get(x_13, 1); +lean_inc(x_79); +lean_dec(x_13); +x_80 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2; +x_81 = l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__6(x_80); +lean_ctor_set(x_17, 1, x_14); +lean_ctor_set(x_17, 0, x_81); +x_9 = lean_box(0); +x_13 = x_79; +x_14 = x_17; goto _start; } else { -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; -lean_dec(x_16); -x_82 = lean_ctor_get(x_12, 1); -lean_inc(x_82); -lean_dec(x_12); -x_83 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2; -x_84 = l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__6(x_83); -x_85 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_85, 0, x_84); -lean_ctor_set(x_85, 1, x_13); -x_8 = lean_box(0); -x_12 = x_82; -x_13 = x_85; +lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +lean_dec(x_17); +x_83 = lean_ctor_get(x_13, 1); +lean_inc(x_83); +lean_dec(x_13); +x_84 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2; +x_85 = l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__6(x_84); +x_86 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_14); +x_9 = lean_box(0); +x_13 = x_83; +x_14 = x_86; goto _start; } } @@ -19730,7 +19730,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___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, uint8_t 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_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___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, uint8_t 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) { _start: { 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; uint8_t x_29; @@ -19748,7 +19748,7 @@ x_25 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match x_26 = l_List_filterTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__4(x_1, x_21, x_23); lean_inc(x_4); x_27 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__5(x_2, x_5, x_6, x_7, x_8, x_9, lean_box(0), x_4, x_10, x_14, x_26, x_23); -x_28 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7(x_2, x_11, x_5, x_6, x_7, x_8, x_9, lean_box(0), x_1, x_10, x_14, x_27, x_23); +x_28 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7(x_2, x_11, x_5, x_6, x_7, x_6, x_8, x_9, lean_box(0), x_1, x_10, x_14, x_27, x_23); x_29 = !lean_is_exclusive(x_2); if (x_29 == 0) { @@ -19788,7 +19788,7 @@ return x_38; } } } -static lean_object* _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1() { _start: { lean_object* x_1; @@ -19796,16 +19796,16 @@ x_1 = lean_mk_string_unchecked("processValue subst: ", 20, 20); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2() { +static lean_object* _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1; +x_1 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3() { +static lean_object* _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3() { _start: { lean_object* x_1; @@ -19813,16 +19813,16 @@ x_1 = lean_mk_string_unchecked(", ", 2, 2); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4() { +static lean_object* _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3; +x_1 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___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) { _start: { lean_object* x_17; uint8_t x_18; @@ -19909,7 +19909,7 @@ lean_dec(x_39); x_43 = lean_box(0); x_44 = lean_unbox(x_40); lean_dec(x_40); -x_45 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(x_36, x_3, x_8, x_38, x_9, x_2, x_4, x_10, x_11, x_44, x_1, x_6, x_37, x_43, x_12, x_13, x_14, x_15, x_42); +x_45 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(x_36, x_3, x_8, x_38, x_9, x_2, x_4, x_10, x_11, x_44, x_1, x_6, x_37, x_43, x_12, x_13, x_14, x_15, x_42); lean_dec(x_4); return x_45; } @@ -19929,11 +19929,11 @@ lean_inc(x_49); x_51 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__9(x_49, x_50); x_52 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_51, x_50); x_53 = l_Lean_MessageData_ofList(x_52); -x_54 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2; +x_54 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2; lean_ctor_set_tag(x_39, 7); lean_ctor_set(x_39, 1, x_53); lean_ctor_set(x_39, 0, x_54); -x_55 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4; +x_55 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4; x_56 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_56, 0, x_39); lean_ctor_set(x_56, 1, x_55); @@ -19955,7 +19955,7 @@ lean_inc(x_65); lean_dec(x_63); x_66 = lean_unbox(x_40); lean_dec(x_40); -x_67 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(x_36, x_3, x_8, x_38, x_9, x_2, x_4, x_10, x_11, x_66, x_1, x_6, x_37, x_64, x_12, x_13, x_14, x_15, x_65); +x_67 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(x_36, x_3, x_8, x_38, x_9, x_2, x_4, x_10, x_11, x_66, x_1, x_6, x_37, x_64, x_12, x_13, x_14, x_15, x_65); lean_dec(x_64); lean_dec(x_4); return x_67; @@ -19972,11 +19972,11 @@ lean_inc(x_69); x_71 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__9(x_69, x_70); x_72 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_71, x_70); x_73 = l_Lean_MessageData_ofList(x_72); -x_74 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2; +x_74 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2; 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_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4; +x_76 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4; x_77 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_77, 0, x_75); lean_ctor_set(x_77, 1, x_76); @@ -19998,7 +19998,7 @@ lean_inc(x_86); lean_dec(x_84); x_87 = lean_unbox(x_40); lean_dec(x_40); -x_88 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(x_36, x_3, x_8, x_38, x_9, x_2, x_4, x_10, x_11, x_87, x_1, x_6, x_37, x_85, x_12, x_13, x_14, x_15, x_86); +x_88 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(x_36, x_3, x_8, x_38, x_9, x_2, x_4, x_10, x_11, x_87, x_1, x_6, x_37, x_85, x_12, x_13, x_14, x_15, x_86); lean_dec(x_85); lean_dec(x_4); return x_88; @@ -20007,7 +20007,7 @@ return x_88; } } } -static lean_object* _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1() { _start: { lean_object* x_1; @@ -20015,16 +20015,16 @@ x_1 = lean_mk_string_unchecked("processValue subgoal\n", 21, 21); return x_1; } } -static lean_object* _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2() { +static lean_object* _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1; +x_1 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___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, lean_object* x_8, lean_object* x_9, 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_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___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, lean_object* x_8, lean_object* x_9, 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; @@ -20055,7 +20055,7 @@ lean_inc(x_2); lean_inc(x_4); lean_inc(x_3); lean_inc(x_1); -x_29 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(x_5, x_10, x_1, x_22, x_3, x_4, x_2, x_6, x_7, x_28, x_27, x_13, x_14, x_15, x_16, x_26); +x_29 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(x_5, x_10, x_1, x_22, x_3, x_4, x_2, x_6, x_7, x_28, x_27, x_13, x_14, x_15, x_16, x_26); x_30 = lean_ctor_get(x_29, 0); lean_inc(x_30); x_31 = lean_ctor_get(x_29, 1); @@ -20085,7 +20085,7 @@ x_38 = lean_ctor_get(x_22, 0); lean_inc(x_38); x_39 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_39, 0, x_38); -x_40 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2; +x_40 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2; lean_ctor_set_tag(x_23, 7); lean_ctor_set(x_23, 1, x_39); lean_ctor_set(x_23, 0, x_40); @@ -20106,7 +20106,7 @@ lean_inc(x_2); lean_inc(x_4); lean_inc(x_3); lean_inc(x_1); -x_47 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(x_5, x_10, x_1, x_22, x_3, x_4, x_2, x_6, x_7, x_46, x_44, x_13, x_14, x_15, x_16, x_45); +x_47 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(x_5, x_10, x_1, x_22, x_3, x_4, x_2, x_6, x_7, x_46, x_44, x_13, x_14, x_15, x_16, x_45); lean_dec(x_44); x_48 = lean_ctor_get(x_47, 0); lean_inc(x_48); @@ -20133,7 +20133,7 @@ x_54 = lean_ctor_get(x_22, 0); lean_inc(x_54); x_55 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_55, 0, x_54); -x_56 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2; +x_56 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2; x_57 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_57, 0, x_56); lean_ctor_set(x_57, 1, x_55); @@ -20154,7 +20154,7 @@ lean_inc(x_2); lean_inc(x_4); lean_inc(x_3); lean_inc(x_1); -x_64 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(x_5, x_10, x_1, x_22, x_3, x_4, x_2, x_6, x_7, x_63, x_61, x_13, x_14, x_15, x_16, x_62); +x_64 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(x_5, x_10, x_1, x_22, x_3, x_4, x_2, x_6, x_7, x_63, x_61, x_13, x_14, x_15, x_16, x_62); lean_dec(x_61); x_65 = lean_ctor_get(x_64, 0); lean_inc(x_65); @@ -20250,7 +20250,7 @@ lean_dec(x_19); x_22 = lean_array_get_size(x_20); x_23 = lean_mk_empty_array_with_capacity(x_22); x_24 = lean_unsigned_to_nat(0u); -x_25 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11(x_1, x_2, x_12, x_13, x_14, x_16, x_20, x_20, x_22, x_24, lean_box(0), x_23, x_4, x_5, x_6, x_7, x_21); +x_25 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11(x_1, x_2, x_12, x_13, x_14, x_16, x_20, x_20, x_22, x_24, lean_box(0), x_23, x_4, x_5, x_6, x_7, x_21); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -20397,26 +20397,27 @@ lean_dec(x_1); return x_15; } } -LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___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, 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_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___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, 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_14; uint8_t x_15; lean_object* x_16; -x_14 = lean_unbox(x_6); -lean_dec(x_6); -x_15 = lean_unbox(x_10); -lean_dec(x_10); -x_16 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7(x_1, x_2, x_3, x_4, x_5, x_14, x_7, x_8, x_9, x_15, x_11, x_12, x_13); -lean_dec(x_11); +uint8_t x_15; uint8_t x_16; lean_object* x_17; +x_15 = lean_unbox(x_7); lean_dec(x_7); +x_16 = lean_unbox(x_11); +lean_dec(x_11); +x_17 = l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7(x_1, x_2, x_3, x_4, x_5, x_6, x_15, x_8, x_9, x_10, x_16, x_12, x_13, x_14); +lean_dec(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); lean_dec(x_1); -return x_16; +return x_17; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -20443,7 +20444,7 @@ x_20 = lean_unbox(x_8); lean_dec(x_8); x_21 = lean_unbox(x_10); lean_dec(x_10); -x_22 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_20, x_9, x_21, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19); +x_22 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_20, x_9, x_21, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -20458,13 +20459,13 @@ lean_dec(x_3); return x_22; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___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_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___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_17; lean_object* x_18; x_17 = lean_unbox(x_10); lean_dec(x_10); -x_18 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17, x_11, x_12, x_13, x_14, x_15, x_16); +x_18 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -20477,7 +20478,7 @@ lean_dec(x_1); return x_18; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -20498,7 +20499,7 @@ lean_object* x_17 = _args[16]; _start: { lean_object* x_18; -x_18 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11(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 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11(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_16); lean_dec(x_15); lean_dec(x_14); @@ -22413,7 +22414,7 @@ return x_161; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___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, lean_object* x_8, lean_object* x_9, 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_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___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, lean_object* x_8, lean_object* x_9, 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; @@ -22784,7 +22785,7 @@ lean_dec(x_18); x_21 = lean_array_get_size(x_19); x_22 = lean_mk_empty_array_with_capacity(x_21); x_23 = lean_unsigned_to_nat(0u); -x_24 = l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__9(x_1, x_11, x_12, x_13, x_15, x_19, x_19, x_21, x_23, lean_box(0), x_22, x_3, x_4, x_5, x_6, x_20); +x_24 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__9(x_1, x_11, x_12, x_13, x_15, x_19, x_19, x_21, x_23, lean_box(0), x_22, x_3, x_4, x_5, x_6, x_20); lean_dec(x_19); lean_dec(x_15); lean_dec(x_13); @@ -22917,11 +22918,11 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___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, 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_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___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, 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_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__9(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 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__9(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); @@ -49014,18 +49015,18 @@ l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_proces lean_mark_persistent(l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__1); l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2 = _init_l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2(); lean_mark_persistent(l_List_mapTR_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__7___closed__2); -l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1 = _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1); -l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2 = _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2(); -lean_mark_persistent(l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2); -l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3 = _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3(); -lean_mark_persistent(l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3); -l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4 = _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4(); -lean_mark_persistent(l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4); -l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1 = _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1); -l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2 = _init_l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2(); -lean_mark_persistent(l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2); +l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1 = _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__1); +l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2 = _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__2); +l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3 = _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__3); +l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4 = _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___lambda__2___closed__4); +l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1 = _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__1); +l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2 = _init_l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__11___closed__2); l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___lambda__1___closed__1 = _init_l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___lambda__1___closed__1(); lean_mark_persistent(l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___lambda__1___closed__1); l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___closed__1 = _init_l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___closed__1(); diff --git a/stage0/stdlib/Lean/Meta/Tactic/AC/Main.c b/stage0/stdlib/Lean/Meta/Tactic/AC/Main.c index 86751a894eda..76a69f296fba 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/AC/Main.c +++ b/stage0/stdlib/Lean/Meta/Tactic/AC/Main.c @@ -17,19 +17,24 @@ static lean_object* l_Std_DHashMap_Internal_AssocList_get_x21___at_Lean_Meta_AC_ lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__9; lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_abstractAtoms_go___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___lambda__3___boxed(lean_object*); lean_object* l_Lean_mkNatLit(lean_object*); LEAN_EXPORT lean_object* l_Array_insertionSort_traverse___at_Lean_Meta_AC_toACExpr___spec__7(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*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__2(size_t, size_t, lean_object*); static lean_object* l_Lean_Meta_AC_buildNormProof_convert___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_AC_toACExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_DHashMap_Internal_AssocList_get_x21___at_Lean_Meta_AC_toACExpr___spec__10___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_AC_acRflTactic___rarg___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_Meta_AC_acRflTactic_declRange__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_AC_instEvalInformationPreContextACExpr___lambda__1(lean_object*); +static lean_object* l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__3; static lean_object* l_Lean_Meta_AC_getInstance___closed__6; static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__6; +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__13; LEAN_EXPORT lean_object* l_Std_HashMap_get_x21___at_Lean_Meta_AC_toACExpr___spec__9___boxed(lean_object*, lean_object*, lean_object*); uint32_t l_UInt32_ofNatTruncate(lean_object*); lean_object* l_Lean_mkApp7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -38,6 +43,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_AC_acNfTargetTactic(lean_object*, lean_obje LEAN_EXPORT lean_object* l_Lean_Meta_AC_acRflTactic(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_AC_buildNormProof___lambda__1(lean_object*, 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_ForEachExpr_visit___spec__2(lean_object*, lean_object*); 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_AC_getInstance___closed__1; @@ -45,22 +51,27 @@ size_t lean_uint64_to_usize(uint64_t); lean_object* lean_array_fswap(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_preContext___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_AC_rewriteUnnormalized___lambda__4(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_isAppOfArity(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_expandLocation(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_rewriteUnnormalized___lambda__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_Elab_Tactic_tacticElabAttribute; static lean_object* l_Lean_Meta_AC_acNfTargetTactic___closed__1; -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__8; lean_object* lean_array_push(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_rewriteUnnormalized___closed__12; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__1(size_t, size_t, lean_object*); +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__3; +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__14; lean_object* lean_mk_array(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__8; uint8_t lean_usize_dec_eq(size_t, size_t); extern uint8_t l_instInhabitedBool; LEAN_EXPORT lean_object* l_Lean_Meta_AC_acNfHypMeta___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_rewriteUnnormalized___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_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_convert(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304_(lean_object*); static lean_object* l_Lean_Meta_AC_getInstance___lambda__2___closed__1; +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__5; +lean_object* l_Lean_Meta_mkExpectedTypeHint(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_bvar___override(lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* l_Lean_Meta_Simp_main(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -71,6 +82,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_AC_evalNf0___lambda__4___boxed(lean_object* static lean_object* l_Lean_Meta_AC_rewriteUnnormalized___closed__10; 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*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_AC_toACExpr___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__10; static lean_object* l_Lean_Meta_AC_buildNormProof___closed__1; static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic_declRange__1___closed__2; @@ -78,7 +90,6 @@ static lean_object* l_Lean_Meta_AC_preContext___closed__6; static lean_object* l_Lean_Meta_AC_evalNf0___lambda__4___closed__1; static lean_object* l_Lean_Meta_AC_toACExpr___closed__1; lean_object* l_Lean_MVarId_refl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__3; static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___closed__3; @@ -98,28 +109,31 @@ static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic_declRange__1___close lean_object* l_Lean_mkApp4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_getFVarIds(lean_object*, 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_AC_acNfHypTactic___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_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__10; +LEAN_EXPORT lean_object* l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__3(lean_object*, lean_object*); lean_object* l_Lean_Meta_getSimpCongrTheorems___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_getInstance___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_evalNf0___closed__3; -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__2; +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__11; +lean_object* l_Lean_Expr_appArg_x21(lean_object*); static lean_object* l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___closed__4; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x21___at_Lean_Meta_AC_toACExpr___spec__10___boxed(lean_object*, lean_object*, lean_object*); extern lean_object* l_instInhabitedNat; -LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__2___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_preContext___closed__5; -LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__2(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_buildNormProof___lambda__1___closed__3; +static lean_object* l_Lean_Meta_AC_buildNormProof___lambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic_declRange__1___closed__4; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Meta_AC_toACExpr___spec__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___lambda__1(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__4; size_t lean_usize_of_nat(lean_object*); +static lean_object* l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__2; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2; -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__11; +static lean_object* l_Lean_Meta_AC_buildNormProof___lambda__1___closed__1; lean_object* l_Lean_MVarId_getNondepPropHyps(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___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_Lean_Meta_AC_buildNormProof_mkContext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__3___boxed(lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_ForEachExpr_visit___spec__3(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_rewriteUnnormalized___lambda__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_AC_evalNf0___closed__1; @@ -132,12 +146,10 @@ LEAN_EXPORT lean_object* l_Lean_Meta_AC_rewriteUnnormalized___lambda__2___boxed( static lean_object* l_Lean_Meta_AC_getInstance___closed__2; static lean_object* l_Lean_Meta_AC_getInstance___closed__7; uint64_t lean_uint64_shift_right(uint64_t, uint64_t); -lean_object* l_Array_unzip___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_AC_toACExpr___spec__11(lean_object*, size_t, size_t, lean_object*); lean_object* lean_nat_div(lean_object*, lean_object*); lean_object* l_Lean_MVarId_getType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895_(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4; static lean_object* l_Lean_Meta_AC_buildNormProof_convert___closed__5; LEAN_EXPORT uint8_t l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___lambda__3(lean_object*); @@ -145,12 +157,13 @@ static lean_object* l_Lean_Meta_AC_getInstance___lambda__2___closed__2; lean_object* l_Lean_registerTraceClass(lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__7; static lean_object* l_Lean_Meta_AC_acNfHypMeta___lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__6(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic_declRange__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_AC_evalNf0___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_AC_buildNormProof_mkContext___closed__8; static lean_object* l_Lean_Meta_AC_buildNormProof___closed__3; static lean_object* l_Lean_Meta_AC_evalNf0___closed__2; -LEAN_EXPORT lean_object* l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__1___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__4; 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_foldlMUnsafe_fold___at_Lean_Meta_AC_evalNf0___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___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__2; @@ -164,13 +177,14 @@ static uint32_t l_Lean_Meta_AC_rewriteUnnormalized___closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Meta_AC_toACExpr___spec__4(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_evalNf0___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_mkAppM(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__12; +static lean_object* l_Lean_Meta_AC_buildNormProof___lambda__1___closed__6; static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__1; +static lean_object* l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__4; static lean_object* l___regBuiltin_Lean_Meta_AC_evalNf0__1___closed__2; lean_object* lean_array_to_list(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_convertTarget(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_mkEq(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_AC_evalNf0___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_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3(lean_object*, lean_object*); lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_withMainContext___spec__1___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_Name_num___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_evalNf0___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -179,19 +193,21 @@ static lean_object* l_Lean_Meta_AC_rewriteUnnormalized___closed__4; static lean_object* l_Lean_Meta_AC_acNfHypMeta___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Meta_AC_toACExpr___spec__6(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_buildNormProof___closed__2; -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__16; static lean_object* l_Lean_Meta_AC_buildNormProof_convert___closed__2; static lean_object* l_Lean_Meta_AC_acNfHypMeta___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___lambda__2___boxed(lean_object*); static lean_object* l_Lean_Meta_AC_instEvalInformationPreContextACExpr___closed__4; extern lean_object* l_Lean_instInhabitedExpr; +static lean_object* l_Lean_Meta_AC_abstractAtoms_go___closed__2; uint64_t l_Lean_Expr_hash(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5(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_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Meta_AC_buildNormProof___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Meta_AC_toACExpr___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_AC_toACExpr___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_acNfHypMeta___lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms_go___lambda__1___boxed(lean_object**); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__7; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -201,26 +217,33 @@ uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_rewriteUnnormalized___closed__9; LEAN_EXPORT lean_object* l_Lean_Meta_AC_acNfHypTactic(lean_object*, 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_AC_instEvalInformationPreContextACExpr___lambda__3(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__9; static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__3; static lean_object* l___regBuiltin_Lean_Meta_AC_evalNf0__1___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_getInstance___lambda__1___boxed(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_AC_toACExpr___spec__12(lean_object*, size_t, size_t, lean_object*); static lean_object* l___regBuiltin_Lean_Meta_AC_evalNf0__1___closed__3; -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__13; LEAN_EXPORT lean_object* l_Lean_Meta_AC_rewriteUnnormalized___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_AC_rewriteUnnormalized___closed__3; static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic_declRange__1___closed__1; +lean_object* l_Lean_Meta_instInhabitedMetaM___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_rewriteUnnormalizedRefl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__15; +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__8; +lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Meta_AC_toACExpr___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_buildNormProof___lambda__1___closed__5; +LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof___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_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__6___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_toACExpr___closed__4; static lean_object* l_Lean_Meta_AC_preContext___closed__7; uint8_t lean_expr_lt(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__7; +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms_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_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__15; LEAN_EXPORT lean_object* l_Lean_Meta_AC_post(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_AC_instEvalInformationPreContextACExpr; +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__1; lean_object* l_Lean_Data_AC_mergeIdem(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_acRflTactic___rarg(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_AC_buildNormProof_mkContext___spec__1(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_object*, lean_object*, lean_object*); @@ -234,28 +257,32 @@ LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_convertTarget___boxed(lea static lean_object* l_Lean_Meta_AC_toACExpr___closed__3; 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_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_AC_preContext___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_applySimpResultToLocalDecl(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_toACExpr___closed__2; +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__2; 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*); 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_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__4(lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_instEvalInformationPreContextACExpr___closed__3; -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_AC_toACExpr_toPreExpr___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___closed__2; lean_object* l_Lean_Meta_mkEqRefl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms_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*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_indentExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_rewriteUnnormalized___lambda__3(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_AC_buildNormProof___spec__7___closed__1; +static lean_object* l_Lean_Meta_AC_buildNormProof___lambda__1___closed__2; lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__4___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_preContext___closed__3; static lean_object* l_Lean_Meta_AC_buildNormProof_convert___closed__1; static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__3; uint64_t lean_uint64_xor(uint64_t, uint64_t); uint8_t l_Lean_Syntax_isNone(lean_object*); -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__9; +lean_object* lean_panic_fn(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_preContext___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__10; static lean_object* l_Lean_Meta_AC_getInstance___closed__3; @@ -263,25 +290,32 @@ lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Meta_AC_toACExpr___spec__2(lean_object*, lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_instEvalInformationPreContextACExpr___lambda__1___closed__1; +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__16; LEAN_EXPORT lean_object* l_Lean_Meta_AC_getInstance___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__6; lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_rewriteUnnormalized___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_Meta_AC_instEvalInformationPreContextACExpr___closed__2; LEAN_EXPORT lean_object* l_Array_insertionSort_swapLoop___at_Lean_Meta_AC_toACExpr___spec__8(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_toACExpr_toPreExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__12; +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms_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_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__6; size_t lean_usize_sub(size_t, size_t); lean_object* lean_array_mk(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_acRflTactic___rarg___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_AC_toACExpr_toACExpr(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__13; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x21___at_Lean_Meta_AC_toACExpr___spec__10(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__2___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_rewriteUnnormalized___closed__11; LEAN_EXPORT lean_object* l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool; static lean_object* l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___closed__1; LEAN_EXPORT uint8_t l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___lambda__2(lean_object*); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Meta_AC_toACExpr___spec__3(lean_object*); -static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__11; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_instInhabitedPreContext___closed__2; static lean_object* l_Lean_Meta_AC_rewriteUnnormalized___closed__8; LEAN_EXPORT lean_object* l_Lean_Meta_AC_instInhabitedPreContext; @@ -296,25 +330,24 @@ LEAN_EXPORT lean_object* l_Lean_Meta_AC_instEvalInformationPreContextACExpr___la static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__6; static lean_object* l___regBuiltin_Lean_Meta_AC_acRflTactic_declRange__1___closed__5; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__8; -static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__12; LEAN_EXPORT lean_object* l_Lean_Meta_AC_acRflTactic___boxed(lean_object*); static lean_object* l_Lean_Meta_AC_preContext___closed__8; 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 lean_object* l_Lean_Meta_AC_post___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___regBuiltin_Lean_Meta_AC_evalNf0__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__4___boxed(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AC_preContext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__9; -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_AC_getInstance___lambda__2___boxed(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*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Meta_AC_acNfTargetTactic___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_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__4(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_buildNormProof___closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_AC_instEvalInformationPreContextACExpr___lambda__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_buildNormProof___closed__6; +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*); static lean_object* l_Std_DHashMap_Internal_AssocList_get_x21___at_Lean_Meta_AC_toACExpr___spec__10___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_AC_toACExpr_toPreExpr___lambda__1___boxed(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*); @@ -324,6 +357,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_AC_evalNf0___lambda__1(lean_object*, lean_o lean_object* l_Lean_Data_AC_sort(lean_object*); static lean_object* l_Std_DHashMap_Internal_AssocList_get_x21___at_Lean_Meta_AC_toACExpr___spec__10___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_AC_instEvalInformationPreContextACExpr___lambda__3___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AC_buildNormProof_mkContext___closed__7; static lean_object* l_Lean_Meta_AC_getInstance___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_AC_getInstance(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -333,13 +367,11 @@ lean_object* lean_array_uset(lean_object*, size_t, lean_object*); 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_Meta_AC_buildNormProof_convert___closed__3; static lean_object* l_Lean_Meta_AC_instInhabitedPreContext___closed__1; -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__14; static lean_object* l_Lean_Meta_AC_buildNormProof_convert___closed__7; static lean_object* l_Lean_Meta_AC_preContext___closed__4; size_t lean_usize_land(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Meta_AC_post___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_AC_getInstance___closed__5; -static lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___lambda__1___boxed(lean_object*, lean_object*); static lean_object* _init_l_Lean_Meta_AC_instInhabitedPreContext___closed__1() { _start: @@ -3496,7 +3528,44 @@ lean_dec(x_1); return x_7; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms_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, 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_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_unsigned_to_nat(1u); +x_21 = lean_nat_add(x_1, x_20); +lean_inc(x_14); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_14); +lean_inc(x_2); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_2); +lean_ctor_set(x_23, 1, x_22); +x_24 = lean_array_push(x_3, x_23); +lean_inc(x_4); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_14); +lean_ctor_set(x_25, 1, x_4); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_2); +lean_ctor_set(x_26, 1, x_25); +x_27 = lean_array_mk(x_26); +x_28 = l_Array_append___rarg(x_5, x_27); +lean_dec(x_27); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_6); +lean_ctor_set(x_29, 1, x_4); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_7); +lean_ctor_set(x_30, 1, x_29); +x_31 = lean_array_mk(x_30); +x_32 = l_Array_append___rarg(x_8, x_31); +lean_dec(x_31); +x_33 = l_Lean_Meta_AC_abstractAtoms_go(x_9, x_10, x_11, x_12, x_13, x_21, x_24, x_28, x_32, x_15, x_16, x_17, x_18, x_19); +return x_33; +} +} +static lean_object* _init_l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__1() { _start: { lean_object* x_1; @@ -3504,481 +3573,425 @@ x_1 = lean_mk_string_unchecked("LawfulIdentity", 14, 14); return x_1; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2() { +static lean_object* _init_l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Meta_AC_preContext___closed__1; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; +x_2 = l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__1; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3() { +static lean_object* _init_l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("Lean", 4, 4); +x_1 = lean_mk_string_unchecked("inst", 4, 4); return x_1; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4() { +static lean_object* _init_l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Data", 4, 4); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__5() { +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms_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, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Variable", 8, 8); -return x_1; -} -} -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__6() { -_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; +x_16 = lean_ctor_get(x_1, 1); +lean_inc(x_16); +x_17 = lean_array_fget(x_2, x_3); +x_18 = lean_box(0); +lean_inc(x_17); +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_inc(x_16); +x_20 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_20, 0, x_16); +lean_ctor_set(x_20, 1, x_19); +x_21 = lean_array_mk(x_20); +x_22 = l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__2; +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +x_23 = l_Lean_Meta_AC_getInstance(x_22, x_21, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("mk", 2, 2); -return x_1; -} +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; 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_16); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_unsigned_to_nat(1u); +x_27 = lean_nat_add(x_3, x_26); +lean_dec(x_3); +x_28 = lean_box(0); +lean_inc(x_10); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_10); +lean_ctor_set(x_29, 1, x_28); +x_30 = lean_array_push(x_4, x_29); +x_31 = lean_array_push(x_5, x_10); +x_32 = lean_array_push(x_6, x_17); +x_33 = l_Lean_Meta_AC_abstractAtoms_go(x_1, x_2, x_7, x_8, x_9, x_27, x_30, x_31, x_32, x_11, x_12, x_13, x_14, x_25); +return x_33; } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__7() { -_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; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4; -x_3 = l_Lean_Meta_AC_getInstance___closed__2; -x_4 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__5; -x_5 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__6; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; +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; uint8_t x_42; lean_object* x_43; +x_34 = lean_ctor_get(x_23, 1); +lean_inc(x_34); +lean_dec(x_23); +x_35 = lean_ctor_get(x_24, 0); +lean_inc(x_35); +lean_dec(x_24); +lean_inc(x_9); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_9); +lean_ctor_set(x_36, 1, x_18); +x_37 = l_Lean_Expr_const___override(x_22, x_36); +lean_inc(x_10); +lean_inc(x_8); +x_38 = l_Lean_mkApp3(x_37, x_8, x_16, x_10); +x_39 = lean_alloc_closure((void*)(l_Lean_Meta_AC_abstractAtoms_go___lambda__1___boxed), 19, 13); +lean_closure_set(x_39, 0, x_3); +lean_closure_set(x_39, 1, x_10); +lean_closure_set(x_39, 2, x_4); +lean_closure_set(x_39, 3, x_18); +lean_closure_set(x_39, 4, x_5); +lean_closure_set(x_39, 5, x_35); +lean_closure_set(x_39, 6, x_17); +lean_closure_set(x_39, 7, x_6); +lean_closure_set(x_39, 8, x_1); +lean_closure_set(x_39, 9, x_2); +lean_closure_set(x_39, 10, x_7); +lean_closure_set(x_39, 11, x_8); +lean_closure_set(x_39, 12, x_9); +x_40 = l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__4; +x_41 = 0; +x_42 = 0; +x_43 = l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__2___rarg(x_40, x_41, x_38, x_39, x_42, x_11, x_12, x_13, x_14, x_34); +return x_43; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__8() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Option", 6, 6); -return x_1; -} +uint8_t x_44; +lean_dec(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_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_23); +if (x_44 == 0) +{ +return x_23; } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__9() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("none", 4, 4); -return x_1; +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_23, 0); +x_46 = lean_ctor_get(x_23, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_23); +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; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__8; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__9; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__11() { +static lean_object* _init_l_Lean_Meta_AC_abstractAtoms_go___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("some", 4, 4); +x_1 = lean_mk_string_unchecked("x", 1, 1); return x_1; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__12() { +static lean_object* _init_l_Lean_Meta_AC_abstractAtoms_go___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__8; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__11; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); +x_1 = lean_box(0); +x_2 = l_Lean_Meta_AC_abstractAtoms_go___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___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, size_t x_8, size_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_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms_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_object* x_13, lean_object* x_14) { _start: { -uint8_t x_16; -x_16 = lean_usize_dec_lt(x_9, x_8); +lean_object* x_15; uint8_t x_16; +x_15 = lean_array_get_size(x_2); +x_16 = lean_nat_dec_lt(x_6, x_15); +lean_dec(x_15); if (x_16 == 0) { lean_object* x_17; -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -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_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_10); -lean_ctor_set(x_17, 1, x_15); -return x_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; lean_object* x_26; lean_object* x_27; -x_18 = lean_array_uget(x_10, x_9); -x_19 = lean_unsigned_to_nat(0u); -x_20 = lean_array_uset(x_10, x_9, x_19); -x_21 = lean_ctor_get(x_1, 1); -lean_inc(x_21); -x_22 = lean_box(0); -lean_inc(x_18); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_18); -lean_ctor_set(x_23, 1, x_22); -lean_inc(x_21); -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); -x_26 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2; -lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -x_27 = l_Lean_Meta_AC_getInstance(x_26, x_25, x_11, x_12, x_13, x_14, x_15); -if (lean_obj_tag(x_27) == 0) +lean_inc(x_10); +x_17 = lean_apply_6(x_3, x_7, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_17) == 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_27, 0); -lean_inc(x_28); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -lean_inc(x_4); -lean_inc(x_3); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_3); -lean_ctor_set(x_30, 1, x_4); -lean_inc(x_30); -x_31 = l_Lean_Expr_const___override(x_26, x_30); +lean_object* x_18; lean_object* x_19; uint8_t x_20; uint8_t x_21; uint8_t x_22; lean_object* x_23; +x_18 = lean_ctor_get(x_17, 0); lean_inc(x_18); -lean_inc(x_21); -lean_inc(x_2); -x_32 = l_Lean_mkApp3(x_31, x_2, x_21, x_18); -x_33 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__7; -x_34 = l_Lean_Expr_const___override(x_33, x_30); -if (lean_obj_tag(x_28) == 0) +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = 0; +x_21 = 1; +x_22 = 1; +x_23 = l_Lean_Meta_mkLambdaFVars(x_8, x_18, x_20, x_21, x_20, x_22, x_10, x_11, x_12, x_13, x_19); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +if (lean_obj_tag(x_23) == 0) { -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; size_t x_43; size_t x_44; lean_object* x_45; -x_35 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10; -lean_inc(x_5); -x_36 = l_Lean_Expr_const___override(x_35, x_5); -lean_inc(x_6); -x_37 = l_Lean_Expr_app___override(x_6, x_32); -x_38 = l_Lean_Expr_app___override(x_36, x_37); -lean_inc(x_2); -x_39 = l_Lean_mkApp4(x_34, x_2, x_21, x_18, x_38); -x_40 = 0; -x_41 = lean_box(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_39); -x_43 = 1; -x_44 = lean_usize_add(x_9, x_43); -x_45 = lean_array_uset(x_20, x_9, x_42); -x_9 = x_44; -x_10 = x_45; -x_15 = x_29; -goto _start; +uint8_t x_24; +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); +x_26 = l_Lean_mkAppN(x_25, x_9); +lean_dec(x_9); +lean_ctor_set(x_23, 0, x_26); +return x_23; } 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; uint8_t x_54; lean_object* x_55; lean_object* x_56; size_t x_57; size_t x_58; lean_object* x_59; -x_47 = lean_ctor_get(x_28, 0); -lean_inc(x_47); -lean_dec(x_28); -x_48 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__12; -lean_inc(x_5); -x_49 = l_Lean_Expr_const___override(x_48, x_5); -lean_inc(x_32); -lean_inc(x_6); -x_50 = l_Lean_Expr_app___override(x_6, x_32); -lean_inc(x_7); -x_51 = l_Lean_mkAppB(x_7, x_32, x_47); -x_52 = l_Lean_mkAppB(x_49, x_50, x_51); -lean_inc(x_2); -x_53 = l_Lean_mkApp4(x_34, x_2, x_21, x_18, x_52); -x_54 = 1; -x_55 = lean_box(x_54); -x_56 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_56, 0, x_55); -lean_ctor_set(x_56, 1, x_53); -x_57 = 1; -x_58 = lean_usize_add(x_9, x_57); -x_59 = lean_array_uset(x_20, x_9, x_56); -x_9 = x_58; -x_10 = x_59; -x_15 = x_29; -goto _start; +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_27 = lean_ctor_get(x_23, 0); +x_28 = lean_ctor_get(x_23, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_23); +x_29 = l_Lean_mkAppN(x_27, x_9); +lean_dec(x_9); +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_61; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_18); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -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_61 = !lean_is_exclusive(x_27); -if (x_61 == 0) +uint8_t x_31; +lean_dec(x_9); +x_31 = !lean_is_exclusive(x_23); +if (x_31 == 0) { -return x_27; +return x_23; } else { -lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_62 = lean_ctor_get(x_27, 0); -x_63 = lean_ctor_get(x_27, 1); -lean_inc(x_63); -lean_inc(x_62); -lean_dec(x_27); -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_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_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; } } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("PLift", 5, 5); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___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_AC_buildNormProof_mkContext___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = lean_box(0); -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_Meta_AC_buildNormProof_mkContext___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__2; -x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__3; -x_3 = l_Lean_Expr_const___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("up", 2, 2); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__6() { -_start: +uint8_t x_35; +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_35 = !lean_is_exclusive(x_17); +if (x_35 == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__1; -x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__5; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} +return x_17; } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__7() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__6; -x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__3; -x_3 = l_Lean_Expr_const___override(x_1, x_2); -return x_3; -} +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_17, 0); +x_37 = lean_ctor_get(x_17, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_17); +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_Lean_Meta_AC_buildNormProof_mkContext___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_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4; -x_3 = l_Lean_Meta_AC_getInstance___closed__2; -x_4 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___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_AC_buildNormProof_mkContext___closed__9() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Context", 7, 7); -return x_1; -} +lean_object* x_39; lean_object* x_40; uint8_t x_41; uint8_t x_42; lean_object* x_43; +lean_inc(x_4); +x_39 = lean_alloc_closure((void*)(l_Lean_Meta_AC_abstractAtoms_go___lambda__2), 15, 9); +lean_closure_set(x_39, 0, x_1); +lean_closure_set(x_39, 1, x_2); +lean_closure_set(x_39, 2, x_6); +lean_closure_set(x_39, 3, x_7); +lean_closure_set(x_39, 4, x_8); +lean_closure_set(x_39, 5, x_9); +lean_closure_set(x_39, 6, x_3); +lean_closure_set(x_39, 7, x_4); +lean_closure_set(x_39, 8, x_5); +x_40 = l_Lean_Meta_AC_abstractAtoms_go___closed__2; +x_41 = 0; +x_42 = 0; +x_43 = l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__2___rarg(x_40, x_41, x_4, x_39, x_42, x_10, x_11, x_12, x_13, x_14); +return x_43; } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___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_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4; -x_3 = l_Lean_Meta_AC_getInstance___closed__2; -x_4 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__9; -x_5 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__6; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10; -x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__3; -x_3 = l_Lean_Expr_const___override(x_1, x_2); -return x_3; +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms_go___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_object* x_18 = _args[17]; +lean_object* x_19 = _args[18]; +_start: +{ +lean_object* x_20; +x_20 = l_Lean_Meta_AC_abstractAtoms_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, x_14, x_15, x_16, x_17, x_18, x_19); +lean_dec(x_1); +return x_20; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__12() { +LEAN_EXPORT lean_object* l_Lean_Meta_AC_abstractAtoms(lean_object* x_1, lean_object* x_2, 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_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__12; -x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__3; -x_3 = l_Lean_Expr_const___override(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_mkContext(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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; lean_object* x_10; uint8_t x_11; +x_9 = lean_array_get_size(x_2); +x_10 = lean_unsigned_to_nat(0u); +x_11 = lean_nat_dec_lt(x_10, x_9); +lean_dec(x_9); +if (x_11 == 0) { -lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_object* x_13; size_t x_14; size_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; -x_10 = lean_array_get_size(x_4); -x_11 = lean_unsigned_to_nat(0u); -x_12 = lean_nat_dec_lt(x_11, x_10); -lean_dec(x_10); -x_13 = lean_box(0); -x_14 = lean_array_size(x_4); -x_15 = 0; -x_16 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__3; -x_17 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__4; -x_18 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__7; -lean_inc(x_8); +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = l_Lean_instInhabitedExpr; +x_13 = l_outOfBounds___rarg(x_12); 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_19 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1(x_1, x_2, x_3, x_13, x_16, x_17, x_18, x_14, x_15, x_4, x_5, x_6, x_7, x_8, x_9); -if (x_12 == 0) +x_14 = lean_infer_type(x_13, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_14) == 0) { -lean_dec(x_4); -if (lean_obj_tag(x_19) == 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); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_15); +x_17 = l_Lean_Meta_getLevel(x_15, x_4, x_5, x_6, x_7, x_16); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; -x_185 = lean_ctor_get(x_19, 0); -lean_inc(x_185); -x_186 = lean_ctor_get(x_19, 1); -lean_inc(x_186); -lean_dec(x_19); -x_187 = l_Lean_instInhabitedExpr; -x_188 = l_outOfBounds___rarg(x_187); -x_20 = x_188; -x_21 = x_185; -x_22 = x_186; -goto block_184; +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +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_AC_toACExpr___closed__4; +x_21 = l_Lean_Meta_AC_abstractAtoms_go(x_1, x_2, x_3, x_15, x_18, x_10, x_20, x_20, x_20, x_4, x_5, x_6, x_7, x_19); +return x_21; } else { -uint8_t x_189; -lean_dec(x_8); +uint8_t x_22; +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_189 = !lean_is_exclusive(x_19); -if (x_189 == 0) +x_22 = !lean_is_exclusive(x_17); +if (x_22 == 0) { -return x_19; +return x_17; } else { -lean_object* x_190; lean_object* x_191; lean_object* x_192; -x_190 = lean_ctor_get(x_19, 0); -x_191 = lean_ctor_get(x_19, 1); -lean_inc(x_191); -lean_inc(x_190); -lean_dec(x_19); -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_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; } } -else -{ -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_193; lean_object* x_194; lean_object* x_195; -x_193 = lean_ctor_get(x_19, 0); -lean_inc(x_193); -x_194 = lean_ctor_get(x_19, 1); -lean_inc(x_194); -lean_dec(x_19); -x_195 = lean_array_fget(x_4, x_11); -lean_dec(x_4); -x_20 = x_195; -x_21 = x_193; -x_22 = x_194; -goto block_184; } else { -uint8_t x_196; -lean_dec(x_8); +uint8_t x_26; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -3986,948 +3999,1945 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_196 = !lean_is_exclusive(x_19); -if (x_196 == 0) +x_26 = !lean_is_exclusive(x_14); +if (x_26 == 0) { -return x_19; +return x_14; } else { -lean_object* x_197; lean_object* x_198; lean_object* x_199; -x_197 = lean_ctor_get(x_19, 0); -x_198 = lean_ctor_get(x_19, 1); -lean_inc(x_198); -lean_inc(x_197); -lean_dec(x_19); -x_199 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_199, 0, x_197); -lean_ctor_set(x_199, 1, x_198); -return x_199; +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_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; } } } -block_184: -{ -lean_object* x_23; uint8_t x_24; -x_23 = l_Array_unzip___rarg(x_21); -lean_dec(x_21); -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) +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; -x_25 = lean_ctor_get(x_23, 0); -x_26 = lean_ctor_get(x_23, 1); -x_27 = lean_array_to_list(x_26); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_3); -lean_ctor_set(x_28, 1, x_13); -x_29 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__8; -lean_inc(x_28); -x_30 = l_Lean_Expr_const___override(x_29, x_28); -x_31 = lean_ctor_get(x_1, 1); -lean_inc(x_31); -lean_inc(x_31); -lean_inc(x_2); -x_32 = l_Lean_mkAppB(x_30, x_2, x_31); -x_33 = l_Lean_Meta_mkListLit(x_32, x_27, x_5, x_6, x_7, x_8, x_22); -if (lean_obj_tag(x_33) == 0) +lean_object* x_30; lean_object* x_31; +x_30 = lean_array_fget(x_2, x_10); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_31 = lean_infer_type(x_30, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_31) == 0) { -uint8_t x_34; -x_34 = !lean_is_exclusive(x_33); -if (x_34 == 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_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_32); +x_34 = l_Lean_Meta_getLevel(x_32, x_4, x_5, x_6, x_7, 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; -x_35 = lean_ctor_get(x_33, 0); -x_36 = l_Lean_Meta_AC_preContext___closed__6; -lean_inc(x_28); -x_37 = l_Lean_Expr_const___override(x_36, x_28); -lean_inc(x_31); -lean_inc(x_2); -x_38 = l_Lean_mkAppB(x_37, x_2, x_31); -x_39 = lean_ctor_get(x_1, 3); -lean_inc(x_39); -x_40 = l_Lean_Meta_AC_preContext___closed__8; -lean_inc(x_28); -x_41 = l_Lean_Expr_const___override(x_40, x_28); -lean_inc(x_31); -lean_inc(x_2); -x_42 = l_Lean_mkAppB(x_41, x_2, x_31); -x_43 = lean_ctor_get(x_1, 4); -lean_inc(x_43); -x_44 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__10; -x_45 = l_Lean_Expr_const___override(x_44, x_28); -if (lean_obj_tag(x_39) == 0) +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +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_Lean_Meta_AC_toACExpr___closed__4; +x_38 = l_Lean_Meta_AC_abstractAtoms_go(x_1, x_2, x_3, x_32, x_35, x_10, x_37, x_37, x_37, x_4, x_5, x_6, x_7, x_36); +return x_38; +} +else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_46 = lean_ctor_get(x_1, 2); -lean_inc(x_46); +uint8_t x_39; +lean_dec(x_32); +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 = l_Lean_Expr_app___override(x_17, x_38); -x_48 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; -x_49 = l_Lean_Expr_app___override(x_48, x_47); -if (lean_obj_tag(x_43) == 0) +x_39 = !lean_is_exclusive(x_34); +if (x_39 == 0) { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = l_Lean_Expr_app___override(x_17, x_42); -x_51 = l_Lean_Expr_app___override(x_48, x_50); -x_52 = l_Lean_mkApp7(x_45, x_2, x_31, x_46, x_49, x_51, x_35, x_20); -lean_ctor_set(x_23, 1, x_52); -lean_ctor_set(x_33, 0, x_23); -return x_33; +return x_34; } 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; -x_53 = lean_ctor_get(x_43, 0); -lean_inc(x_53); -lean_dec(x_43); -lean_inc(x_42); -x_54 = l_Lean_Expr_app___override(x_17, x_42); -x_55 = l_Lean_mkAppB(x_18, x_42, x_53); -x_56 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; -x_57 = l_Lean_mkAppB(x_56, x_54, x_55); -x_58 = l_Lean_mkApp7(x_45, x_2, x_31, x_46, x_49, x_57, x_35, x_20); -lean_ctor_set(x_23, 1, x_58); -lean_ctor_set(x_33, 0, x_23); -return x_33; +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_34, 0); +x_41 = lean_ctor_get(x_34, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_34); +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_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_1, 2); -lean_inc(x_59); -lean_dec(x_1); -x_60 = lean_ctor_get(x_39, 0); -lean_inc(x_60); -lean_dec(x_39); -lean_inc(x_38); -x_61 = l_Lean_Expr_app___override(x_17, x_38); -x_62 = l_Lean_mkAppB(x_18, x_38, x_60); -x_63 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; -x_64 = l_Lean_mkAppB(x_63, x_61, x_62); -if (lean_obj_tag(x_43) == 0) -{ -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_65 = l_Lean_Expr_app___override(x_17, x_42); -x_66 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; -x_67 = l_Lean_Expr_app___override(x_66, x_65); -x_68 = l_Lean_mkApp7(x_45, x_2, x_31, x_59, x_64, x_67, x_35, x_20); -lean_ctor_set(x_23, 1, x_68); -lean_ctor_set(x_33, 0, x_23); -return x_33; -} -else -{ -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_43, 0); -lean_inc(x_69); -lean_dec(x_43); -lean_inc(x_42); -x_70 = l_Lean_Expr_app___override(x_17, x_42); -x_71 = l_Lean_mkAppB(x_18, x_42, x_69); -x_72 = l_Lean_mkAppB(x_63, x_70, x_71); -x_73 = l_Lean_mkApp7(x_45, x_2, x_31, x_59, x_64, x_72, x_35, x_20); -lean_ctor_set(x_23, 1, x_73); -lean_ctor_set(x_33, 0, x_23); -return x_33; -} -} -} -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; lean_object* x_85; -x_74 = lean_ctor_get(x_33, 0); -x_75 = lean_ctor_get(x_33, 1); -lean_inc(x_75); -lean_inc(x_74); -lean_dec(x_33); -x_76 = l_Lean_Meta_AC_preContext___closed__6; -lean_inc(x_28); -x_77 = l_Lean_Expr_const___override(x_76, x_28); -lean_inc(x_31); -lean_inc(x_2); -x_78 = l_Lean_mkAppB(x_77, x_2, x_31); -x_79 = lean_ctor_get(x_1, 3); -lean_inc(x_79); -x_80 = l_Lean_Meta_AC_preContext___closed__8; -lean_inc(x_28); -x_81 = l_Lean_Expr_const___override(x_80, x_28); -lean_inc(x_31); -lean_inc(x_2); -x_82 = l_Lean_mkAppB(x_81, x_2, x_31); -x_83 = lean_ctor_get(x_1, 4); -lean_inc(x_83); -x_84 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__10; -x_85 = l_Lean_Expr_const___override(x_84, x_28); -if (lean_obj_tag(x_79) == 0) -{ -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_86 = lean_ctor_get(x_1, 2); -lean_inc(x_86); -lean_dec(x_1); -x_87 = l_Lean_Expr_app___override(x_17, x_78); -x_88 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; -x_89 = l_Lean_Expr_app___override(x_88, x_87); -if (lean_obj_tag(x_83) == 0) -{ -lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_90 = l_Lean_Expr_app___override(x_17, x_82); -x_91 = l_Lean_Expr_app___override(x_88, x_90); -x_92 = l_Lean_mkApp7(x_85, x_2, x_31, x_86, x_89, x_91, x_74, x_20); -lean_ctor_set(x_23, 1, x_92); -x_93 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_93, 0, x_23); -lean_ctor_set(x_93, 1, x_75); -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; -x_94 = lean_ctor_get(x_83, 0); -lean_inc(x_94); -lean_dec(x_83); -lean_inc(x_82); -x_95 = l_Lean_Expr_app___override(x_17, x_82); -x_96 = l_Lean_mkAppB(x_18, x_82, x_94); -x_97 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; -x_98 = l_Lean_mkAppB(x_97, x_95, x_96); -x_99 = l_Lean_mkApp7(x_85, x_2, x_31, x_86, x_89, x_98, x_74, x_20); -lean_ctor_set(x_23, 1, x_99); -x_100 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_100, 0, x_23); -lean_ctor_set(x_100, 1, x_75); -return x_100; -} -} -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; -x_101 = lean_ctor_get(x_1, 2); -lean_inc(x_101); -lean_dec(x_1); -x_102 = lean_ctor_get(x_79, 0); -lean_inc(x_102); -lean_dec(x_79); -lean_inc(x_78); -x_103 = l_Lean_Expr_app___override(x_17, x_78); -x_104 = l_Lean_mkAppB(x_18, x_78, x_102); -x_105 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; -x_106 = l_Lean_mkAppB(x_105, x_103, x_104); -if (lean_obj_tag(x_83) == 0) -{ -lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_107 = l_Lean_Expr_app___override(x_17, x_82); -x_108 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; -x_109 = l_Lean_Expr_app___override(x_108, x_107); -x_110 = l_Lean_mkApp7(x_85, x_2, x_31, x_101, x_106, x_109, x_74, x_20); -lean_ctor_set(x_23, 1, x_110); -x_111 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_111, 0, x_23); -lean_ctor_set(x_111, 1, x_75); -return x_111; -} -else -{ -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_83, 0); -lean_inc(x_112); -lean_dec(x_83); -lean_inc(x_82); -x_113 = l_Lean_Expr_app___override(x_17, x_82); -x_114 = l_Lean_mkAppB(x_18, x_82, x_112); -x_115 = l_Lean_mkAppB(x_105, x_113, x_114); -x_116 = l_Lean_mkApp7(x_85, x_2, x_31, x_101, x_106, x_115, x_74, x_20); -lean_ctor_set(x_23, 1, x_116); -x_117 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_117, 0, x_23); -lean_ctor_set(x_117, 1, x_75); -return x_117; -} -} -} -} -else -{ -uint8_t x_118; -lean_dec(x_31); -lean_dec(x_28); -lean_free_object(x_23); -lean_dec(x_25); -lean_dec(x_20); +uint8_t x_43; +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_is_exclusive(x_33); -if (x_118 == 0) -{ -return x_33; -} -else -{ -lean_object* x_119; lean_object* x_120; lean_object* x_121; -x_119 = lean_ctor_get(x_33, 0); -x_120 = lean_ctor_get(x_33, 1); -lean_inc(x_120); -lean_inc(x_119); -lean_dec(x_33); -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; -} -} -} -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; lean_object* x_129; lean_object* x_130; -x_122 = lean_ctor_get(x_23, 0); -x_123 = lean_ctor_get(x_23, 1); -lean_inc(x_123); -lean_inc(x_122); -lean_dec(x_23); -x_124 = lean_array_to_list(x_123); -x_125 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_125, 0, x_3); -lean_ctor_set(x_125, 1, x_13); -x_126 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__8; -lean_inc(x_125); -x_127 = l_Lean_Expr_const___override(x_126, x_125); -x_128 = lean_ctor_get(x_1, 1); -lean_inc(x_128); -lean_inc(x_128); -lean_inc(x_2); -x_129 = l_Lean_mkAppB(x_127, x_2, x_128); -x_130 = l_Lean_Meta_mkListLit(x_129, x_124, x_5, x_6, x_7, x_8, x_22); -if (lean_obj_tag(x_130) == 0) -{ -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; -x_131 = lean_ctor_get(x_130, 0); -lean_inc(x_131); -x_132 = lean_ctor_get(x_130, 1); -lean_inc(x_132); -if (lean_is_exclusive(x_130)) { - lean_ctor_release(x_130, 0); - lean_ctor_release(x_130, 1); - x_133 = x_130; -} else { - lean_dec_ref(x_130); - x_133 = lean_box(0); -} -x_134 = l_Lean_Meta_AC_preContext___closed__6; -lean_inc(x_125); -x_135 = l_Lean_Expr_const___override(x_134, x_125); -lean_inc(x_128); -lean_inc(x_2); -x_136 = l_Lean_mkAppB(x_135, x_2, x_128); -x_137 = lean_ctor_get(x_1, 3); -lean_inc(x_137); -x_138 = l_Lean_Meta_AC_preContext___closed__8; -lean_inc(x_125); -x_139 = l_Lean_Expr_const___override(x_138, x_125); -lean_inc(x_128); -lean_inc(x_2); -x_140 = l_Lean_mkAppB(x_139, x_2, x_128); -x_141 = lean_ctor_get(x_1, 4); -lean_inc(x_141); -x_142 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__10; -x_143 = l_Lean_Expr_const___override(x_142, x_125); -if (lean_obj_tag(x_137) == 0) -{ -lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; -x_144 = lean_ctor_get(x_1, 2); -lean_inc(x_144); -lean_dec(x_1); -x_145 = l_Lean_Expr_app___override(x_17, x_136); -x_146 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; -x_147 = l_Lean_Expr_app___override(x_146, x_145); -if (lean_obj_tag(x_141) == 0) -{ -lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; -x_148 = l_Lean_Expr_app___override(x_17, x_140); -x_149 = l_Lean_Expr_app___override(x_146, x_148); -x_150 = l_Lean_mkApp7(x_143, x_2, x_128, x_144, x_147, x_149, x_131, x_20); -x_151 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_151, 0, x_122); -lean_ctor_set(x_151, 1, x_150); -if (lean_is_scalar(x_133)) { - x_152 = lean_alloc_ctor(0, 2, 0); -} else { - x_152 = x_133; -} -lean_ctor_set(x_152, 0, x_151); -lean_ctor_set(x_152, 1, x_132); -return x_152; -} -else +x_43 = !lean_is_exclusive(x_31); +if (x_43 == 0) { -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; -x_153 = lean_ctor_get(x_141, 0); -lean_inc(x_153); -lean_dec(x_141); -lean_inc(x_140); -x_154 = l_Lean_Expr_app___override(x_17, x_140); -x_155 = l_Lean_mkAppB(x_18, x_140, x_153); -x_156 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; -x_157 = l_Lean_mkAppB(x_156, x_154, x_155); -x_158 = l_Lean_mkApp7(x_143, x_2, x_128, x_144, x_147, x_157, x_131, x_20); -x_159 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_159, 0, x_122); -lean_ctor_set(x_159, 1, x_158); -if (lean_is_scalar(x_133)) { - x_160 = lean_alloc_ctor(0, 2, 0); -} else { - x_160 = x_133; -} -lean_ctor_set(x_160, 0, x_159); -lean_ctor_set(x_160, 1, x_132); -return x_160; -} +return x_31; } 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_1, 2); -lean_inc(x_161); -lean_dec(x_1); -x_162 = lean_ctor_get(x_137, 0); -lean_inc(x_162); -lean_dec(x_137); -lean_inc(x_136); -x_163 = l_Lean_Expr_app___override(x_17, x_136); -x_164 = l_Lean_mkAppB(x_18, x_136, x_162); -x_165 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; -x_166 = l_Lean_mkAppB(x_165, x_163, x_164); -if (lean_obj_tag(x_141) == 0) -{ -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_167 = l_Lean_Expr_app___override(x_17, x_140); -x_168 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; -x_169 = l_Lean_Expr_app___override(x_168, x_167); -x_170 = l_Lean_mkApp7(x_143, x_2, x_128, x_161, x_166, x_169, x_131, x_20); -x_171 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_171, 0, x_122); -lean_ctor_set(x_171, 1, x_170); -if (lean_is_scalar(x_133)) { - x_172 = lean_alloc_ctor(0, 2, 0); -} else { - x_172 = x_133; -} -lean_ctor_set(x_172, 0, x_171); -lean_ctor_set(x_172, 1, x_132); -return x_172; +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 -{ -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_173 = lean_ctor_get(x_141, 0); -lean_inc(x_173); -lean_dec(x_141); -lean_inc(x_140); -x_174 = l_Lean_Expr_app___override(x_17, x_140); -x_175 = l_Lean_mkAppB(x_18, x_140, x_173); -x_176 = l_Lean_mkAppB(x_165, x_174, x_175); -x_177 = l_Lean_mkApp7(x_143, x_2, x_128, x_161, x_166, x_176, x_131, x_20); -x_178 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_178, 0, x_122); -lean_ctor_set(x_178, 1, x_177); -if (lean_is_scalar(x_133)) { - x_179 = lean_alloc_ctor(0, 2, 0); -} else { - x_179 = x_133; } -lean_ctor_set(x_179, 0, x_178); -lean_ctor_set(x_179, 1, x_132); -return x_179; } } } -else +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1() { +_start: { -lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; -lean_dec(x_128); -lean_dec(x_125); -lean_dec(x_122); -lean_dec(x_20); -lean_dec(x_2); -lean_dec(x_1); -x_180 = lean_ctor_get(x_130, 0); -lean_inc(x_180); -x_181 = lean_ctor_get(x_130, 1); -lean_inc(x_181); -if (lean_is_exclusive(x_130)) { - lean_ctor_release(x_130, 0); - lean_ctor_release(x_130, 1); - x_182 = x_130; -} else { - lean_dec_ref(x_130); - x_182 = lean_box(0); -} -if (lean_is_scalar(x_182)) { - x_183 = lean_alloc_ctor(1, 2, 0); -} else { - x_183 = x_182; -} -lean_ctor_set(x_183, 0, x_180); -lean_ctor_set(x_183, 1, x_181); -return x_183; -} -} -} +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean", 4, 4); +return x_1; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___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) { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2() { _start: { -size_t x_16; size_t x_17; lean_object* x_18; -x_16 = lean_unbox_usize(x_8); -lean_dec(x_8); -x_17 = lean_unbox_usize(x_9); -lean_dec(x_9); -x_18 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_16, x_17, x_10, x_11, x_12, x_13, x_14, x_15); -return x_18; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Data", 4, 4); +return x_1; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__1() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("Expr", 4, 4); +x_1 = lean_mk_string_unchecked("Variable", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__2() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("var", 3, 3); +x_1 = lean_mk_string_unchecked("mk", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__3() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__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; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2; x_3 = l_Lean_Meta_AC_getInstance___closed__2; -x_4 = l_Lean_Meta_AC_buildNormProof_convert___closed__1; -x_5 = l_Lean_Meta_AC_buildNormProof_convert___closed__2; +x_4 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; +x_5 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__4() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__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_AC_buildNormProof_convert___closed__3; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Option", 6, 6); +return x_1; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__5() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__7() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("op", 2, 2); +x_1 = lean_mk_string_unchecked("none", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__6() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___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; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4; -x_3 = l_Lean_Meta_AC_getInstance___closed__2; -x_4 = l_Lean_Meta_AC_buildNormProof_convert___closed__1; -x_5 = l_Lean_Meta_AC_buildNormProof_convert___closed__5; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); -return x_6; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__6; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__7; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__7() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("some", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__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_Meta_AC_buildNormProof_convert___closed__6; -x_3 = l_Lean_Expr_const___override(x_2, x_1); +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__6; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__9; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_convert(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___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, size_t x_8, size_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) { _start: { -if (lean_obj_tag(x_1) == 0) +uint8_t x_16; +x_16 = lean_usize_dec_lt(x_9, x_8); +if (x_16 == 0) { -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = lean_ctor_get(x_1, 0); -lean_inc(x_2); +lean_object* x_17; +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_3 = l_Lean_mkNatLit(x_2); -x_4 = l_Lean_Meta_AC_buildNormProof_convert___closed__4; -x_5 = l_Lean_Expr_app___override(x_4, x_3); -return x_5; +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_10); +lean_ctor_set(x_17, 1, x_15); +return x_17; } else { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_6 = lean_ctor_get(x_1, 0); +lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_18 = lean_array_uget(x_10, x_9); +x_19 = lean_unsigned_to_nat(0u); +x_20 = lean_array_uset(x_10, x_9, x_19); +x_21 = !lean_is_exclusive(x_18); +if (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_18, 0); +x_23 = lean_ctor_get(x_18, 1); +lean_inc(x_4); +lean_inc(x_3); +lean_ctor_set_tag(x_18, 1); +lean_ctor_set(x_18, 1, x_4); +lean_ctor_set(x_18, 0, x_3); +x_24 = l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__2; +lean_inc(x_18); +x_25 = l_Lean_Expr_const___override(x_24, x_18); +x_26 = lean_ctor_get(x_1, 1); +lean_inc(x_26); +lean_inc(x_22); +lean_inc(x_26); +lean_inc(x_2); +x_27 = l_Lean_mkApp3(x_25, x_2, x_26, x_22); +x_28 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__5; +x_29 = l_Lean_Expr_const___override(x_28, x_18); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; size_t x_35; size_t x_36; lean_object* x_37; +x_30 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__8; +lean_inc(x_5); +x_31 = l_Lean_Expr_const___override(x_30, x_5); lean_inc(x_6); -x_7 = lean_ctor_get(x_1, 1); -lean_inc(x_7); -lean_dec(x_1); -x_8 = l_Lean_Meta_AC_buildNormProof_convert(x_6); -x_9 = l_Lean_Meta_AC_buildNormProof_convert(x_7); -x_10 = l_Lean_Meta_AC_buildNormProof_convert___closed__7; -x_11 = l_Lean_mkAppB(x_10, x_8, x_9); -return x_11; -} -} +x_32 = l_Lean_Expr_app___override(x_6, x_27); +x_33 = l_Lean_Expr_app___override(x_31, x_32); +lean_inc(x_2); +x_34 = l_Lean_mkApp4(x_29, x_2, x_26, x_22, x_33); +x_35 = 1; +x_36 = lean_usize_add(x_9, x_35); +x_37 = lean_array_uset(x_20, x_9, x_34); +x_9 = x_36; +x_10 = x_37; +goto _start; } -LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_convertTarget(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -if (lean_obj_tag(x_3) == 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; size_t x_46; size_t x_47; lean_object* x_48; +x_39 = lean_ctor_get(x_23, 0); +lean_inc(x_39); +lean_dec(x_23); +x_40 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10; +lean_inc(x_5); +x_41 = l_Lean_Expr_const___override(x_40, x_5); +lean_inc(x_27); +lean_inc(x_6); +x_42 = l_Lean_Expr_app___override(x_6, x_27); +lean_inc(x_7); +x_43 = l_Lean_mkAppB(x_7, x_27, x_39); +x_44 = l_Lean_mkAppB(x_41, x_42, x_43); +lean_inc(x_2); +x_45 = l_Lean_mkApp4(x_29, x_2, x_26, x_22, x_44); +x_46 = 1; +x_47 = lean_usize_add(x_9, x_46); +x_48 = lean_array_uset(x_20, x_9, x_45); +x_9 = x_47; +x_10 = x_48; +goto _start; +} +} +else { -lean_object* x_4; lean_object* x_5; uint8_t x_6; -lean_dec(x_1); -x_4 = lean_ctor_get(x_3, 0); -x_5 = lean_array_get_size(x_2); -x_6 = lean_nat_dec_lt(x_4, x_5); -lean_dec(x_5); -if (x_6 == 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; +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); +lean_inc(x_4); +lean_inc(x_3); +x_52 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_52, 0, x_3); +lean_ctor_set(x_52, 1, x_4); +x_53 = l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__2; +lean_inc(x_52); +x_54 = l_Lean_Expr_const___override(x_53, x_52); +x_55 = lean_ctor_get(x_1, 1); +lean_inc(x_55); +lean_inc(x_50); +lean_inc(x_55); +lean_inc(x_2); +x_56 = l_Lean_mkApp3(x_54, x_2, x_55, x_50); +x_57 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__5; +x_58 = l_Lean_Expr_const___override(x_57, x_52); +if (lean_obj_tag(x_51) == 0) { -lean_object* x_7; lean_object* x_8; -x_7 = l_Lean_instInhabitedExpr; -x_8 = l_outOfBounds___rarg(x_7); -return x_8; +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; size_t x_64; size_t x_65; lean_object* x_66; +x_59 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__8; +lean_inc(x_5); +x_60 = l_Lean_Expr_const___override(x_59, x_5); +lean_inc(x_6); +x_61 = l_Lean_Expr_app___override(x_6, x_56); +x_62 = l_Lean_Expr_app___override(x_60, x_61); +lean_inc(x_2); +x_63 = l_Lean_mkApp4(x_58, x_2, x_55, x_50, x_62); +x_64 = 1; +x_65 = lean_usize_add(x_9, x_64); +x_66 = lean_array_uset(x_20, x_9, x_63); +x_9 = x_65; +x_10 = x_66; +goto _start; } else { -lean_object* x_9; -x_9 = lean_array_fget(x_2, x_4); -return x_9; +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; size_t x_75; size_t x_76; lean_object* x_77; +x_68 = lean_ctor_get(x_51, 0); +lean_inc(x_68); +lean_dec(x_51); +x_69 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10; +lean_inc(x_5); +x_70 = l_Lean_Expr_const___override(x_69, x_5); +lean_inc(x_56); +lean_inc(x_6); +x_71 = l_Lean_Expr_app___override(x_6, x_56); +lean_inc(x_7); +x_72 = l_Lean_mkAppB(x_7, x_56, x_68); +x_73 = l_Lean_mkAppB(x_70, x_71, x_72); +lean_inc(x_2); +x_74 = l_Lean_mkApp4(x_58, x_2, x_55, x_50, x_73); +x_75 = 1; +x_76 = lean_usize_add(x_9, x_75); +x_77 = lean_array_uset(x_20, x_9, x_74); +x_9 = x_76; +x_10 = x_77; +goto _start; } } -else -{ -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_3, 0); -x_11 = lean_ctor_get(x_3, 1); -x_12 = lean_ctor_get(x_1, 1); -lean_inc(x_12); -lean_inc(x_1); -x_13 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_2, x_10); -x_14 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_2, x_11); -x_15 = l_Lean_mkAppB(x_12, x_13, x_14); -return x_15; } } } -LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_convertTarget___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__1() { _start: { -lean_object* x_4; -x_4 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_2, x_3); -lean_dec(x_3); -lean_dec(x_2); -return x_4; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_instInhabitedExpr; +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_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__2() { _start: { -if (lean_obj_tag(x_2) == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("PLift", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__3() { +_start: { -lean_object* x_3; -x_3 = lean_box(0); +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__2; +x_3 = l_Lean_Name_str___override(x_1, x_2); 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; 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_1, 1); -x_8 = lean_array_get_size(x_7); -x_9 = lean_nat_dec_lt(x_5, x_8); -lean_dec(x_8); -if (x_9 == 0) -{ -uint8_t x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = l_instInhabitedBool; -x_11 = lean_box(x_10); -x_12 = l_outOfBounds___rarg(x_11); -x_13 = lean_unbox(x_12); -lean_dec(x_12); -if (x_13 == 0) -{ -lean_object* x_14; -x_14 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3(x_1, x_6); -lean_ctor_set(x_2, 1, x_14); -return x_2; } -else +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__4() { +_start: { -lean_free_object(x_2); -lean_dec(x_5); -x_2 = x_6; -goto _start; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = lean_box(0); +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; } } -else -{ -lean_object* x_16; uint8_t x_17; -x_16 = lean_array_fget(x_7, x_5); -x_17 = lean_unbox(x_16); -lean_dec(x_16); -if (x_17 == 0) +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__5() { +_start: { -lean_object* x_18; -x_18 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3(x_1, x_6); -lean_ctor_set(x_2, 1, x_18); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__3; +x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__4; +x_3 = l_Lean_Expr_const___override(x_1, x_2); +return x_3; } -else -{ -lean_free_object(x_2); -lean_dec(x_5); -x_2 = x_6; -goto _start; } +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("up", 2, 2); +return x_1; } } -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_2, 0); -x_21 = lean_ctor_get(x_2, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_2); -x_22 = lean_ctor_get(x_1, 1); -x_23 = lean_array_get_size(x_22); -x_24 = lean_nat_dec_lt(x_20, x_23); -lean_dec(x_23); -if (x_24 == 0) -{ -uint8_t x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_25 = l_instInhabitedBool; -x_26 = lean_box(x_25); -x_27 = l_outOfBounds___rarg(x_26); -x_28 = lean_unbox(x_27); -lean_dec(x_27); -if (x_28 == 0) +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__7() { +_start: { -lean_object* x_29; lean_object* x_30; -x_29 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3(x_1, x_21); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_20); -lean_ctor_set(x_30, 1, x_29); -return x_30; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__2; +x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__6; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } -else +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__8() { +_start: { -lean_dec(x_20); -x_2 = x_21; -goto _start; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__7; +x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__4; +x_3 = l_Lean_Expr_const___override(x_1, x_2); +return x_3; } } -else -{ -lean_object* x_32; uint8_t x_33; -x_32 = lean_array_fget(x_22, x_20); -x_33 = lean_unbox(x_32); -lean_dec(x_32); -if (x_33 == 0) +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__9() { +_start: { -lean_object* x_34; lean_object* x_35; -x_34 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3(x_1, x_21); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_20); -lean_ctor_set(x_35, 1, x_34); -return x_35; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2; +x_3 = l_Lean_Meta_AC_getInstance___closed__2; +x_4 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } -else +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__10() { +_start: { -lean_dec(x_20); -x_2 = x_21; -goto _start; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Context", 7, 7); +return x_1; } } +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__11() { +_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_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2; +x_3 = l_Lean_Meta_AC_getInstance___closed__2; +x_4 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__10; +x_5 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; } } +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__8; +x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__4; +x_3 = l_Lean_Expr_const___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__2(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__13() { _start: { -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_3; -x_3 = lean_box(0); +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10; +x_2 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__4; +x_3 = l_Lean_Expr_const___override(x_1, x_2); return x_3; } +} +LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_mkContext(lean_object* x_1, lean_object* x_2, lean_object* x_3, 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; lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_10 = lean_array_get_size(x_4); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_nat_dec_lt(x_11, x_10); +lean_dec(x_10); +x_13 = lean_box(0); +x_14 = lean_array_size(x_4); +x_15 = 0; +x_16 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__4; +x_17 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__5; +x_18 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__8; +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1(x_1, x_2, x_3, x_13, x_16, x_17, x_18, x_14, x_15, x_4, x_5, x_6, x_7, x_8, x_9); +if (x_12 == 0) +{ +lean_object* x_179; lean_object* x_180; +lean_dec(x_4); +x_179 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__1; +x_180 = l_outOfBounds___rarg(x_179); +x_20 = x_180; +goto block_178; +} +else +{ +lean_object* x_181; +x_181 = lean_array_fget(x_4, x_11); +lean_dec(x_4); +x_20 = x_181; +goto block_178; +} +block_178: +{ +uint8_t x_21; +x_21 = !lean_is_exclusive(x_19); +if (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; lean_object* x_30; +x_22 = lean_ctor_get(x_19, 0); +x_23 = lean_ctor_get(x_19, 1); +x_24 = lean_ctor_get(x_20, 0); +lean_inc(x_24); +lean_dec(x_20); +x_25 = lean_array_to_list(x_22); +lean_ctor_set_tag(x_19, 1); +lean_ctor_set(x_19, 1, x_13); +lean_ctor_set(x_19, 0, x_3); +x_26 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__9; +lean_inc(x_19); +x_27 = l_Lean_Expr_const___override(x_26, x_19); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +lean_inc(x_28); +lean_inc(x_2); +x_29 = l_Lean_mkAppB(x_27, x_2, x_28); +x_30 = l_Lean_Meta_mkListLit(x_29, x_25, x_5, x_6, x_7, x_8, x_23); +if (lean_obj_tag(x_30) == 0) +{ +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; 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_32 = lean_ctor_get(x_30, 0); +x_33 = l_Lean_Meta_AC_preContext___closed__6; +lean_inc(x_19); +x_34 = l_Lean_Expr_const___override(x_33, x_19); +lean_inc(x_28); +lean_inc(x_2); +x_35 = l_Lean_mkAppB(x_34, x_2, x_28); +x_36 = lean_ctor_get(x_1, 3); +lean_inc(x_36); +x_37 = l_Lean_Meta_AC_preContext___closed__8; +lean_inc(x_19); +x_38 = l_Lean_Expr_const___override(x_37, x_19); +lean_inc(x_28); +lean_inc(x_2); +x_39 = l_Lean_mkAppB(x_38, x_2, x_28); +x_40 = lean_ctor_get(x_1, 4); +lean_inc(x_40); +x_41 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; +x_42 = l_Lean_Expr_const___override(x_41, x_19); +if (lean_obj_tag(x_36) == 0) +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_43 = lean_ctor_get(x_1, 2); +lean_inc(x_43); +lean_dec(x_1); +x_44 = l_Lean_Expr_app___override(x_17, x_35); +x_45 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; +x_46 = l_Lean_Expr_app___override(x_45, x_44); +if (lean_obj_tag(x_40) == 0) +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = l_Lean_Expr_app___override(x_17, x_39); +x_48 = l_Lean_Expr_app___override(x_45, x_47); +x_49 = l_Lean_mkApp7(x_42, x_2, x_28, x_43, x_46, x_48, x_32, x_24); +lean_ctor_set(x_30, 0, x_49); +return x_30; +} +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_40, 0); +lean_inc(x_50); +lean_dec(x_40); +lean_inc(x_39); +x_51 = l_Lean_Expr_app___override(x_17, x_39); +x_52 = l_Lean_mkAppB(x_18, x_39, x_50); +x_53 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__13; +x_54 = l_Lean_mkAppB(x_53, x_51, x_52); +x_55 = l_Lean_mkApp7(x_42, x_2, x_28, x_43, x_46, x_54, x_32, x_24); +lean_ctor_set(x_30, 0, x_55); +return x_30; +} +} +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_1, 2); +lean_inc(x_56); +lean_dec(x_1); +x_57 = lean_ctor_get(x_36, 0); +lean_inc(x_57); +lean_dec(x_36); +lean_inc(x_35); +x_58 = l_Lean_Expr_app___override(x_17, x_35); +x_59 = l_Lean_mkAppB(x_18, x_35, x_57); +x_60 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__13; +x_61 = l_Lean_mkAppB(x_60, x_58, x_59); +if (lean_obj_tag(x_40) == 0) +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_62 = l_Lean_Expr_app___override(x_17, x_39); +x_63 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; +x_64 = l_Lean_Expr_app___override(x_63, x_62); +x_65 = l_Lean_mkApp7(x_42, x_2, x_28, x_56, x_61, x_64, x_32, x_24); +lean_ctor_set(x_30, 0, x_65); +return x_30; +} +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_40, 0); +lean_inc(x_66); +lean_dec(x_40); +lean_inc(x_39); +x_67 = l_Lean_Expr_app___override(x_17, x_39); +x_68 = l_Lean_mkAppB(x_18, x_39, x_66); +x_69 = l_Lean_mkAppB(x_60, x_67, x_68); +x_70 = l_Lean_mkApp7(x_42, x_2, x_28, x_56, x_61, x_69, x_32, x_24); +lean_ctor_set(x_30, 0, x_70); +return x_30; +} +} +} +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; +x_71 = lean_ctor_get(x_30, 0); +x_72 = lean_ctor_get(x_30, 1); +lean_inc(x_72); +lean_inc(x_71); +lean_dec(x_30); +x_73 = l_Lean_Meta_AC_preContext___closed__6; +lean_inc(x_19); +x_74 = l_Lean_Expr_const___override(x_73, x_19); +lean_inc(x_28); +lean_inc(x_2); +x_75 = l_Lean_mkAppB(x_74, x_2, x_28); +x_76 = lean_ctor_get(x_1, 3); +lean_inc(x_76); +x_77 = l_Lean_Meta_AC_preContext___closed__8; +lean_inc(x_19); +x_78 = l_Lean_Expr_const___override(x_77, x_19); +lean_inc(x_28); +lean_inc(x_2); +x_79 = l_Lean_mkAppB(x_78, x_2, x_28); +x_80 = lean_ctor_get(x_1, 4); +lean_inc(x_80); +x_81 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; +x_82 = l_Lean_Expr_const___override(x_81, x_19); +if (lean_obj_tag(x_76) == 0) +{ +lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_83 = lean_ctor_get(x_1, 2); +lean_inc(x_83); +lean_dec(x_1); +x_84 = l_Lean_Expr_app___override(x_17, x_75); +x_85 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; +x_86 = l_Lean_Expr_app___override(x_85, x_84); +if (lean_obj_tag(x_80) == 0) +{ +lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; +x_87 = l_Lean_Expr_app___override(x_17, x_79); +x_88 = l_Lean_Expr_app___override(x_85, x_87); +x_89 = l_Lean_mkApp7(x_82, x_2, x_28, x_83, x_86, x_88, x_71, x_24); +x_90 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_90, 0, x_89); +lean_ctor_set(x_90, 1, x_72); +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_80, 0); +lean_inc(x_91); +lean_dec(x_80); +lean_inc(x_79); +x_92 = l_Lean_Expr_app___override(x_17, x_79); +x_93 = l_Lean_mkAppB(x_18, x_79, x_91); +x_94 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__13; +x_95 = l_Lean_mkAppB(x_94, x_92, x_93); +x_96 = l_Lean_mkApp7(x_82, x_2, x_28, x_83, x_86, x_95, x_71, x_24); +x_97 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_97, 0, x_96); +lean_ctor_set(x_97, 1, x_72); +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; +x_98 = lean_ctor_get(x_1, 2); +lean_inc(x_98); +lean_dec(x_1); +x_99 = lean_ctor_get(x_76, 0); +lean_inc(x_99); +lean_dec(x_76); +lean_inc(x_75); +x_100 = l_Lean_Expr_app___override(x_17, x_75); +x_101 = l_Lean_mkAppB(x_18, x_75, x_99); +x_102 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__13; +x_103 = l_Lean_mkAppB(x_102, x_100, x_101); +if (lean_obj_tag(x_80) == 0) +{ +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_104 = l_Lean_Expr_app___override(x_17, x_79); +x_105 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; +x_106 = l_Lean_Expr_app___override(x_105, x_104); +x_107 = l_Lean_mkApp7(x_82, x_2, x_28, x_98, x_103, x_106, x_71, x_24); +x_108 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_108, 0, x_107); +lean_ctor_set(x_108, 1, x_72); +return x_108; +} +else +{ +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +x_109 = lean_ctor_get(x_80, 0); +lean_inc(x_109); +lean_dec(x_80); +lean_inc(x_79); +x_110 = l_Lean_Expr_app___override(x_17, x_79); +x_111 = l_Lean_mkAppB(x_18, x_79, x_109); +x_112 = l_Lean_mkAppB(x_102, x_110, x_111); +x_113 = l_Lean_mkApp7(x_82, x_2, x_28, x_98, x_103, x_112, x_71, x_24); +x_114 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_114, 0, x_113); +lean_ctor_set(x_114, 1, x_72); +return x_114; +} +} +} +} +else +{ +uint8_t x_115; +lean_dec(x_28); +lean_dec(x_19); +lean_dec(x_24); +lean_dec(x_2); +lean_dec(x_1); +x_115 = !lean_is_exclusive(x_30); +if (x_115 == 0) +{ +return x_30; +} +else +{ +lean_object* x_116; lean_object* x_117; lean_object* x_118; +x_116 = lean_ctor_get(x_30, 0); +x_117 = lean_ctor_get(x_30, 1); +lean_inc(x_117); +lean_inc(x_116); +lean_dec(x_30); +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_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_119 = lean_ctor_get(x_19, 0); +x_120 = lean_ctor_get(x_19, 1); +lean_inc(x_120); +lean_inc(x_119); +lean_dec(x_19); +x_121 = lean_ctor_get(x_20, 0); +lean_inc(x_121); +lean_dec(x_20); +x_122 = lean_array_to_list(x_119); +x_123 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_123, 0, x_3); +lean_ctor_set(x_123, 1, x_13); +x_124 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__9; +lean_inc(x_123); +x_125 = l_Lean_Expr_const___override(x_124, x_123); +x_126 = lean_ctor_get(x_1, 1); +lean_inc(x_126); +lean_inc(x_126); +lean_inc(x_2); +x_127 = l_Lean_mkAppB(x_125, x_2, x_126); +x_128 = l_Lean_Meta_mkListLit(x_127, x_122, x_5, x_6, x_7, x_8, x_120); +if (lean_obj_tag(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; lean_object* x_139; lean_object* x_140; lean_object* x_141; +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); +} +x_132 = l_Lean_Meta_AC_preContext___closed__6; +lean_inc(x_123); +x_133 = l_Lean_Expr_const___override(x_132, x_123); +lean_inc(x_126); +lean_inc(x_2); +x_134 = l_Lean_mkAppB(x_133, x_2, x_126); +x_135 = lean_ctor_get(x_1, 3); +lean_inc(x_135); +x_136 = l_Lean_Meta_AC_preContext___closed__8; +lean_inc(x_123); +x_137 = l_Lean_Expr_const___override(x_136, x_123); +lean_inc(x_126); +lean_inc(x_2); +x_138 = l_Lean_mkAppB(x_137, x_2, x_126); +x_139 = lean_ctor_get(x_1, 4); +lean_inc(x_139); +x_140 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__11; +x_141 = l_Lean_Expr_const___override(x_140, x_123); +if (lean_obj_tag(x_135) == 0) +{ +lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; +x_142 = lean_ctor_get(x_1, 2); +lean_inc(x_142); +lean_dec(x_1); +x_143 = l_Lean_Expr_app___override(x_17, x_134); +x_144 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; +x_145 = l_Lean_Expr_app___override(x_144, x_143); +if (lean_obj_tag(x_139) == 0) +{ +lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; +x_146 = l_Lean_Expr_app___override(x_17, x_138); +x_147 = l_Lean_Expr_app___override(x_144, x_146); +x_148 = l_Lean_mkApp7(x_141, x_2, x_126, x_142, x_145, x_147, x_129, x_121); +if (lean_is_scalar(x_131)) { + x_149 = lean_alloc_ctor(0, 2, 0); +} else { + x_149 = x_131; +} +lean_ctor_set(x_149, 0, x_148); +lean_ctor_set(x_149, 1, x_130); +return x_149; +} +else +{ +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_150 = lean_ctor_get(x_139, 0); +lean_inc(x_150); +lean_dec(x_139); +lean_inc(x_138); +x_151 = l_Lean_Expr_app___override(x_17, x_138); +x_152 = l_Lean_mkAppB(x_18, x_138, x_150); +x_153 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__13; +x_154 = l_Lean_mkAppB(x_153, x_151, x_152); +x_155 = l_Lean_mkApp7(x_141, x_2, x_126, x_142, x_145, x_154, x_129, x_121); +if (lean_is_scalar(x_131)) { + x_156 = lean_alloc_ctor(0, 2, 0); +} else { + x_156 = x_131; +} +lean_ctor_set(x_156, 0, x_155); +lean_ctor_set(x_156, 1, x_130); +return x_156; +} +} +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; +x_157 = lean_ctor_get(x_1, 2); +lean_inc(x_157); +lean_dec(x_1); +x_158 = lean_ctor_get(x_135, 0); +lean_inc(x_158); +lean_dec(x_135); +lean_inc(x_134); +x_159 = l_Lean_Expr_app___override(x_17, x_134); +x_160 = l_Lean_mkAppB(x_18, x_134, x_158); +x_161 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__13; +x_162 = l_Lean_mkAppB(x_161, x_159, x_160); +if (lean_obj_tag(x_139) == 0) +{ +lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; +x_163 = l_Lean_Expr_app___override(x_17, x_138); +x_164 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__12; +x_165 = l_Lean_Expr_app___override(x_164, x_163); +x_166 = l_Lean_mkApp7(x_141, x_2, x_126, x_157, x_162, x_165, x_129, x_121); +if (lean_is_scalar(x_131)) { + x_167 = lean_alloc_ctor(0, 2, 0); +} else { + x_167 = x_131; +} +lean_ctor_set(x_167, 0, x_166); +lean_ctor_set(x_167, 1, x_130); +return x_167; +} +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; +x_168 = lean_ctor_get(x_139, 0); +lean_inc(x_168); +lean_dec(x_139); +lean_inc(x_138); +x_169 = l_Lean_Expr_app___override(x_17, x_138); +x_170 = l_Lean_mkAppB(x_18, x_138, x_168); +x_171 = l_Lean_mkAppB(x_161, x_169, x_170); +x_172 = l_Lean_mkApp7(x_141, x_2, x_126, x_157, x_162, x_171, x_129, x_121); +if (lean_is_scalar(x_131)) { + x_173 = lean_alloc_ctor(0, 2, 0); +} else { + x_173 = x_131; +} +lean_ctor_set(x_173, 0, x_172); +lean_ctor_set(x_173, 1, x_130); +return x_173; +} +} +} +else +{ +lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; +lean_dec(x_126); +lean_dec(x_123); +lean_dec(x_121); +lean_dec(x_2); +lean_dec(x_1); +x_174 = lean_ctor_get(x_128, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_128, 1); +lean_inc(x_175); +if (lean_is_exclusive(x_128)) { + lean_ctor_release(x_128, 0); + lean_ctor_release(x_128, 1); + x_176 = x_128; +} else { + lean_dec_ref(x_128); + x_176 = lean_box(0); +} +if (lean_is_scalar(x_176)) { + x_177 = lean_alloc_ctor(1, 2, 0); +} else { + x_177 = x_176; +} +lean_ctor_set(x_177, 0, x_174); +lean_ctor_set(x_177, 1, x_175); +return x_177; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___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_8); +lean_dec(x_8); +x_17 = lean_unbox_usize(x_9); +lean_dec(x_9); +x_18 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_16, x_17, 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); +return x_18; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Expr", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("var", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___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_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2; +x_3 = l_Lean_Meta_AC_getInstance___closed__2; +x_4 = l_Lean_Meta_AC_buildNormProof_convert___closed__1; +x_5 = l_Lean_Meta_AC_buildNormProof_convert___closed__2; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___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_AC_buildNormProof_convert___closed__3; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("op", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___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; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2; +x_3 = l_Lean_Meta_AC_getInstance___closed__2; +x_4 = l_Lean_Meta_AC_buildNormProof_convert___closed__1; +x_5 = l_Lean_Meta_AC_buildNormProof_convert___closed__5; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof_convert___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_AC_buildNormProof_convert___closed__6; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_convert(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +lean_dec(x_1); +x_3 = l_Lean_mkNatLit(x_2); +x_4 = l_Lean_Meta_AC_buildNormProof_convert___closed__4; +x_5 = l_Lean_Expr_app___override(x_4, x_3); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +lean_dec(x_1); +x_8 = l_Lean_Meta_AC_buildNormProof_convert(x_6); +x_9 = l_Lean_Meta_AC_buildNormProof_convert(x_7); +x_10 = l_Lean_Meta_AC_buildNormProof_convert___closed__7; +x_11 = l_Lean_mkAppB(x_10, x_8, x_9); +return x_11; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_convertTarget(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_object* x_5; uint8_t x_6; +lean_dec(x_1); +x_4 = lean_ctor_get(x_3, 0); +x_5 = lean_array_get_size(x_2); +x_6 = lean_nat_dec_lt(x_4, x_5); +lean_dec(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; +x_7 = l_Lean_instInhabitedExpr; +x_8 = l_outOfBounds___rarg(x_7); +return x_8; +} +else +{ +lean_object* x_9; +x_9 = lean_array_fget(x_2, x_4); +return x_9; +} +} +else +{ +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_3, 0); +x_11 = lean_ctor_get(x_3, 1); +x_12 = lean_ctor_get(x_1, 1); +lean_inc(x_12); +lean_inc(x_1); +x_13 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_2, x_10); +x_14 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_2, x_11); +x_15 = l_Lean_mkAppB(x_12, x_13, x_14); +return x_15; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof_convertTarget___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_2, x_3); +lean_dec(x_3); +lean_dec(x_2); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__1(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; +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); +if (lean_obj_tag(x_8) == 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_array_uset(x_7, x_2, x_12); +x_2 = x_10; +x_3 = x_13; +goto _start; +} +else +{ +uint8_t x_15; lean_object* x_16; lean_object* x_17; +lean_dec(x_8); +x_15 = 1; +x_16 = lean_box(x_15); +x_17 = lean_array_uset(x_7, x_2, x_16); +x_2 = x_10; +x_3 = x_17; +goto _start; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__2(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, 0); +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; +goto _start; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5(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; lean_object* 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_1, 1); +x_8 = lean_array_get_size(x_7); +x_9 = lean_nat_dec_lt(x_5, x_8); +lean_dec(x_8); +if (x_9 == 0) +{ +uint8_t x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = l_instInhabitedBool; +x_11 = lean_box(x_10); +x_12 = l_outOfBounds___rarg(x_11); +x_13 = lean_unbox(x_12); +lean_dec(x_12); +if (x_13 == 0) +{ +lean_object* x_14; +x_14 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5(x_1, x_6); +lean_ctor_set(x_2, 1, x_14); +return x_2; +} +else +{ +lean_free_object(x_2); +lean_dec(x_5); +x_2 = x_6; +goto _start; +} +} +else +{ +lean_object* x_16; uint8_t x_17; +x_16 = lean_array_fget(x_7, x_5); +x_17 = lean_unbox(x_16); +lean_dec(x_16); +if (x_17 == 0) +{ +lean_object* x_18; +x_18 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5(x_1, x_6); +lean_ctor_set(x_2, 1, x_18); +return x_2; +} +else +{ +lean_free_object(x_2); +lean_dec(x_5); +x_2 = x_6; +goto _start; +} +} +} +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_2, 0); +x_21 = lean_ctor_get(x_2, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_2); +x_22 = lean_ctor_get(x_1, 1); +x_23 = lean_array_get_size(x_22); +x_24 = lean_nat_dec_lt(x_20, x_23); +lean_dec(x_23); +if (x_24 == 0) +{ +uint8_t x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_25 = l_instInhabitedBool; +x_26 = lean_box(x_25); +x_27 = l_outOfBounds___rarg(x_26); +x_28 = lean_unbox(x_27); +lean_dec(x_27); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +x_29 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5(x_1, x_21); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_20); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} +else +{ +lean_dec(x_20); +x_2 = x_21; +goto _start; +} +} +else +{ +lean_object* x_32; uint8_t x_33; +x_32 = lean_array_fget(x_22, x_20); +x_33 = lean_unbox(x_32); +lean_dec(x_32); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; +x_34 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5(x_1, x_21); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_20); +lean_ctor_set(x_35, 1, x_34); +return x_35; +} +else +{ +lean_dec(x_20); +x_2 = x_21; +goto _start; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__4(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; +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5(x_1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_box(0); +x_8 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_8, 0, x_5); +lean_ctor_set(x_8, 1, x_7); +return x_8; +} +else +{ +lean_dec(x_5); +return x_6; +} +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_ctor_get(x_2, 0); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +lean_inc(x_9); +lean_dec(x_2); +lean_inc(x_9); +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 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5(x_1, x_11); +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_13; lean_object* x_14; +x_13 = lean_box(0); +x_14 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_14, 0, x_9); +lean_ctor_set(x_14, 1, x_13); +return x_14; +} +else +{ +lean_dec(x_9); +return x_12; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__3(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; +x_3 = l_Lean_Data_AC_Expr_toList(x_2); +x_4 = l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__4(x_1, x_3); +x_5 = lean_ctor_get(x_1, 0); +x_6 = lean_ctor_get(x_5, 3); +if (lean_obj_tag(x_6) == 0) +{ +lean_object* x_7; +x_7 = lean_ctor_get(x_5, 4); +if (lean_obj_tag(x_7) == 0) +{ +return x_4; +} +else +{ +lean_object* x_8; +x_8 = l_Lean_Data_AC_mergeIdem(x_4); +return x_8; +} +} +else +{ +lean_object* x_9; +x_9 = lean_ctor_get(x_5, 4); +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_10; +x_10 = l_Lean_Data_AC_sort(x_4); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; +x_11 = l_Lean_Data_AC_sort(x_4); +x_12 = l_Lean_Data_AC_mergeIdem(x_11); +return x_12; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__6(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_3; +x_3 = l_Lean_Meta_AC_instEvalInformationPreContextACExpr___lambda__1___closed__1; +return x_3; +} +else +{ +lean_object* x_4; +x_4 = lean_ctor_get(x_2, 1); +lean_inc(x_4); +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_5; lean_object* x_6; +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); +return x_6; +} +else +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t 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); +lean_inc(x_4); +x_9 = l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__6(x_1, x_4); +x_10 = !lean_is_exclusive(x_4); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_4, 1); +lean_dec(x_11); +x_12 = lean_ctor_get(x_4, 0); +lean_dec(x_12); +lean_ctor_set(x_4, 1, x_9); +lean_ctor_set(x_4, 0, x_8); +return x_4; +} +else +{ +lean_object* x_13; +lean_dec(x_4); +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_8); +lean_ctor_set(x_13, 1, x_9); +return x_13; +} +} +} +} +} +static lean_object* _init_l_panic___at_Lean_Meta_AC_buildNormProof___spec__7___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_AC_buildNormProof___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) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = l_panic___at_Lean_Meta_AC_buildNormProof___spec__7___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_Lean_Meta_AC_buildNormProof___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_Meta_AC_buildNormProof___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_Meta_AC_buildNormProof___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_AC_buildNormProof___lambda__1___closed__1; +x_2 = l_Lean_Meta_AC_buildNormProof___lambda__1___closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof___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_Meta_AC_buildNormProof___lambda__1___closed__3; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("eq_of_norm", 10, 10); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_AC_buildNormProof___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; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2; +x_3 = l_Lean_Meta_AC_getInstance___closed__2; +x_4 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__10; +x_5 = l_Lean_Meta_AC_buildNormProof___lambda__1___closed__5; +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_AC_buildNormProof___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_79; lean_object* x_80; uint8_t x_81; +x_79 = lean_array_get_size(x_3); +x_80 = lean_unsigned_to_nat(0u); +x_81 = lean_nat_dec_lt(x_80, x_79); +lean_dec(x_79); +if (x_81 == 0) +{ +lean_object* x_82; lean_object* x_83; +x_82 = l_Lean_instInhabitedExpr; +x_83 = l_outOfBounds___rarg(x_82); +x_10 = x_83; +goto block_78; +} +else +{ +lean_object* x_84; +x_84 = lean_array_fget(x_3, x_80); +x_10 = x_84; +goto block_78; +} +block_78: +{ +lean_object* x_11; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_11 = lean_infer_type(x_10, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* 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); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_12); +x_14 = l_Lean_Meta_getLevel(x_12, x_5, x_6, x_7, x_8, x_13); +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); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_15); +lean_inc(x_12); +lean_inc(x_1); +x_17 = l_Lean_Meta_AC_buildNormProof_mkContext(x_1, x_12, x_15, x_4, x_5, x_6, x_7, x_8, x_16); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; size_t x_20; size_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; +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_array_size(x_4); +x_21 = 0; +lean_inc(x_4); +x_22 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__1(x_20, x_21, x_4); +x_23 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__2(x_20, x_21, x_4); +lean_inc(x_1); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_1); +lean_ctor_set(x_24, 1, x_22); +x_25 = l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__3(x_24, x_2); +lean_dec(x_24); +x_26 = l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__6(x_1, x_25); +lean_inc(x_2); +x_27 = l_Lean_Meta_AC_buildNormProof_convert(x_2); +lean_inc(x_26); +x_28 = l_Lean_Meta_AC_buildNormProof_convert(x_26); +x_29 = lean_box(0); +x_30 = l_Lean_Meta_AC_buildNormProof___lambda__1___closed__4; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_31 = l_Lean_Meta_mkEqRefl(x_30, x_5, x_6, x_7, x_8, x_19); +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; 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_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_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_15); +lean_ctor_set(x_34, 1, x_29); +x_35 = l_Lean_Meta_AC_buildNormProof___lambda__1___closed__6; +x_36 = l_Lean_Expr_const___override(x_35, x_34); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_32); +lean_ctor_set(x_37, 1, x_29); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_28); +lean_ctor_set(x_38, 1, x_37); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_27); +lean_ctor_set(x_39, 1, x_38); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_18); +lean_ctor_set(x_40, 1, x_39); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_12); +lean_ctor_set(x_41, 1, x_40); +x_42 = lean_array_mk(x_41); +x_43 = l_Lean_mkAppN(x_36, x_42); +lean_dec(x_42); +lean_inc(x_1); +x_44 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_23, x_2); +lean_dec(x_2); +x_45 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_23, x_26); +lean_dec(x_26); +lean_dec(x_23); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_46 = l_Lean_Meta_mkEq(x_44, x_45, x_5, x_6, x_7, x_8, x_33); +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_Lean_Meta_mkExpectedTypeHint(x_43, x_47, x_5, x_6, x_7, x_8, x_48); +if (lean_obj_tag(x_49) == 0) +{ +uint8_t x_50; +x_50 = !lean_is_exclusive(x_49); +if (x_50 == 0) +{ +return x_49; +} else { -uint8_t x_4; -x_4 = !lean_is_exclusive(x_2); -if (x_4 == 0) +lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_51 = lean_ctor_get(x_49, 0); +x_52 = lean_ctor_get(x_49, 1); +lean_inc(x_52); +lean_inc(x_51); +lean_dec(x_49); +x_53 = lean_alloc_ctor(0, 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_5; lean_object* x_6; -x_5 = lean_ctor_get(x_2, 0); -lean_inc(x_5); -x_6 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3(x_1, x_2); -if (lean_obj_tag(x_6) == 0) +uint8_t x_54; +x_54 = !lean_is_exclusive(x_49); +if (x_54 == 0) { -lean_object* x_7; lean_object* x_8; -x_7 = lean_box(0); -x_8 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_8, 0, x_5); -lean_ctor_set(x_8, 1, x_7); -return x_8; +return x_49; } else { -lean_dec(x_5); -return x_6; +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; +} } } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_ctor_get(x_2, 0); -x_10 = lean_ctor_get(x_2, 1); -lean_inc(x_10); -lean_inc(x_9); -lean_dec(x_2); -lean_inc(x_9); -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 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3(x_1, x_11); -if (lean_obj_tag(x_12) == 0) +uint8_t x_58; +lean_dec(x_43); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_58 = !lean_is_exclusive(x_46); +if (x_58 == 0) { -lean_object* x_13; lean_object* x_14; -x_13 = lean_box(0); -x_14 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_14, 0, x_9); -lean_ctor_set(x_14, 1, x_13); -return x_14; +return x_46; } else { -lean_dec(x_9); -return x_12; -} -} +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; } } } -LEAN_EXPORT lean_object* l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__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; -x_3 = l_Lean_Data_AC_Expr_toList(x_2); -x_4 = l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__2(x_1, x_3); -x_5 = lean_ctor_get(x_1, 0); -x_6 = lean_ctor_get(x_5, 3); -if (lean_obj_tag(x_6) == 0) +else { -lean_object* x_7; -x_7 = lean_ctor_get(x_5, 4); -if (lean_obj_tag(x_7) == 0) +uint8_t x_62; +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_23); +lean_dec(x_18); +lean_dec(x_15); +lean_dec(x_12); +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_62 = !lean_is_exclusive(x_31); +if (x_62 == 0) { -return x_4; +return x_31; } else { -lean_object* x_8; -x_8 = l_Lean_Data_AC_mergeIdem(x_4); -return x_8; +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_31, 0); +x_64 = lean_ctor_get(x_31, 1); +lean_inc(x_64); +lean_inc(x_63); +lean_dec(x_31); +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_9; -x_9 = lean_ctor_get(x_5, 4); -if (lean_obj_tag(x_9) == 0) +uint8_t x_66; +lean_dec(x_15); +lean_dec(x_12); +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_66 = !lean_is_exclusive(x_17); +if (x_66 == 0) { -lean_object* x_10; -x_10 = l_Lean_Data_AC_sort(x_4); -return x_10; +return x_17; } else { -lean_object* x_11; lean_object* x_12; -x_11 = l_Lean_Data_AC_sort(x_4); -x_12 = l_Lean_Data_AC_mergeIdem(x_11); -return x_12; -} +lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_67 = lean_ctor_get(x_17, 0); +x_68 = lean_ctor_get(x_17, 1); +lean_inc(x_68); +lean_inc(x_67); +lean_dec(x_17); +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_EXPORT lean_object* l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__4(lean_object* x_1, lean_object* x_2) { -_start: +else { -if (lean_obj_tag(x_2) == 0) +uint8_t x_70; +lean_dec(x_12); +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_70 = !lean_is_exclusive(x_14); +if (x_70 == 0) { -lean_object* x_3; -x_3 = l_Lean_Meta_AC_instEvalInformationPreContextACExpr___lambda__1___closed__1; -return x_3; +return x_14; } else { -lean_object* x_4; -x_4 = lean_ctor_get(x_2, 1); -lean_inc(x_4); -if (lean_obj_tag(x_4) == 0) -{ -lean_object* x_5; lean_object* x_6; -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); -return x_6; +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_ctor_get(x_14, 0); +x_72 = lean_ctor_get(x_14, 1); +lean_inc(x_72); +lean_inc(x_71); +lean_dec(x_14); +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_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_7 = lean_ctor_get(x_2, 0); -lean_inc(x_7); +uint8_t x_74; +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_8 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_8, 0, x_7); -lean_inc(x_4); -x_9 = l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__4(x_1, x_4); -x_10 = !lean_is_exclusive(x_4); -if (x_10 == 0) +lean_dec(x_1); +x_74 = !lean_is_exclusive(x_11); +if (x_74 == 0) { -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_4, 1); -lean_dec(x_11); -x_12 = lean_ctor_get(x_4, 0); -lean_dec(x_12); -lean_ctor_set(x_4, 1, x_9); -lean_ctor_set(x_4, 0, x_8); -return x_4; +return x_11; } else { -lean_object* x_13; -lean_dec(x_4); -x_13 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_13, 0, x_8); -lean_ctor_set(x_13, 1, x_9); -return x_13; +lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_75 = lean_ctor_get(x_11, 0); +x_76 = lean_ctor_get(x_11, 1); +lean_inc(x_76); +lean_inc(x_75); +lean_dec(x_11); +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; } } } @@ -4937,43 +5947,41 @@ static lean_object* _init_l_Lean_Meta_AC_buildNormProof___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("Bool", 4, 4); +x_1 = lean_mk_string_unchecked("Eq", 2, 2); return x_1; } } static lean_object* _init_l_Lean_Meta_AC_buildNormProof___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("true", 4, 4); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_AC_buildNormProof___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } static lean_object* _init_l_Lean_Meta_AC_buildNormProof___closed__3() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_buildNormProof___closed__1; -x_2 = l_Lean_Meta_AC_buildNormProof___closed__2; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Meta.Tactic.AC.Main", 24, 24); +return x_1; } } static lean_object* _init_l_Lean_Meta_AC_buildNormProof___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_AC_buildNormProof___closed__3; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Meta.AC.buildNormProof", 27, 27); +return x_1; } } static lean_object* _init_l_Lean_Meta_AC_buildNormProof___closed__5() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("eq_of_norm", 10, 10); +x_1 = lean_mk_string_unchecked("unexpected proof type", 21, 21); return x_1; } } @@ -4981,12 +5989,12 @@ static lean_object* _init_l_Lean_Meta_AC_buildNormProof___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; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__4; -x_3 = l_Lean_Meta_AC_getInstance___closed__2; -x_4 = l_Lean_Meta_AC_buildNormProof_mkContext___closed__9; +x_1 = l_Lean_Meta_AC_buildNormProof___closed__3; +x_2 = l_Lean_Meta_AC_buildNormProof___closed__4; +x_3 = lean_unsigned_to_nat(129u); +x_4 = lean_unsigned_to_nat(52u); x_5 = l_Lean_Meta_AC_buildNormProof___closed__5; -x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } @@ -5003,51 +6011,29 @@ lean_inc(x_4); x_10 = l_Lean_Meta_AC_toACExpr(x_9, x_2, x_3, x_4, x_5, x_6, x_7, 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_111; lean_object* x_112; uint8_t x_113; +lean_object* x_11; lean_object* x_12; uint8_t 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_ctor_get(x_11, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_11, 1); -lean_inc(x_14); -if (lean_is_exclusive(x_11)) { - lean_ctor_release(x_11, 0); - lean_ctor_release(x_11, 1); - x_15 = x_11; -} else { - lean_dec_ref(x_11); - x_15 = lean_box(0); -} -x_111 = lean_array_get_size(x_13); -x_112 = lean_unsigned_to_nat(0u); -x_113 = lean_nat_dec_lt(x_112, x_111); -lean_dec(x_111); -if (x_113 == 0) -{ -lean_object* x_114; lean_object* x_115; -x_114 = l_Lean_instInhabitedExpr; -x_115 = l_outOfBounds___rarg(x_114); -x_16 = x_115; -goto block_110; -} -else -{ -lean_object* x_116; -x_116 = lean_array_fget(x_13, x_112); -x_16 = x_116; -goto block_110; -} -block_110: +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 0) { -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_11, 0); +x_15 = lean_ctor_get(x_11, 1); +lean_inc(x_14); +lean_inc(x_1); +x_16 = lean_alloc_closure((void*)(l_Lean_Meta_AC_buildNormProof___lambda__1___boxed), 9, 3); +lean_closure_set(x_16, 0, x_1); +lean_closure_set(x_16, 1, x_15); +lean_closure_set(x_16, 2, x_14); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_17 = lean_infer_type(x_16, x_4, x_5, x_6, x_7, x_12); +x_17 = l_Lean_Meta_AC_abstractAtoms(x_1, x_14, x_16, x_4, x_5, x_6, x_7, x_12); if (lean_obj_tag(x_17) == 0) { lean_object* x_18; lean_object* x_19; lean_object* x_20; @@ -5060,439 +6046,384 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_18); -x_20 = l_Lean_Meta_getLevel(x_18, x_4, x_5, x_6, x_7, 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_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_13); -lean_inc(x_21); -lean_inc(x_18); -lean_inc(x_1); -x_23 = l_Lean_Meta_AC_buildNormProof_mkContext(x_1, x_18, x_21, x_13, x_4, x_5, x_6, x_7, x_22); -if (lean_obj_tag(x_23) == 0) -{ -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) -{ -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; -x_27 = lean_ctor_get(x_24, 0); -x_28 = lean_ctor_get(x_24, 1); -lean_inc(x_1); -lean_ctor_set(x_24, 1, x_27); -lean_ctor_set(x_24, 0, x_1); -x_29 = l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__1(x_24, x_14); -lean_dec(x_24); -x_30 = l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__4(x_1, x_29); -x_31 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_13, x_30); -lean_dec(x_13); -x_32 = l_Lean_Meta_AC_buildNormProof_convert(x_14); -x_33 = l_Lean_Meta_AC_buildNormProof_convert(x_30); -x_34 = lean_box(0); -x_35 = l_Lean_Meta_AC_buildNormProof___closed__4; -x_36 = l_Lean_Meta_mkEqRefl(x_35, x_4, x_5, x_6, x_7, x_25); -if (lean_obj_tag(x_36) == 0) +lean_inc(x_18); +x_20 = lean_infer_type(x_18, x_4, x_5, x_6, x_7, x_19); +if (lean_obj_tag(x_20) == 0) { -uint8_t x_37; -x_37 = !lean_is_exclusive(x_36); -if (x_37 == 0) +uint8_t x_21; +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 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; -x_38 = lean_ctor_get(x_36, 0); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_21); -lean_ctor_set(x_39, 1, x_34); -x_40 = l_Lean_Meta_AC_buildNormProof___closed__6; -x_41 = l_Lean_Expr_const___override(x_40, x_39); -x_42 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_42, 0, x_38); -lean_ctor_set(x_42, 1, x_34); -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_33); -lean_ctor_set(x_43, 1, x_42); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_32); -lean_ctor_set(x_44, 1, x_43); -x_45 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_45, 0, x_28); -lean_ctor_set(x_45, 1, x_44); -x_46 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_46, 0, x_18); -lean_ctor_set(x_46, 1, x_45); -x_47 = lean_array_mk(x_46); -x_48 = l_Lean_mkAppN(x_41, x_47); -lean_dec(x_47); -if (lean_is_scalar(x_15)) { - x_49 = lean_alloc_ctor(0, 2, 0); -} else { - x_49 = x_15; -} -lean_ctor_set(x_49, 0, x_48); -lean_ctor_set(x_49, 1, x_31); -lean_ctor_set(x_36, 0, x_49); -return x_36; +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_20, 0); +x_23 = lean_ctor_get(x_20, 1); +x_24 = l_Lean_Meta_AC_buildNormProof___closed__2; +x_25 = lean_unsigned_to_nat(3u); +x_26 = l_Lean_Expr_isAppOfArity(x_22, x_24, x_25); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; +lean_free_object(x_20); +lean_dec(x_22); +lean_dec(x_18); +lean_free_object(x_11); +x_27 = l_Lean_Meta_AC_buildNormProof___closed__6; +x_28 = l_panic___at_Lean_Meta_AC_buildNormProof___spec__7(x_27, x_4, x_5, x_6, x_7, x_23); +return x_28; } 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; lean_object* x_62; lean_object* x_63; -x_50 = lean_ctor_get(x_36, 0); -x_51 = lean_ctor_get(x_36, 1); -lean_inc(x_51); -lean_inc(x_50); -lean_dec(x_36); -x_52 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_52, 0, x_21); -lean_ctor_set(x_52, 1, x_34); -x_53 = l_Lean_Meta_AC_buildNormProof___closed__6; -x_54 = l_Lean_Expr_const___override(x_53, x_52); -x_55 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_55, 0, x_50); -lean_ctor_set(x_55, 1, x_34); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_33); -lean_ctor_set(x_56, 1, x_55); -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_28); -lean_ctor_set(x_58, 1, x_57); -x_59 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_59, 0, x_18); -lean_ctor_set(x_59, 1, x_58); -x_60 = lean_array_mk(x_59); -x_61 = l_Lean_mkAppN(x_54, x_60); -lean_dec(x_60); -if (lean_is_scalar(x_15)) { - x_62 = lean_alloc_ctor(0, 2, 0); -} else { - x_62 = x_15; -} -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_31); -x_63 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_63, 0, x_62); -lean_ctor_set(x_63, 1, x_51); -return x_63; +lean_object* x_29; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_29 = l_Lean_Expr_appArg_x21(x_22); +lean_dec(x_22); +lean_ctor_set(x_11, 1, x_29); +lean_ctor_set(x_11, 0, x_18); +lean_ctor_set(x_20, 0, x_11); +return x_20; } } else { -uint8_t x_64; -lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_31); -lean_dec(x_28); -lean_dec(x_21); -lean_dec(x_18); -lean_dec(x_15); -x_64 = !lean_is_exclusive(x_36); -if (x_64 == 0) +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +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 = l_Lean_Meta_AC_buildNormProof___closed__2; +x_33 = lean_unsigned_to_nat(3u); +x_34 = l_Lean_Expr_isAppOfArity(x_30, x_32, x_33); +if (x_34 == 0) { +lean_object* x_35; lean_object* x_36; +lean_dec(x_30); +lean_dec(x_18); +lean_free_object(x_11); +x_35 = l_Lean_Meta_AC_buildNormProof___closed__6; +x_36 = l_panic___at_Lean_Meta_AC_buildNormProof___spec__7(x_35, x_4, x_5, x_6, x_7, x_31); return x_36; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_65 = lean_ctor_get(x_36, 0); -x_66 = lean_ctor_get(x_36, 1); -lean_inc(x_66); -lean_inc(x_65); -lean_dec(x_36); -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_37; lean_object* x_38; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_37 = l_Lean_Expr_appArg_x21(x_30); +lean_dec(x_30); +lean_ctor_set(x_11, 1, x_37); +lean_ctor_set(x_11, 0, x_18); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_11); +lean_ctor_set(x_38, 1, x_31); +return x_38; } } } 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; -x_68 = lean_ctor_get(x_24, 0); -x_69 = lean_ctor_get(x_24, 1); -lean_inc(x_69); -lean_inc(x_68); -lean_dec(x_24); -lean_inc(x_1); -x_70 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_70, 0, x_1); -lean_ctor_set(x_70, 1, x_68); -x_71 = l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__1(x_70, x_14); -lean_dec(x_70); -x_72 = l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__4(x_1, x_71); -x_73 = l_Lean_Meta_AC_buildNormProof_convertTarget(x_1, x_13, x_72); -lean_dec(x_13); -x_74 = l_Lean_Meta_AC_buildNormProof_convert(x_14); -x_75 = l_Lean_Meta_AC_buildNormProof_convert(x_72); -x_76 = lean_box(0); -x_77 = l_Lean_Meta_AC_buildNormProof___closed__4; -x_78 = l_Lean_Meta_mkEqRefl(x_77, x_4, x_5, x_6, x_7, x_25); -if (lean_obj_tag(x_78) == 0) +uint8_t x_39; +lean_dec(x_18); +lean_free_object(x_11); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_39 = !lean_is_exclusive(x_20); +if (x_39 == 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; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; -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); -} -x_82 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_82, 0, x_21); -lean_ctor_set(x_82, 1, x_76); -x_83 = l_Lean_Meta_AC_buildNormProof___closed__6; -x_84 = l_Lean_Expr_const___override(x_83, x_82); -x_85 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_85, 0, x_79); -lean_ctor_set(x_85, 1, x_76); -x_86 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_86, 0, x_75); -lean_ctor_set(x_86, 1, x_85); -x_87 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_87, 0, x_74); -lean_ctor_set(x_87, 1, x_86); -x_88 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_88, 0, x_69); -lean_ctor_set(x_88, 1, x_87); -x_89 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_89, 0, x_18); -lean_ctor_set(x_89, 1, x_88); -x_90 = lean_array_mk(x_89); -x_91 = l_Lean_mkAppN(x_84, x_90); -lean_dec(x_90); -if (lean_is_scalar(x_15)) { - x_92 = lean_alloc_ctor(0, 2, 0); -} else { - x_92 = x_15; -} -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_73); -if (lean_is_scalar(x_81)) { - x_93 = lean_alloc_ctor(0, 2, 0); -} else { - x_93 = x_81; -} -lean_ctor_set(x_93, 0, x_92); -lean_ctor_set(x_93, 1, x_80); -return x_93; +return x_20; } else { -lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; -lean_dec(x_75); -lean_dec(x_74); -lean_dec(x_73); -lean_dec(x_69); -lean_dec(x_21); -lean_dec(x_18); -lean_dec(x_15); -x_94 = lean_ctor_get(x_78, 0); -lean_inc(x_94); -x_95 = lean_ctor_get(x_78, 1); -lean_inc(x_95); -if (lean_is_exclusive(x_78)) { - lean_ctor_release(x_78, 0); - lean_ctor_release(x_78, 1); - x_96 = x_78; -} else { - lean_dec_ref(x_78); - x_96 = lean_box(0); -} -if (lean_is_scalar(x_96)) { - x_97 = lean_alloc_ctor(1, 2, 0); -} else { - x_97 = x_96; -} -lean_ctor_set(x_97, 0, x_94); -lean_ctor_set(x_97, 1, x_95); -return x_97; +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_20, 0); +x_41 = lean_ctor_get(x_20, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_20); +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 { -uint8_t x_98; -lean_dec(x_21); -lean_dec(x_18); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +uint8_t x_43; +lean_free_object(x_11); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_1); -x_98 = !lean_is_exclusive(x_23); -if (x_98 == 0) +x_43 = !lean_is_exclusive(x_17); +if (x_43 == 0) { -return x_23; +return x_17; } else { -lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_99 = lean_ctor_get(x_23, 0); -x_100 = lean_ctor_get(x_23, 1); -lean_inc(x_100); -lean_inc(x_99); -lean_dec(x_23); -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_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; } } } else { -uint8_t x_102; -lean_dec(x_18); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +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_dec(x_11); +lean_inc(x_47); +lean_inc(x_1); +x_49 = lean_alloc_closure((void*)(l_Lean_Meta_AC_buildNormProof___lambda__1___boxed), 9, 3); +lean_closure_set(x_49, 0, x_1); +lean_closure_set(x_49, 1, x_48); +lean_closure_set(x_49, 2, x_47); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_50 = l_Lean_Meta_AC_abstractAtoms(x_1, x_47, x_49, x_4, x_5, x_6, x_7, x_12); +if (lean_obj_tag(x_50) == 0) +{ +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); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_51); +x_53 = lean_infer_type(x_51, x_4, x_5, x_6, x_7, 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; lean_object* x_58; uint8_t x_59; +x_54 = lean_ctor_get(x_53, 0); +lean_inc(x_54); +x_55 = lean_ctor_get(x_53, 1); +lean_inc(x_55); +if (lean_is_exclusive(x_53)) { + lean_ctor_release(x_53, 0); + lean_ctor_release(x_53, 1); + x_56 = x_53; +} else { + lean_dec_ref(x_53); + x_56 = lean_box(0); +} +x_57 = l_Lean_Meta_AC_buildNormProof___closed__2; +x_58 = lean_unsigned_to_nat(3u); +x_59 = l_Lean_Expr_isAppOfArity(x_54, x_57, x_58); +if (x_59 == 0) +{ +lean_object* x_60; lean_object* x_61; +lean_dec(x_56); +lean_dec(x_54); +lean_dec(x_51); +x_60 = l_Lean_Meta_AC_buildNormProof___closed__6; +x_61 = l_panic___at_Lean_Meta_AC_buildNormProof___spec__7(x_60, x_4, x_5, x_6, x_7, x_55); +return x_61; +} +else +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_1); -x_102 = !lean_is_exclusive(x_20); -if (x_102 == 0) -{ -return x_20; +x_62 = l_Lean_Expr_appArg_x21(x_54); +lean_dec(x_54); +x_63 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_63, 0, x_51); +lean_ctor_set(x_63, 1, x_62); +if (lean_is_scalar(x_56)) { + x_64 = lean_alloc_ctor(0, 2, 0); +} else { + x_64 = x_56; +} +lean_ctor_set(x_64, 0, x_63); +lean_ctor_set(x_64, 1, x_55); +return x_64; +} } else { -lean_object* x_103; lean_object* x_104; lean_object* x_105; -x_103 = lean_ctor_get(x_20, 0); -x_104 = lean_ctor_get(x_20, 1); -lean_inc(x_104); -lean_inc(x_103); -lean_dec(x_20); -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_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +lean_dec(x_51); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_65 = lean_ctor_get(x_53, 0); +lean_inc(x_65); +x_66 = lean_ctor_get(x_53, 1); +lean_inc(x_66); +if (lean_is_exclusive(x_53)) { + lean_ctor_release(x_53, 0); + lean_ctor_release(x_53, 1); + x_67 = x_53; +} else { + lean_dec_ref(x_53); + 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 { -uint8_t x_106; -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_1); -x_106 = !lean_is_exclusive(x_17); -if (x_106 == 0) -{ -return x_17; +x_69 = lean_ctor_get(x_50, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_50, 1); +lean_inc(x_70); +if (lean_is_exclusive(x_50)) { + lean_ctor_release(x_50, 0); + lean_ctor_release(x_50, 1); + x_71 = x_50; +} else { + lean_dec_ref(x_50); + x_71 = lean_box(0); } -else -{ -lean_object* x_107; lean_object* x_108; lean_object* x_109; -x_107 = lean_ctor_get(x_17, 0); -x_108 = lean_ctor_get(x_17, 1); -lean_inc(x_108); -lean_inc(x_107); -lean_dec(x_17); -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; +if (lean_is_scalar(x_71)) { + x_72 = lean_alloc_ctor(1, 2, 0); +} else { + x_72 = x_71; } +lean_ctor_set(x_72, 0, x_69); +lean_ctor_set(x_72, 1, x_70); +return x_72; } } } else { -uint8_t x_117; +uint8_t x_73; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_117 = !lean_is_exclusive(x_10); -if (x_117 == 0) +x_73 = !lean_is_exclusive(x_10); +if (x_73 == 0) { return x_10; } else { -lean_object* x_118; lean_object* x_119; lean_object* x_120; -x_118 = lean_ctor_get(x_10, 0); -x_119 = lean_ctor_get(x_10, 1); -lean_inc(x_119); -lean_inc(x_118); +lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_74 = lean_ctor_get(x_10, 0); +x_75 = lean_ctor_get(x_10, 1); +lean_inc(x_75); +lean_inc(x_74); lean_dec(x_10); -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; +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_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__1___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_6 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__1(x_4, x_5, x_3); +return x_6; } } +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__2___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_6 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof___spec__2(x_4, x_5, x_3); +return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__3(x_1, x_2); +x_3 = l_Lean_Data_AC_removeNeutrals_loop___at_Lean_Meta_AC_buildNormProof___spec__5(x_1, x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__2___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__4___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__2(x_1, x_2); +x_3 = l_Lean_Data_AC_removeNeutrals___at_Lean_Meta_AC_buildNormProof___spec__4(x_1, x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__3___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__1(x_1, x_2); +x_3 = l_Lean_Data_AC_norm___at_Lean_Meta_AC_buildNormProof___spec__3(x_1, x_2); lean_dec(x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__4___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__6___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__4(x_1, x_2); +x_3 = l_Lean_Data_AC_evalList___at_Lean_Meta_AC_buildNormProof___spec__6(x_1, x_2); lean_dec(x_1); return x_3; } } +LEAN_EXPORT lean_object* l_Lean_Meta_AC_buildNormProof___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_Meta_AC_buildNormProof___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_3); +return x_10; +} +} LEAN_EXPORT lean_object* l_Lean_Meta_AC_post___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: { @@ -7756,7 +8687,7 @@ static lean_object* _init_l___regBuiltin_Lean_Meta_AC_acRflTactic__1___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_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; x_2 = l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__1; x_3 = l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__2; x_4 = l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__3; @@ -7776,7 +8707,7 @@ static lean_object* _init_l___regBuiltin_Lean_Meta_AC_acRflTactic__1___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_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; x_2 = l_Lean_Meta_AC_getInstance___closed__1; x_3 = l_Lean_Meta_AC_getInstance___closed__2; x_4 = l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__5; @@ -9131,7 +10062,7 @@ static lean_object* _init_l_Lean_Meta_AC_evalNf0___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_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; x_2 = l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__1; x_3 = l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__2; x_4 = l_Lean_Meta_AC_evalNf0___closed__1; @@ -9266,7 +10197,7 @@ static lean_object* _init_l___regBuiltin_Lean_Meta_AC_evalNf0__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_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; x_2 = l_Lean_Meta_AC_getInstance___closed__1; x_3 = l_Lean_Meta_AC_getInstance___closed__2; x_4 = l___regBuiltin_Lean_Meta_AC_evalNf0__1___closed__1; @@ -9294,37 +10225,37 @@ x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__1() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____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_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__2() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__1; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__1; x_2 = l_Lean_Meta_AC_getInstance___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__3() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__2; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__2; x_2 = l_Lean_Meta_AC_getInstance___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__4() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__4() { _start: { lean_object* x_1; @@ -9332,17 +10263,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__5() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__3; -x_2 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__4; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__3; +x_2 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__6() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__6() { _start: { lean_object* x_1; @@ -9350,57 +10281,57 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__7() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__5; -x_2 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__6; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__5; +x_2 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__8() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__7; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__3; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__7; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__9() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__8; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__8; x_2 = l_Lean_Meta_AC_getInstance___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__10() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__9; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__9; x_2 = l___regBuiltin_Lean_Meta_AC_acRflTactic__1___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__11() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__10; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__10; x_2 = l_Lean_Meta_AC_getInstance___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__12() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__12() { _start: { lean_object* x_1; @@ -9408,17 +10339,17 @@ x_1 = lean_mk_string_unchecked("Main", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__13() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__11; -x_2 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__12; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__11; +x_2 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__14() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__14() { _start: { lean_object* x_1; @@ -9426,33 +10357,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__15() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__13; -x_2 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__14; +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__13; +x_2 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__14; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__16() { +static lean_object* _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__15; -x_2 = lean_unsigned_to_nat(2895u); +x_1 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__15; +x_2 = lean_unsigned_to_nat(6304u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304_(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_AC_getInstance___closed__3; x_3 = 0; -x_4 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__16; +x_4 = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__16; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -9560,6 +10491,18 @@ l_Lean_Meta_AC_toACExpr___closed__3 = _init_l_Lean_Meta_AC_toACExpr___closed__3( lean_mark_persistent(l_Lean_Meta_AC_toACExpr___closed__3); l_Lean_Meta_AC_toACExpr___closed__4 = _init_l_Lean_Meta_AC_toACExpr___closed__4(); lean_mark_persistent(l_Lean_Meta_AC_toACExpr___closed__4); +l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__1 = _init_l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__1); +l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__2 = _init_l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__2); +l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__3 = _init_l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__3); +l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__4 = _init_l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__4(); +lean_mark_persistent(l_Lean_Meta_AC_abstractAtoms_go___lambda__2___closed__4); +l_Lean_Meta_AC_abstractAtoms_go___closed__1 = _init_l_Lean_Meta_AC_abstractAtoms_go___closed__1(); +lean_mark_persistent(l_Lean_Meta_AC_abstractAtoms_go___closed__1); +l_Lean_Meta_AC_abstractAtoms_go___closed__2 = _init_l_Lean_Meta_AC_abstractAtoms_go___closed__2(); +lean_mark_persistent(l_Lean_Meta_AC_abstractAtoms_go___closed__2); l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1(); lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__1); l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__2(); @@ -9580,10 +10523,6 @@ l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___cl lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__9); l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10(); lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__10); -l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__11 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__11(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__11); -l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__12 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__12(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_AC_buildNormProof_mkContext___spec__1___closed__12); l_Lean_Meta_AC_buildNormProof_mkContext___closed__1 = _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__1(); lean_mark_persistent(l_Lean_Meta_AC_buildNormProof_mkContext___closed__1); l_Lean_Meta_AC_buildNormProof_mkContext___closed__2 = _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__2(); @@ -9608,6 +10547,8 @@ l_Lean_Meta_AC_buildNormProof_mkContext___closed__11 = _init_l_Lean_Meta_AC_buil lean_mark_persistent(l_Lean_Meta_AC_buildNormProof_mkContext___closed__11); l_Lean_Meta_AC_buildNormProof_mkContext___closed__12 = _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__12(); lean_mark_persistent(l_Lean_Meta_AC_buildNormProof_mkContext___closed__12); +l_Lean_Meta_AC_buildNormProof_mkContext___closed__13 = _init_l_Lean_Meta_AC_buildNormProof_mkContext___closed__13(); +lean_mark_persistent(l_Lean_Meta_AC_buildNormProof_mkContext___closed__13); l_Lean_Meta_AC_buildNormProof_convert___closed__1 = _init_l_Lean_Meta_AC_buildNormProof_convert___closed__1(); lean_mark_persistent(l_Lean_Meta_AC_buildNormProof_convert___closed__1); l_Lean_Meta_AC_buildNormProof_convert___closed__2 = _init_l_Lean_Meta_AC_buildNormProof_convert___closed__2(); @@ -9622,6 +10563,20 @@ l_Lean_Meta_AC_buildNormProof_convert___closed__6 = _init_l_Lean_Meta_AC_buildNo lean_mark_persistent(l_Lean_Meta_AC_buildNormProof_convert___closed__6); l_Lean_Meta_AC_buildNormProof_convert___closed__7 = _init_l_Lean_Meta_AC_buildNormProof_convert___closed__7(); lean_mark_persistent(l_Lean_Meta_AC_buildNormProof_convert___closed__7); +l_panic___at_Lean_Meta_AC_buildNormProof___spec__7___closed__1 = _init_l_panic___at_Lean_Meta_AC_buildNormProof___spec__7___closed__1(); +lean_mark_persistent(l_panic___at_Lean_Meta_AC_buildNormProof___spec__7___closed__1); +l_Lean_Meta_AC_buildNormProof___lambda__1___closed__1 = _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Meta_AC_buildNormProof___lambda__1___closed__1); +l_Lean_Meta_AC_buildNormProof___lambda__1___closed__2 = _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Meta_AC_buildNormProof___lambda__1___closed__2); +l_Lean_Meta_AC_buildNormProof___lambda__1___closed__3 = _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Meta_AC_buildNormProof___lambda__1___closed__3); +l_Lean_Meta_AC_buildNormProof___lambda__1___closed__4 = _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Meta_AC_buildNormProof___lambda__1___closed__4); +l_Lean_Meta_AC_buildNormProof___lambda__1___closed__5 = _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Meta_AC_buildNormProof___lambda__1___closed__5); +l_Lean_Meta_AC_buildNormProof___lambda__1___closed__6 = _init_l_Lean_Meta_AC_buildNormProof___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Meta_AC_buildNormProof___lambda__1___closed__6); l_Lean_Meta_AC_buildNormProof___closed__1 = _init_l_Lean_Meta_AC_buildNormProof___closed__1(); lean_mark_persistent(l_Lean_Meta_AC_buildNormProof___closed__1); l_Lean_Meta_AC_buildNormProof___closed__2 = _init_l_Lean_Meta_AC_buildNormProof___closed__2(); @@ -9720,39 +10675,39 @@ lean_mark_persistent(l___regBuiltin_Lean_Meta_AC_evalNf0__1___closed__3); if (builtin) {res = l___regBuiltin_Lean_Meta_AC_evalNf0__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__1 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__1(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__1); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__2 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__2(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__2); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__3 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__3(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__3); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__4 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__4(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__4); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__5 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__5(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__5); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__6 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__6(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__6); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__7 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__7(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__7); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__8 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__8(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__8); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__9 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__9(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__9); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__10 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__10(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__10); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__11 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__11(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__11); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__12 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__12(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__12); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__13 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__13(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__13); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__14 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__14(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__14); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__15 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__15(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__15); -l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__16 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__16(); -lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895____closed__16); -if (builtin) {res = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_2895_(lean_io_mk_world()); +}l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__1 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__1(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__1); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__2 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__2(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__2); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__3 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__3(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__3); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__4 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__4(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__4); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__5 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__5(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__5); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__6 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__6(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__6); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__7 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__7(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__7); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__8 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__8(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__8); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__9 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__9(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__9); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__10 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__10(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__10); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__11 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__11(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__11); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__12 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__12(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__12); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__13 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__13(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__13); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__14 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__14(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__14); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__15 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__15(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__15); +l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__16 = _init_l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__16(); +lean_mark_persistent(l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304____closed__16); +if (builtin) {res = l_Lean_Meta_AC_initFn____x40_Lean_Meta_Tactic_AC_Main___hyg_6304_(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/Backtrack.c b/stage0/stdlib/Lean/Meta/Tactic/Backtrack.c index 2b86a6dc16c7..39075f92a4a7 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Backtrack.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Backtrack.c @@ -27,6 +27,7 @@ lean_object* l_Lean_MVarId_getType___boxed(lean_object*, lean_object*, lean_obje LEAN_EXPORT lean_object* l_ReaderT_pure___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run___spec__2(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run___lambda__1___closed__4; static lean_object* l___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run___lambda__10___closed__1; +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_processIndependentGoals___spec__7(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_processIndependentGoals___lambda__1___closed__6; static lean_object* l___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_processIndependentGoals___lambda__4___closed__2; double lean_float_div(double, double); @@ -68,7 +69,6 @@ static lean_object* l___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_B LEAN_EXPORT lean_object* l_Lean_withTraceNode___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run___spec__6___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_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_pure___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_processIndependentGoals___spec__7(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterMapTR_go___at_Lean_Meta_Tactic_Backtrack_Backtrack_tryAllM___spec__2(lean_object*, lean_object*); lean_object* l_List_appendTR___rarg(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_run___lambda__1___closed__3; @@ -5553,7 +5553,7 @@ return x_26; } } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_processIndependentGoals___spec__7(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_processIndependentGoals___spec__7(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -6418,7 +6418,7 @@ lean_inc(x_19); x_20 = lean_ctor_get(x_17, 1); lean_inc(x_20); lean_dec(x_17); -x_21 = l_List_bindTR_go___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_processIndependentGoals___spec__7(x_20, x_3); +x_21 = l_List_flatMapTR_go___at___private_Lean_Meta_Tactic_Backtrack_0__Lean_Meta_Tactic_Backtrack_Backtrack_processIndependentGoals___spec__7(x_20, x_3); lean_inc(x_4); lean_inc(x_21); lean_inc(x_19); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Cases.c b/stage0/stdlib/Lean/Meta/Tactic/Cases.c index 95c82dff9dff..ac7fa2be1cd0 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Cases.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Cases.c @@ -223,6 +223,7 @@ lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_hasIndepIndices___spec__44(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_hasIndepIndices___spec__14(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_hasIndepIndices___spec__10(lean_object*, lean_object*, lean_object*, size_t, size_t); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___spec__1(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_Array_anyMUnsafe_any___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_hasIndepIndices___spec__52(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_hasIndepIndices___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at_Lean_MVarId_casesRec___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -300,7 +301,6 @@ lean_object* l_Array_extract___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_withNewEqs___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_exactlyOne(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MVarId_casesRec___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___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_Cases_cases___closed__1; lean_object* l_Lean_Meta_introNCore(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_Cases___hyg_3709____closed__12; @@ -375,6 +375,7 @@ lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0_ LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at_Lean_MVarId_casesRec___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_EXPORT lean_object* l_Lean_Meta_Cases_cases___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_generalizeIndices___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_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___spec__1___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_mapTR_loop___at_Lean_MVarId_casesRec___spec__1(lean_object*, lean_object*); uint8_t l_Lean_Expr_hasFVar(lean_object*); @@ -393,7 +394,6 @@ lean_object* l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(lean LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_generalizeIndices___spec__1___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_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_throwInductiveTypeExpected___spec__1(lean_object*); static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_Cases___hyg_3709____closed__4; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___spec__1(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_Array_anyMUnsafe_any___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_hasIndepIndices___spec__49(lean_object*, lean_object*, lean_object*, size_t, size_t); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Cases_cases___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -12595,7 +12595,7 @@ lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___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_Array_mapFinIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___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; @@ -12749,15 +12749,15 @@ lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; x_6 = lean_array_get_size(x_1); x_7 = lean_mk_empty_array_with_capacity(x_6); x_8 = lean_unsigned_to_nat(0u); -x_9 = l_Array_mapIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___spec__1(x_1, x_2, x_3, x_4, x_5, x_1, x_6, x_8, lean_box(0), x_7); +x_9 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___spec__1(x_1, x_2, x_3, x_4, x_5, x_1, x_6, x_8, lean_box(0), x_7); return x_9; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___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_Array_mapFinIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___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_Array_mapIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Array_mapFinIdxM_map___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_toCasesSubgoals___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_6); lean_dec(x_5); lean_dec(x_2); diff --git a/stage0/stdlib/Lean/Meta/Tactic/FunInd.c b/stage0/stdlib/Lean/Meta/Tactic/FunInd.c index 5e6a7ee4e351..d18e78d2de53 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/FunInd.c +++ b/stage0/stdlib/Lean/Meta/Tactic/FunInd.c @@ -13,11 +13,13 @@ #ifdef __cplusplus extern "C" { #endif +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__11; static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__9___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescope___at_Lean_Tactic_FunInd_deriveUnaryInduction___spec__3___rarg(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_Lean_Tactic_FunInd_buildInductionCase(lean_object*, lean_object*, lean_object*, lean_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_Tactic_FunInd_abstractIndependentMVars___spec__1(lean_object*, size_t, size_t, 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_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__3; static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__13___closed__5; lean_object* l_Lean_log___at_Lean_Elab_Term_reportUnsolvedGoals___spec__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkEqHEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -26,22 +28,24 @@ lean_object* l_StateRefT_x27_instMonadExceptOf___rarg(lean_object*); lean_object* l_Lean_registerReservedNameAction(lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__43___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*); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__8; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__19___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Tactic_FunInd_buildInductionBody___spec__4___rarg___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_inferArgumentTypesN(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__5; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__1(lean_object*); static lean_object* l_Lean_isTracingEnabledFor___at_Lean_Tactic_FunInd_buildInductionCase___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___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_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__5(lean_object*, 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*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_buildInductionBody___spec__6___closed__1; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__2; static lean_object* l_Lean_Tactic_FunInd_buildInductionCase___closed__7; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__17___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__4(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_Tactic_FunInd_buildInductionBody___spec__26(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__5; LEAN_EXPORT lean_object* l_StateT_bind___at_Lean_Tactic_FunInd_buildInductionBody___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_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_buildInductionBody___spec__6___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_Meta_ArgsPacker_curryParam___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -57,32 +61,29 @@ LEAN_EXPORT lean_object* l_Lean_Meta_MatcherApp_withUserNames___at_Lean_Tactic_F LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__25___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__22(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_Tactic_FunInd_unpackMutualInduction___spec__1___lambda__2___closed__4; -LEAN_EXPORT lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616_(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_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___closed__3; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__5___closed__5; static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__10___closed__1; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Meta_Tactic_Simp_SimpTheorems_0__Lean_Meta_isPerm___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__5; lean_object* lean_mk_empty_array_with_capacity(lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__4___closed__4; static lean_object* l_Lean_getConstInfo___at_Lean_Tactic_FunInd_foldAndCollect___spec__3___closed__3; static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__13___closed__4; extern lean_object* l_Lean_Elab_WF_instInhabitedEqnInfo; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__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_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__38(lean_object*, size_t, 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* l_Lean_Meta_mkPProdFst(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Tactic_FunInd_foldAndCollect___spec__6___closed__3; lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__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_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__17(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__12___closed__1; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___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*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__2; +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____closed__1; LEAN_EXPORT uint8_t l_Lean_logAt___at_Lean_Tactic_FunInd_buildInductionBody___spec__41___lambda__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__11(lean_object*, lean_object*, 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_Tactic_FunInd_buildInductionBody___lambda__26___closed__2; @@ -147,7 +148,6 @@ uint8_t l_Lean_Expr_isAppOfArity(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Tactic_FunInd_foldAndCollect___spec__9___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_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__24(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_MatcherApp_withUserNames___at_Lean_Meta_MatcherApp_inferMatchType___spec__10___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8___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_Tactic_FunInd_buildInductionBody___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*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_StateT_pure___at_Lean_Tactic_FunInd_buildInductionBody___spec__46___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isApp(lean_object*); @@ -172,8 +172,8 @@ static lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_fold LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__12___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___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*); uint8_t l_Array_contains___at_Lean_findField_x3f___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___lambda__4___closed__3; -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__4(lean_object*, lean_object*, lean_object*, size_t, 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*); static lean_object* l_Lean_logAt___at_Lean_Tactic_FunInd_buildInductionBody___spec__41___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___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*); @@ -196,10 +196,10 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildI static lean_object* l_Lean_Tactic_FunInd_deriveInduction___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__10___boxed(lean_object**); lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__19___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f___spec__5(lean_object*, lean_object*, uint8_t, 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_Elab_Structural_getRecArgInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_M_run___rarg___closed__1; lean_object* l_Lean_replaceRef(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f___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*); @@ -220,7 +220,6 @@ lean_object* l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27__ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__35___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_Tactic_FunInd_deriveInduction___lambda__1___closed__2; extern lean_object* l_Lean_casesOnSuffix; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); lean_object* l_Lean_Meta_Match_MatcherInfo_arity(lean_object*); lean_object* l_Lean_ConstantInfo_name(lean_object*); @@ -264,7 +263,6 @@ lean_object* l_Lean_MessageData_hasSyntheticSorry(lean_object*); static lean_object* l_Lean_Expr_withAppAux___at_Lean_Tactic_FunInd_unpackMutualInduction___spec__1___lambda__2___closed__2; static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___closed__1; LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Tactic_FunInd_mkLambdaFVarsMasked___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__10; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__4___boxed(lean_object**); static lean_object* l_Lean_Tactic_FunInd_deriveInduction___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -278,10 +276,10 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_buildInd LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_assertIHs___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__18(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_elimOptParam___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__10; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f___boxed(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_List_get___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__1; lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); static lean_object* l_Lean_Elab_Structural_Positions_groupAndSort___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__3___closed__1; LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f___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*); @@ -291,7 +289,6 @@ static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__8___closed LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__18(lean_object*); lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Meta_MatcherApp_inferMatchType___spec__4(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_Lean_Tactic_FunInd_deriveInductionStructural___lambda__11(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*); -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__3; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__43___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__6___boxed(lean_object**); uint8_t l___private_Lean_Util_Trace_0__Lean_checkTraceOption(lean_object*, lean_object*, lean_object*); @@ -301,7 +298,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunIn lean_object* l_Lean_mkApp4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_MatcherApp_inferMatchType___spec__9(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedLevel; -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__11; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__12___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_Lean_Tactic_FunInd_unpackMutualInduction___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_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__26___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -348,6 +344,7 @@ extern lean_object* l_instInhabitedNat; extern lean_object* l_Lean_Elab_WF_eqnInfoExt; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_index(lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Tactic_FunInd_deriveUnaryInduction___spec__4___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_buildInductionBody___spec__39___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -357,7 +354,6 @@ extern lean_object* l_instInhabitedPUnit; LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_buildInductionBody___spec__6___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_Tactic_FunInd_unpackMutualInduction(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_removeLamda___at_Lean_Tactic_FunInd_buildInductionBody___spec__15___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__15; static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__12___closed__4; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___lambda__2___closed__1; @@ -376,6 +372,7 @@ static lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__5___closed__3 LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_cleanupAfter_allHeqToEq___spec__3(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_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at___private_Lean_Meta_InferType_0__Lean_Meta_checkInferTypeCache___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___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_EXPORT lean_object* l___private_Lean_Meta_Match_MatcherApp_Transform_0__Lean_Meta_MatcherApp_forallAltTelescope_x27___at_Lean_Tactic_FunInd_buildInductionBody___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*); @@ -384,7 +381,6 @@ lean_object* l_Lean_Meta_isTypeCorrect(lean_object*, lean_object*, lean_object*, static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__13___closed__8; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__12(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*); extern lean_object* l_Lean_Elab_Structural_eqnInfoExt; -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__12; size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_foldAndCollect___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_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__17___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -407,6 +403,7 @@ static lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__5___closed__1 lean_object* l_Array_reverse___rarg(lean_object*); uint8_t l_instDecidableNot___rarg(uint8_t); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___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 lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__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_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionCase___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_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_assertIHs___spec__1___closed__1; LEAN_EXPORT lean_object* l_StateT_lift___at_Lean_Tactic_FunInd_buildInductionBody___spec__1(lean_object*); @@ -433,7 +430,6 @@ uint8_t lean_expr_eqv(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_cleanupAfter_allHeqToEq___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* l_Lean_Meta_Match_Extension_getMatcherInfo_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__38___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_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__22___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_zip___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__38___lambda__1(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -444,15 +440,16 @@ lean_object* l_ReaderT_instMonadFunctor(lean_object*, lean_object*, lean_object* static lean_object* l_Lean_Tactic_FunInd_buildInductionCase___closed__2; static double l_Lean_addTrace___at_Lean_Tactic_FunInd_buildInductionCase___spec__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_M_eval(lean_object*); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__1; static lean_object* l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda__3___closed__2; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__2___closed__4; LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Tactic_FunInd_buildInductionBody___spec__41___lambda__2___boxed(lean_object*); lean_object* l_Lean_Meta_PProdN_proj(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_Tactic_FunInd_foldAndCollect___spec__15___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Tactic_FunInd_buildInductionBody___spec__40___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__6; lean_object* l_Lean_MVarId_getType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__8___closed__4; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__6(size_t, size_t, lean_object*); static lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___closed__4; static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__16___closed__1; static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__14___closed__4; @@ -467,7 +464,6 @@ static lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__13___closed__2 LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___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_registerTraceClass(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__16___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__7___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Tactic_FunInd_buildInductionBody___spec__4(lean_object*); lean_object* l_Lean_Meta_kabstract(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkHEqRefl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -484,6 +480,7 @@ lean_object* l_Lean_Name_getPrefix(lean_object*); static lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Nat_foldRevM_loop___at_Lean_Tactic_FunInd_foldAndCollect___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_M_branch___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__8; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__35(lean_object*, size_t, size_t, 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*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_M_tell___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -524,8 +521,8 @@ LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Tactic_FunInd_deriveIndu LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f___spec__1(lean_object*, 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_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__43___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_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___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_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8___rarg___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_Tactic_FunInd_buildInductionBody___lambda__8___closed__2; +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__13; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___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_object*, lean_object*); @@ -543,7 +540,6 @@ LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Tactic_FunInd_foldAndCollec LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Tactic_FunInd_unpackMutualInduction___spec__1___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_foldAndCollect___spec__1___lambda__2___closed__1; lean_object* lean_array_pop(lean_object*); -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__8; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Tactic_FunInd_buildInductionBody___spec__4___rarg(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_Lean_Tactic_FunInd_buildInductionBody___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_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -557,7 +553,6 @@ LEAN_EXPORT lean_object* l_Lean_getConstInfoDefn___at_Lean_Tactic_FunInd_deriveU static lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___lambda__6___closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_buildInductionBody___spec__6___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_array_to_list(lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__7; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__16___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_unpackMutualInduction___lambda__6___closed__11; static lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__10___closed__2; @@ -591,6 +586,7 @@ LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Tactic_FunInd_unpackMu LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_inferType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_logAt___at_Lean_Tactic_FunInd_buildInductionBody___spec__41___lambda__2___closed__4; +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__11; extern lean_object* l_Lean_levelZero; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__16(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_Array_foldlMUnsafe_fold___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -610,7 +606,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveIn static lean_object* l_Lean_Tactic_FunInd_removeLamda___rarg___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_withLetDecls_go(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_M_exec(lean_object*); -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__6; lean_object* l_Lean_Meta_whnfD(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deduplicateIHs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -631,8 +626,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_abstra LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at_Lean_Tactic_FunInd_foldAndCollect___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_EXPORT lean_object* l_Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__1; -static lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__23(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__9___closed__1; static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__16___closed__3; @@ -674,7 +667,6 @@ LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__3(lea 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_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_maskArray___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_unpackMutualInduction___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_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__2; static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__9___closed__1; static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__11___closed__1; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -683,6 +675,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveIn LEAN_EXPORT lean_object* l_Lean_Meta_withErasedFVars___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__20(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_PProdN_packLambdas(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkNot(lean_object*); +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*); static lean_object* l_Lean_Tactic_FunInd_unpackMutualInduction___closed__1; uint8_t l_Lean_LocalDecl_isLet(lean_object*); static lean_object* l_Lean_Expr_withAppAux___at_Lean_Tactic_FunInd_unpackMutualInduction___spec__1___lambda__2___closed__3; @@ -702,7 +695,6 @@ static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__7___closed lean_object* l_Lean_Expr_appFn_x21(lean_object*); static lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__8___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Tactic_FunInd_buildInductionBody___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_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Tactic_FunInd_withLetDecls___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__5___closed__4; LEAN_EXPORT lean_object* l_StateT_bind___at_Lean_Tactic_FunInd_buildInductionBody___spec__3(lean_object*, lean_object*); @@ -721,7 +713,6 @@ static lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__17___closed__1 static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__12___closed__5; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_cleanupAfter_allHeqToEq___spec__5(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_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__17(lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__43___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*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_buildInductionBody___spec__31(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_assert(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -740,6 +731,7 @@ static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__14_ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__17___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_buildInductionBody___spec__39(lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_forallTelescopeCompatibleAux___spec__15___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__10; static lean_object* l_Lean_Tactic_FunInd_isFunInductName___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_isFunInductName___lambda__3(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_instInhabitedMetaM___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -748,7 +740,8 @@ LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Tactic_FunInd_mkLambda static lean_object* l_Lean_Tactic_FunInd_abstractIndependentMVars___closed__2; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___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* l_Lean_mkConstWithLevelParams___at_Lean_Meta_mkSimpCongrTheorem___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__4; +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__9; lean_object* l_Array_append___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_unpackMutualInduction___lambda__6___closed__8; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__43(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*); @@ -759,7 +752,7 @@ LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda lean_object* l_Lean_throwError___at_Lean_LMVarId_getLevel___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_inheritedTraceOptions; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__13; +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__12; lean_object* l_Lean_MessageData_ofExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__28___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_buildInductionBody___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -796,7 +789,6 @@ static lean_object* l_Lean_Tactic_FunInd_abstractIndependentMVars___closed__4; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_unpackMutualInduction___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_name_append_index_after(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__8___boxed(lean_object**); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__14; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionCase___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_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__20___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isFVarOf(lean_object*, lean_object*); @@ -855,12 +847,11 @@ LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_M2_branch(lean_object*); static lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__10___closed__6; lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__9(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_withLocalDecls___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__7(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__24___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448_(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__20___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_mkLambdaFVarsMasked(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mapErrorImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__6___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__13___closed__2; static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__13___closed__2; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -871,7 +862,6 @@ LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda static lean_object* l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__15(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___lambda__2___closed__4; -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__8; static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__11___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_projectMutualInduct___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*); extern lean_object* l_Lean_brecOnSuffix; @@ -892,25 +882,28 @@ lean_object* l_Lean_Meta_getLocalInstances(lean_object*, lean_object*, lean_obje static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__10___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_observing_x3f___at_Lean_MVarId_iffOfEq___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f___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*); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__15; static lean_object* l_Lean_getConstInfo___at_Lean_Tactic_FunInd_foldAndCollect___spec__3___closed__1; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__19(lean_object*, lean_object*, lean_object*, lean_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_Tactic_FunInd_deriveInductionStructural___spec__14(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__2(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_Lean_Tactic_FunInd_abstractIndependentMVars___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__11; LEAN_EXPORT lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___lambda__3___boxed(lean_object**); lean_object* l_Lean_Meta_mkEqRefl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_unpackMutualInduction___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_Match_MatcherApp_Transform_0__Lean_Meta_MatcherApp_forallAltTelescope_x27___at_Lean_Tactic_FunInd_buildInductionBody___spec__42___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*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___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*); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at_Lean_Tactic_FunInd_foldAndCollect___spec__10(lean_object*); lean_object* l_Lean_indentExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__11(lean_object*, lean_object*, 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_isHEq(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___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_Tactic_FunInd_deriveUnaryInduction___lambda__17(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__7; static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__16___closed__5; static lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__25___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -939,7 +932,6 @@ lean_object* l_Lean_mkFreshFVarId___at___private_Lean_Meta_Basic_0__Lean_Meta_fo 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_Lean_Meta_MatcherApp_toExpr(lean_object*); static lean_object* l_Lean_Elab_Structural_Positions_groupAndSort___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__3___closed__3; -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__12; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_isFunInductName___lambda__1___boxed(lean_object*); @@ -950,20 +942,18 @@ LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Tactic_FunInd_foldA LEAN_EXPORT lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___lambda__6(lean_object*, lean_object*, size_t, 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_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_foldAndCollect___spec__1___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_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Tactic_FunInd_buildInductionBody___spec__14___rarg(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_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__4; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__24___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_M_localM(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); 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*); static lean_object* l_Lean_Elab_Structural_Positions_groupAndSort___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__3___closed__2; -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__5(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f___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_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getAppFn(lean_object*); lean_object* l_Lean_Meta_withLCtx___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_projectMutualInduct___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_Tactic_FunInd_deriveInductionStructural___lambda__15(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*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__6; static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__12___closed__3; static lean_object* l_Lean_Tactic_FunInd_M_branch___rarg___closed__1; static lean_object* l_Lean_Elab_Structural_Positions_groupAndSort___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__3___closed__4; @@ -973,6 +963,7 @@ LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__6(lean_o LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__4___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_foldAndCollect___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_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Tactic_FunInd_unpackMutualInduction___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_EXPORT lean_object* l_Lean_Tactic_FunInd_cleanPackedArgs___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__3___closed__3; @@ -991,10 +982,8 @@ lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_obj lean_object* l_Array_ofSubarray___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_withLetDecls_go___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*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__19___lambda__3___closed__5; -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470_(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe___at_Lean_Tactic_FunInd_M_localMapM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___closed__2; -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__9; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___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_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__7___boxed(lean_object**); lean_object* l_Array_back___rarg(lean_object*, lean_object*); @@ -1010,13 +999,14 @@ static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__15_ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_projectMutualInduct___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_Tactic_FunInd_deriveInductionStructural___lambda__10___closed__2; static lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___lambda__2___closed__2; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_Tactic_FunInd_buildInductionBody___spec__34___rarg(lean_object*, lean_object*, uint8_t, 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_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__16___closed__4; static lean_object* l_Lean_getConstInfo___at_Lean_Tactic_FunInd_foldAndCollect___spec__3___closed__4; LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Tactic_FunInd_unpackMutualInduction___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__12; lean_object* l_Lean_instantiateMVarsCore(lean_object*, lean_object*); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__9; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_isFunInductName___lambda__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getMatcherInfo_x3f___at_Lean_Tactic_FunInd_foldAndCollect___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1031,24 +1021,24 @@ lean_object* l_Lean_Meta_elimOptParam___lambda__1___boxed(lean_object*, lean_obj size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Tactic_FunInd_foldAndCollect___spec__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__5___closed__1; -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__5; static lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__13___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_buildInductionBody___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*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___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_Tactic_FunInd_buildInductionBody___lambda__9___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_PersistentArray_forInAux___at_Lean_Tactic_FunInd_cleanupAfter_allHeqToEq___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__43___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_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__4; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__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_Tactic_FunInd_maskArray___rarg___boxed(lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedName; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_unpackMutualInduction___lambda__5(lean_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_loop___at_Lean_Tactic_FunInd_foldAndCollect___spec__6(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); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvar___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__24___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1; size_t lean_array_size(lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_withAppAux___at_Lean_Tactic_FunInd_unpackMutualInduction___spec__1___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__19___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__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_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_buildInductionBody___spec__44(lean_object*, size_t, size_t, lean_object*); @@ -1066,11 +1056,11 @@ lean_object* l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(lean lean_object* l___private_Lean_Meta_Match_MatcherApp_Transform_0__Lean_Meta_MatcherApp_withUserNamesImpl___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__17(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*, lean_object*); lean_object* l_Lean_hasConst___at_Lean_Elab_Structural_getRecArgInfo___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__7; static lean_object* l_Lean_Expr_withAppAux___at_Lean_Tactic_FunInd_unpackMutualInduction___spec__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__7(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*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_cleanupAfter_cleanupAfter_x3f___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_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___lambda__2___closed__3; +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1; lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAux___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__14(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_EXPORT lean_object* l_Lean_Tactic_FunInd_projectMutualInduct___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1113,17 +1103,17 @@ LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda uint8_t l_Lean_isAuxRecursorWithSuffix(lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__9___boxed(lean_object**); +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__2; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__4(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_Tactic_FunInd_buildInductionBody___spec__27___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___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_Lean_Tactic_FunInd_foldAndCollect___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* l_Lean_Meta_Match_forallAltTelescope___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__1; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__22___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_isTracingEnabledFor___at_Lean_Tactic_FunInd_buildInductionCase___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_buildInductionBody___spec__38___lambda__3(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_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Tactic_FunInd_cleanupAfter_allHeqToEq___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1; lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Tactic_FunInd_buildInductionBody___spec__14___rarg___lambda__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*); @@ -1144,6 +1134,7 @@ static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__17___clo 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_Lean_log___at_Lean_Tactic_FunInd_buildInductionBody___spec__40(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__10(lean_object*, lean_object*, 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_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__14; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__10(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* lean_nat_add(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__5(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -1158,7 +1149,6 @@ LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__2(l LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___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* 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_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__9; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_cleanupAfter_go(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_Tactic_FunInd_deriveInductionStructural___spec__21(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_Structural_Positions_mapMwith___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__12___closed__6; @@ -1184,12 +1174,12 @@ lean_object* l_Lean_Expr_mvarId_x21(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__8(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_StateT_lift___at_Lean_Tactic_FunInd_buildInductionBody___spec__2(lean_object*); lean_object* l_Lean_InductiveVal_numCtors(lean_object*); -static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_foldAndCollect___spec__23___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Split_0__Lean_Meta_Split_generalizeMatchDiscrs___spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__3___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveInductionStructural___lambda__3(lean_object*, lean_object*, lean_object*, size_t, 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_EXPORT lean_object* l_Lean_throwError___at_Lean_Tactic_FunInd_buildInductionBody___spec__25(lean_object*); +LEAN_EXPORT lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody___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_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___lambda__6___closed__1; static lean_object* l_Lean_Tactic_FunInd_unpackMutualInduction___lambda__6___closed__2; @@ -1201,6 +1191,7 @@ LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Tactic_FunInd_buildInductionBody LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_removeLamda___at_Lean_Tactic_FunInd_foldAndCollect___spec__14(lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_buildInductionBody(lean_object*, 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_Tactic_FunInd_deriveUnaryInduction___lambda__17___closed__2; +static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__6; LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Tactic_FunInd_buildInductionCase___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_expr_instantiate1(lean_object*, lean_object*); lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); @@ -1208,10 +1199,12 @@ LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__13___boxe static lean_object* l_Lean_Meta_MatcherApp_transform___at_Lean_Tactic_FunInd_buildInductionBody___spec__29___lambda__2___closed__1; lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___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*); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__10; uint8_t l___private_Lean_Message_0__Lean_beqMessageSeverity____x40_Lean_Message___hyg_106_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__19___boxed(lean_object**); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__16___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_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Tactic_FunInd_buildInductionCase___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__3; static lean_object* l_Lean_Elab_Structural_Positions_groupAndSort___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__3___closed__6; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_isFunInductName___lambda__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_Tactic_FunInd_buildInductionBody___spec__34(lean_object*); @@ -1226,7 +1219,6 @@ static lean_object* l_Lean_Tactic_FunInd_withLetDecls___rarg___closed__1; static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___lambda__3___closed__4; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__5___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_deriveUnaryInduction___lambda__12___closed__2; -static lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__1; lean_object* l_Lean_mkFreshFVarId___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Tactic_FunInd_buildInductionBody___closed__2; LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_foldAndCollect___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -42536,7 +42528,7 @@ return x_33; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___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) { _start: { lean_object* x_8; @@ -42544,7 +42536,7 @@ x_8 = l_Lean_MVarId_getType(x_1, x_3, x_4, x_5, x_6, x_7); return x_8; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1() { _start: { lean_object* x_1; @@ -42552,7 +42544,7 @@ x_1 = lean_mk_string_unchecked("case", 4, 4); return x_1; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___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_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___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_7; uint8_t x_8; @@ -42569,14 +42561,14 @@ x_12 = lean_nat_add(x_4, x_9); lean_dec(x_4); lean_inc(x_12); x_13 = l___private_Init_Data_Repr_0__Nat_reprFast(x_12); -x_14 = l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1; +x_14 = l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1; x_15 = lean_string_append(x_14, x_13); lean_dec(x_13); x_16 = l_Lean_Tactic_FunInd_removeLamda___rarg___lambda__2___closed__3; x_17 = lean_string_append(x_15, x_16); x_18 = lean_box(0); x_19 = l_Lean_Name_str___override(x_18, x_17); -x_20 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1___boxed), 7, 1); +x_20 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1___boxed), 7, 1); lean_closure_set(x_20, 0, x_11); x_21 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_21, 0, x_19); @@ -42881,208 +42873,6 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__6(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; size_t x_8; size_t x_9; uint8_t x_10; -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 = 1; -x_9 = lean_usize_add(x_2, x_8); -x_10 = !lean_is_exclusive(x_5); -if (x_10 == 0) -{ -lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = lean_ctor_get(x_5, 0); -x_12 = 0; -x_13 = lean_box(x_12); -lean_ctor_set(x_5, 0, x_13); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_11); -lean_ctor_set(x_14, 1, x_5); -x_15 = lean_array_uset(x_7, x_2, x_14); -x_2 = x_9; -x_3 = x_15; -goto _start; -} -else -{ -lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_17 = lean_ctor_get(x_5, 0); -x_18 = lean_ctor_get(x_5, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_5); -x_19 = 0; -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_18); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_17); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_array_uset(x_7, x_2, x_22); -x_2 = x_9; -x_3 = x_23; -goto _start; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8___rarg___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_array_push(x_1, x_5); -x_12 = l_Lean_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8___rarg(x_2, x_3, x_4, x_11, x_6, x_7, x_8, x_9, x_10); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8___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; uint8_t x_12; -x_10 = lean_array_get_size(x_4); -x_11 = lean_array_get_size(x_1); -x_12 = lean_nat_dec_lt(x_10, x_11); -lean_dec(x_11); -if (x_12 == 0) -{ -lean_object* x_13; -lean_dec(x_10); -lean_dec(x_3); -lean_dec(x_1); -x_13 = lean_apply_6(x_2, x_4, x_5, x_6, x_7, x_8, x_9); -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; -x_14 = lean_array_fget(x_1, x_10); -lean_dec(x_10); -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 0); -lean_inc(x_16); -lean_dec(x_14); -x_17 = lean_ctor_get(x_15, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_dec(x_15); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_19 = lean_apply_6(x_18, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; uint8_t 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 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8___rarg___lambda__1), 10, 4); -lean_closure_set(x_22, 0, x_4); -lean_closure_set(x_22, 1, x_1); -lean_closure_set(x_22, 2, x_2); -lean_closure_set(x_22, 3, x_3); -x_23 = 0; -x_24 = lean_unbox(x_17); -lean_dec(x_17); -x_25 = l_Lean_Meta_withLocalDecl___at_Lean_Meta_forallTelescopeCompatibleAux___spec__15___rarg(x_16, x_24, x_20, x_22, x_23, x_5, x_6, x_7, x_8, x_21); -return x_25; -} -else -{ -uint8_t x_26; -lean_dec(x_17); -lean_dec(x_16); -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_19); -if (x_26 == 0) -{ -return x_19; -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_19, 0); -x_28 = lean_ctor_get(x_19, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_19); -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_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8___rarg), 9, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__7___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 = l_Lean_Tactic_FunInd_M_run___rarg___closed__1; -x_10 = l_Lean_Meta_withLocalDecls_loop___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__8___rarg(x_2, x_3, x_1, x_9, x_4, x_5, x_6, x_7, x_8); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__7(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__7___rarg), 8, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__5___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: -{ -size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_array_size(x_2); -x_10 = 0; -x_11 = l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__6(x_9, x_10, x_2); -x_12 = l_Lean_Meta_withLocalDecls___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__7___rarg(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__5(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDeclsD___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__5___rarg), 8, 0); -return x_2; -} -} LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_abstractIndependentMVars___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_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { @@ -43116,14 +42906,14 @@ lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean x_10 = lean_array_get_size(x_1); x_11 = lean_mk_empty_array_with_capacity(x_10); x_12 = lean_unsigned_to_nat(0u); -x_13 = l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2(x_1, x_1, x_10, x_12, lean_box(0), x_11); +x_13 = l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2(x_1, x_1, x_10, x_12, lean_box(0), x_11); x_14 = lean_box_usize(x_2); x_15 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda__1___boxed), 9, 3); lean_closure_set(x_15, 0, x_1); lean_closure_set(x_15, 1, x_14); lean_closure_set(x_15, 2, x_3); x_16 = l_Lean_instInhabitedExpr; -x_17 = l_Lean_Meta_withLocalDeclsD___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__5___rarg(x_16, x_13, x_15, x_5, x_6, x_7, x_8, x_9); +x_17 = l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(x_16, x_13, x_15, x_5, x_6, x_7, x_8, x_9); return x_17; } } @@ -43438,11 +43228,11 @@ x_12 = l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_abstractIndependentMVars__ return x_12; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___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) { _start: { lean_object* x_8; -x_8 = l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___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); @@ -43451,11 +43241,11 @@ lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___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_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_2); lean_dec(x_1); return x_7; @@ -43490,18 +43280,6 @@ lean_dec(x_1); return x_12; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__6___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_6 = l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__6(x_4, x_5, x_3); -return x_6; -} -} LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_abstractIndependentMVars___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: { @@ -52927,7 +52705,7 @@ return x_35; } } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1() { _start: { lean_object* x_1; @@ -52935,7 +52713,7 @@ x_1 = lean_mk_string_unchecked("motive_", 7, 7); return x_1; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___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, 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_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___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, 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; @@ -52960,7 +52738,7 @@ x_21 = lean_nat_add(x_5, x_15); lean_dec(x_5); lean_inc(x_21); x_22 = l___private_Init_Data_Repr_0__Nat_reprFast(x_21); -x_23 = l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1; +x_23 = l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1; x_24 = lean_string_append(x_23, x_22); lean_dec(x_22); x_25 = l_Lean_Tactic_FunInd_removeLamda___rarg___lambda__2___closed__3; @@ -60948,7 +60726,7 @@ lean_dec(x_25); x_28 = lean_array_get_size(x_23); x_29 = lean_mk_empty_array_with_capacity(x_28); x_30 = lean_unsigned_to_nat(0u); -x_31 = l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9(x_5, x_23, x_23, x_28, x_30, lean_box(0), x_29, x_17, x_18, x_19, x_20, x_27); +x_31 = l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9(x_5, x_23, x_23, x_28, x_30, lean_box(0), x_29, x_17, x_18, x_19, x_20, x_27); lean_dec(x_23); x_32 = lean_ctor_get(x_31, 0); lean_inc(x_32); @@ -60976,7 +60754,7 @@ lean_closure_set(x_36, 14, x_26); lean_closure_set(x_36, 15, x_15); lean_closure_set(x_36, 16, x_16); x_37 = l_Lean_instInhabitedExpr; -x_38 = l_Lean_Meta_withLocalDeclsD___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__5___rarg(x_37, x_32, x_36, x_17, x_18, x_19, x_20, x_33); +x_38 = l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(x_37, x_32, x_36, x_17, x_18, x_19, x_20, x_33); return x_38; } else @@ -63513,11 +63291,11 @@ lean_dec(x_1); return x_12; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___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, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___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, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; -x_13 = l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9(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 = l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9(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); @@ -65073,7 +64851,7 @@ lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { uint8_t x_5; lean_object* x_6; lean_object* x_7; @@ -65085,15 +64863,15 @@ lean_ctor_set(x_7, 1, x_4); return x_7; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__1() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__1___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__1___boxed), 4, 0); return x_1; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__2() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__2() { _start: { uint8_t x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; @@ -65118,7 +64896,7 @@ lean_ctor_set_uint8(x_5, 12, x_2); return x_5; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__3() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__3() { _start: { lean_object* x_1; @@ -65126,17 +64904,17 @@ x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); return x_1; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__3; +x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___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_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__5() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -65145,23 +64923,23 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__6() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__5; +x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___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_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__7() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___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_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__6; -x_3 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__5; +x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__6; +x_3 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___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); @@ -65172,25 +64950,25 @@ lean_ctor_set_usize(x_5, 4, x_1); return x_5; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__8() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4; -x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__7; +x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__4; +x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____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; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__9() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__9() { _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; x_1 = lean_box(0); -x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__2; -x_3 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__8; +x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__2; +x_3 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__8; x_4 = l_Lean_Tactic_FunInd_M_run___rarg___closed__1; x_5 = lean_unsigned_to_nat(0u); x_6 = 0; @@ -65206,12 +64984,12 @@ lean_ctor_set_uint8(x_7, sizeof(void*)*6 + 1, x_6); return x_7; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__10() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_unsigned_to_nat(0u); -x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4; +x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__4; x_3 = lean_alloc_ctor(0, 9, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_1); @@ -65225,22 +65003,22 @@ lean_ctor_set(x_3, 8, x_2); return x_3; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__11() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__11() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4; +x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__4; 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_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__12() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4; +x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__4; x_2 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_2, 0, x_1); lean_ctor_set(x_2, 1, x_1); @@ -65249,13 +65027,13 @@ lean_ctor_set(x_2, 3, x_1); return x_2; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__13() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__11; -x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4; -x_3 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__12; +x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__11; +x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__4; +x_3 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__12; x_4 = lean_alloc_ctor(0, 7, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -65267,11 +65045,11 @@ lean_ctor_set(x_4, 6, x_3); return x_4; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__14() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__14() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4; +x_1 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__4; x_2 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_2, 0, x_1); lean_ctor_set(x_2, 1, x_1); @@ -65280,15 +65058,15 @@ lean_ctor_set(x_2, 3, x_1); return x_2; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__15() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__15() { _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_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__10; -x_3 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__13; -x_4 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__7; -x_5 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__14; +x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__10; +x_3 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__13; +x_4 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__7; +x_5 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__14; x_6 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_6, 0, x_2); lean_ctor_set(x_6, 1, x_3); @@ -65298,7 +65076,7 @@ lean_ctor_set(x_6, 4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; uint8_t x_6; @@ -65312,7 +65090,7 @@ x_8 = lean_ctor_get(x_5, 1); x_9 = lean_ctor_get(x_7, 0); lean_inc(x_9); lean_dec(x_7); -x_10 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__1; +x_10 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__1; lean_inc(x_1); x_11 = l_Lean_Tactic_FunInd_isFunInductName(x_9, x_1); lean_dec(x_9); @@ -65336,14 +65114,14 @@ lean_free_object(x_5); x_15 = lean_ctor_get(x_1, 0); lean_inc(x_15); lean_dec(x_1); -x_16 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__15; +x_16 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__15; x_17 = lean_st_mk_ref(x_16, x_8); 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_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__9; +x_20 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__9; lean_inc(x_18); x_21 = l_Lean_Tactic_FunInd_deriveInduction(x_15, x_20, x_18, x_2, x_3, x_19); if (lean_obj_tag(x_21) == 0) @@ -65427,7 +65205,7 @@ lean_dec(x_5); x_40 = lean_ctor_get(x_38, 0); lean_inc(x_40); lean_dec(x_38); -x_41 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__1; +x_41 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__1; lean_inc(x_1); x_42 = l_Lean_Tactic_FunInd_isFunInductName(x_40, x_1); lean_dec(x_40); @@ -65449,14 +65227,14 @@ lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean x_46 = lean_ctor_get(x_1, 0); lean_inc(x_46); lean_dec(x_1); -x_47 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__15; +x_47 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__15; x_48 = lean_st_mk_ref(x_47, x_39); 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 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__9; +x_51 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__9; lean_inc(x_49); x_52 = l_Lean_Tactic_FunInd_deriveInduction(x_46, x_51, x_49, x_2, x_3, x_50); if (lean_obj_tag(x_52) == 0) @@ -65531,7 +65309,7 @@ return x_66; } } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__1() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____closed__1() { _start: { lean_object* x_1; @@ -65539,19 +65317,19 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_isFunInductName___boxed), return x_1; } } -static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__2() { +static lean_object* _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2), 4, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__1; +x_2 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____closed__1; x_3 = l_Lean_registerReservedNamePredicate(x_2, x_1); if (lean_obj_tag(x_3) == 0) { @@ -65559,7 +65337,7 @@ lean_object* x_4; lean_object* x_5; lean_object* x_6; x_4 = lean_ctor_get(x_3, 1); lean_inc(x_4); lean_dec(x_3); -x_5 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__2; +x_5 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____closed__2; x_6 = l_Lean_registerReservedNameAction(x_5, x_4); return x_6; } @@ -65587,18 +65365,18 @@ return x_10; } } } -LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__1___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_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); return x_5; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__1() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__1() { _start: { lean_object* x_1; @@ -65606,17 +65384,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__2() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__1; +x_2 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__3() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__3() { _start: { lean_object* x_1; @@ -65624,17 +65402,17 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__4() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__2; -x_2 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__3; +x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__2; +x_2 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__5() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__5() { _start: { lean_object* x_1; @@ -65642,47 +65420,47 @@ x_1 = lean_mk_string_unchecked("Lean", 4, 4); return x_1; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__6() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__4; -x_2 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__5; +x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__4; +x_2 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__7() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__6; +x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__6; x_2 = l_Lean_Tactic_FunInd_buildInductionCase___closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__8() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__7; +x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__7; x_2 = l_Lean_logAt___at_Lean_Tactic_FunInd_buildInductionBody___spec__41___lambda__2___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__9() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__8; +x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__8; x_2 = l_Lean_Tactic_FunInd_buildInductionCase___closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__10() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__10() { _start: { lean_object* x_1; @@ -65690,33 +65468,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__11() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__9; -x_2 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__10; +x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__9; +x_2 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__10; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__12() { +static lean_object* _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__11; -x_2 = lean_unsigned_to_nat(16616u); +x_1 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__11; +x_2 = lean_unsigned_to_nat(16594u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594_(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_Tactic_FunInd_buildInductionCase___closed__5; x_3 = 0; -x_4 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__12; +x_4 = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__12; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -65991,8 +65769,8 @@ l_Lean_Tactic_FunInd_buildInductionBody___closed__1 = _init_l_Lean_Tactic_FunInd lean_mark_persistent(l_Lean_Tactic_FunInd_buildInductionBody___closed__1); l_Lean_Tactic_FunInd_buildInductionBody___closed__2 = _init_l_Lean_Tactic_FunInd_buildInductionBody___closed__2(); lean_mark_persistent(l_Lean_Tactic_FunInd_buildInductionBody___closed__2); -l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1 = _init_l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1); +l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1 = _init_l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_abstractIndependentMVars___spec__2___closed__1); l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda__3___closed__1 = _init_l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda__3___closed__1(); lean_mark_persistent(l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda__3___closed__1); l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda__3___closed__2 = _init_l_Lean_Tactic_FunInd_abstractIndependentMVars___lambda__3___closed__2(); @@ -66183,8 +65961,8 @@ l_Lean_Elab_Structural_Positions_groupAndSort___at_Lean_Tactic_FunInd_deriveIndu lean_mark_persistent(l_Lean_Elab_Structural_Positions_groupAndSort___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__3___closed__6); l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__8___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__8___closed__1(); lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__8___closed__1); -l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1 = _init_l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1); +l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1 = _init_l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__9___closed__1); l_panic___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__13___closed__1 = _init_l_panic___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__13___closed__1(); lean_mark_persistent(l_panic___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__13___closed__1); l_Lean_Elab_Structural_Positions_mapMwith___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__12___closed__1 = _init_l_Lean_Elab_Structural_Positions_mapMwith___at_Lean_Tactic_FunInd_deriveInductionStructural___spec__12___closed__1(); @@ -66321,68 +66099,68 @@ l_Lean_Tactic_FunInd_isFunInductName___lambda__2___closed__1 = _init_l_Lean_Tact lean_mark_persistent(l_Lean_Tactic_FunInd_isFunInductName___lambda__2___closed__1); l_Lean_Tactic_FunInd_isFunInductName___lambda__2___closed__2 = _init_l_Lean_Tactic_FunInd_isFunInductName___lambda__2___closed__2(); lean_mark_persistent(l_Lean_Tactic_FunInd_isFunInductName___lambda__2___closed__2); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__1 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__1); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__2 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__2); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__3 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__3(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__3); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__4); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__5 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__5(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__5); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__6 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__6(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__6); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__7 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__7(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__7); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__8 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__8(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__8); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__9 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__9(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__9); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__10 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__10(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__10); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__11 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__11(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__11); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__12 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__12(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__12); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__13 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__13(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__13); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__14 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__14(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__14); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__15 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__15(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____lambda__2___closed__15); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__1 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__1(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__1); -l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__2 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__2(); -lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470____closed__2); -if (builtin) {res = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16470_(lean_io_mk_world()); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__1 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__1); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__2 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__2); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__3 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__3); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__4 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__4(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__4); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__5 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__5(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__5); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__6 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__6(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__6); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__7 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__7(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__7); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__8 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__8(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__8); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__9 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__9(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__9); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__10 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__10(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__10); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__11 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__11(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__11); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__12 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__12(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__12); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__13 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__13(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__13); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__14 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__14(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__14); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__15 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__15(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____lambda__2___closed__15); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____closed__1 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____closed__1(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____closed__1); +l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____closed__2 = _init_l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____closed__2(); +lean_mark_persistent(l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448____closed__2); +if (builtin) {res = l_Lean_Tactic_FunInd_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16448_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__1 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__1(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__1); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__2 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__2(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__2); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__3 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__3(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__3); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__4 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__4(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__4); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__5 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__5(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__5); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__6 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__6(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__6); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__7 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__7(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__7); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__8 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__8(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__8); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__9 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__9(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__9); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__10 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__10(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__10); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__11 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__11(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__11); -l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__12 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__12(); -lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616____closed__12); -if (builtin) {res = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16616_(lean_io_mk_world()); +}l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__1 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__1(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__1); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__2 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__2(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__2); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__3 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__3(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__3); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__4 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__4(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__4); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__5 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__5(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__5); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__6 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__6(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__6); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__7 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__7(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__7); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__8 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__8(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__8); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__9 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__9(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__9); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__10 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__10(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__10); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__11 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__11(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__11); +l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__12 = _init_l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__12(); +lean_mark_persistent(l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594____closed__12); +if (builtin) {res = l_initFn____x40_Lean_Meta_Tactic_FunInd___hyg_16594_(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/LinearArith/Nat/Simp.c b/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Simp.c index 2ae55d3c7f2a..f8cbf25be59b 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Simp.c +++ b/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Simp.c @@ -16,73 +16,91 @@ extern "C" { 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; lean_object* l_Lean_Meta_Linear_Nat_toContextExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__9; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f(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__7; 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*); -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__10; uint8_t l_Lean_Expr_isAppOfArity(lean_object*, lean_object*, 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_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_simpCnstrPos_x3f___closed__15; 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; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__2; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__3; +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_mkApp4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__8; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__13; +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*); +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; lean_object* l_Nat_Linear_PolyCnstr_norm(lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__3; uint8_t l_Nat_Linear_PolyCnstr_isUnsat(lean_object*); +static lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg___closed__1; 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; +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_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; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__14; 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*); extern lean_object* l_Lean_levelZero; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__12; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__14; lean_object* l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(lean_object*); lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__4; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__9; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__5; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__18; +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*); 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; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__11; +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; 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*); -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__4; +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__9; +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; @@ -90,13 +108,25 @@ lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__17; lean_object* l_Nat_Linear_PolyCnstr_toExpr(lean_object*); lean_object* l_Nat_Linear_ExprCnstr_toPoly(lean_object*); -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__7; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__17; +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_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; +static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__3; +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__1; +lean_object* lean_array_mk(lean_object*); +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__13; +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__2; +lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__2___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__4; +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*); 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; @@ -104,12 +134,18 @@ static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__2 lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Nat_Linear_PolyCnstr_isValid(lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__8; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__16; +lean_object* lean_array_get_size(lean_object*); +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__10; +static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__1; +uint8_t lean_usize_dec_lt(size_t, size_t); +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*); +static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__3; 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; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__6; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__12; -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1() { +lean_object* l_Lean_Expr_beta(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* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1() { _start: { lean_object* x_1; @@ -117,83 +153,907 @@ x_1 = lean_mk_string_unchecked("Nat", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__2() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Linear", 6, 6); -return x_1; +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_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___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_Meta_Linear_Nat_withAbstractAtoms___spec__1___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_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___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_Linear_Nat_simpCnstrPos_x3f___closed__3() { +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___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) { +_start: +{ +lean_object* x_7; lean_object* x_8; +x_7 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__3; +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_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("ExprCnstr", 9, 9); +x_1 = lean_mk_string_unchecked("x", 1, 1); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__4() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___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_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___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_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("eq_of_toNormPoly_eq", 19, 19); +x_1 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___boxed), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__5() { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___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: { -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_Linear_Nat_simpCnstrPos_x3f___closed__1; -x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__2; -x_3 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__3; -x_4 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__4; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +uint8_t x_9; +x_9 = lean_usize_dec_lt(x_2, x_1); +if (x_9 == 0) +{ +lean_object* x_10; +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; uint8_t x_15; +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_3, x_2, x_11); +x_13 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__2; +x_14 = l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(x_13, x_6, x_7, x_8); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; size_t x_18; size_t x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_14, 1); +x_17 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__3; +lean_ctor_set(x_14, 1, x_17); +x_18 = 1; +x_19 = lean_usize_add(x_2, x_18); +x_20 = lean_array_uset(x_12, x_2, x_14); +x_2 = x_19; +x_3 = x_20; +x_8 = x_16; +goto _start; } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__6() { +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; size_t x_26; size_t x_27; lean_object* x_28; +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 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__3; +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_22); +lean_ctor_set(x_25, 1, x_24); +x_26 = 1; +x_27 = lean_usize_add(x_2, x_26); +x_28 = lean_array_uset(x_12, x_2, x_25); +x_2 = x_27; +x_3 = x_28; +x_8 = x_23; +goto _start; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__3(size_t x_1, size_t x_2, lean_object* x_3) { _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_simpCnstrPos_x3f___closed__5; -x_3 = l_Lean_Expr_const___override(x_2, x_1); +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; size_t x_8; size_t x_9; uint8_t x_10; +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 = 1; +x_9 = lean_usize_add(x_2, x_8); +x_10 = !lean_is_exclusive(x_5); +if (x_10 == 0) +{ +lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_11 = lean_ctor_get(x_5, 0); +x_12 = 0; +x_13 = lean_box(x_12); +lean_ctor_set(x_5, 0, x_13); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_11); +lean_ctor_set(x_14, 1, x_5); +x_15 = lean_array_uset(x_7, x_2, x_14); +x_2 = x_9; +x_3 = x_15; +goto _start; +} +else +{ +lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_17 = lean_ctor_get(x_5, 0); +x_18 = lean_ctor_get(x_5, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_5); +x_19 = 0; +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_18); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_17); +lean_ctor_set(x_22, 1, x_21); +x_23 = lean_array_uset(x_7, x_2, x_22); +x_2 = x_9; +x_3 = x_23; +goto _start; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5___rarg___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_array_push(x_1, x_5); +x_12 = l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5___rarg(x_2, x_3, x_4, x_11, x_6, x_7, x_8, x_9, x_10); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5___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; uint8_t x_12; +x_10 = lean_array_get_size(x_4); +x_11 = lean_array_get_size(x_1); +x_12 = lean_nat_dec_lt(x_10, x_11); +lean_dec(x_11); +if (x_12 == 0) +{ +lean_object* x_13; +lean_dec(x_10); +lean_dec(x_3); +lean_dec(x_1); +x_13 = lean_apply_6(x_2, x_4, x_5, x_6, x_7, x_8, x_9); +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; +x_14 = lean_array_fget(x_1, x_10); +lean_dec(x_10); +x_15 = lean_ctor_get(x_14, 1); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_dec(x_14); +x_17 = lean_ctor_get(x_15, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_15, 1); +lean_inc(x_18); +lean_dec(x_15); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_19 = lean_apply_6(x_18, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; uint8_t 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 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5___rarg___lambda__1), 10, 4); +lean_closure_set(x_22, 0, x_4); +lean_closure_set(x_22, 1, x_1); +lean_closure_set(x_22, 2, x_2); +lean_closure_set(x_22, 3, x_3); +x_23 = 0; +x_24 = lean_unbox(x_17); +lean_dec(x_17); +x_25 = l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__2___rarg(x_16, x_24, x_20, x_22, x_23, x_5, x_6, x_7, x_8, x_21); +return x_25; +} +else +{ +uint8_t x_26; +lean_dec(x_17); +lean_dec(x_16); +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_19); +if (x_26 == 0) +{ +return x_19; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_19, 0); +x_28 = lean_ctor_get(x_19, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_19); +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_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5___rarg), 9, 0); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg___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_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___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) { +_start: +{ +lean_object* x_9; lean_object* x_10; +x_9 = l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg___closed__1; +x_10 = l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5___rarg(x_2, x_3, x_1, x_9, x_4, x_5, x_6, x_7, x_8); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg), 8, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___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: +{ +size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_array_size(x_2); +x_10 = 0; +x_11 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__3(x_9, x_10, x_2); +x_12 = l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg), 8, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_withAbstractAtoms___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_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_10 = lean_apply_6(x_1, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_10) == 0) +{ +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_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +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_2); +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_2); +lean_ctor_set(x_15, 1, x_14); +return x_15; +} +} +else +{ +uint8_t x_16; +lean_dec(x_2); +x_16 = !lean_is_exclusive(x_11); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_17 = lean_ctor_get(x_11, 0); +x_18 = lean_ctor_get(x_10, 1); +lean_inc(x_18); +lean_dec(x_10); +x_19 = !lean_is_exclusive(x_17); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; uint8_t x_22; uint8_t x_23; uint8_t x_24; lean_object* x_25; +x_20 = lean_ctor_get(x_17, 0); +x_21 = lean_ctor_get(x_17, 1); +x_22 = 0; +x_23 = 1; +x_24 = 1; +lean_inc(x_4); +x_25 = l_Lean_Meta_mkLambdaFVars(x_4, x_20, x_22, x_23, x_22, x_24, x_5, x_6, x_7, x_8, x_18); +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, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +lean_inc(x_3); +x_28 = l_Lean_Expr_beta(x_26, x_3); +x_29 = l_Lean_Meta_mkLambdaFVars(x_4, x_21, x_22, x_23, x_22, x_24, x_5, x_6, x_7, x_8, x_27); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +if (lean_obj_tag(x_29) == 0) +{ +uint8_t x_30; +x_30 = !lean_is_exclusive(x_29); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; +x_31 = lean_ctor_get(x_29, 0); +x_32 = l_Lean_mkAppN(x_31, x_3); +lean_dec(x_3); +lean_ctor_set(x_17, 1, x_32); +lean_ctor_set(x_17, 0, x_28); +lean_ctor_set(x_29, 0, x_11); +return x_29; +} +else +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_33 = lean_ctor_get(x_29, 0); +x_34 = lean_ctor_get(x_29, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_29); +x_35 = l_Lean_mkAppN(x_33, x_3); +lean_dec(x_3); +lean_ctor_set(x_17, 1, x_35); +lean_ctor_set(x_17, 0, x_28); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_11); +lean_ctor_set(x_36, 1, x_34); +return x_36; +} +} +else +{ +uint8_t x_37; +lean_dec(x_28); +lean_free_object(x_17); +lean_free_object(x_11); +lean_dec(x_3); +x_37 = !lean_is_exclusive(x_29); +if (x_37 == 0) +{ +return x_29; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; +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_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_free_object(x_17); +lean_dec(x_21); +lean_free_object(x_11); +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_25); +if (x_41 == 0) +{ +return x_25; +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_25, 0); +x_43 = lean_ctor_get(x_25, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_25); +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; uint8_t x_47; uint8_t x_48; uint8_t x_49; lean_object* x_50; +x_45 = lean_ctor_get(x_17, 0); +x_46 = lean_ctor_get(x_17, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_17); +x_47 = 0; +x_48 = 1; +x_49 = 1; +lean_inc(x_4); +x_50 = l_Lean_Meta_mkLambdaFVars(x_4, x_45, x_47, x_48, x_47, x_49, x_5, x_6, x_7, x_8, x_18); +if (lean_obj_tag(x_50) == 0) +{ +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +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); +lean_inc(x_3); +x_53 = l_Lean_Expr_beta(x_51, x_3); +x_54 = l_Lean_Meta_mkLambdaFVars(x_4, x_46, x_47, x_48, x_47, x_49, x_5, x_6, x_7, x_8, x_52); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +if (lean_obj_tag(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; +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); +} +x_58 = l_Lean_mkAppN(x_55, x_3); +lean_dec(x_3); +x_59 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_59, 0, x_53); +lean_ctor_set(x_59, 1, x_58); +lean_ctor_set(x_11, 0, x_59); +if (lean_is_scalar(x_57)) { + x_60 = lean_alloc_ctor(0, 2, 0); +} else { + x_60 = x_57; +} +lean_ctor_set(x_60, 0, x_11); +lean_ctor_set(x_60, 1, x_56); +return x_60; +} +else +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +lean_dec(x_53); +lean_free_object(x_11); +lean_dec(x_3); +x_61 = lean_ctor_get(x_54, 0); +lean_inc(x_61); +x_62 = lean_ctor_get(x_54, 1); +lean_inc(x_62); +if (lean_is_exclusive(x_54)) { + lean_ctor_release(x_54, 0); + lean_ctor_release(x_54, 1); + x_63 = x_54; +} else { + lean_dec_ref(x_54); + 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_46); +lean_free_object(x_11); +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_50, 0); +lean_inc(x_65); +x_66 = lean_ctor_get(x_50, 1); +lean_inc(x_66); +if (lean_is_exclusive(x_50)) { + lean_ctor_release(x_50, 0); + lean_ctor_release(x_50, 1); + x_67 = x_50; +} else { + lean_dec_ref(x_50); + 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_object* x_71; lean_object* x_72; lean_object* x_73; uint8_t x_74; uint8_t x_75; uint8_t x_76; lean_object* x_77; +x_69 = lean_ctor_get(x_11, 0); +lean_inc(x_69); +lean_dec(x_11); +x_70 = lean_ctor_get(x_10, 1); +lean_inc(x_70); +lean_dec(x_10); +x_71 = lean_ctor_get(x_69, 0); +lean_inc(x_71); +x_72 = lean_ctor_get(x_69, 1); +lean_inc(x_72); +if (lean_is_exclusive(x_69)) { + lean_ctor_release(x_69, 0); + lean_ctor_release(x_69, 1); + x_73 = x_69; +} else { + lean_dec_ref(x_69); + x_73 = lean_box(0); +} +x_74 = 0; +x_75 = 1; +x_76 = 1; +lean_inc(x_4); +x_77 = l_Lean_Meta_mkLambdaFVars(x_4, x_71, x_74, x_75, x_74, x_76, x_5, x_6, x_7, x_8, x_70); +if (lean_obj_tag(x_77) == 0) +{ +lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +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); +lean_inc(x_3); +x_80 = l_Lean_Expr_beta(x_78, x_3); +x_81 = l_Lean_Meta_mkLambdaFVars(x_4, x_72, x_74, x_75, x_74, x_76, x_5, x_6, x_7, x_8, x_79); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +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; +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); +} +x_85 = l_Lean_mkAppN(x_82, x_3); +lean_dec(x_3); +if (lean_is_scalar(x_73)) { + x_86 = lean_alloc_ctor(0, 2, 0); +} else { + x_86 = x_73; +} +lean_ctor_set(x_86, 0, x_80); +lean_ctor_set(x_86, 1, x_85); +x_87 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_87, 0, x_86); +if (lean_is_scalar(x_84)) { + x_88 = lean_alloc_ctor(0, 2, 0); +} else { + x_88 = x_84; +} +lean_ctor_set(x_88, 0, x_87); +lean_ctor_set(x_88, 1, x_83); +return x_88; +} +else +{ +lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; +lean_dec(x_80); +lean_dec(x_73); +lean_dec(x_3); +x_89 = lean_ctor_get(x_81, 0); +lean_inc(x_89); +x_90 = lean_ctor_get(x_81, 1); +lean_inc(x_90); +if (lean_is_exclusive(x_81)) { + lean_ctor_release(x_81, 0); + lean_ctor_release(x_81, 1); + x_91 = x_81; +} else { + lean_dec_ref(x_81); + x_91 = lean_box(0); } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__7() { +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; +} +} +else +{ +lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; +lean_dec(x_73); +lean_dec(x_72); +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_93 = lean_ctor_get(x_77, 0); +lean_inc(x_93); +x_94 = lean_ctor_get(x_77, 1); +lean_inc(x_94); +if (lean_is_exclusive(x_77)) { + lean_ctor_release(x_77, 0); + lean_ctor_release(x_77, 1); + x_95 = x_77; +} else { + lean_dec_ref(x_77); + 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 +{ +uint8_t x_97; +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_97 = !lean_is_exclusive(x_10); +if (x_97 == 0) +{ +return x_10; +} +else +{ +lean_object* x_98; lean_object* x_99; lean_object* x_100; +x_98 = lean_ctor_get(x_10, 0); +x_99 = lean_ctor_get(x_10, 1); +lean_inc(x_99); +lean_inc(x_98); +lean_dec(x_10); +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_EXPORT lean_object* l_Lean_Meta_Linear_Nat_withAbstractAtoms(lean_object* x_1, 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; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_8 = lean_array_size(x_1); +x_9 = 0; +lean_inc(x_1); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1(x_8, x_9, x_1, x_3, x_4, x_5, x_6, x_7); +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_closure((void*)(l_Lean_Meta_Linear_Nat_withAbstractAtoms___lambda__1), 9, 3); +lean_closure_set(x_14, 0, x_2); +lean_closure_set(x_14, 1, x_13); +lean_closure_set(x_14, 2, x_1); +x_15 = l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(x_13, x_11, x_14, x_3, x_4, x_5, x_6, x_12); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___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) { +_start: +{ +lean_object* x_7; +x_7 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___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); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___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_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1(x_9, x_10, 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); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___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_6 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__3(x_4, x_5, x_3); +return x_6; +} +} +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("eq_true_of_isValid", 18, 18); +x_1 = lean_mk_string_unchecked("Linear", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ExprCnstr", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__8() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("eq_of_toNormPoly_eq", 19, 19); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___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; -x_1 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1; -x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__2; -x_3 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__3; -x_4 = l_Lean_Meta_Linear_Nat_simpCnstrPos_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_simpCnstrPos_x3f___lambda__1___closed__1; +x_3 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__2; +x_4 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___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_Linear_Nat_simpCnstrPos_x3f___closed__9() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___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_Meta_Linear_Nat_simpCnstrPos_x3f___closed__8; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__4; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__10() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__6() { _start: { lean_object* x_1; @@ -201,57 +1061,57 @@ x_1 = lean_mk_string_unchecked("True", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__11() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___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_Meta_Linear_Nat_simpCnstrPos_x3f___closed__10; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__12() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___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_Meta_Linear_Nat_simpCnstrPos_x3f___closed__11; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__7; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__13() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__9() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("eq_false_of_isUnsat", 19, 19); +x_1 = lean_mk_string_unchecked("eq_true_of_isValid", 18, 18); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__14() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___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; -x_1 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1; -x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__2; -x_3 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__3; -x_4 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__13; +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_simpCnstrPos_x3f___lambda__1___closed__1; +x_3 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__2; +x_4 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___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_Linear_Nat_simpCnstrPos_x3f___closed__15() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___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_Meta_Linear_Nat_simpCnstrPos_x3f___closed__14; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__10; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__16() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__12() { _start: { lean_object* x_1; @@ -259,381 +1119,418 @@ x_1 = lean_mk_string_unchecked("False", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__17() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___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_Linear_Nat_simpCnstrPos_x3f___closed__16; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__18() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___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_Linear_Nat_simpCnstrPos_x3f___closed__17; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__13; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_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) { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__15() { _start: { -lean_object* x_7; lean_object* x_8; -lean_inc(x_1); -x_7 = lean_alloc_closure((void*)(l_Lean_Meta_Linear_Nat_ToLinear_toLinearCnstr_x3f), 7, 1); -lean_closure_set(x_7, 0, x_1); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_8 = l_Lean_Meta_Linear_Nat_ToLinear_run___rarg(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; -x_9 = lean_ctor_get(x_8, 0); -lean_inc(x_9); -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_9); -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_8); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; -x_12 = lean_ctor_get(x_8, 0); -lean_dec(x_12); -x_13 = lean_box(0); -lean_ctor_set(x_8, 0, x_13); -return x_8; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("eq_false_of_isUnsat", 19, 19); +return x_1; } -else +} +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__16() { +_start: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_8, 1); -lean_inc(x_14); -lean_dec(x_8); -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; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +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_simpCnstrPos_x3f___lambda__1___closed__1; +x_3 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__2; +x_4 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__15; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -else +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__17() { +_start: { -lean_object* x_17; uint8_t x_18; -x_17 = lean_ctor_get(x_8, 1); -lean_inc(x_17); -lean_dec(x_8); -x_18 = !lean_is_exclusive(x_9); -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_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__16; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_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) { +_start: { -lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_19 = lean_ctor_get(x_9, 1); -x_20 = lean_ctor_get(x_9, 0); -lean_dec(x_20); -x_21 = !lean_is_exclusive(x_10); -if (x_21 == 0) +lean_object* x_8; uint8_t x_9; +lean_inc(x_1); +x_8 = l_Lean_Meta_Linear_Nat_LinearCnstr_toArith(x_2, x_1, x_3, x_4, x_5, x_6, x_7); +x_9 = !lean_is_exclusive(x_8); +if (x_9 == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_22 = lean_ctor_get(x_10, 0); -lean_inc(x_22); -x_23 = l_Nat_Linear_ExprCnstr_toPoly(x_22); -x_24 = l_Nat_Linear_PolyCnstr_norm(x_23); -x_25 = l_Nat_Linear_PolyCnstr_isUnsat(x_24); -if (x_25 == 0) +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_10 = lean_ctor_get(x_8, 0); +x_11 = lean_ctor_get(x_8, 1); +lean_inc(x_1); +x_12 = l_Nat_Linear_ExprCnstr_toPoly(x_1); +x_13 = l_Nat_Linear_PolyCnstr_norm(x_12); +x_14 = l_Nat_Linear_PolyCnstr_isUnsat(x_13); +if (x_14 == 0) { -uint8_t x_26; -x_26 = l_Nat_Linear_PolyCnstr_isValid(x_24); -if (x_26 == 0) +uint8_t x_15; +x_15 = l_Nat_Linear_PolyCnstr_isValid(x_13); +if (x_15 == 0) { -lean_object* x_27; lean_object* x_28; uint8_t x_29; -x_27 = l_Nat_Linear_PolyCnstr_toExpr(x_24); -lean_inc(x_27); -x_28 = l_Lean_Meta_Linear_Nat_LinearCnstr_toArith(x_19, x_27, x_2, x_3, x_4, x_5, x_17); -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) -{ -lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_30 = lean_ctor_get(x_28, 0); -x_31 = lean_ctor_get(x_28, 1); -x_32 = lean_expr_eqv(x_30, x_1); -if (x_32 == 0) +lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_16 = l_Nat_Linear_PolyCnstr_toExpr(x_13); +lean_inc(x_16); +x_17 = l_Lean_Meta_Linear_Nat_LinearCnstr_toArith(x_2, x_16, x_3, x_4, x_5, x_6, x_11); +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 = lean_ctor_get(x_17, 1); +x_21 = lean_expr_eqv(x_19, x_10); +if (x_21 == 0) { -lean_object* x_33; -lean_free_object(x_28); +lean_object* x_22; +lean_free_object(x_17); +lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -x_33 = l_Lean_Meta_Linear_Nat_toContextExpr(x_19, x_2, x_3, x_4, x_5, x_31); -if (lean_obj_tag(x_33) == 0) +x_22 = l_Lean_Meta_Linear_Nat_toContextExpr(x_2, x_3, x_4, x_5, x_6, x_20); +if (lean_obj_tag(x_22) == 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; -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_Linear_Nat_LinearCnstr_toExpr(x_22); -x_37 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_27); -x_38 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__6; -x_39 = l_Lean_Meta_Linear_Nat_reflTrue; -x_40 = l_Lean_mkApp4(x_38, x_34, x_36, x_37, x_39); +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_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_Linear_Nat_LinearCnstr_toExpr(x_1); +x_26 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_16); +x_27 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__5; +x_28 = l_Lean_Meta_Linear_Nat_reflTrue; +x_29 = l_Lean_mkApp4(x_27, x_23, x_25, x_26, x_28); +lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_30); -x_41 = l_Lean_Meta_mkEq(x_1, x_30, x_2, x_3, x_4, x_5, x_35); -if (lean_obj_tag(x_41) == 0) -{ -lean_object* x_42; lean_object* x_43; lean_object* x_44; -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_Meta_mkExpectedTypeHint(x_40, x_42, x_2, x_3, x_4, x_5, x_43); -if (lean_obj_tag(x_44) == 0) +lean_inc(x_19); +x_30 = l_Lean_Meta_mkEq(x_10, x_19, x_3, x_4, x_5, x_6, x_24); +if (lean_obj_tag(x_30) == 0) { -uint8_t x_45; -x_45 = !lean_is_exclusive(x_44); -if (x_45 == 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); +x_33 = l_Lean_Meta_mkExpectedTypeHint(x_29, x_31, x_3, x_4, x_5, x_6, x_32); +if (lean_obj_tag(x_33) == 0) { -lean_object* x_46; -x_46 = lean_ctor_get(x_44, 0); -lean_ctor_set(x_9, 1, x_46); -lean_ctor_set(x_9, 0, x_30); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set(x_44, 0, x_10); -return x_44; +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, 0); +lean_ctor_set(x_8, 1, x_35); +lean_ctor_set(x_8, 0, x_19); +x_36 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_36, 0, x_8); +lean_ctor_set(x_33, 0, x_36); +return x_33; } else { -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_9, 1, x_47); -lean_ctor_set(x_9, 0, x_30); -lean_ctor_set(x_10, 0, x_9); -x_49 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_49, 0, x_10); -lean_ctor_set(x_49, 1, x_48); -return x_49; +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_37 = lean_ctor_get(x_33, 0); +x_38 = lean_ctor_get(x_33, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_33); +lean_ctor_set(x_8, 1, x_37); +lean_ctor_set(x_8, 0, x_19); +x_39 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_39, 0, x_8); +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_50; -lean_dec(x_30); -lean_free_object(x_10); -lean_free_object(x_9); -x_50 = !lean_is_exclusive(x_44); -if (x_50 == 0) +uint8_t x_41; +lean_dec(x_19); +lean_free_object(x_8); +x_41 = !lean_is_exclusive(x_33); +if (x_41 == 0) { -return x_44; +return x_33; } else { -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; +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_33, 0); +x_43 = lean_ctor_get(x_33, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_33); +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_54; -lean_dec(x_40); -lean_dec(x_30); -lean_free_object(x_10); -lean_free_object(x_9); +uint8_t x_45; +lean_dec(x_29); +lean_dec(x_19); +lean_free_object(x_8); +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_41); -if (x_54 == 0) +x_45 = !lean_is_exclusive(x_30); +if (x_45 == 0) { -return x_41; +return x_30; } 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_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_30, 0); +x_47 = lean_ctor_get(x_30, 1); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_30); +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_58; -lean_dec(x_30); -lean_dec(x_27); -lean_free_object(x_10); -lean_dec(x_22); -lean_free_object(x_9); +uint8_t x_49; +lean_dec(x_19); +lean_dec(x_16); +lean_free_object(x_8); +lean_dec(x_10); +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_33); -if (x_58 == 0) +x_49 = !lean_is_exclusive(x_22); +if (x_49 == 0) { -return x_33; +return x_22; } else { -lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_59 = lean_ctor_get(x_33, 0); -x_60 = lean_ctor_get(x_33, 1); -lean_inc(x_60); -lean_inc(x_59); -lean_dec(x_33); -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_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_22, 0); +x_51 = lean_ctor_get(x_22, 1); +lean_inc(x_51); +lean_inc(x_50); +lean_dec(x_22); +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_62; -lean_dec(x_30); -lean_dec(x_27); -lean_free_object(x_10); -lean_dec(x_22); -lean_free_object(x_9); +lean_object* x_53; lean_dec(x_19); +lean_dec(x_16); +lean_free_object(x_8); +lean_dec(x_10); +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_62 = lean_box(0); -lean_ctor_set(x_28, 0, x_62); -return x_28; +x_53 = lean_box(0); +lean_ctor_set(x_17, 0, x_53); +return x_17; } } else { -lean_object* x_63; lean_object* x_64; uint8_t x_65; -x_63 = lean_ctor_get(x_28, 0); -x_64 = lean_ctor_get(x_28, 1); -lean_inc(x_64); -lean_inc(x_63); -lean_dec(x_28); -x_65 = lean_expr_eqv(x_63, x_1); -if (x_65 == 0) +lean_object* x_54; lean_object* x_55; uint8_t x_56; +x_54 = lean_ctor_get(x_17, 0); +x_55 = lean_ctor_get(x_17, 1); +lean_inc(x_55); +lean_inc(x_54); +lean_dec(x_17); +x_56 = lean_expr_eqv(x_54, x_10); +if (x_56 == 0) { -lean_object* x_66; +lean_object* x_57; +lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -x_66 = l_Lean_Meta_Linear_Nat_toContextExpr(x_19, x_2, x_3, x_4, x_5, x_64); -if (lean_obj_tag(x_66) == 0) +x_57 = l_Lean_Meta_Linear_Nat_toContextExpr(x_2, x_3, x_4, x_5, x_6, x_55); +if (lean_obj_tag(x_57) == 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_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_Meta_Linear_Nat_LinearCnstr_toExpr(x_22); -x_70 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_27); -x_71 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__6; -x_72 = l_Lean_Meta_Linear_Nat_reflTrue; -x_73 = l_Lean_mkApp4(x_71, x_67, x_69, x_70, x_72); +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_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_Linear_Nat_LinearCnstr_toExpr(x_1); +x_61 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_16); +x_62 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__5; +x_63 = l_Lean_Meta_Linear_Nat_reflTrue; +x_64 = l_Lean_mkApp4(x_62, x_58, x_60, x_61, x_63); +lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_63); -x_74 = l_Lean_Meta_mkEq(x_1, x_63, x_2, x_3, x_4, x_5, x_68); -if (lean_obj_tag(x_74) == 0) +lean_inc(x_54); +x_65 = l_Lean_Meta_mkEq(x_10, x_54, x_3, x_4, x_5, x_6, x_59); +if (lean_obj_tag(x_65) == 0) { -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_74, 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_Lean_Meta_mkExpectedTypeHint(x_64, x_66, x_3, x_4, x_5, x_6, 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; +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); +} +lean_ctor_set(x_8, 1, x_69); +lean_ctor_set(x_8, 0, x_54); +x_72 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_72, 0, x_8); +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_dec(x_54); +lean_free_object(x_8); +x_74 = lean_ctor_get(x_68, 0); +lean_inc(x_74); +x_75 = lean_ctor_get(x_68, 1); 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_mkExpectedTypeHint(x_73, x_75, x_2, x_3, x_4, x_5, x_76); -if (lean_obj_tag(x_77) == 0) +if (lean_is_exclusive(x_68)) { + lean_ctor_release(x_68, 0); + lean_ctor_release(x_68, 1); + x_76 = x_68; +} else { + lean_dec_ref(x_68); + x_76 = lean_box(0); +} +if (lean_is_scalar(x_76)) { + x_77 = lean_alloc_ctor(1, 2, 0); +} else { + x_77 = x_76; +} +lean_ctor_set(x_77, 0, x_74); +lean_ctor_set(x_77, 1, x_75); +return x_77; +} +} +else { lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_78 = lean_ctor_get(x_77, 0); +lean_dec(x_64); +lean_dec(x_54); +lean_free_object(x_8); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_78 = lean_ctor_get(x_65, 0); lean_inc(x_78); -x_79 = lean_ctor_get(x_77, 1); +x_79 = lean_ctor_get(x_65, 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; +if (lean_is_exclusive(x_65)) { + lean_ctor_release(x_65, 0); + lean_ctor_release(x_65, 1); + x_80 = x_65; } else { - lean_dec_ref(x_77); + lean_dec_ref(x_65); x_80 = lean_box(0); } -lean_ctor_set(x_9, 1, x_78); -lean_ctor_set(x_9, 0, x_63); -lean_ctor_set(x_10, 0, x_9); if (lean_is_scalar(x_80)) { - x_81 = lean_alloc_ctor(0, 2, 0); + x_81 = lean_alloc_ctor(1, 2, 0); } else { x_81 = x_80; } -lean_ctor_set(x_81, 0, x_10); +lean_ctor_set(x_81, 0, x_78); 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; -lean_dec(x_63); -lean_free_object(x_10); -lean_free_object(x_9); -x_82 = lean_ctor_get(x_77, 0); +lean_dec(x_54); +lean_dec(x_16); +lean_free_object(x_8); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_82 = lean_ctor_get(x_57, 0); lean_inc(x_82); -x_83 = lean_ctor_get(x_77, 1); +x_83 = lean_ctor_get(x_57, 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; +if (lean_is_exclusive(x_57)) { + lean_ctor_release(x_57, 0); + lean_ctor_release(x_57, 1); + x_84 = x_57; } else { - lean_dec_ref(x_77); + lean_dec_ref(x_57); x_84 = lean_box(0); } if (lean_is_scalar(x_84)) { @@ -648,992 +1545,942 @@ return x_85; } else { -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; -lean_dec(x_73); -lean_dec(x_63); -lean_free_object(x_10); -lean_free_object(x_9); +lean_object* x_86; lean_object* x_87; +lean_dec(x_54); +lean_dec(x_16); +lean_free_object(x_8); +lean_dec(x_10); +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_74, 0); -lean_inc(x_86); -x_87 = lean_ctor_get(x_74, 1); -lean_inc(x_87); -if (lean_is_exclusive(x_74)) { - lean_ctor_release(x_74, 0); - lean_ctor_release(x_74, 1); - x_88 = x_74; -} else { - lean_dec_ref(x_74); - x_88 = lean_box(0); +lean_dec(x_1); +x_86 = lean_box(0); +x_87 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_87, 0, x_86); +lean_ctor_set(x_87, 1, x_55); +return x_87; } -if (lean_is_scalar(x_88)) { - x_89 = lean_alloc_ctor(1, 2, 0); -} else { - x_89 = x_88; } -lean_ctor_set(x_89, 0, x_86); -lean_ctor_set(x_89, 1, x_87); -return x_89; +} +else +{ +lean_object* x_88; +lean_dec(x_13); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_88 = l_Lean_Meta_Linear_Nat_toContextExpr(x_2, x_3, x_4, x_5, x_6, x_11); +if (lean_obj_tag(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; +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_Meta_Linear_Nat_LinearCnstr_toExpr(x_1); +x_92 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__11; +x_93 = l_Lean_Meta_Linear_Nat_reflTrue; +x_94 = l_Lean_mkApp3(x_92, x_89, x_91, x_93); +x_95 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__8; +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_96 = l_Lean_Meta_mkEq(x_10, x_95, x_3, x_4, x_5, x_6, x_90); +if (lean_obj_tag(x_96) == 0) +{ +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); +x_99 = l_Lean_Meta_mkExpectedTypeHint(x_94, x_97, x_3, x_4, x_5, x_6, x_98); +if (lean_obj_tag(x_99) == 0) +{ +uint8_t x_100; +x_100 = !lean_is_exclusive(x_99); +if (x_100 == 0) +{ +lean_object* x_101; lean_object* x_102; +x_101 = lean_ctor_get(x_99, 0); +lean_ctor_set(x_8, 1, x_101); +lean_ctor_set(x_8, 0, x_95); +x_102 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_102, 0, x_8); +lean_ctor_set(x_99, 0, x_102); +return x_99; +} +else +{ +lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; +x_103 = lean_ctor_get(x_99, 0); +x_104 = lean_ctor_get(x_99, 1); +lean_inc(x_104); +lean_inc(x_103); +lean_dec(x_99); +lean_ctor_set(x_8, 1, x_103); +lean_ctor_set(x_8, 0, x_95); +x_105 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_105, 0, x_8); +x_106 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_106, 0, x_105); +lean_ctor_set(x_106, 1, x_104); +return x_106; } } else { -lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; -lean_dec(x_63); -lean_dec(x_27); -lean_free_object(x_10); -lean_dec(x_22); -lean_free_object(x_9); +uint8_t x_107; +lean_free_object(x_8); +x_107 = !lean_is_exclusive(x_99); +if (x_107 == 0) +{ +return x_99; +} +else +{ +lean_object* x_108; lean_object* x_109; lean_object* x_110; +x_108 = lean_ctor_get(x_99, 0); +x_109 = lean_ctor_get(x_99, 1); +lean_inc(x_109); +lean_inc(x_108); +lean_dec(x_99); +x_110 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_110, 0, x_108); +lean_ctor_set(x_110, 1, x_109); +return x_110; +} +} +} +else +{ +uint8_t x_111; +lean_dec(x_94); +lean_free_object(x_8); +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_90 = lean_ctor_get(x_66, 0); -lean_inc(x_90); -x_91 = lean_ctor_get(x_66, 1); -lean_inc(x_91); -if (lean_is_exclusive(x_66)) { - lean_ctor_release(x_66, 0); - lean_ctor_release(x_66, 1); - x_92 = x_66; -} else { - lean_dec_ref(x_66); - x_92 = lean_box(0); +x_111 = !lean_is_exclusive(x_96); +if (x_111 == 0) +{ +return x_96; } -if (lean_is_scalar(x_92)) { - x_93 = lean_alloc_ctor(1, 2, 0); -} else { - x_93 = x_92; +else +{ +lean_object* x_112; lean_object* x_113; lean_object* x_114; +x_112 = lean_ctor_get(x_96, 0); +x_113 = lean_ctor_get(x_96, 1); +lean_inc(x_113); +lean_inc(x_112); +lean_dec(x_96); +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; } -lean_ctor_set(x_93, 0, x_90); -lean_ctor_set(x_93, 1, x_91); -return x_93; } } else { -lean_object* x_94; lean_object* x_95; -lean_dec(x_63); -lean_dec(x_27); -lean_free_object(x_10); -lean_dec(x_22); -lean_free_object(x_9); -lean_dec(x_19); +uint8_t x_115; +lean_free_object(x_8); +lean_dec(x_10); +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_94 = lean_box(0); -x_95 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_95, 0, x_94); -lean_ctor_set(x_95, 1, x_64); -return x_95; +x_115 = !lean_is_exclusive(x_88); +if (x_115 == 0) +{ +return x_88; +} +else +{ +lean_object* x_116; lean_object* x_117; lean_object* x_118; +x_116 = lean_ctor_get(x_88, 0); +x_117 = lean_ctor_get(x_88, 1); +lean_inc(x_117); +lean_inc(x_116); +lean_dec(x_88); +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_96; -lean_dec(x_24); -lean_dec(x_1); -x_96 = l_Lean_Meta_Linear_Nat_toContextExpr(x_19, x_2, x_3, x_4, x_5, x_17); -if (lean_obj_tag(x_96) == 0) -{ -uint8_t x_97; -x_97 = !lean_is_exclusive(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; -x_98 = lean_ctor_get(x_96, 0); -x_99 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_22); -x_100 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__9; -x_101 = l_Lean_Meta_Linear_Nat_reflTrue; -x_102 = l_Lean_mkApp3(x_100, x_98, x_99, x_101); -x_103 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__12; -lean_ctor_set(x_9, 1, x_102); -lean_ctor_set(x_9, 0, x_103); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set(x_96, 0, x_10); -return x_96; +lean_object* x_119; +lean_dec(x_13); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_119 = l_Lean_Meta_Linear_Nat_toContextExpr(x_2, x_3, x_4, x_5, x_6, x_11); +if (lean_obj_tag(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; +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_Meta_Linear_Nat_LinearCnstr_toExpr(x_1); +x_123 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__17; +x_124 = l_Lean_Meta_Linear_Nat_reflTrue; +x_125 = l_Lean_mkApp3(x_123, x_120, x_122, x_124); +x_126 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__14; +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_127 = l_Lean_Meta_mkEq(x_10, x_126, x_3, x_4, x_5, x_6, x_121); +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_Lean_Meta_mkExpectedTypeHint(x_125, x_128, x_3, x_4, x_5, x_6, x_129); +if (lean_obj_tag(x_130) == 0) +{ +uint8_t x_131; +x_131 = !lean_is_exclusive(x_130); +if (x_131 == 0) +{ +lean_object* x_132; lean_object* x_133; +x_132 = lean_ctor_get(x_130, 0); +lean_ctor_set(x_8, 1, x_132); +lean_ctor_set(x_8, 0, x_126); +x_133 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_133, 0, x_8); +lean_ctor_set(x_130, 0, x_133); +return x_130; } else { -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_104 = lean_ctor_get(x_96, 0); -x_105 = lean_ctor_get(x_96, 1); -lean_inc(x_105); -lean_inc(x_104); -lean_dec(x_96); -x_106 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_22); -x_107 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__9; -x_108 = l_Lean_Meta_Linear_Nat_reflTrue; -x_109 = l_Lean_mkApp3(x_107, x_104, x_106, x_108); -x_110 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__12; -lean_ctor_set(x_9, 1, x_109); -lean_ctor_set(x_9, 0, x_110); -lean_ctor_set(x_10, 0, x_9); -x_111 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_111, 0, x_10); -lean_ctor_set(x_111, 1, x_105); -return x_111; +lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; +x_134 = lean_ctor_get(x_130, 0); +x_135 = lean_ctor_get(x_130, 1); +lean_inc(x_135); +lean_inc(x_134); +lean_dec(x_130); +lean_ctor_set(x_8, 1, x_134); +lean_ctor_set(x_8, 0, x_126); +x_136 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_136, 0, x_8); +x_137 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_137, 0, x_136); +lean_ctor_set(x_137, 1, x_135); +return x_137; } } else { -uint8_t x_112; -lean_free_object(x_10); -lean_dec(x_22); -lean_free_object(x_9); -x_112 = !lean_is_exclusive(x_96); -if (x_112 == 0) +uint8_t x_138; +lean_free_object(x_8); +x_138 = !lean_is_exclusive(x_130); +if (x_138 == 0) { -return x_96; +return x_130; } else { -lean_object* x_113; lean_object* x_114; lean_object* x_115; -x_113 = lean_ctor_get(x_96, 0); -x_114 = lean_ctor_get(x_96, 1); -lean_inc(x_114); -lean_inc(x_113); -lean_dec(x_96); -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; -} +lean_object* x_139; lean_object* x_140; lean_object* x_141; +x_139 = lean_ctor_get(x_130, 0); +x_140 = lean_ctor_get(x_130, 1); +lean_inc(x_140); +lean_inc(x_139); +lean_dec(x_130); +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; } } } else { -lean_object* x_116; -lean_dec(x_24); -lean_dec(x_1); -x_116 = l_Lean_Meta_Linear_Nat_toContextExpr(x_19, x_2, x_3, x_4, x_5, x_17); -if (lean_obj_tag(x_116) == 0) -{ -uint8_t x_117; -x_117 = !lean_is_exclusive(x_116); -if (x_117 == 0) +uint8_t x_142; +lean_dec(x_125); +lean_free_object(x_8); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_142 = !lean_is_exclusive(x_127); +if (x_142 == 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; -x_118 = lean_ctor_get(x_116, 0); -x_119 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_22); -x_120 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__15; -x_121 = l_Lean_Meta_Linear_Nat_reflTrue; -x_122 = l_Lean_mkApp3(x_120, x_118, x_119, x_121); -x_123 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__18; -lean_ctor_set(x_9, 1, x_122); -lean_ctor_set(x_9, 0, x_123); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set(x_116, 0, x_10); -return x_116; +return x_127; } 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_object* x_130; lean_object* x_131; -x_124 = lean_ctor_get(x_116, 0); -x_125 = lean_ctor_get(x_116, 1); -lean_inc(x_125); -lean_inc(x_124); -lean_dec(x_116); -x_126 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_22); -x_127 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__15; -x_128 = l_Lean_Meta_Linear_Nat_reflTrue; -x_129 = l_Lean_mkApp3(x_127, x_124, x_126, x_128); -x_130 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__18; -lean_ctor_set(x_9, 1, x_129); -lean_ctor_set(x_9, 0, x_130); -lean_ctor_set(x_10, 0, x_9); -x_131 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_131, 0, x_10); -lean_ctor_set(x_131, 1, x_125); -return x_131; +lean_object* x_143; lean_object* x_144; lean_object* x_145; +x_143 = lean_ctor_get(x_127, 0); +x_144 = lean_ctor_get(x_127, 1); +lean_inc(x_144); +lean_inc(x_143); +lean_dec(x_127); +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 { -uint8_t x_132; -lean_free_object(x_10); -lean_dec(x_22); -lean_free_object(x_9); -x_132 = !lean_is_exclusive(x_116); -if (x_132 == 0) +uint8_t x_146; +lean_free_object(x_8); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_146 = !lean_is_exclusive(x_119); +if (x_146 == 0) { -return x_116; +return x_119; } else { -lean_object* x_133; lean_object* x_134; lean_object* x_135; -x_133 = lean_ctor_get(x_116, 0); -x_134 = lean_ctor_get(x_116, 1); -lean_inc(x_134); -lean_inc(x_133); -lean_dec(x_116); -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_147; lean_object* x_148; lean_object* x_149; +x_147 = lean_ctor_get(x_119, 0); +x_148 = lean_ctor_get(x_119, 1); +lean_inc(x_148); +lean_inc(x_147); +lean_dec(x_119); +x_149 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_149, 0, x_147); +lean_ctor_set(x_149, 1, x_148); +return x_149; } } } } else { -lean_object* x_136; lean_object* x_137; lean_object* x_138; uint8_t x_139; -x_136 = lean_ctor_get(x_10, 0); -lean_inc(x_136); -lean_dec(x_10); -lean_inc(x_136); -x_137 = l_Nat_Linear_ExprCnstr_toPoly(x_136); -x_138 = l_Nat_Linear_PolyCnstr_norm(x_137); -x_139 = l_Nat_Linear_PolyCnstr_isUnsat(x_138); -if (x_139 == 0) -{ -uint8_t x_140; -x_140 = l_Nat_Linear_PolyCnstr_isValid(x_138); -if (x_140 == 0) -{ -lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; uint8_t x_146; -x_141 = l_Nat_Linear_PolyCnstr_toExpr(x_138); -lean_inc(x_141); -x_142 = l_Lean_Meta_Linear_Nat_LinearCnstr_toArith(x_19, x_141, x_2, x_3, x_4, x_5, x_17); -x_143 = lean_ctor_get(x_142, 0); -lean_inc(x_143); -x_144 = lean_ctor_get(x_142, 1); -lean_inc(x_144); -if (lean_is_exclusive(x_142)) { - lean_ctor_release(x_142, 0); - lean_ctor_release(x_142, 1); - x_145 = x_142; +lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; uint8_t x_154; +x_150 = lean_ctor_get(x_8, 0); +x_151 = lean_ctor_get(x_8, 1); +lean_inc(x_151); +lean_inc(x_150); +lean_dec(x_8); +lean_inc(x_1); +x_152 = l_Nat_Linear_ExprCnstr_toPoly(x_1); +x_153 = l_Nat_Linear_PolyCnstr_norm(x_152); +x_154 = l_Nat_Linear_PolyCnstr_isUnsat(x_153); +if (x_154 == 0) +{ +uint8_t x_155; +x_155 = l_Nat_Linear_PolyCnstr_isValid(x_153); +if (x_155 == 0) +{ +lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; uint8_t x_161; +x_156 = l_Nat_Linear_PolyCnstr_toExpr(x_153); +lean_inc(x_156); +x_157 = l_Lean_Meta_Linear_Nat_LinearCnstr_toArith(x_2, x_156, x_3, x_4, x_5, x_6, x_151); +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_142); - x_145 = lean_box(0); + lean_dec_ref(x_157); + x_160 = lean_box(0); } -x_146 = lean_expr_eqv(x_143, x_1); -if (x_146 == 0) +x_161 = lean_expr_eqv(x_158, x_150); +if (x_161 == 0) { -lean_object* x_147; -lean_dec(x_145); +lean_object* x_162; +lean_dec(x_160); +lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -x_147 = l_Lean_Meta_Linear_Nat_toContextExpr(x_19, x_2, x_3, x_4, x_5, x_144); -if (lean_obj_tag(x_147) == 0) +x_162 = l_Lean_Meta_Linear_Nat_toContextExpr(x_2, x_3, x_4, x_5, x_6, x_159); +if (lean_obj_tag(x_162) == 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; -x_148 = lean_ctor_get(x_147, 0); -lean_inc(x_148); -x_149 = lean_ctor_get(x_147, 1); -lean_inc(x_149); -lean_dec(x_147); -x_150 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_136); -x_151 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_141); -x_152 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__6; -x_153 = l_Lean_Meta_Linear_Nat_reflTrue; -x_154 = l_Lean_mkApp4(x_152, x_148, x_150, x_151, x_153); +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; +x_163 = lean_ctor_get(x_162, 0); +lean_inc(x_163); +x_164 = lean_ctor_get(x_162, 1); +lean_inc(x_164); +lean_dec(x_162); +x_165 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_1); +x_166 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_156); +x_167 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__5; +x_168 = l_Lean_Meta_Linear_Nat_reflTrue; +x_169 = l_Lean_mkApp4(x_167, x_163, x_165, x_166, x_168); +lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_143); -x_155 = l_Lean_Meta_mkEq(x_1, x_143, x_2, x_3, x_4, x_5, x_149); -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); -x_157 = lean_ctor_get(x_155, 1); -lean_inc(x_157); -lean_dec(x_155); -x_158 = l_Lean_Meta_mkExpectedTypeHint(x_154, x_156, x_2, x_3, x_4, x_5, 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); -x_160 = lean_ctor_get(x_158, 1); -lean_inc(x_160); -if (lean_is_exclusive(x_158)) { - lean_ctor_release(x_158, 0); - lean_ctor_release(x_158, 1); - x_161 = x_158; +lean_inc(x_158); +x_170 = l_Lean_Meta_mkEq(x_150, x_158, x_3, x_4, x_5, x_6, x_164); +if (lean_obj_tag(x_170) == 0) +{ +lean_object* x_171; lean_object* x_172; lean_object* x_173; +x_171 = lean_ctor_get(x_170, 0); +lean_inc(x_171); +x_172 = lean_ctor_get(x_170, 1); +lean_inc(x_172); +lean_dec(x_170); +x_173 = l_Lean_Meta_mkExpectedTypeHint(x_169, x_171, x_3, x_4, x_5, x_6, x_172); +if (lean_obj_tag(x_173) == 0) +{ +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_174 = lean_ctor_get(x_173, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_173, 1); +lean_inc(x_175); +if (lean_is_exclusive(x_173)) { + lean_ctor_release(x_173, 0); + lean_ctor_release(x_173, 1); + x_176 = x_173; } else { - lean_dec_ref(x_158); - x_161 = lean_box(0); -} -lean_ctor_set(x_9, 1, x_159); -lean_ctor_set(x_9, 0, x_143); -x_162 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_162, 0, x_9); -if (lean_is_scalar(x_161)) { - x_163 = lean_alloc_ctor(0, 2, 0); + lean_dec_ref(x_173); + x_176 = lean_box(0); +} +x_177 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_177, 0, x_158); +lean_ctor_set(x_177, 1, x_174); +x_178 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_178, 0, x_177); +if (lean_is_scalar(x_176)) { + x_179 = lean_alloc_ctor(0, 2, 0); } else { - x_163 = x_161; + x_179 = x_176; } -lean_ctor_set(x_163, 0, x_162); -lean_ctor_set(x_163, 1, x_160); -return x_163; +lean_ctor_set(x_179, 0, x_178); +lean_ctor_set(x_179, 1, x_175); +return x_179; } else { -lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; -lean_dec(x_143); -lean_free_object(x_9); -x_164 = lean_ctor_get(x_158, 0); -lean_inc(x_164); -x_165 = lean_ctor_get(x_158, 1); -lean_inc(x_165); -if (lean_is_exclusive(x_158)) { - lean_ctor_release(x_158, 0); - lean_ctor_release(x_158, 1); - x_166 = x_158; +lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; +lean_dec(x_158); +x_180 = lean_ctor_get(x_173, 0); +lean_inc(x_180); +x_181 = lean_ctor_get(x_173, 1); +lean_inc(x_181); +if (lean_is_exclusive(x_173)) { + lean_ctor_release(x_173, 0); + lean_ctor_release(x_173, 1); + x_182 = x_173; } else { - lean_dec_ref(x_158); - x_166 = lean_box(0); + lean_dec_ref(x_173); + x_182 = lean_box(0); } -if (lean_is_scalar(x_166)) { - x_167 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_182)) { + x_183 = lean_alloc_ctor(1, 2, 0); } else { - x_167 = x_166; + x_183 = x_182; } -lean_ctor_set(x_167, 0, x_164); -lean_ctor_set(x_167, 1, x_165); -return x_167; +lean_ctor_set(x_183, 0, x_180); +lean_ctor_set(x_183, 1, x_181); +return x_183; } } else { -lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; -lean_dec(x_154); -lean_dec(x_143); -lean_free_object(x_9); +lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; +lean_dec(x_169); +lean_dec(x_158); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -x_168 = lean_ctor_get(x_155, 0); -lean_inc(x_168); -x_169 = lean_ctor_get(x_155, 1); -lean_inc(x_169); -if (lean_is_exclusive(x_155)) { - lean_ctor_release(x_155, 0); - lean_ctor_release(x_155, 1); - x_170 = x_155; +x_184 = lean_ctor_get(x_170, 0); +lean_inc(x_184); +x_185 = lean_ctor_get(x_170, 1); +lean_inc(x_185); +if (lean_is_exclusive(x_170)) { + lean_ctor_release(x_170, 0); + lean_ctor_release(x_170, 1); + x_186 = x_170; } else { - lean_dec_ref(x_155); - x_170 = lean_box(0); + lean_dec_ref(x_170); + x_186 = lean_box(0); } -if (lean_is_scalar(x_170)) { - x_171 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_186)) { + x_187 = lean_alloc_ctor(1, 2, 0); } else { - x_171 = x_170; + x_187 = x_186; } -lean_ctor_set(x_171, 0, x_168); -lean_ctor_set(x_171, 1, x_169); -return x_171; +lean_ctor_set(x_187, 0, x_184); +lean_ctor_set(x_187, 1, x_185); +return x_187; } } else { -lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; -lean_dec(x_143); -lean_dec(x_141); -lean_dec(x_136); -lean_free_object(x_9); +lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; +lean_dec(x_158); +lean_dec(x_156); +lean_dec(x_150); +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_172 = lean_ctor_get(x_147, 0); -lean_inc(x_172); -x_173 = lean_ctor_get(x_147, 1); -lean_inc(x_173); -if (lean_is_exclusive(x_147)) { - lean_ctor_release(x_147, 0); - lean_ctor_release(x_147, 1); - x_174 = x_147; +x_188 = lean_ctor_get(x_162, 0); +lean_inc(x_188); +x_189 = lean_ctor_get(x_162, 1); +lean_inc(x_189); +if (lean_is_exclusive(x_162)) { + lean_ctor_release(x_162, 0); + lean_ctor_release(x_162, 1); + x_190 = x_162; } else { - lean_dec_ref(x_147); - x_174 = lean_box(0); + lean_dec_ref(x_162); + x_190 = lean_box(0); } -if (lean_is_scalar(x_174)) { - x_175 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_190)) { + x_191 = lean_alloc_ctor(1, 2, 0); } else { - x_175 = x_174; + x_191 = x_190; } -lean_ctor_set(x_175, 0, x_172); -lean_ctor_set(x_175, 1, x_173); -return x_175; +lean_ctor_set(x_191, 0, x_188); +lean_ctor_set(x_191, 1, x_189); +return x_191; } } else { -lean_object* x_176; lean_object* x_177; -lean_dec(x_143); -lean_dec(x_141); -lean_dec(x_136); -lean_free_object(x_9); -lean_dec(x_19); +lean_object* x_192; lean_object* x_193; +lean_dec(x_158); +lean_dec(x_156); +lean_dec(x_150); +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_176 = lean_box(0); -if (lean_is_scalar(x_145)) { - x_177 = lean_alloc_ctor(0, 2, 0); +x_192 = lean_box(0); +if (lean_is_scalar(x_160)) { + x_193 = lean_alloc_ctor(0, 2, 0); } else { - x_177 = x_145; + x_193 = x_160; } -lean_ctor_set(x_177, 0, x_176); -lean_ctor_set(x_177, 1, x_144); -return x_177; +lean_ctor_set(x_193, 0, x_192); +lean_ctor_set(x_193, 1, x_159); +return x_193; } } else { -lean_object* x_178; -lean_dec(x_138); -lean_dec(x_1); -x_178 = l_Lean_Meta_Linear_Nat_toContextExpr(x_19, x_2, x_3, x_4, x_5, x_17); -if (lean_obj_tag(x_178) == 0) +lean_object* x_194; +lean_dec(x_153); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_194 = l_Lean_Meta_Linear_Nat_toContextExpr(x_2, x_3, x_4, x_5, x_6, x_151); +if (lean_obj_tag(x_194) == 0) { -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; -x_179 = lean_ctor_get(x_178, 0); -lean_inc(x_179); -x_180 = lean_ctor_get(x_178, 1); -lean_inc(x_180); -if (lean_is_exclusive(x_178)) { - lean_ctor_release(x_178, 0); - lean_ctor_release(x_178, 1); - x_181 = x_178; -} else { - lean_dec_ref(x_178); - x_181 = lean_box(0); -} -x_182 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_136); -x_183 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__9; -x_184 = l_Lean_Meta_Linear_Nat_reflTrue; -x_185 = l_Lean_mkApp3(x_183, x_179, x_182, x_184); -x_186 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__12; -lean_ctor_set(x_9, 1, x_185); -lean_ctor_set(x_9, 0, x_186); -x_187 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_187, 0, x_9); -if (lean_is_scalar(x_181)) { - x_188 = lean_alloc_ctor(0, 2, 0); -} else { - x_188 = x_181; -} -lean_ctor_set(x_188, 0, x_187); -lean_ctor_set(x_188, 1, x_180); -return x_188; -} -else -{ -lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; -lean_dec(x_136); -lean_free_object(x_9); -x_189 = lean_ctor_get(x_178, 0); -lean_inc(x_189); -x_190 = lean_ctor_get(x_178, 1); -lean_inc(x_190); -if (lean_is_exclusive(x_178)) { - lean_ctor_release(x_178, 0); - lean_ctor_release(x_178, 1); - x_191 = x_178; +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; +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 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_1); +x_198 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__11; +x_199 = l_Lean_Meta_Linear_Nat_reflTrue; +x_200 = l_Lean_mkApp3(x_198, x_195, x_197, x_199); +x_201 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__8; +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_202 = l_Lean_Meta_mkEq(x_150, x_201, x_3, x_4, x_5, x_6, x_196); +if (lean_obj_tag(x_202) == 0) +{ +lean_object* x_203; lean_object* x_204; lean_object* x_205; +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_Meta_mkExpectedTypeHint(x_200, x_203, x_3, x_4, x_5, x_6, x_204); +if (lean_obj_tag(x_205) == 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_205, 0); +lean_inc(x_206); +x_207 = lean_ctor_get(x_205, 1); +lean_inc(x_207); +if (lean_is_exclusive(x_205)) { + lean_ctor_release(x_205, 0); + lean_ctor_release(x_205, 1); + x_208 = x_205; +} else { + lean_dec_ref(x_205); + x_208 = lean_box(0); +} +x_209 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_209, 0, x_201); +lean_ctor_set(x_209, 1, x_206); +x_210 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_210, 0, x_209); +if (lean_is_scalar(x_208)) { + x_211 = lean_alloc_ctor(0, 2, 0); } else { - lean_dec_ref(x_178); - x_191 = lean_box(0); + x_211 = x_208; } -if (lean_is_scalar(x_191)) { - x_192 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_211, 0, x_210); +lean_ctor_set(x_211, 1, x_207); +return x_211; +} +else +{ +lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; +x_212 = lean_ctor_get(x_205, 0); +lean_inc(x_212); +x_213 = lean_ctor_get(x_205, 1); +lean_inc(x_213); +if (lean_is_exclusive(x_205)) { + lean_ctor_release(x_205, 0); + lean_ctor_release(x_205, 1); + x_214 = x_205; } else { - x_192 = x_191; + lean_dec_ref(x_205); + x_214 = lean_box(0); } -lean_ctor_set(x_192, 0, x_189); -lean_ctor_set(x_192, 1, x_190); -return x_192; +if (lean_is_scalar(x_214)) { + x_215 = lean_alloc_ctor(1, 2, 0); +} else { + x_215 = x_214; } +lean_ctor_set(x_215, 0, x_212); +lean_ctor_set(x_215, 1, x_213); +return x_215; } } else { -lean_object* x_193; -lean_dec(x_138); -lean_dec(x_1); -x_193 = l_Lean_Meta_Linear_Nat_toContextExpr(x_19, x_2, x_3, x_4, x_5, x_17); -if (lean_obj_tag(x_193) == 0) -{ -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; -x_194 = lean_ctor_get(x_193, 0); -lean_inc(x_194); -x_195 = lean_ctor_get(x_193, 1); -lean_inc(x_195); -if (lean_is_exclusive(x_193)) { - lean_ctor_release(x_193, 0); - lean_ctor_release(x_193, 1); - x_196 = x_193; +lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; +lean_dec(x_200); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_216 = lean_ctor_get(x_202, 0); +lean_inc(x_216); +x_217 = lean_ctor_get(x_202, 1); +lean_inc(x_217); +if (lean_is_exclusive(x_202)) { + lean_ctor_release(x_202, 0); + lean_ctor_release(x_202, 1); + x_218 = x_202; } else { - lean_dec_ref(x_193); - x_196 = lean_box(0); + lean_dec_ref(x_202); + x_218 = lean_box(0); } -x_197 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_136); -x_198 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__15; -x_199 = l_Lean_Meta_Linear_Nat_reflTrue; -x_200 = l_Lean_mkApp3(x_198, x_194, x_197, x_199); -x_201 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__18; -lean_ctor_set(x_9, 1, x_200); -lean_ctor_set(x_9, 0, x_201); -x_202 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_202, 0, x_9); -if (lean_is_scalar(x_196)) { - x_203 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_218)) { + x_219 = lean_alloc_ctor(1, 2, 0); } else { - x_203 = x_196; + x_219 = x_218; +} +lean_ctor_set(x_219, 0, x_216); +lean_ctor_set(x_219, 1, x_217); +return x_219; } -lean_ctor_set(x_203, 0, x_202); -lean_ctor_set(x_203, 1, x_195); -return x_203; } else { -lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; -lean_dec(x_136); -lean_free_object(x_9); -x_204 = lean_ctor_get(x_193, 0); -lean_inc(x_204); -x_205 = lean_ctor_get(x_193, 1); -lean_inc(x_205); -if (lean_is_exclusive(x_193)) { - lean_ctor_release(x_193, 0); - lean_ctor_release(x_193, 1); - x_206 = x_193; +lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; +lean_dec(x_150); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_220 = lean_ctor_get(x_194, 0); +lean_inc(x_220); +x_221 = lean_ctor_get(x_194, 1); +lean_inc(x_221); +if (lean_is_exclusive(x_194)) { + lean_ctor_release(x_194, 0); + lean_ctor_release(x_194, 1); + x_222 = x_194; } else { - lean_dec_ref(x_193); - x_206 = lean_box(0); + lean_dec_ref(x_194); + x_222 = lean_box(0); } -if (lean_is_scalar(x_206)) { - x_207 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_222)) { + x_223 = lean_alloc_ctor(1, 2, 0); } else { - x_207 = x_206; -} -lean_ctor_set(x_207, 0, x_204); -lean_ctor_set(x_207, 1, x_205); -return x_207; + 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_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; uint8_t x_213; -x_208 = lean_ctor_get(x_9, 1); -lean_inc(x_208); -lean_dec(x_9); -x_209 = lean_ctor_get(x_10, 0); -lean_inc(x_209); -if (lean_is_exclusive(x_10)) { - lean_ctor_release(x_10, 0); - x_210 = x_10; -} else { - lean_dec_ref(x_10); - x_210 = lean_box(0); -} -lean_inc(x_209); -x_211 = l_Nat_Linear_ExprCnstr_toPoly(x_209); -x_212 = l_Nat_Linear_PolyCnstr_norm(x_211); -x_213 = l_Nat_Linear_PolyCnstr_isUnsat(x_212); -if (x_213 == 0) -{ -uint8_t x_214; -x_214 = l_Nat_Linear_PolyCnstr_isValid(x_212); -if (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; -x_215 = l_Nat_Linear_PolyCnstr_toExpr(x_212); -lean_inc(x_215); -x_216 = l_Lean_Meta_Linear_Nat_LinearCnstr_toArith(x_208, x_215, x_2, x_3, x_4, x_5, x_17); -x_217 = lean_ctor_get(x_216, 0); -lean_inc(x_217); -x_218 = lean_ctor_get(x_216, 1); -lean_inc(x_218); -if (lean_is_exclusive(x_216)) { - lean_ctor_release(x_216, 0); - lean_ctor_release(x_216, 1); - x_219 = x_216; -} else { - lean_dec_ref(x_216); - x_219 = lean_box(0); -} -x_220 = lean_expr_eqv(x_217, x_1); -if (x_220 == 0) -{ -lean_object* x_221; -lean_dec(x_219); +lean_object* x_224; +lean_dec(x_153); +lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -x_221 = l_Lean_Meta_Linear_Nat_toContextExpr(x_208, x_2, x_3, x_4, x_5, x_218); -if (lean_obj_tag(x_221) == 0) -{ -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; -x_222 = lean_ctor_get(x_221, 0); -lean_inc(x_222); -x_223 = lean_ctor_get(x_221, 1); -lean_inc(x_223); -lean_dec(x_221); -x_224 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_209); -x_225 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_215); -x_226 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__6; -x_227 = l_Lean_Meta_Linear_Nat_reflTrue; -x_228 = l_Lean_mkApp4(x_226, x_222, x_224, x_225, x_227); +x_224 = l_Lean_Meta_Linear_Nat_toContextExpr(x_2, x_3, x_4, x_5, x_6, x_151); +if (lean_obj_tag(x_224) == 0) +{ +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; +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_Meta_Linear_Nat_LinearCnstr_toExpr(x_1); +x_228 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__17; +x_229 = l_Lean_Meta_Linear_Nat_reflTrue; +x_230 = l_Lean_mkApp3(x_228, x_225, x_227, x_229); +x_231 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__14; +lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_217); -x_229 = l_Lean_Meta_mkEq(x_1, x_217, x_2, x_3, x_4, x_5, x_223); -if (lean_obj_tag(x_229) == 0) -{ -lean_object* x_230; lean_object* x_231; lean_object* x_232; -x_230 = lean_ctor_get(x_229, 0); -lean_inc(x_230); -x_231 = lean_ctor_get(x_229, 1); -lean_inc(x_231); -lean_dec(x_229); -x_232 = l_Lean_Meta_mkExpectedTypeHint(x_228, x_230, x_2, x_3, x_4, x_5, x_231); +x_232 = l_Lean_Meta_mkEq(x_150, x_231, x_3, x_4, x_5, x_6, 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_233; lean_object* x_234; lean_object* x_235; 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_alloc_ctor(0, 2, 0); -lean_ctor_set(x_236, 0, x_217); -lean_ctor_set(x_236, 1, x_233); -if (lean_is_scalar(x_210)) { - x_237 = lean_alloc_ctor(1, 1, 0); -} else { - x_237 = x_210; -} -lean_ctor_set(x_237, 0, x_236); -if (lean_is_scalar(x_235)) { - x_238 = lean_alloc_ctor(0, 2, 0); -} else { +lean_dec(x_232); +x_235 = l_Lean_Meta_mkExpectedTypeHint(x_230, x_233, x_3, x_4, x_5, x_6, x_234); +if (lean_obj_tag(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; +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; -} -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; -lean_dec(x_217); -lean_dec(x_210); -x_239 = lean_ctor_get(x_232, 0); -lean_inc(x_239); -x_240 = lean_ctor_get(x_232, 1); -lean_inc(x_240); -if (lean_is_exclusive(x_232)) { - lean_ctor_release(x_232, 0); - lean_ctor_release(x_232, 1); - x_241 = x_232; } else { - lean_dec_ref(x_232); - x_241 = lean_box(0); -} -if (lean_is_scalar(x_241)) { - x_242 = lean_alloc_ctor(1, 2, 0); + lean_dec_ref(x_235); + x_238 = lean_box(0); +} +x_239 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_239, 0, x_231); +lean_ctor_set(x_239, 1, x_236); +x_240 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_240, 0, x_239); +if (lean_is_scalar(x_238)) { + x_241 = lean_alloc_ctor(0, 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; + x_241 = x_238; } +lean_ctor_set(x_241, 0, x_240); +lean_ctor_set(x_241, 1, x_237); +return x_241; } else { -lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; -lean_dec(x_228); -lean_dec(x_217); -lean_dec(x_210); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_243 = lean_ctor_get(x_229, 0); +lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; +x_242 = lean_ctor_get(x_235, 0); +lean_inc(x_242); +x_243 = lean_ctor_get(x_235, 1); lean_inc(x_243); -x_244 = lean_ctor_get(x_229, 1); -lean_inc(x_244); -if (lean_is_exclusive(x_229)) { - lean_ctor_release(x_229, 0); - lean_ctor_release(x_229, 1); - x_245 = x_229; +if (lean_is_exclusive(x_235)) { + lean_ctor_release(x_235, 0); + lean_ctor_release(x_235, 1); + x_244 = x_235; } else { - lean_dec_ref(x_229); - x_245 = lean_box(0); + lean_dec_ref(x_235); + x_244 = lean_box(0); } -if (lean_is_scalar(x_245)) { - x_246 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_244)) { + x_245 = lean_alloc_ctor(1, 2, 0); } else { - x_246 = x_245; + x_245 = x_244; } -lean_ctor_set(x_246, 0, x_243); -lean_ctor_set(x_246, 1, x_244); -return x_246; +lean_ctor_set(x_245, 0, x_242); +lean_ctor_set(x_245, 1, x_243); +return x_245; } } else { -lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; -lean_dec(x_217); -lean_dec(x_215); -lean_dec(x_210); -lean_dec(x_209); +lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; +lean_dec(x_230); +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_ctor_get(x_221, 0); +x_246 = lean_ctor_get(x_232, 0); +lean_inc(x_246); +x_247 = lean_ctor_get(x_232, 1); lean_inc(x_247); -x_248 = lean_ctor_get(x_221, 1); -lean_inc(x_248); -if (lean_is_exclusive(x_221)) { - lean_ctor_release(x_221, 0); - lean_ctor_release(x_221, 1); - x_249 = x_221; +if (lean_is_exclusive(x_232)) { + lean_ctor_release(x_232, 0); + lean_ctor_release(x_232, 1); + x_248 = x_232; } else { - lean_dec_ref(x_221); - x_249 = lean_box(0); + lean_dec_ref(x_232); + x_248 = lean_box(0); } -if (lean_is_scalar(x_249)) { - x_250 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_248)) { + x_249 = lean_alloc_ctor(1, 2, 0); } else { - x_250 = x_249; + x_249 = x_248; } -lean_ctor_set(x_250, 0, x_247); -lean_ctor_set(x_250, 1, x_248); -return x_250; +lean_ctor_set(x_249, 0, x_246); +lean_ctor_set(x_249, 1, x_247); +return x_249; } } else { -lean_object* x_251; lean_object* x_252; -lean_dec(x_217); -lean_dec(x_215); -lean_dec(x_210); -lean_dec(x_209); -lean_dec(x_208); +lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; +lean_dec(x_150); +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_251 = lean_box(0); -if (lean_is_scalar(x_219)) { - x_252 = lean_alloc_ctor(0, 2, 0); -} else { - x_252 = x_219; -} -lean_ctor_set(x_252, 0, x_251); -lean_ctor_set(x_252, 1, x_218); -return x_252; -} -} -else -{ -lean_object* x_253; -lean_dec(x_212); lean_dec(x_1); -x_253 = l_Lean_Meta_Linear_Nat_toContextExpr(x_208, x_2, x_3, x_4, x_5, x_17); -if (lean_obj_tag(x_253) == 0) -{ -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_254 = lean_ctor_get(x_253, 0); -lean_inc(x_254); -x_255 = lean_ctor_get(x_253, 1); -lean_inc(x_255); -if (lean_is_exclusive(x_253)) { - lean_ctor_release(x_253, 0); - lean_ctor_release(x_253, 1); - x_256 = x_253; -} else { - lean_dec_ref(x_253); - x_256 = lean_box(0); -} -x_257 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_209); -x_258 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__9; -x_259 = l_Lean_Meta_Linear_Nat_reflTrue; -x_260 = l_Lean_mkApp3(x_258, x_254, x_257, x_259); -x_261 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__12; -x_262 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_262, 0, x_261); -lean_ctor_set(x_262, 1, x_260); -if (lean_is_scalar(x_210)) { - x_263 = lean_alloc_ctor(1, 1, 0); +x_250 = lean_ctor_get(x_224, 0); +lean_inc(x_250); +x_251 = lean_ctor_get(x_224, 1); +lean_inc(x_251); +if (lean_is_exclusive(x_224)) { + lean_ctor_release(x_224, 0); + lean_ctor_release(x_224, 1); + x_252 = x_224; } else { - x_263 = x_210; + lean_dec_ref(x_224); + x_252 = lean_box(0); } -lean_ctor_set(x_263, 0, x_262); -if (lean_is_scalar(x_256)) { - x_264 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_252)) { + x_253 = lean_alloc_ctor(1, 2, 0); } else { - x_264 = x_256; -} -lean_ctor_set(x_264, 0, x_263); -lean_ctor_set(x_264, 1, x_255); -return x_264; + x_253 = x_252; } -else -{ -lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; -lean_dec(x_210); -lean_dec(x_209); -x_265 = lean_ctor_get(x_253, 0); -lean_inc(x_265); -x_266 = lean_ctor_get(x_253, 1); -lean_inc(x_266); -if (lean_is_exclusive(x_253)) { - lean_ctor_release(x_253, 0); - lean_ctor_release(x_253, 1); - x_267 = x_253; -} else { - lean_dec_ref(x_253); - x_267 = lean_box(0); +lean_ctor_set(x_253, 0, x_250); +lean_ctor_set(x_253, 1, x_251); +return x_253; } -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_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_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_269; -lean_dec(x_212); -lean_dec(x_1); -x_269 = l_Lean_Meta_Linear_Nat_toContextExpr(x_208, x_2, x_3, x_4, x_5, x_17); -if (lean_obj_tag(x_269) == 0) +lean_object* x_7; lean_object* x_8; +x_7 = lean_alloc_closure((void*)(l_Lean_Meta_Linear_Nat_ToLinear_toLinearCnstr_x3f), 7, 1); +lean_closure_set(x_7, 0, x_1); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_8 = l_Lean_Meta_Linear_Nat_ToLinear_run___rarg(x_7, x_2, x_3, x_4, x_5, x_6); +if (lean_obj_tag(x_8) == 0) { -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; -x_270 = lean_ctor_get(x_269, 0); -lean_inc(x_270); -x_271 = lean_ctor_get(x_269, 1); -lean_inc(x_271); -if (lean_is_exclusive(x_269)) { - lean_ctor_release(x_269, 0); - lean_ctor_release(x_269, 1); - x_272 = x_269; -} else { - lean_dec_ref(x_269); - x_272 = lean_box(0); -} -x_273 = l_Lean_Meta_Linear_Nat_LinearCnstr_toExpr(x_209); -x_274 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__15; -x_275 = l_Lean_Meta_Linear_Nat_reflTrue; -x_276 = l_Lean_mkApp3(x_274, x_270, x_273, x_275); -x_277 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__18; -x_278 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_278, 0, x_277); -lean_ctor_set(x_278, 1, x_276); -if (lean_is_scalar(x_210)) { - x_279 = lean_alloc_ctor(1, 1, 0); -} else { - x_279 = x_210; -} -lean_ctor_set(x_279, 0, x_278); -if (lean_is_scalar(x_272)) { - x_280 = lean_alloc_ctor(0, 2, 0); -} else { - x_280 = x_272; -} -lean_ctor_set(x_280, 0, x_279); -lean_ctor_set(x_280, 1, x_271); -return x_280; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +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_9); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_11 = !lean_is_exclusive(x_8); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_8, 0); +lean_dec(x_12); +x_13 = lean_box(0); +lean_ctor_set(x_8, 0, x_13); +return x_8; } else { -lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; -lean_dec(x_210); -lean_dec(x_209); -x_281 = lean_ctor_get(x_269, 0); -lean_inc(x_281); -x_282 = lean_ctor_get(x_269, 1); -lean_inc(x_282); -if (lean_is_exclusive(x_269)) { - lean_ctor_release(x_269, 0); - lean_ctor_release(x_269, 1); - x_283 = x_269; -} else { - lean_dec_ref(x_269); - 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; -} +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_8, 1); +lean_inc(x_14); +lean_dec(x_8); +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; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_17 = lean_ctor_get(x_8, 1); +lean_inc(x_17); +lean_dec(x_8); +x_18 = lean_ctor_get(x_9, 1); +lean_inc(x_18); +lean_dec(x_9); +x_19 = lean_ctor_get(x_10, 0); +lean_inc(x_19); +lean_dec(x_10); +x_20 = lean_alloc_closure((void*)(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1), 7, 1); +lean_closure_set(x_20, 0, x_19); +x_21 = l_Lean_Meta_Linear_Nat_withAbstractAtoms(x_18, x_20, x_2, x_3, x_4, x_5, x_17); +return x_21; } } else { -uint8_t x_285; +uint8_t x_22; lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_285 = !lean_is_exclusive(x_8); -if (x_285 == 0) +x_22 = !lean_is_exclusive(x_8); +if (x_22 == 0) { return x_8; } else { -lean_object* x_286; lean_object* x_287; lean_object* x_288; -x_286 = lean_ctor_get(x_8, 0); -x_287 = lean_ctor_get(x_8, 1); -lean_inc(x_287); -lean_inc(x_286); +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_8, 0); +x_24 = lean_ctor_get(x_8, 1); +lean_inc(x_24); +lean_inc(x_23); lean_dec(x_8); -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; +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; } } } @@ -2225,7 +3072,7 @@ static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1; +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; @@ -2243,7 +3090,7 @@ static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1; +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_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; @@ -2270,7 +3117,7 @@ static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__21() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1; +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_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; @@ -2288,7 +3135,7 @@ static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__23() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1; +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_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; @@ -2719,10 +3566,10 @@ static lean_object* _init_l_Lean_Meta_Linear_Nat_simpExpr_x3f___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_Linear_Nat_simpCnstrPos_x3f___closed__1; -x_2 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__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_simpCnstrPos_x3f___lambda__1___closed__1; x_3 = l_Lean_Meta_Linear_Nat_simpExpr_x3f___closed__1; -x_4 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__4; +x_4 = l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__3; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -3184,42 +4031,54 @@ _G_initialized = true; res = initialize_Lean_Meta_Tactic_LinearArith_Nat_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__2 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__2(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__2); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__3 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__3(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__3); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__4 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__4(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__4); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__5 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__5(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__5); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__6 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__6(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__6); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__7 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__7(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__7); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__8 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__8(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__8); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__9 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__9(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__9); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__10 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__10(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__10); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__11 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__11(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__11); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__12 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__12(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__12); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__13 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__13(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__13); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__14 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__14(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__14); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__15 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__15(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__15); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__16 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__16(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__16); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__17 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__17(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__17); -l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__18 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__18(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__18); +l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1); +l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__2 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__2(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__2); +l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__3 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__3(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__3); +l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__1); +l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__2 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__2(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__2); +l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__3 = _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__3(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__3); +l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg___closed__1 = _init_l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg___closed__1(); +lean_mark_persistent(l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg___closed__1); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__1 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__1); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__2 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__2); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__3 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__3); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__4 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__4); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__5 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__5); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__6 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__6); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__7 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__7); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__8 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__8); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__9 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__9); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__10 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__10); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__11 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__11(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__11); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__12 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__12(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__12); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__13 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__13(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__13); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__14 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__14(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__14); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__15 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__15(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__15); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__16 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__16(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__16); +l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__17 = _init_l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__17(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__17); l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__1 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__1(); lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__1); l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__2 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__2(); diff --git a/stage0/stdlib/Lean/Meta/Tactic/SplitIf.c b/stage0/stdlib/Lean/Meta/Tactic/SplitIf.c index f912d4a7a065..614c73219b72 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/SplitIf.c +++ b/stage0/stdlib/Lean/Meta/Tactic/SplitIf.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean.Meta.Tactic.SplitIf -// Imports: Lean.LazyInitExtension Lean.Meta.Tactic.Cases Lean.Meta.Tactic.Simp.Main +// Imports: Lean.Meta.Tactic.Cases Lean.Meta.Tactic.Simp.Main #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -14,18 +14,20 @@ extern "C" { #endif static lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__5; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__11; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__5; -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__5; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__9; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__12; +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__11; static lean_object* l_Lean_Meta_simpIfTarget___closed__9; -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__8; LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___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_Meta_splitIfLocalDecl_x3f___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_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__2; lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_simpIfLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__9; uint8_t l_Lean_Expr_isDIte(lean_object*); +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__8; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__4; LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___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*); static lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__4; @@ -43,85 +45,80 @@ LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_ uint8_t l_Lean_Expr_isAppOfArity(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_LocalContext_findDeclRevM_x3f___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_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*); static lean_object* l_Lean_Meta_simpIfLocalDecl___closed__1; -static lean_object* l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__2; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__10; LEAN_EXPORT lean_object* l_Lean_commitWhenSome_x3f___at_Lean_Meta_splitIfLocalDecl_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_LocalContext_findDeclRevM_x3f___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___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_Meta_SplitIf_splitIfAt_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_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_mkDischarge_x3f___elambda__1(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_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__7; +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__10; lean_object* lean_array_fget(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635_(lean_object*); lean_object* l_Lean_MVarId_byCasesDec(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instantiateMVars___at_Lean_Meta_Simp_synthesizeArgs___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_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__4; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__7; static lean_object* l_Lean_Meta_simpIfTarget___closed__11; LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_findIfToSplit_x3f___lambda__1(lean_object*); -lean_object* l_Lean_registerLazyInitExtension___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Meta_SplitIf_splitIfAt_x3f___lambda__2___closed__1; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__10; lean_object* l_Lean_stringToMessageData(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__2___closed__5; static lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__3; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__12; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__8; +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__9; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__14; static lean_object* l_Lean_Meta_simpIfTarget___closed__6; lean_object* l_Lean_Meta_getSimpCongrTheorems___rarg(lean_object*, lean_object*); lean_object* l_Lean_Expr_appArg_x21(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__2___closed__6; -LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4_(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__2___closed__1; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__5; lean_object* l_Lean_LocalDecl_index(lean_object*); static lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__2; uint8_t l_Lean_Expr_hasMVar(lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_EnvExtension_getState___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__5; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__2___closed__4; -static lean_object* l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__3; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__1; extern lean_object* l_Lean_PersistentHashMap_empty___at_Lean_Meta_instInhabitedSimpTheorems___spec__1; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__1; -lean_object* lean_st_ref_take(lean_object*, lean_object*); lean_object* l_Lean_Expr_getRevArg_x21(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__7; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__5; static lean_object* l_Lean_Meta_simpIfTarget___closed__3; static lean_object* l_Lean_Meta_simpIfTarget___closed__8; +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__12; +static uint32_t l_Lean_Meta_SplitIf_getSimpContext___closed__14; static lean_object* l_Lean_Meta_simpIfTarget___closed__5; lean_object* l_Lean_MVarId_getType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_registerTraceClass(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeRevM_x3f___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___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_SplitIf_getSimpContext___closed__3; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_findIfToSplit_x3f___lambda__1___closed__2; lean_object* l_Lean_Meta_SavedState_restore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_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*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__11; lean_object* l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_SplitIf_splitIfAt_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_simpIfTarget___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__1; lean_object* l_Lean_MessageData_ofFormat(lean_object*); -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_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_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_object* l_Lean_Meta_simpTarget(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_DiscrTree_empty(lean_object*); -lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_splitIfTarget_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_SplitIf_splitIfAt_x3f___closed__2; LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeRevMAux___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___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_splitIfLocalDecl_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_splitIfAt_x3f___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_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__7; uint8_t l_Lean_Expr_hasLooseBVars(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_ext; LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___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* l_Lean_Name_num___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_getSimpContext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Simp_congrArgs___spec__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_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__2___closed__2; static lean_object* l_Lean_Meta_simpIfLocalDecl___closed__2; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_mkDischarge_x3f(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkDecide(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_findIfToSplit_x3f___boxed(lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); @@ -131,67 +128,56 @@ LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_mkDischarge_x3f___elambda__1___boxe LEAN_EXPORT lean_object* l_Lean_Meta_simpIfTarget(lean_object*, uint8_t, 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*); uint8_t l_Lean_Expr_isIte(lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__6; lean_object* l_Lean_Meta_saveState___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__4; uint8_t l_Lean_LocalDecl_isAuxDecl(lean_object*); -static lean_object* l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__4; static lean_object* l_Lean_Meta_simpIfTarget___closed__2; static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_mkDischarge_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__14; static lean_object* l_Lean_Meta_simpIfTarget___closed__7; -static lean_object* l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__1; -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__10; LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___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*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__3; -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__6; -LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611_(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_findIfToSplit_x3f(lean_object*); static lean_object* l_Lean_Meta_simpIfTarget___closed__10; 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_EnvExtension_setState___rarg(lean_object*, lean_object*, lean_object*); 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_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__1; -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__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_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__3; lean_object* l_Lean_Meta_mkEqRefl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_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*); uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); static lean_object* l_Lean_Meta_simpIfTarget___closed__4; lean_object* l_Lean_LocalDecl_type(lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__9; -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__4; lean_object* l_Lean_addTrace___at_Lean_Meta_Simp_congrArgs___spec__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_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__2; lean_object* lean_nat_sub(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__2___closed__3; -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_findIfToSplit_x3f___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_commitWhenSome_x3f___at_Lean_Meta_splitIfTarget_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); lean_object* l_Lean_Meta_SimpTheorems_addConst(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_Meta_SplitIf_getSimpContext___closed__7; lean_object* lean_array_mk(lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___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*); +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__6; extern lean_object* l_Lean_Meta_Simp_defaultMaxSteps; uint8_t l_Lean_Expr_hasFVar(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__2(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_Expr_fvar___override(lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__13; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__13; lean_object* l_Lean_Meta_simpLocalDecl(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_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_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__8; lean_object* lean_local_ctx_num_indices(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_splitIfAt_x3f___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_SplitIf_getSimpContext___closed__5; LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeRevMAux___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___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*); static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__3; -static uint32_t l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__8; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__13; extern lean_object* l_Lean_PersistentHashMap_empty___at_Lean_KeyedDeclsAttribute_instInhabitedExtensionState___spec__1; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_findIfToSplit_x3f___closed__1; 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_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__2; lean_object* lean_array_get_size(lean_object*); lean_object* l_Lean_LocalDecl_toExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeRevM_x3f___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_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*); @@ -199,20 +185,81 @@ lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_obje lean_object* lean_find_expr(lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_findIfToSplit_x3f___lambda__1___boxed(lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__12; -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__1; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___lambda__2___closed__7; +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__4; uint8_t l_Lean_Exception_isRuntime(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_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_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__15; -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__3; +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__13; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__15; LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_splitIfAt_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_SplitIf_getSimpContext___closed__2; lean_object* l_panic___at_Lean_Meta_subst_substEq___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__4; static lean_object* l_Lean_Meta_simpIfTarget___closed__1; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__6; static lean_object* l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_findIfToSplit_x3f___closed__3; -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___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_Meta_SplitIf_getSimpContext___closed__2() { +_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_SplitIf_getSimpContext___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_SplitIf_getSimpContext___closed__2; +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_SplitIf_getSimpContext___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_SplitIf_getSimpContext___closed__1; +x_2 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_instInhabitedSimpTheorems___spec__1; +x_3 = l_Lean_PersistentHashMap_empty___at_Lean_KeyedDeclsAttribute_instInhabitedExtensionState___spec__1; +x_4 = l_Lean_Meta_SplitIf_getSimpContext___closed__3; +x_5 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_1); +lean_ctor_set(x_5, 2, x_2); +lean_ctor_set(x_5, 3, x_3); +lean_ctor_set(x_5, 4, x_2); +lean_ctor_set(x_5, 5, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("if_pos", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___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_SplitIf_getSimpContext___closed__5; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__7() { _start: { lean_object* x_1; @@ -220,17 +267,17 @@ x_1 = lean_mk_string_unchecked("if_neg", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___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_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__1; +x_2 = l_Lean_Meta_SplitIf_getSimpContext___closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__9() { _start: { lean_object* x_1; @@ -238,17 +285,17 @@ x_1 = lean_mk_string_unchecked("dif_pos", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___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_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__3; +x_2 = l_Lean_Meta_SplitIf_getSimpContext___closed__9; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__11() { _start: { lean_object* x_1; @@ -256,17 +303,17 @@ x_1 = lean_mk_string_unchecked("dif_neg", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___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_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__5; +x_2 = l_Lean_Meta_SplitIf_getSimpContext___closed__11; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__13() { _start: { lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; @@ -300,7 +347,7 @@ lean_ctor_set_uint8(x_6, sizeof(void*)*2 + 18, x_4); return x_6; } } -static uint32_t _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__8() { +static uint32_t _init_l_Lean_Meta_SplitIf_getSimpContext___closed__14() { _start: { lean_object* x_1; uint32_t x_2; @@ -309,18 +356,20 @@ x_2 = l_UInt32_ofNatTruncate(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_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_EXPORT lean_object* l_Lean_Meta_SplitIf_getSimpContext(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; uint8_t x_9; lean_object* x_10; lean_object* x_11; +lean_object* x_6; lean_object* x_7; uint8_t x_8; uint8_t x_9; lean_object* x_10; lean_object* x_11; +x_6 = l_Lean_Meta_SplitIf_getSimpContext___closed__4; +x_7 = l_Lean_Meta_SplitIf_getSimpContext___closed__6; x_8 = 1; x_9 = 0; x_10 = lean_unsigned_to_nat(1000u); -lean_inc(x_6); -lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_11 = l_Lean_Meta_SimpTheorems_addConst(x_1, x_2, x_8, x_9, x_10, x_3, x_4, x_5, x_6, x_7); +lean_inc(x_2); +lean_inc(x_1); +x_11 = l_Lean_Meta_SimpTheorems_addConst(x_6, x_7, x_8, x_9, x_10, x_1, x_2, x_3, x_4, x_5); if (lean_obj_tag(x_11) == 0) { lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; @@ -329,12 +378,12 @@ 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_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__2; -lean_inc(x_6); -lean_inc(x_5); +x_14 = l_Lean_Meta_SplitIf_getSimpContext___closed__8; lean_inc(x_4); lean_inc(x_3); -x_15 = l_Lean_Meta_SimpTheorems_addConst(x_12, x_14, x_8, x_9, x_10, x_3, x_4, x_5, x_6, x_13); +lean_inc(x_2); +lean_inc(x_1); +x_15 = l_Lean_Meta_SimpTheorems_addConst(x_12, x_14, x_8, x_9, x_10, x_1, x_2, x_3, x_4, 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; @@ -343,12 +392,12 @@ 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_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__4; -lean_inc(x_6); -lean_inc(x_5); +x_18 = l_Lean_Meta_SplitIf_getSimpContext___closed__10; lean_inc(x_4); lean_inc(x_3); -x_19 = l_Lean_Meta_SimpTheorems_addConst(x_16, x_18, x_8, x_9, x_10, x_3, x_4, x_5, x_6, x_17); +lean_inc(x_2); +lean_inc(x_1); +x_19 = l_Lean_Meta_SimpTheorems_addConst(x_16, x_18, x_8, x_9, x_10, x_1, x_2, x_3, x_4, x_17); if (lean_obj_tag(x_19) == 0) { lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; @@ -357,9 +406,9 @@ 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_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__6; -lean_inc(x_6); -x_23 = l_Lean_Meta_SimpTheorems_addConst(x_20, x_22, x_8, x_9, x_10, x_3, x_4, x_5, x_6, x_21); +x_22 = l_Lean_Meta_SplitIf_getSimpContext___closed__12; +lean_inc(x_4); +x_23 = l_Lean_Meta_SimpTheorems_addConst(x_20, x_22, x_8, x_9, x_10, x_1, x_2, x_3, x_4, x_21); if (lean_obj_tag(x_23) == 0) { lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; @@ -368,8 +417,8 @@ 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_getSimpCongrTheorems___rarg(x_6, x_25); -lean_dec(x_6); +x_26 = l_Lean_Meta_getSimpCongrTheorems___rarg(x_4, x_25); +lean_dec(x_4); x_27 = !lean_is_exclusive(x_26); if (x_27 == 0) { @@ -382,8 +431,8 @@ lean_ctor_set(x_30, 1, x_29); x_31 = lean_array_mk(x_30); x_32 = lean_box(0); x_33 = 0; -x_34 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__7; -x_35 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__8; +x_34 = l_Lean_Meta_SplitIf_getSimpContext___closed__13; +x_35 = l_Lean_Meta_SplitIf_getSimpContext___closed__14; x_36 = lean_unsigned_to_nat(0u); x_37 = lean_alloc_ctor(0, 5, 9); lean_ctor_set(x_37, 0, x_34); @@ -412,8 +461,8 @@ lean_ctor_set(x_41, 1, x_40); x_42 = lean_array_mk(x_41); x_43 = lean_box(0); x_44 = 0; -x_45 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__7; -x_46 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__8; +x_45 = l_Lean_Meta_SplitIf_getSimpContext___closed__13; +x_46 = l_Lean_Meta_SplitIf_getSimpContext___closed__14; x_47 = lean_unsigned_to_nat(0u); x_48 = lean_alloc_ctor(0, 5, 9); lean_ctor_set(x_48, 0, x_45); @@ -433,7 +482,7 @@ return x_49; else { uint8_t x_50; -lean_dec(x_6); +lean_dec(x_4); x_50 = !lean_is_exclusive(x_23); if (x_50 == 0) { @@ -457,10 +506,10 @@ return x_53; else { uint8_t x_54; -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_19); if (x_54 == 0) { @@ -484,10 +533,10 @@ return x_57; else { uint8_t x_58; -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_15); if (x_58 == 0) { @@ -509,644 +558,31 @@ return x_61; } } else -{ -uint8_t x_62; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_62 = !lean_is_exclusive(x_11); -if (x_62 == 0) -{ -return x_11; -} -else -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_63 = lean_ctor_get(x_11, 0); -x_64 = lean_ctor_get(x_11, 1); -lean_inc(x_64); -lean_inc(x_63); -lean_dec(x_11); -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; -} -} -} -} -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____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_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__2() { -_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_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__2; -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_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____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_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__1; -x_2 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_instInhabitedSimpTheorems___spec__1; -x_3 = l_Lean_PersistentHashMap_empty___at_Lean_KeyedDeclsAttribute_instInhabitedExtensionState___spec__1; -x_4 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3; -x_5 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_5, 0, x_1); -lean_ctor_set(x_5, 1, x_1); -lean_ctor_set(x_5, 2, x_2); -lean_ctor_set(x_5, 3, x_3); -lean_ctor_set(x_5, 4, x_2); -lean_ctor_set(x_5, 5, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("if_pos", 6, 6); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____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_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__5; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4_(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_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__4; -x_3 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__6; -x_4 = lean_alloc_closure((void*)(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1), 7, 2); -lean_closure_set(x_4, 0, x_2); -lean_closure_set(x_4, 1, x_3); -x_5 = l_Lean_registerLazyInitExtension___rarg(x_4, x_1); -return x_5; -} -} -static lean_object* _init_l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3; -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_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3; -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_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3; -x_2 = lean_alloc_ctor(0, 4, 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); -return x_2; -} -} -static lean_object* _init_l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__2; -x_2 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3; -x_3 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__3; -x_4 = lean_alloc_ctor(0, 7, 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_2); -lean_ctor_set(x_4, 4, x_2); -lean_ctor_set(x_4, 5, x_3); -lean_ctor_set(x_4, 6, x_3); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___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) { -_start: -{ -lean_object* x_7; uint8_t x_8; -x_7 = lean_st_ref_get(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; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_9 = lean_ctor_get(x_7, 0); -x_10 = lean_ctor_get(x_7, 1); -x_11 = lean_ctor_get(x_9, 0); -lean_inc(x_11); -lean_dec(x_9); -x_12 = lean_box(0); -x_13 = lean_ctor_get(x_1, 0); -lean_inc(x_13); -x_14 = l_Lean_EnvExtension_getState___rarg(x_12, x_13, x_11); -lean_dec(x_11); -if (lean_obj_tag(x_14) == 0) -{ -lean_object* x_15; lean_object* x_16; -lean_free_object(x_7); -x_15 = lean_ctor_get(x_1, 1); -lean_inc(x_15); -lean_dec(x_1); -lean_inc(x_5); -lean_inc(x_3); -x_16 = lean_apply_5(x_15, x_2, x_3, x_4, x_5, x_10); -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; uint8_t 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_take(x_5, 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_is_exclusive(x_20); -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; uint8_t x_33; -x_23 = lean_ctor_get(x_20, 0); -x_24 = lean_ctor_get(x_20, 4); -lean_dec(x_24); -lean_inc(x_17); -x_25 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_25, 0, x_17); -x_26 = l_Lean_EnvExtension_setState___rarg(x_13, x_23, x_25); -lean_dec(x_13); -x_27 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__1; -lean_ctor_set(x_20, 4, x_27); -lean_ctor_set(x_20, 0, x_26); -x_28 = lean_st_ref_set(x_5, x_20, x_21); -lean_dec(x_5); -x_29 = lean_ctor_get(x_28, 1); -lean_inc(x_29); -lean_dec(x_28); -x_30 = lean_st_ref_take(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_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; uint8_t x_37; -x_34 = lean_ctor_get(x_31, 1); -lean_dec(x_34); -x_35 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__4; -lean_ctor_set(x_31, 1, x_35); -x_36 = lean_st_ref_set(x_3, x_31, x_32); -lean_dec(x_3); -x_37 = !lean_is_exclusive(x_36); -if (x_37 == 0) -{ -lean_object* x_38; -x_38 = lean_ctor_get(x_36, 0); -lean_dec(x_38); -lean_ctor_set(x_36, 0, x_17); -return x_36; -} -else -{ -lean_object* x_39; lean_object* x_40; -x_39 = lean_ctor_get(x_36, 1); -lean_inc(x_39); -lean_dec(x_36); -x_40 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_40, 0, x_17); -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_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_41 = lean_ctor_get(x_31, 0); -x_42 = lean_ctor_get(x_31, 2); -x_43 = lean_ctor_get(x_31, 3); -x_44 = lean_ctor_get(x_31, 4); -lean_inc(x_44); -lean_inc(x_43); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_31); -x_45 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__4; -x_46 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_46, 0, x_41); -lean_ctor_set(x_46, 1, x_45); -lean_ctor_set(x_46, 2, x_42); -lean_ctor_set(x_46, 3, x_43); -lean_ctor_set(x_46, 4, x_44); -x_47 = lean_st_ref_set(x_3, x_46, x_32); -lean_dec(x_3); -x_48 = lean_ctor_get(x_47, 1); -lean_inc(x_48); -if (lean_is_exclusive(x_47)) { - lean_ctor_release(x_47, 0); - lean_ctor_release(x_47, 1); - x_49 = x_47; -} else { - lean_dec_ref(x_47); - x_49 = lean_box(0); -} -if (lean_is_scalar(x_49)) { - x_50 = lean_alloc_ctor(0, 2, 0); -} else { - x_50 = x_49; -} -lean_ctor_set(x_50, 0, x_17); -lean_ctor_set(x_50, 1, x_48); -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; 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_51 = lean_ctor_get(x_20, 0); -x_52 = lean_ctor_get(x_20, 1); -x_53 = lean_ctor_get(x_20, 2); -x_54 = lean_ctor_get(x_20, 3); -x_55 = lean_ctor_get(x_20, 5); -x_56 = lean_ctor_get(x_20, 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_dec(x_20); -lean_inc(x_17); -x_57 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_57, 0, x_17); -x_58 = l_Lean_EnvExtension_setState___rarg(x_13, x_51, x_57); -lean_dec(x_13); -x_59 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__1; -x_60 = lean_alloc_ctor(0, 7, 0); -lean_ctor_set(x_60, 0, x_58); -lean_ctor_set(x_60, 1, x_52); -lean_ctor_set(x_60, 2, x_53); -lean_ctor_set(x_60, 3, x_54); -lean_ctor_set(x_60, 4, x_59); -lean_ctor_set(x_60, 5, x_55); -lean_ctor_set(x_60, 6, x_56); -x_61 = lean_st_ref_set(x_5, x_60, x_21); -lean_dec(x_5); -x_62 = lean_ctor_get(x_61, 1); -lean_inc(x_62); -lean_dec(x_61); -x_63 = lean_st_ref_take(x_3, 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_64, 0); -lean_inc(x_66); -x_67 = lean_ctor_get(x_64, 2); -lean_inc(x_67); -x_68 = lean_ctor_get(x_64, 3); -lean_inc(x_68); -x_69 = lean_ctor_get(x_64, 4); -lean_inc(x_69); -if (lean_is_exclusive(x_64)) { - lean_ctor_release(x_64, 0); - lean_ctor_release(x_64, 1); - lean_ctor_release(x_64, 2); - lean_ctor_release(x_64, 3); - lean_ctor_release(x_64, 4); - x_70 = x_64; -} else { - lean_dec_ref(x_64); - x_70 = lean_box(0); -} -x_71 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__4; -if (lean_is_scalar(x_70)) { - x_72 = lean_alloc_ctor(0, 5, 0); -} else { - x_72 = x_70; -} -lean_ctor_set(x_72, 0, x_66); -lean_ctor_set(x_72, 1, x_71); -lean_ctor_set(x_72, 2, x_67); -lean_ctor_set(x_72, 3, x_68); -lean_ctor_set(x_72, 4, x_69); -x_73 = lean_st_ref_set(x_3, x_72, x_65); -lean_dec(x_3); -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); -} -if (lean_is_scalar(x_75)) { - x_76 = lean_alloc_ctor(0, 2, 0); -} else { - x_76 = x_75; -} -lean_ctor_set(x_76, 0, x_17); -lean_ctor_set(x_76, 1, x_74); -return x_76; -} -} -else -{ -uint8_t x_77; -lean_dec(x_13); -lean_dec(x_5); -lean_dec(x_3); -x_77 = !lean_is_exclusive(x_16); -if (x_77 == 0) -{ -return x_16; -} -else -{ -lean_object* x_78; lean_object* x_79; lean_object* x_80; -x_78 = lean_ctor_get(x_16, 0); -x_79 = lean_ctor_get(x_16, 1); -lean_inc(x_79); -lean_inc(x_78); -lean_dec(x_16); -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_dec(x_13); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_81 = lean_ctor_get(x_14, 0); -lean_inc(x_81); -lean_dec(x_14); -lean_ctor_set(x_7, 0, x_81); -return x_7; -} -} -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_7, 0); -x_83 = lean_ctor_get(x_7, 1); -lean_inc(x_83); -lean_inc(x_82); -lean_dec(x_7); -x_84 = lean_ctor_get(x_82, 0); -lean_inc(x_84); -lean_dec(x_82); -x_85 = lean_box(0); -x_86 = lean_ctor_get(x_1, 0); -lean_inc(x_86); -x_87 = l_Lean_EnvExtension_getState___rarg(x_85, x_86, x_84); -lean_dec(x_84); -if (lean_obj_tag(x_87) == 0) -{ -lean_object* x_88; lean_object* x_89; -x_88 = lean_ctor_get(x_1, 1); -lean_inc(x_88); -lean_dec(x_1); -lean_inc(x_5); -lean_inc(x_3); -x_89 = lean_apply_5(x_88, x_2, x_3, x_4, x_5, x_83); -if (lean_obj_tag(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; 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; -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_st_ref_take(x_5, x_91); -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 = 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); -x_98 = lean_ctor_get(x_93, 3); -lean_inc(x_98); -x_99 = lean_ctor_get(x_93, 5); -lean_inc(x_99); -x_100 = lean_ctor_get(x_93, 6); -lean_inc(x_100); -if (lean_is_exclusive(x_93)) { - lean_ctor_release(x_93, 0); - lean_ctor_release(x_93, 1); - lean_ctor_release(x_93, 2); - lean_ctor_release(x_93, 3); - lean_ctor_release(x_93, 4); - lean_ctor_release(x_93, 5); - lean_ctor_release(x_93, 6); - x_101 = x_93; -} else { - lean_dec_ref(x_93); - x_101 = lean_box(0); -} -lean_inc(x_90); -x_102 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_102, 0, x_90); -x_103 = l_Lean_EnvExtension_setState___rarg(x_86, x_95, x_102); -lean_dec(x_86); -x_104 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__1; -if (lean_is_scalar(x_101)) { - x_105 = lean_alloc_ctor(0, 7, 0); -} else { - x_105 = x_101; -} -lean_ctor_set(x_105, 0, x_103); -lean_ctor_set(x_105, 1, x_96); -lean_ctor_set(x_105, 2, x_97); -lean_ctor_set(x_105, 3, x_98); -lean_ctor_set(x_105, 4, x_104); -lean_ctor_set(x_105, 5, x_99); -lean_ctor_set(x_105, 6, x_100); -x_106 = lean_st_ref_set(x_5, x_105, x_94); -lean_dec(x_5); -x_107 = lean_ctor_get(x_106, 1); -lean_inc(x_107); -lean_dec(x_106); -x_108 = lean_st_ref_take(x_3, 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_109, 0); -lean_inc(x_111); -x_112 = lean_ctor_get(x_109, 2); -lean_inc(x_112); -x_113 = lean_ctor_get(x_109, 3); -lean_inc(x_113); -x_114 = lean_ctor_get(x_109, 4); -lean_inc(x_114); -if (lean_is_exclusive(x_109)) { - lean_ctor_release(x_109, 0); - lean_ctor_release(x_109, 1); - lean_ctor_release(x_109, 2); - lean_ctor_release(x_109, 3); - lean_ctor_release(x_109, 4); - x_115 = x_109; -} else { - lean_dec_ref(x_109); - x_115 = lean_box(0); -} -x_116 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__4; -if (lean_is_scalar(x_115)) { - x_117 = lean_alloc_ctor(0, 5, 0); -} else { - x_117 = x_115; -} -lean_ctor_set(x_117, 0, x_111); -lean_ctor_set(x_117, 1, x_116); -lean_ctor_set(x_117, 2, x_112); -lean_ctor_set(x_117, 3, x_113); -lean_ctor_set(x_117, 4, x_114); -x_118 = lean_st_ref_set(x_3, x_117, x_110); -lean_dec(x_3); -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); -} -if (lean_is_scalar(x_120)) { - x_121 = lean_alloc_ctor(0, 2, 0); -} else { - x_121 = x_120; -} -lean_ctor_set(x_121, 0, x_90); -lean_ctor_set(x_121, 1, x_119); -return x_121; -} -else -{ -lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; -lean_dec(x_86); -lean_dec(x_5); -lean_dec(x_3); -x_122 = lean_ctor_get(x_89, 0); -lean_inc(x_122); -x_123 = lean_ctor_get(x_89, 1); -lean_inc(x_123); -if (lean_is_exclusive(x_89)) { - lean_ctor_release(x_89, 0); - lean_ctor_release(x_89, 1); - x_124 = x_89; -} else { - lean_dec_ref(x_89); - x_124 = lean_box(0); -} -if (lean_is_scalar(x_124)) { - x_125 = lean_alloc_ctor(1, 2, 0); -} else { - x_125 = x_124; -} -lean_ctor_set(x_125, 0, x_122); -lean_ctor_set(x_125, 1, x_123); -return x_125; -} -} -else -{ -lean_object* x_126; lean_object* x_127; -lean_dec(x_86); -lean_dec(x_5); +{ +uint8_t x_62; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_126 = lean_ctor_get(x_87, 0); -lean_inc(x_126); -lean_dec(x_87); -x_127 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_127, 0, x_126); -lean_ctor_set(x_127, 1, x_83); -return x_127; -} -} -} +x_62 = !lean_is_exclusive(x_11); +if (x_62 == 0) +{ +return x_11; } -static lean_object* _init_l_Lean_Meta_SplitIf_getSimpContext___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = l_Lean_Meta_SplitIf_ext; -return x_1; +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_11, 0); +x_64 = lean_ctor_get(x_11, 1); +lean_inc(x_64); +lean_inc(x_63); +lean_dec(x_11); +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_Meta_SplitIf_getSimpContext(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 = l_Lean_Meta_SplitIf_getSimpContext___closed__1; -x_7 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1(x_6, x_1, x_2, x_3, x_4, x_5); -return x_7; } } static lean_object* _init_l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__1() { @@ -4131,7 +3567,7 @@ static lean_object* _init_l_Lean_Meta_simpIfTarget___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3; +x_1 = l_Lean_Meta_SplitIf_getSimpContext___closed__3; x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4179,7 +3615,7 @@ static lean_object* _init_l_Lean_Meta_simpIfTarget___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3; +x_1 = l_Lean_Meta_SplitIf_getSimpContext___closed__3; x_2 = l_Lean_Meta_simpIfTarget___closed__5; x_3 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_3, 0, x_1); @@ -4231,7 +3667,7 @@ static lean_object* _init_l_Lean_Meta_simpIfTarget___closed__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; x_1 = l_Lean_Meta_simpIfTarget___closed__8; x_2 = l_Lean_Meta_simpIfTarget___closed__9; -x_3 = lean_unsigned_to_nat(101u); +x_3 = lean_unsigned_to_nat(96u); x_4 = lean_unsigned_to_nat(4u); x_5 = l_Lean_Meta_simpIfTarget___closed__10; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -4241,182 +3677,181 @@ return x_6; LEAN_EXPORT lean_object* l_Lean_Meta_simpIfTarget(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) { _start: { -lean_object* x_8; lean_object* x_9; -x_8 = l_Lean_Meta_SplitIf_getSimpContext___closed__1; +lean_object* x_8; lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_9 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1(x_8, x_3, x_4, x_5, x_6, x_7); -if (lean_obj_tag(x_9) == 0) +x_8 = l_Lean_Meta_SplitIf_getSimpContext(x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_8) == 0) { -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_9, 0); +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_8, 1); lean_inc(x_10); -x_11 = lean_ctor_get(x_9, 1); -lean_inc(x_11); -lean_dec(x_9); -x_12 = lean_box(x_2); -x_13 = lean_alloc_closure((void*)(l_Lean_Meta_SplitIf_mkDischarge_x3f___boxed), 6, 1); -lean_closure_set(x_13, 0, x_12); +lean_dec(x_8); +x_11 = lean_box(x_2); +x_12 = lean_alloc_closure((void*)(l_Lean_Meta_SplitIf_mkDischarge_x3f___boxed), 6, 1); +lean_closure_set(x_12, 0, x_11); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_1); -x_14 = l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(x_1, x_13, x_3, x_4, x_5, x_6, x_11); -if (lean_obj_tag(x_14) == 0) +x_13 = l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(x_1, x_12, x_3, x_4, x_5, x_6, x_10); +if (lean_obj_tag(x_13) == 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; lean_object* x_21; -x_15 = lean_ctor_get(x_14, 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_20; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); -lean_inc(x_16); -lean_dec(x_14); -x_17 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_17, 0, x_15); -x_18 = l_Lean_Meta_simpIfTarget___closed__1; -x_19 = 0; -x_20 = l_Lean_Meta_simpIfTarget___closed__7; +lean_dec(x_13); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_14); +x_17 = l_Lean_Meta_simpIfTarget___closed__1; +x_18 = 0; +x_19 = l_Lean_Meta_simpIfTarget___closed__7; lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_21 = l_Lean_Meta_simpTarget(x_1, x_10, x_18, x_17, x_19, x_20, x_3, x_4, x_5, x_6, x_16); -if (lean_obj_tag(x_21) == 0) +x_20 = l_Lean_Meta_simpTarget(x_1, x_9, x_17, x_16, x_18, x_19, x_3, x_4, x_5, x_6, x_15); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_22; lean_object* x_23; +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); x_22 = lean_ctor_get(x_21, 0); lean_inc(x_22); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -lean_dec(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_21, 1); -lean_inc(x_24); lean_dec(x_21); -x_25 = l_Lean_Meta_simpIfTarget___closed__11; -x_26 = l_panic___at_Lean_Meta_subst_substEq___spec__1(x_25, x_3, x_4, x_5, x_6, x_24); -return x_26; +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_20, 1); +lean_inc(x_23); +lean_dec(x_20); +x_24 = l_Lean_Meta_simpIfTarget___closed__11; +x_25 = l_panic___at_Lean_Meta_subst_substEq___spec__1(x_24, x_3, x_4, x_5, x_6, x_23); +return x_25; } else { -uint8_t x_27; +uint8_t x_26; 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) +x_26 = !lean_is_exclusive(x_20); +if (x_26 == 0) { -lean_object* x_28; lean_object* x_29; -x_28 = lean_ctor_get(x_21, 0); -lean_dec(x_28); -x_29 = lean_ctor_get(x_23, 0); -lean_inc(x_29); -lean_dec(x_23); -lean_ctor_set(x_21, 0, x_29); -return x_21; +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_20, 0); +lean_dec(x_27); +x_28 = lean_ctor_get(x_22, 0); +lean_inc(x_28); +lean_dec(x_22); +lean_ctor_set(x_20, 0, x_28); +return x_20; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_21, 1); +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_20, 1); +lean_inc(x_29); +lean_dec(x_20); +x_30 = lean_ctor_get(x_22, 0); lean_inc(x_30); -lean_dec(x_21); -x_31 = lean_ctor_get(x_23, 0); -lean_inc(x_31); -lean_dec(x_23); -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_dec(x_22); +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_33; +uint8_t x_32; lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_33 = !lean_is_exclusive(x_21); -if (x_33 == 0) +x_32 = !lean_is_exclusive(x_20); +if (x_32 == 0) { -return x_21; +return x_20; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_21, 0); -x_35 = lean_ctor_get(x_21, 1); -lean_inc(x_35); +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_20, 0); +x_34 = lean_ctor_get(x_20, 1); lean_inc(x_34); -lean_dec(x_21); -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_20); +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_37; -lean_dec(x_10); +uint8_t x_36; +lean_dec(x_9); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_37 = !lean_is_exclusive(x_14); -if (x_37 == 0) +x_36 = !lean_is_exclusive(x_13); +if (x_36 == 0) { -return x_14; +return x_13; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_14, 0); -x_39 = lean_ctor_get(x_14, 1); -lean_inc(x_39); +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_13, 0); +x_38 = lean_ctor_get(x_13, 1); lean_inc(x_38); -lean_dec(x_14); -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_13); +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_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_41 = !lean_is_exclusive(x_9); -if (x_41 == 0) +x_40 = !lean_is_exclusive(x_8); +if (x_40 == 0) { -return x_9; +return x_8; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_9, 0); -x_43 = lean_ctor_get(x_9, 1); -lean_inc(x_43); +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_8, 0); +x_42 = lean_ctor_get(x_8, 1); lean_inc(x_42); -lean_dec(x_9); -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_8); +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; } } } @@ -4456,7 +3891,7 @@ static lean_object* _init_l_Lean_Meta_simpIfLocalDecl___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_Lean_Meta_simpIfTarget___closed__8; x_2 = l_Lean_Meta_simpIfLocalDecl___closed__2; -x_3 = lean_unsigned_to_nat(108u); +x_3 = lean_unsigned_to_nat(103u); x_4 = lean_unsigned_to_nat(4u); x_5 = l_Lean_Meta_simpIfTarget___closed__10; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -4466,185 +3901,184 @@ return x_6; LEAN_EXPORT lean_object* l_Lean_Meta_simpIfLocalDecl(lean_object* x_1, 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 = l_Lean_Meta_SplitIf_getSimpContext___closed__1; +lean_object* x_8; lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_9 = l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1(x_8, x_3, x_4, x_5, x_6, x_7); -if (lean_obj_tag(x_9) == 0) +x_8 = l_Lean_Meta_SplitIf_getSimpContext(x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_8) == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = lean_ctor_get(x_9, 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); -x_11 = lean_ctor_get(x_9, 1); -lean_inc(x_11); -lean_dec(x_9); -x_12 = l_Lean_Meta_simpIfLocalDecl___closed__1; +lean_dec(x_8); +x_11 = l_Lean_Meta_simpIfLocalDecl___closed__1; lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_1); -x_13 = l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(x_1, x_12, x_3, x_4, x_5, x_6, x_11); -if (lean_obj_tag(x_13) == 0) +x_12 = l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(x_1, x_11, x_3, x_4, x_5, x_6, x_10); +if (lean_obj_tag(x_12) == 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_20; -x_14 = lean_ctor_get(x_13, 0); +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; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_16, 0, x_14); -x_17 = l_Lean_Meta_simpIfTarget___closed__1; -x_18 = 0; -x_19 = l_Lean_Meta_simpIfTarget___closed__7; +lean_dec(x_12); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_13); +x_16 = l_Lean_Meta_simpIfTarget___closed__1; +x_17 = 0; +x_18 = l_Lean_Meta_simpIfTarget___closed__7; lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_20 = l_Lean_Meta_simpLocalDecl(x_1, x_2, x_10, x_17, x_16, x_18, x_19, x_3, x_4, x_5, x_6, x_15); -if (lean_obj_tag(x_20) == 0) +x_19 = l_Lean_Meta_simpLocalDecl(x_1, x_2, x_9, x_16, x_15, x_17, x_18, x_3, x_4, x_5, x_6, x_14); +if (lean_obj_tag(x_19) == 0) { -lean_object* x_21; lean_object* x_22; +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); x_21 = lean_ctor_get(x_20, 0); lean_inc(x_21); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -lean_dec(x_21); -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_20, 1); -lean_inc(x_23); lean_dec(x_20); -x_24 = l_Lean_Meta_simpIfLocalDecl___closed__3; -x_25 = l_panic___at_Lean_Meta_subst_substEq___spec__1(x_24, x_3, x_4, x_5, x_6, x_23); -return x_25; +if (lean_obj_tag(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 = l_Lean_Meta_simpIfLocalDecl___closed__3; +x_24 = l_panic___at_Lean_Meta_subst_substEq___spec__1(x_23, x_3, x_4, x_5, x_6, x_22); +return x_24; } else { -lean_object* x_26; uint8_t x_27; +lean_object* x_25; uint8_t x_26; lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_26 = lean_ctor_get(x_22, 0); -lean_inc(x_26); -lean_dec(x_22); -x_27 = !lean_is_exclusive(x_20); -if (x_27 == 0) +x_25 = lean_ctor_get(x_21, 0); +lean_inc(x_25); +lean_dec(x_21); +x_26 = !lean_is_exclusive(x_19); +if (x_26 == 0) { -lean_object* x_28; lean_object* x_29; -x_28 = lean_ctor_get(x_20, 0); -lean_dec(x_28); -x_29 = lean_ctor_get(x_26, 1); -lean_inc(x_29); -lean_dec(x_26); -lean_ctor_set(x_20, 0, x_29); -return x_20; +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_19, 0); +lean_dec(x_27); +x_28 = lean_ctor_get(x_25, 1); +lean_inc(x_28); +lean_dec(x_25); +lean_ctor_set(x_19, 0, x_28); +return x_19; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_20, 1); +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_19, 1); +lean_inc(x_29); +lean_dec(x_19); +x_30 = lean_ctor_get(x_25, 1); lean_inc(x_30); -lean_dec(x_20); -x_31 = lean_ctor_get(x_26, 1); -lean_inc(x_31); -lean_dec(x_26); -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_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 { -uint8_t x_33; +uint8_t x_32; lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_33 = !lean_is_exclusive(x_20); -if (x_33 == 0) +x_32 = !lean_is_exclusive(x_19); +if (x_32 == 0) { -return x_20; +return x_19; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_20, 0); -x_35 = lean_ctor_get(x_20, 1); -lean_inc(x_35); +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_dec(x_20); -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_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; } } } else { -uint8_t x_37; -lean_dec(x_10); +uint8_t x_36; +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_37 = !lean_is_exclusive(x_13); -if (x_37 == 0) +x_36 = !lean_is_exclusive(x_12); +if (x_36 == 0) { -return x_13; +return x_12; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_13, 0); -x_39 = lean_ctor_get(x_13, 1); -lean_inc(x_39); +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_12, 0); +x_38 = lean_ctor_get(x_12, 1); lean_inc(x_38); -lean_dec(x_13); -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_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; } } } else { -uint8_t x_41; +uint8_t x_40; 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_9); -if (x_41 == 0) +x_40 = !lean_is_exclusive(x_8); +if (x_40 == 0) { -return x_9; +return x_8; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_9, 0); -x_43 = lean_ctor_get(x_9, 1); -lean_inc(x_43); +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_8, 0); +x_42 = lean_ctor_get(x_8, 1); lean_inc(x_42); -lean_dec(x_9); -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_8); +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; } } } @@ -6912,7 +6346,7 @@ x_12 = l_Lean_commitWhenSome_x3f___at_Lean_Meta_splitIfLocalDecl_x3f___spec__1(x return x_12; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__1() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__1() { _start: { lean_object* x_1; @@ -6920,27 +6354,27 @@ x_1 = lean_mk_string_unchecked("Lean", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__2() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____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_Tactic_SplitIf___hyg_1635____closed__1; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____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_Tactic_SplitIf___hyg_1635____closed__3() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__2; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__2; x_2 = l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___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_Tactic_SplitIf___hyg_1635____closed__4() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__4() { _start: { lean_object* x_1; @@ -6948,17 +6382,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__5() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__3; -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__4; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__3; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____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_Tactic_SplitIf___hyg_1635____closed__6() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__6() { _start: { lean_object* x_1; @@ -6966,47 +6400,47 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__7() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__5; -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__6; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__5; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____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_Tactic_SplitIf___hyg_1635____closed__8() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__7; -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__1; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__7; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____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_Tactic_SplitIf___hyg_1635____closed__9() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__8; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__8; x_2 = l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___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_Tactic_SplitIf___hyg_1635____closed__10() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__9; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__9; x_2 = l___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__2; 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_Tactic_SplitIf___hyg_1635____closed__11() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__11() { _start: { lean_object* x_1; @@ -7014,17 +6448,17 @@ x_1 = lean_mk_string_unchecked("SplitIf", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__12() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__10; -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__11; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__10; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__11; 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_Tactic_SplitIf___hyg_1635____closed__13() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__13() { _start: { lean_object* x_1; @@ -7032,38 +6466,37 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__14() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__12; -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__13; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__12; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__13; 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_Tactic_SplitIf___hyg_1635____closed__15() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__14; -x_2 = lean_unsigned_to_nat(1635u); +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__14; +x_2 = lean_unsigned_to_nat(1611u); 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_Tactic_SplitIf___hyg_1635_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611_(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_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___closed__4; x_3 = 0; -x_4 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__15; +x_4 = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__15; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } } -lean_object* initialize_Lean_LazyInitExtension(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_Tactic_Cases(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_Tactic_Simp_Main(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -7071,57 +6504,39 @@ LEAN_EXPORT lean_object* initialize_Lean_Meta_Tactic_SplitIf(uint8_t builtin, le lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Lean_LazyInitExtension(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Lean_Meta_Tactic_Cases(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); res = initialize_Lean_Meta_Tactic_Simp_Main(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__1 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__1); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__2 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__2); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__3 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__3); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__4 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__4); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__5 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__5); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__6 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__6); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__7 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__7); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__8 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____lambda__1___closed__8(); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__1 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__1(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__1); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__2 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__2(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__2); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__3); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__4 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__4(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__4); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__5 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__5(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__5); -l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__6 = _init_l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__6(); -lean_mark_persistent(l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4____closed__6); -if (builtin) {res = l_Lean_Meta_SplitIf_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_4_(lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -l_Lean_Meta_SplitIf_ext = lean_io_result_get_value(res); -lean_mark_persistent(l_Lean_Meta_SplitIf_ext); -lean_dec_ref(res); -}l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__1 = _init_l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__1(); -lean_mark_persistent(l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__1); -l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__2 = _init_l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__2(); -lean_mark_persistent(l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__2); -l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__3 = _init_l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__3(); -lean_mark_persistent(l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__3); -l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__4 = _init_l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__4(); -lean_mark_persistent(l_Lean_LazyInitExtension_get___at_Lean_Meta_SplitIf_getSimpContext___spec__1___closed__4); l_Lean_Meta_SplitIf_getSimpContext___closed__1 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__1(); lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__1); +l_Lean_Meta_SplitIf_getSimpContext___closed__2 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__2(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__2); +l_Lean_Meta_SplitIf_getSimpContext___closed__3 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__3(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__3); +l_Lean_Meta_SplitIf_getSimpContext___closed__4 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__4(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__4); +l_Lean_Meta_SplitIf_getSimpContext___closed__5 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__5(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__5); +l_Lean_Meta_SplitIf_getSimpContext___closed__6 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__6(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__6); +l_Lean_Meta_SplitIf_getSimpContext___closed__7 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__7(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__7); +l_Lean_Meta_SplitIf_getSimpContext___closed__8 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__8(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__8); +l_Lean_Meta_SplitIf_getSimpContext___closed__9 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__9(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__9); +l_Lean_Meta_SplitIf_getSimpContext___closed__10 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__10(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__10); +l_Lean_Meta_SplitIf_getSimpContext___closed__11 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__11(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__11); +l_Lean_Meta_SplitIf_getSimpContext___closed__12 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__12(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__12); +l_Lean_Meta_SplitIf_getSimpContext___closed__13 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__13(); +lean_mark_persistent(l_Lean_Meta_SplitIf_getSimpContext___closed__13); +l_Lean_Meta_SplitIf_getSimpContext___closed__14 = _init_l_Lean_Meta_SplitIf_getSimpContext___closed__14(); l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__1 = _init_l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__1(); lean_mark_persistent(l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__1); l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__2 = _init_l_Array_findSomeRevM_x3f_find___at___private_Lean_Meta_Tactic_SplitIf_0__Lean_Meta_SplitIf_discharge_x3f___spec__3___closed__2(); @@ -7218,37 +6633,37 @@ l_Lean_Meta_simpIfLocalDecl___closed__2 = _init_l_Lean_Meta_simpIfLocalDecl___cl lean_mark_persistent(l_Lean_Meta_simpIfLocalDecl___closed__2); l_Lean_Meta_simpIfLocalDecl___closed__3 = _init_l_Lean_Meta_simpIfLocalDecl___closed__3(); lean_mark_persistent(l_Lean_Meta_simpIfLocalDecl___closed__3); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__1 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__1(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__1); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__2 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__2(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__2); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__3 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__3(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__3); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__4 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__4(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__4); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__5 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__5(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__5); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__6 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__6(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__6); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__7 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__7(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__7); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__8 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__8(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__8); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__9 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__9(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__9); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__10 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__10(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__10); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__11 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__11(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__11); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__12 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__12(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__12); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__13 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__13(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__13); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__14 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__14(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__14); -l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__15 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__15(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635____closed__15); -if (builtin) {res = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1635_(lean_io_mk_world()); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__1 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__1(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__1); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__2 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__2(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__2); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__3 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__3(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__3); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__4 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__4(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__4); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__5 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__5(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__5); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__6 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__6(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__6); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__7 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__7(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__7); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__8 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__8(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__8); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__9 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__9(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__9); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__10 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__10(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__10); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__11 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__11(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__11); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__12 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__12(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__12); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__13 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__13(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__13); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__14 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__14(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__14); +l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__15 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__15(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611____closed__15); +if (builtin) {res = l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_SplitIf___hyg_1611_(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/WHNF.c b/stage0/stdlib/Lean/Meta/WHNF.c index d86180f5a619..d889cee14606 100644 --- a/stage0/stdlib/Lean/Meta/WHNF.c +++ b/stage0/stdlib/Lean/Meta/WHNF.c @@ -96,6 +96,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_Meta_smartUnfoldi lean_object* l_Lean_MetavarContext_getDelayedMVarAssignmentCore_x3f(lean_object*, lean_object*); static lean_object* l_Lean_getConstInfoCtor___at___private_Lean_Meta_WHNF_0__Lean_Meta_toCtorWhenStructure___spec__1___closed__4; static lean_object* l_Lean_withTraceNode___at_Lean_Meta_whnfImp___spec__1___lambda__2___closed__1; +lean_object* l_Lean_RecursorVal_getMajorInduct(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Meta_WHNF_0__Lean_Meta_toCtorWhenK___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_WHNF_0__Lean_Meta_isQuotRecStuck_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_markSmartUnfoldingMatchAlt___closed__2; @@ -470,7 +471,6 @@ static lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_reducePow___spec__ LEAN_EXPORT lean_object* l_Lean_Meta_whnfEasyCases___at_Lean_Meta_whnfImp___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_getStuckMVar_x3f___spec__2(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_reduceBinNatOp___lambda__3___closed__12; -lean_object* l_Lean_RecursorVal_getInduct(lean_object*); lean_object* l_Nat_add___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_reduceBinNatOp___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_reduceBinNatOp___lambda__3___closed__4; @@ -1821,7 +1821,8 @@ lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_180; lea x_16 = lean_ctor_get(x_14, 0); x_17 = lean_ctor_get(x_14, 1); x_180 = l_Lean_Expr_getAppFn(x_16); -x_181 = l_Lean_RecursorVal_getInduct(x_1); +lean_inc(x_1); +x_181 = l_Lean_RecursorVal_getMajorInduct(x_1); x_182 = l_Lean_Expr_isConstOf(x_180, x_181); lean_dec(x_181); lean_dec(x_180); @@ -2791,7 +2792,8 @@ lean_inc(x_213); lean_inc(x_212); lean_dec(x_14); x_293 = l_Lean_Expr_getAppFn(x_212); -x_294 = l_Lean_RecursorVal_getInduct(x_1); +lean_inc(x_1); +x_294 = l_Lean_RecursorVal_getMajorInduct(x_1); x_295 = l_Lean_Expr_isConstOf(x_293, x_294); lean_dec(x_294); lean_dec(x_293); @@ -5161,7 +5163,8 @@ lean_inc(x_17); x_18 = lean_ctor_get(x_16, 1); lean_inc(x_18); lean_dec(x_16); -x_19 = l_Lean_RecursorVal_getInduct(x_1); +lean_inc(x_1); +x_19 = l_Lean_RecursorVal_getMajorInduct(x_1); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); diff --git a/stage0/stdlib/Lean/Parser/Command.c b/stage0/stdlib/Lean/Parser/Command.c index ec0a9399ac07..b9d73a2736da 100644 --- a/stage0/stdlib/Lean/Parser/Command.c +++ b/stage0/stdlib/Lean/Parser/Command.c @@ -26,6 +26,7 @@ static lean_object* l_Lean_Parser_Command_computedFields___closed__13; static lean_object* l_Lean_Parser_Command_derivingClasses___closed__6; static lean_object* l_Lean_Parser_Command_declValSimple___closed__12; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_universe_declRange__1(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__6; lean_object* l_Lean_Parser_many1_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_register__tactic__tag_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_initialize_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -40,6 +41,7 @@ static lean_object* l_Lean_Parser_Tactic_open___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiersT_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_openHiding_formatter___closed__4; static lean_object* l_Lean_Parser_Command_declId_formatter___closed__11; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__53; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_parenthesizer__1(lean_object*); static lean_object* l_Lean_Parser_Command_nonrec_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_deriving_formatter___closed__8; @@ -58,6 +60,7 @@ static lean_object* l_Lean_Parser_Tactic_open_formatter___closed__5; static lean_object* l_Lean_Parser_Command_structure___closed__11; static lean_object* l_Lean_Parser_Command_optDefDeriving_parenthesizer___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_quot_declRange__1(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__15; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declId_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_initialize_declRange__1___closed__6; static lean_object* l_Lean_Parser_Command_openSimple___closed__6; @@ -79,7 +82,6 @@ lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_obj static lean_object* l___regBuiltin_Lean_Parser_Command_attribute_declRange__1___closed__6; static lean_object* l_Lean_Parser_Command_exit_parenthesizer___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structImplicitBinder; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__49; LEAN_EXPORT lean_object* l_Lean_Parser_Command_include; static lean_object* l_Lean_Parser_Command_printEqns_formatter___closed__1; static lean_object* l_Lean_Parser_Command_end___closed__4; @@ -148,11 +150,11 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_eoi; static lean_object* l_Lean_Parser_Command_declSig_formatter___closed__1; static lean_object* l_Lean_Parser_Command_axiom_formatter___closed__4; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__5; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__48; static lean_object* l_Lean_Parser_Command_import___closed__1; static lean_object* l_Lean_Parser_Command_ctor_parenthesizer___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_open_declRange__1___closed__2; lean_object* l_Lean_Parser_Term_matchAlts_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__23; static lean_object* l_Lean_Parser_Command_instance___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_include_formatter__1___closed__2; static lean_object* l_Lean_Parser_Command_variable_formatter___closed__5; @@ -160,7 +162,6 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter static lean_object* l_Lean_Parser_Command_namedPrio___closed__10; static lean_object* l___regBuiltin_Lean_Parser_Command_end_parenthesizer__1___closed__2; static lean_object* l_Lean_Parser_Command_whereStructInst___closed__4; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__17; LEAN_EXPORT lean_object* l_Lean_Parser_Command_classTk; static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_formatter__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_tactic__extension_declRange__1___closed__6; @@ -190,6 +191,7 @@ static lean_object* l_Lean_Parser_Command_extends_parenthesizer___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_structureTk_parenthesizer__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_in; static lean_object* l_Lean_Parser_Command_computedField_formatter___closed__5; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__52; static lean_object* l_Lean_Parser_Command_theorem_parenthesizer___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_mutual_declRange__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_universe_formatter__1___closed__2; @@ -209,7 +211,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_import_parenthesizer__1__ lean_object* l_Lean_Parser_Term_attrInstance_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_check__failure_formatter__1___closed__1; lean_object* l_Lean_addBuiltinDocString(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__2; static lean_object* l_Lean_Parser_Command_declSig_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_computedFields_formatter__1___closed__1; lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -261,6 +263,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_formatter_ static lean_object* l_Lean_Parser_Command_namedPrio___closed__6; static lean_object* l_Lean_Parser_Command_printTacTags_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_tactic__extension___closed__7; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__20; static lean_object* l_Lean_Parser_Command_structImplicitBinder___closed__11; static lean_object* l_Lean_Parser_Command_universe_formatter___closed__2; lean_object* l_Lean_PrettyPrinter_Formatter_orelse_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -269,8 +272,10 @@ static lean_object* l_Lean_Parser_Command_openSimple___closed__2; lean_object* l_Lean_Parser_Term_whereDecls_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_section; static lean_object* l___regBuiltin_Lean_Parser_Command_register__tactic__tag_declRange__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__1; static lean_object* l_Lean_Parser_Command_addDocString___closed__3; static lean_object* l_Lean_Parser_Command_moduleDoc_formatter___closed__8; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__50; static lean_object* l___regBuiltin_Lean_Parser_Command_eval_docString__1___closed__1; static lean_object* l_Lean_Parser_Command_noncomputable_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_tactic__extension_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -279,13 +284,12 @@ static lean_object* l_Lean_Parser_Command_openOnly_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_variable_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__18; static lean_object* l___regBuiltin_Lean_Parser_Command_addDocString_declRange__1___closed__2; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__54; static lean_object* l_Lean_Parser_Command_set__option___closed__4; static lean_object* l_Lean_Parser_Command_print___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_export_declRange__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__2; static lean_object* l_Lean_Parser_Command_declValSimple_parenthesizer___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_declRange__1___closed__5; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__25; static lean_object* l___regBuiltin_Lean_Parser_Command_structure_formatter__1___closed__1; static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__13; static lean_object* l___regBuiltin_Lean_Parser_Command_eval_declRange__1___closed__6; @@ -300,7 +304,6 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__14; static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__9; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__13; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__15; static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_declRange__1___closed__2; static lean_object* l_Lean_Parser_Command_abbrev___closed__9; @@ -366,6 +369,7 @@ static lean_object* l_Lean_Parser_Command_structImplicitBinder_parenthesizer___c static lean_object* l_Lean_Parser_Command_declSig___closed__9; static lean_object* l_Lean_Parser_Command_optDefDeriving_formatter___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_omit_parenthesizer__1(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__36; static lean_object* l_Lean_Parser_Command_deriving___closed__11; static lean_object* l_Lean_Parser_Command_structFields_formatter___closed__6; static lean_object* l_Lean_Parser_Command_structSimpleBinder_formatter___closed__3; @@ -385,6 +389,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_eraseAttr_formatter(lean_object*, static lean_object* l_Lean_Parser_Command_whereStructInst___closed__20; static lean_object* l___regBuiltin_Lean_Parser_Command_opaque_formatter__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_declRange__1___closed__4; +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3092_(lean_object*); static lean_object* l_Lean_Parser_Command_synth_formatter___closed__2; static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__12; static lean_object* l_Lean_Parser_Command_theorem___closed__9; @@ -482,7 +487,6 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_openHiding_parenthesizer_ static lean_object* l___regBuiltin_Lean_Parser_Term_quot__1___closed__1; static lean_object* l_Lean_Parser_Command_initialize_parenthesizer___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_ctor; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__27; static lean_object* l_Lean_Parser_Command_init__quot___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_variable_parenthesizer__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_export_declRange__1___closed__4; @@ -525,7 +529,6 @@ static lean_object* l_Lean_Parser_Term_quot_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiers_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_attribute_parenthesizer___closed__10; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__40; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_ctor_parenthesizer__1(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_noncomputable_formatter__1(lean_object*); static lean_object* l_Lean_Parser_Command_instance___closed__8; @@ -583,6 +586,7 @@ static lean_object* l_Lean_Parser_Command_moduleDoc___closed__4; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__10; static lean_object* l_Lean_Parser_Command_noncomputableSection_formatter___closed__7; static lean_object* l_Lean_Parser_Command_open___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__26; lean_object* l_instDecidableEqChar___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_quot_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_abbrev_formatter___closed__5; @@ -594,6 +598,7 @@ static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___close static lean_object* l_Lean_Parser_Command_structInstBinder___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_declRange__1___closed__3; static lean_object* l_Lean_Parser_Command_openRenaming___closed__4; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__11; static lean_object* l_Lean_Parser_Command_moduleDoc_formatter___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_docString__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_declRange__1___closed__2; @@ -611,6 +616,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_declRange__1_ static lean_object* l_Lean_Parser_Command_end___closed__3; static lean_object* l_Lean_Parser_Command_register__tactic__tag_formatter___closed__2; static lean_object* l_Lean_Parser_Command_computedField___closed__1; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__44; static lean_object* l_Lean_Parser_Command_nonrec___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_quot_declRange__1___closed__2; static lean_object* l_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__2; @@ -624,7 +630,6 @@ static lean_object* l_Lean_Parser_Command_tactic__extension___closed__3; static lean_object* l_Lean_Parser_Command_whereStructField_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_parenthesizer__1___closed__1; static lean_object* l_Lean_Parser_Command_whereStructInst___closed__11; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__47; LEAN_EXPORT lean_object* l_Lean_Parser_Command_print; static lean_object* l_Lean_Parser_Term_precheckedQuot___closed__4; static lean_object* l_Lean_Parser_Command_abbrev_parenthesizer___closed__7; @@ -652,10 +657,11 @@ static lean_object* l_Lean_Parser_Command_noncomputableSection___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_register__tactic__tag_parenthesizer__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_variable_parenthesizer__1(lean_object*); static lean_object* l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__38; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structureTk_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structFields_formatter__1(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_ctor_formatter__1___closed__1; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__44; static lean_object* l_Lean_Parser_Command_structImplicitBinder_formatter___closed__8; static lean_object* l_Lean_Parser_Command_derivingClasses___closed__5; static lean_object* l_Lean_Parser_Command_optDefDeriving_parenthesizer___closed__7; @@ -668,6 +674,7 @@ lean_object* l_Lean_Parser_andthenFn(lean_object*, lean_object*, lean_object*, l static lean_object* l_Lean_Parser_Tactic_set__option_formatter___closed__2; static lean_object* l_Lean_Parser_Command_classInductive___closed__11; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__4; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__45; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___closed__6; static lean_object* l_Lean_Parser_Command_instance___closed__1; static lean_object* l_Lean_Parser_Command_whereStructInst_formatter___closed__3; @@ -679,6 +686,7 @@ static lean_object* l_Lean_Parser_Command_namedPrio___closed__4; static lean_object* l_Lean_Parser_Command_declModifiers___closed__4; static lean_object* l_Lean_Parser_Command_register__tactic__tag_formatter___closed__7; lean_object* l_Lean_Parser_withOpenFn(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__51; lean_object* l_Lean_Parser_withOpen_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_abbrev___closed__8; static lean_object* l_Lean_Parser_Command_theorem_formatter___closed__2; @@ -779,6 +787,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_namespace_declRange__1___ static lean_object* l_Lean_Parser_Command_declId___closed__14; LEAN_EXPORT lean_object* l_Lean_Parser_Command_optDeriving_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_nonrec_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__5; static lean_object* l_Lean_Parser_Command_optNamedPrio___closed__1; static lean_object* l_Lean_Parser_Command_printAxioms___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_import_formatter__1(lean_object*); @@ -791,6 +800,7 @@ static lean_object* l_Lean_Parser_Command_nonrec_formatter___closed__1; static lean_object* l_Lean_Parser_Command_noncomputableSection___closed__4; static lean_object* l_Lean_Parser_Command_optDeriving___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Command_mutual_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__22; static lean_object* l_Lean_Parser_Command_optDeriving_formatter___closed__2; static lean_object* l_Lean_Parser_Command_quot_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_ctor_formatter___closed__11; @@ -837,6 +847,7 @@ static lean_object* l_Lean_Parser_Tactic_set__option___closed__7; lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_check__failure_parenthesizer___closed__2; lean_object* l_Lean_Parser_setExpected(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__33; static lean_object* l_Lean_Parser_Command_in_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_optDefDeriving_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_include___closed__8; @@ -849,6 +860,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_set__option_declRange__1_ static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_structFields_formatter__1___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_exit_formatter__1___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__8; static lean_object* l_Lean_Parser_Command_set__option_formatter___closed__6; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_eoi_formatter___closed__2; @@ -873,11 +885,11 @@ static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__15; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_private_formatter__1(lean_object*); static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__8; static lean_object* l_Lean_Parser_Command_optDeriving_formatter___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1(lean_object*); static lean_object* l_Lean_Parser_Command_initialize_formatter___closed__11; static lean_object* l___regBuiltin_Lean_Parser_Command_import_declRange__1___closed__5; static lean_object* l_Lean_Parser_Command_variable___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_register__tactic__tag_declRange__1___closed__7; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__2; static lean_object* l_Lean_Parser_Command_derivingClasses___closed__8; static lean_object* l_Lean_Parser_Command_partial_formatter___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structInstBinder_parenthesizer__1(lean_object*); @@ -903,6 +915,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_initialize_parenthesizer_ LEAN_EXPORT lean_object* l_Lean_Parser_Command_declValSimple_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_open___closed__3; static lean_object* l_Lean_Parser_Command_declVal_formatter___closed__3; +static lean_object* l_Lean_Parser_Command_version___closed__1; static lean_object* l_Lean_Parser_Command_structFields_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_printTacTags_formatter___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_initialize_formatter__1(lean_object*); @@ -942,9 +955,7 @@ static lean_object* l_Lean_Parser_Command_open_formatter___closed__5; static lean_object* l_Lean_Parser_Term_precheckedQuot___closed__7; static lean_object* l_Lean_Parser_Command_quot___closed__11; static lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_formatter__1___closed__1; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__24; static lean_object* l___regBuiltin_Lean_Parser_Command_classInductive_parenthesizer__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097_(lean_object*); static lean_object* l_Lean_Parser_Command_printAxioms_parenthesizer___closed__3; lean_object* l_Lean_Parser_priorityParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_deriving___closed__8; @@ -953,14 +964,12 @@ static lean_object* l_Lean_Parser_Command_ctor___closed__13; static lean_object* l_Lean_Parser_Command_computedField_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_declaration___closed__8; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__17; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__31; static lean_object* l_Lean_Parser_Command_check_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_structFields___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_end_formatter__1___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_exit__1(lean_object*); static lean_object* l_Lean_Parser_Command_print___closed__9; static lean_object* l_Lean_Parser_Command_computedField___closed__11; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__22; static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_precheckedQuot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_universe_declRange__1___closed__5; @@ -1023,7 +1032,6 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_tactic__extension; static lean_object* l_Lean_Parser_Command_openOnly___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declId_parenthesizer__1(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_exit_declRange__1___closed__6; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__28; static lean_object* l_Lean_Parser_Command_omit___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_printEqns_formatter__1___closed__2; static lean_object* l_Lean_Parser_Command_structure___closed__23; @@ -1073,7 +1081,6 @@ static lean_object* l_Lean_Parser_Command_open_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_synth_parenthesizer__1___closed__2; static lean_object* l_Lean_Parser_Command_structInstBinder___closed__14; static lean_object* l_Lean_Parser_Command_eval___closed__4; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__37; static lean_object* l_Lean_Parser_Command_printEqns_formatter___closed__3; static lean_object* l_Lean_Parser_Command_attribute_formatter___closed__9; static lean_object* l_Lean_Parser_Command_definition_formatter___closed__9; @@ -1146,7 +1153,6 @@ static lean_object* l_Lean_Parser_Command_declValEqns_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__23; static lean_object* l___regBuiltin_Lean_Parser_Command_declaration_declRange__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_tactic__extension_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__46; static lean_object* l_Lean_Parser_Command_derivingClasses_formatter___closed__7; static lean_object* l_Lean_Parser_Term_quot___closed__17; static lean_object* l_Lean_Parser_Command_printEqns___closed__10; @@ -1236,6 +1242,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_structInstBinder_formatte LEAN_EXPORT lean_object* l_Lean_Parser_Command_structFields; static lean_object* l_Lean_Parser_Command_in_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_openScoped_parenthesizer___closed__1; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__24; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_check__failure___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option_declRange__1___closed__4; @@ -1244,14 +1251,15 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_import_declRange__1___clo static lean_object* l_Lean_Parser_Command_classInductive_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_set__option___closed__8; static lean_object* l_Lean_Parser_Command_ctor_parenthesizer___closed__1; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__17; static lean_object* l_Lean_Parser_Command_structure___closed__15; static lean_object* l_Lean_Parser_Command_computedField___closed__7; static lean_object* l_Lean_Parser_Command_optDeriving___closed__2; static lean_object* l_Lean_Parser_Command_optDefDeriving_formatter___closed__4; static lean_object* l_Lean_Parser_Command_attribute___closed__12; static lean_object* l_Lean_Parser_Command_set__option_parenthesizer___closed__8; +static lean_object* l_Lean_Parser_Command_version_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter__1(lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__11; static lean_object* l_Lean_Parser_Command_check___closed__8; static lean_object* l_Lean_Parser_Command_extends___closed__1; static lean_object* l_Lean_Parser_Command_declId___closed__19; @@ -1275,6 +1283,7 @@ static lean_object* l_Lean_Parser_Command_optDeriving___closed__7; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__15; static lean_object* l___regBuiltin_Lean_Parser_Command_print_declRange__1___closed__2; static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__6; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__7; static lean_object* l_Lean_Parser_Command_import_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_structSimpleBinder_formatter___closed__5; static lean_object* l_Lean_Parser_Term_open___closed__1; @@ -1313,7 +1322,6 @@ lean_object* l_Lean_Parser_commandParser_parenthesizer(lean_object*, lean_object static lean_object* l_Lean_Parser_Command_structInstBinder___closed__6; static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__10; static lean_object* l_Lean_Parser_Command_eoi___closed__1; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__30; static lean_object* l_Lean_Parser_Term_set__option___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_declModifiers_docString__1___closed__2; static lean_object* l_Lean_Parser_Command_nonrec___closed__4; @@ -1353,7 +1361,6 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_addDocString_declRange__1 static lean_object* l_Lean_Parser_Command_optDefDeriving_parenthesizer___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_end_declRange__1___closed__7; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__51; static lean_object* l_Lean_Parser_Command_optDefDeriving___closed__5; static lean_object* l_Lean_Parser_Command_quot___closed__14; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__18; @@ -1414,6 +1421,7 @@ static lean_object* l_Lean_Parser_Term_quot___closed__2; static lean_object* l_Lean_Parser_Command_end_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_declSig___closed__6; static lean_object* l_Lean_Parser_Command_moduleDoc_formatter___closed__5; +LEAN_EXPORT lean_object* l_Lean_Parser_Command_version; static lean_object* l_Lean_Parser_Command_whereStructInst___closed__13; static lean_object* l___regBuiltin_Lean_Parser_Command_variable_formatter__1___closed__2; lean_object* l_Lean_Parser_withOpen_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1423,6 +1431,7 @@ static lean_object* l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_init__quot___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_optDeriving_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_computedFields; +static lean_object* l_Lean_Parser_Command_version_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_mutual_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_classInductive___closed__13; static lean_object* l_Lean_Parser_Command_axiom___closed__4; @@ -1434,6 +1443,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection static lean_object* l_Lean_Parser_Command_export___closed__3; static lean_object* l_Lean_Parser_Command_opaque___closed__6; static lean_object* l_Lean_Parser_Command_open_parenthesizer___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__40; static lean_object* l___regBuiltin_Lean_Parser_Command_whereStructField_formatter__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_derivingClasses; static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_declRange__1___closed__1; @@ -1454,6 +1464,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_declRange__1___closed LEAN_EXPORT lean_object* l_Lean_Parser_Term_precheckedQuot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_partial_parenthesizer__1___closed__2; static lean_object* l_Lean_Parser_Command_universe_formatter___closed__4; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__21; static lean_object* l_Lean_Parser_Command_register__tactic__tag_parenthesizer___closed__4; lean_object* l_Lean_Parser_Term_binderIdent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_declVal_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1490,6 +1501,7 @@ static lean_object* l_Lean_Parser_Tactic_set__option___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_printTacTags_formatter__1___closed__2; static lean_object* l_Lean_Parser_Command_openOnly_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_unsafe_formatter__1___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__41; static lean_object* l_Lean_Parser_Command_openRenamingItem_formatter___closed__1; static lean_object* l_Lean_Parser_Command_quot___closed__7; static lean_object* l_Lean_Parser_Command_whereStructField___closed__1; @@ -1528,7 +1540,6 @@ static lean_object* l_Lean_Parser_Command_printTacTags___closed__7; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declaration_declRange__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_check_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_in_parenthesizer__1___closed__2; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__19; static lean_object* l_Lean_Parser_Command_mutual___closed__13; static lean_object* l___regBuiltin_Lean_Parser_Command_open_declRange__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_formatter__1___closed__2; @@ -1621,6 +1632,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_deriving__1(lean_obj LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_tactic__extension_declRange__1(lean_object*); static lean_object* l_Lean_Parser_Command_register__tactic__tag_formatter___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_whereStructInst_parenthesizer__1(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__47; static lean_object* l_Lean_Parser_Command_structureTk_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openOnly_parenthesizer__1(lean_object*); static lean_object* l_Lean_Parser_Command_structSimpleBinder_formatter___closed__4; @@ -1652,7 +1664,6 @@ static lean_object* l_Lean_Parser_Command_structExplicitBinder_parenthesizer___c static lean_object* l_Lean_Parser_Tactic_open_parenthesizer___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_set__option_formatter__1___closed__1; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__24; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__45; static lean_object* l_Lean_Parser_Command_section_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_protected_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_manyIndent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1663,11 +1674,10 @@ extern lean_object* l_Lean_Parser_Term_attrKind; static lean_object* l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_whereStructInst___closed__24; LEAN_EXPORT lean_object* l_Lean_Parser_Command_import_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__42; lean_object* l_Lean_ppLine_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_inductive_formatter__1___closed__1; static lean_object* l_Lean_Parser_Command_structInstBinder___closed__13; -LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3073_(lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__21; static lean_object* l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openDecl_docString__1(lean_object*); static lean_object* l_Lean_Parser_Command_register__tactic__tag___closed__7; @@ -1697,6 +1707,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_export_declRange__1___clo static lean_object* l_Lean_Parser_Command_ctor_parenthesizer___closed__5; LEAN_EXPORT uint8_t l_Lean_Parser_Command_declId___lambda__1(uint32_t); static lean_object* l_Lean_Parser_Command_printAxioms___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_version_docString__1___closed__1; static lean_object* l_Lean_Parser_Command_register__tactic__tag___closed__3; static lean_object* l_Lean_Parser_Command_addDocString___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_set__option_parenthesizer__1___closed__2; @@ -1714,6 +1725,7 @@ LEAN_EXPORT uint8_t l___private_Lean_Parser_Command_0__Lean_Parser_Command_skipU static lean_object* l___regBuiltin_Lean_Parser_Command_structSimpleBinder_formatter__1___closed__1; lean_object* l_Lean_Parser_notFollowedBy(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structCtor_formatter___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__37; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_deriving_declRange__1(lean_object*); static lean_object* l_Lean_Parser_Command_set__option_parenthesizer___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_theorem_formatter__1(lean_object*); @@ -1721,7 +1733,6 @@ static lean_object* l_Lean_Parser_Command_omit_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_structureTk_formatter___closed__3; static lean_object* l_Lean_Parser_Command_declBody___closed__5; static lean_object* l_Lean_Parser_Command_abbrev___closed__6; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__34; static lean_object* l_Lean_Parser_Command_noncomputable___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_formatter__1___closed__1; static lean_object* l_Lean_Parser_Command_attribute___closed__7; @@ -1743,7 +1754,6 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_formatter__1___c static lean_object* l_Lean_Parser_Command_axiom_formatter___closed__5; lean_object* l_Lean_Parser_symbol(lean_object*); static lean_object* l_Lean_Parser_Command_printAxioms_parenthesizer___closed__5; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__9; static lean_object* l_Lean_Parser_Command_namedPrio___closed__11; static lean_object* l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_opaque_formatter__1___closed__2; @@ -1751,10 +1761,11 @@ static lean_object* l_Lean_Parser_Command_export_parenthesizer___closed__4; lean_object* l_Lean_Parser_Term_typeSpec_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_precheckedQuot_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_initializeKeyword_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_version___closed__5; static lean_object* l_Lean_Parser_Command_definition_formatter___closed__4; static lean_object* l_Lean_Parser_Command_structFields___closed__13; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__12; static lean_object* l_Lean_Parser_Command_declVal___closed__4; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__32; LEAN_EXPORT lean_object* l_Lean_Parser_Command_addDocString; static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__7; static lean_object* l_Lean_Parser_Command_set__option_formatter___closed__1; @@ -1781,7 +1792,6 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputable_formatter__ extern lean_object* l_Lean_Parser_Tactic_tacticSeq; static lean_object* l_Lean_Parser_Term_quot___closed__3; static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__4; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__15; static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_parenthesizer__1___closed__1; static lean_object* l_Lean_Parser_Command_check_formatter___closed__4; static lean_object* l_Lean_Parser_Command_printAxioms___closed__1; @@ -1826,6 +1836,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_quot_parenthesizer__1(l static lean_object* l___regBuiltin_Lean_Parser_Command_inductive_parenthesizer__1___closed__2; static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__1; static lean_object* l_Lean_Parser_Command_structImplicitBinder_formatter___closed__3; +static lean_object* l_Lean_Parser_Command_version_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_set__option_parenthesizer___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_export_parenthesizer__1___closed__1; static lean_object* l_Lean_Parser_Command_universe_parenthesizer___closed__2; @@ -1841,6 +1852,7 @@ static lean_object* l_Lean_Parser_Tactic_open___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structExplicitBinder_formatter__1(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_parenthesizer__1___closed__2; static lean_object* l_Lean_Parser_Command_derivingClasses_parenthesizer___closed__6; +static lean_object* l_Lean_Parser_Command_version___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Command_register__tactic__tag_declRange__1___closed__2; static lean_object* l_Lean_Parser_Command_partial___closed__3; static lean_object* l_Lean_Parser_Command_moduleDoc___closed__2; @@ -1849,6 +1861,7 @@ static lean_object* l_Lean_Parser_Command_attribute_formatter___closed__4; static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__14; static lean_object* l___regBuiltin_Lean_Parser_Command_declaration_declRange__1___closed__2; static lean_object* l_Lean_Parser_Command_noncomputableSection_formatter___closed__1; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__49; static lean_object* l_Lean_Parser_Command_inductive___closed__10; static lean_object* l___regBuiltin_Lean_Parser_Tactic_open__1___closed__2; static lean_object* l_Lean_Parser_Command_printAxioms_parenthesizer___closed__2; @@ -1864,6 +1877,7 @@ static lean_object* l_Lean_Parser_Command_instance_parenthesizer___closed__11; static lean_object* l_Lean_Parser_Command_openRenamingItem_formatter___closed__2; static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Command_include___closed__3; +static lean_object* l_Lean_Parser_Command_version___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_variable_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_export_formatter___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_declRange__1___closed__4; @@ -1882,13 +1896,14 @@ static lean_object* l_Lean_Parser_Command_evalBang___closed__5; static lean_object* l_Lean_Parser_Command_quot_formatter___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter__1___closed__1; static lean_object* l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__11; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__12; static lean_object* l_Lean_Parser_Command_openRenaming___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structCtor; static lean_object* l___regBuiltin_Lean_Parser_Command_abbrev_parenthesizer__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openDecl_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__29; extern lean_object* l_Lean_Parser_Command_docComment; static lean_object* l_Lean_Parser_Command_openRenaming___closed__12; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__50; static lean_object* l_Lean_Parser_Command_deriving_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_variable_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_tactic__extension_parenthesizer___closed__4; @@ -1920,6 +1935,7 @@ static lean_object* l_Lean_Parser_Command_eoi_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_declRange__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_openDecl_docString__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declBody; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__25; static lean_object* l_Lean_Parser_Command_unsafe_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_parenthesizer__1(lean_object*); static lean_object* l_Lean_Parser_Term_quot_formatter___closed__4; @@ -1965,6 +1981,7 @@ static lean_object* l_Lean_Parser_Command_structFields___closed__11; static lean_object* l_Lean_Parser_Command_ctor_parenthesizer___closed__11; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiersF; static lean_object* l_Lean_Parser_Command_deriving___closed__15; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__9; static lean_object* l_Lean_Parser_Tactic_set__option_formatter___closed__3; static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__2; static lean_object* l_Lean_Parser_Command_tactic__extension___closed__4; @@ -1981,6 +1998,7 @@ static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__15; static lean_object* l_Lean_Parser_Command_attribute___closed__4; static lean_object* l_Lean_Parser_Command_set__option_formatter___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_section_parenthesizer__1(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__54; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_export_formatter__1(lean_object*); static lean_object* l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_classInductive___closed__15; @@ -2017,7 +2035,6 @@ static lean_object* l_Lean_Parser_Command_initialize___closed__5; static lean_object* l_Lean_Parser_Tactic_open_parenthesizer___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_openRenamingItem_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__10; static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_parenthesizer__1___closed__1; lean_object* l_Lean_Parser_Term_attrKind_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_partial___closed__4; @@ -2033,10 +2050,12 @@ static lean_object* l_Lean_Parser_Command_print_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declValEqns_formatter__1(lean_object*); static lean_object* l_Lean_Parser_Command_initialize___closed__11; static lean_object* l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer__1___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__46; static lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option_formatter__1___closed__1; static lean_object* l_Lean_Parser_Command_noncomputable_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_optDeriving___closed__4; +static lean_object* l_Lean_Parser_Command_version___closed__6; static lean_object* l_Lean_Parser_Command_namespace_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_namedPrio_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_declaration_formatter__1___closed__1; @@ -2052,6 +2071,7 @@ static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__ lean_object* l_Lean_Parser_many_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__7; lean_object* l_Lean_Parser_Term_attributes_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structExplicitBinder; static lean_object* l_Lean_Parser_Command_initialize_formatter___closed__5; static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__5; @@ -2073,6 +2093,7 @@ static lean_object* l_Lean_Parser_Command_structureTk___closed__7; static lean_object* l_Lean_Parser_Command_definition_parenthesizer___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_declRange__1___closed__7; static lean_object* l_Lean_Parser_Command_ctor___closed__5; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__13; static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter__1___closed__2; static lean_object* l_Lean_Parser_Command_axiom___closed__9; static lean_object* l_Lean_Parser_Command_initialize_formatter___closed__1; @@ -2117,7 +2138,6 @@ static lean_object* l_Lean_Parser_Command_openSimple_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_quot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_printTacTags___closed__1; static lean_object* l_Lean_Parser_Command_declValSimple_formatter___closed__10; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__35; static lean_object* l_Lean_Parser_Command_declSig___closed__3; static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_computedFields___closed__12; @@ -2133,6 +2153,7 @@ static lean_object* l_Lean_Parser_Command_instance_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_quot___closed__4; static lean_object* l_Lean_Parser_Command_printTacTags_formatter___closed__5; static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__8; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__28; static lean_object* l_Lean_Parser_Command_structSimpleBinder___closed__1; static lean_object* l_Lean_Parser_Command_opaque___closed__8; static lean_object* l_Lean_Parser_Command_inductive___closed__12; @@ -2313,7 +2334,6 @@ static lean_object* l_Lean_Parser_Command_abbrev___closed__5; static lean_object* l_Lean_Parser_Command_namespace___closed__1; static lean_object* l_Lean_Parser_Command_whereStructInst_formatter___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_register__tactic__tag_declRange__1(lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__52; static lean_object* l_Lean_Parser_Command_printTacTags___closed__9; static lean_object* l_Lean_Parser_Command_openRenaming_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_openSimple_formatter__1___closed__2; @@ -2371,6 +2391,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_universe_formatter__ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declId_formatter__1(lean_object*); static lean_object* l_Lean_Parser_Command_moduleDoc_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_omit_formatter__1(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_declVal_docString__1___closed__3; static lean_object* l_Lean_Parser_Command_opaque_formatter___closed__4; static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__1; @@ -2397,13 +2418,11 @@ static lean_object* l_Lean_Parser_Command_whereStructInst___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declVal_docString__1(lean_object*); static lean_object* l_Lean_Parser_Command_eraseAttr_formatter___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_classTk_formatter__1(lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__6; static lean_object* l_Lean_Parser_Command_openHiding_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_check__failure_formatter___closed__3; lean_object* l_Lean_Parser_many(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openRenamingItem_formatter__1(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_register__tactic__tag_docString__1(lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__8; static lean_object* l___regBuiltin_Lean_Parser_Command_eoi_parenthesizer__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_synth_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_moduleDoc___closed__3; @@ -2479,6 +2498,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_openSimple_parenthesizer_ static lean_object* l_Lean_Parser_Command_exit_formatter___closed__3; static lean_object* l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__7; lean_object* l_Lean_ppSpace_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__31; LEAN_EXPORT lean_object* l_Lean_Parser_Command_initialize; static lean_object* l_Lean_Parser_Command_openDecl___closed__4; static lean_object* l_Lean_Parser_Command_declValSimple_formatter___closed__4; @@ -2490,6 +2510,7 @@ static lean_object* l_Lean_Parser_Command_extends___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Command_classTk_formatter__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_theorem_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_version_docString__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_import; static lean_object* l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_quot_parenthesizer___closed__2; @@ -2536,6 +2557,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_universe_parenthesizer(lean_objec LEAN_EXPORT lean_object* l_Lean_Parser_Command_printTacTags_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_initialize_declRange__1___closed__5; static lean_object* l_Lean_Parser_Tactic_open_parenthesizer___closed__8; +static lean_object* l_Lean_Parser_Command_version___closed__4; static lean_object* l_Lean_Parser_Command_openScoped_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_inductive___closed__4; static lean_object* l_Lean_Parser_Command_attribute___closed__5; @@ -2563,20 +2585,18 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_structInstBinder_formatter(lean_o static lean_object* l___regBuiltin_Lean_Parser_Command_printTacTags_declRange__1___closed__4; static lean_object* l_Lean_Parser_Command_declId_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_classInductive___closed__12; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__20; LEAN_EXPORT lean_object* l_Lean_Parser_Command_namespace_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_namedPrio_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__3; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__53; static lean_object* l___regBuiltin_Lean_Parser_Command_quot_docString__1___closed__1; static lean_object* l_Lean_Parser_Command_declId_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_classTk___closed__5; static lean_object* l_Lean_Parser_Command_tactic__extension_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_nonrec_formatter__1___closed__2; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_declRange__1___closed__5; static lean_object* l_Lean_Parser_Command_printTacTags___closed__12; lean_object* l_Lean_Parser_sepBy1_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__27; static lean_object* l_Lean_Parser_Command_theorem_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_section_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_optDeriving___closed__6; @@ -2640,11 +2660,12 @@ static lean_object* l_Lean_Parser_Command_eoi_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_printEqns; static lean_object* l___regBuiltin_Lean_Parser_Command_mutual_parenthesizer__1___closed__1; static lean_object* l_Lean_Parser_Command_tactic__extension___closed__5; +static lean_object* l_Lean_Parser_Command_version___closed__2; static lean_object* l_Lean_Parser_Command_structImplicitBinder___closed__5; static lean_object* l_Lean_Parser_Command_mutual___closed__14; static lean_object* l_Lean_Parser_Command_ctor_parenthesizer___closed__2; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__32; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer__1(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_open_declRange__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_eval; static lean_object* l_Lean_Parser_Command_whereStructField___closed__5; @@ -2673,6 +2694,7 @@ static lean_object* l_Lean_Parser_Command_openDecl___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_example_parenthesizer__1___closed__2; static lean_object* l_Lean_Parser_Command_definition___closed__12; static lean_object* l_Lean_Parser_Command_definition___closed__5; +LEAN_EXPORT lean_object* l_Lean_Parser_Command_version_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Command_optionValue_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_check__failure_formatter___closed__4; @@ -2745,6 +2767,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Parser_Command_0__Lean_Parser_Command_ extern lean_object* l_Lean_PrettyPrinter_Parenthesizer_parenthesizerAliasesRef; static lean_object* l_Lean_Parser_Command_declValSimple_parenthesizer___closed__7; lean_object* l_Lean_Parser_withAntiquotSpliceAndSuffix(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__35; static lean_object* l_Lean_Parser_Command_evalBang_formatter___closed__4; static lean_object* l_Lean_Parser_Command_set__option_formatter___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_quot_formatter__1___closed__2; @@ -2777,7 +2800,6 @@ lean_object* l_Lean_Parser_Term_instBinder_parenthesizer(lean_object*, lean_obje lean_object* l_Lean_Parser_withoutPosition_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_addDocString_formatter___closed__5; static lean_object* l_Lean_Parser_Term_precheckedQuot___closed__2; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__48; static lean_object* l_Lean_Parser_Command_variable___closed__6; static lean_object* l_Lean_Parser_Command_initialize___closed__13; static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__12; @@ -2873,6 +2895,7 @@ static lean_object* l_Lean_Parser_Command_export_formatter___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_private_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_register__tactic__tag__1(lean_object*); static lean_object* l_Lean_Parser_Command_structFields___closed__16; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__16; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structCtor_parenthesizer__1(lean_object*); static lean_object* l_Lean_Parser_Command_in_formatter___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_tactic__extension_declRange__1___closed__7; @@ -2882,6 +2905,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_openRenaming; static lean_object* l___regBuiltin_Lean_Parser_Command_optDeriving_formatter__1___closed__2; static lean_object* l_Lean_Parser_Command_structInstBinder_formatter___closed__6; static lean_object* l_Lean_Parser_Command_openScoped___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_version_formatter__1(lean_object*); static lean_object* l_Lean_Parser_Command_initialize_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Tactic_set__option_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_quot_parenthesizer___closed__3; @@ -2915,12 +2939,10 @@ static lean_object* l_Lean_Parser_Command_open_formatter___closed__2; static lean_object* l_Lean_Parser_Command_axiom___closed__10; static lean_object* l_Lean_Parser_Command_computedField___closed__5; static lean_object* l_Lean_Parser_Command_namedPrio_formatter___closed__6; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__16; LEAN_EXPORT lean_object* l_Lean_Parser_Command_eraseAttr; static lean_object* l_Lean_Parser_Command_declId_formatter___closed__4; static lean_object* l_Lean_Parser_Command_synth___closed__2; static lean_object* l_Lean_Parser_Command_structImplicitBinder___closed__7; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_formatter__1___closed__2; static lean_object* l_Lean_Parser_Command_structure___closed__8; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_end_parenthesizer__1(lean_object*); @@ -2928,13 +2950,11 @@ static lean_object* l_Lean_Parser_Command_eoi_formatter___closed__6; static lean_object* l_Lean_Parser_Command_namedPrio_formatter___closed__2; static lean_object* l_Lean_Parser_Command_openSimple___closed__5; static lean_object* l_Lean_Parser_Command_initialize_formatter___closed__6; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__26; LEAN_EXPORT lean_object* l_Lean_Parser_Command_register__tactic__tag_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_computedField_parenthesizer___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Command_namespace_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__16; static lean_object* l_Lean_Parser_Command_namedPrio_formatter___closed__12; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__41; static lean_object* l_Lean_Parser_Command_printAxioms_parenthesizer___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_open_formatter__1(lean_object*); static lean_object* l_Lean_Parser_Command_exit___closed__1; @@ -2993,6 +3013,7 @@ static lean_object* l_Lean_Parser_Command_quot___closed__5; static lean_object* l_Lean_Parser_Command_check___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_protected; static lean_object* l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__39; static lean_object* l_Lean_Parser_Command_derivingClasses_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_print_formatter___closed__1; @@ -3018,6 +3039,7 @@ static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__3; lean_object* l_Lean_Parser_Tactic_tacticSeq_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_quot_formatter___closed__6; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__14; static lean_object* l_Lean_Parser_Command_print___closed__10; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_computedFields_parenthesizer__1(lean_object*); static lean_object* l_Lean_Parser_Term_precheckedQuot___closed__8; @@ -3075,12 +3097,11 @@ static lean_object* l_Lean_Parser_Command_derivingClasses_formatter___closed__5; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___closed__8; static lean_object* l_Lean_Parser_Command_moduleDoc_formatter___closed__3; static lean_object* l_Lean_Parser_Command_import___closed__5; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__42; static lean_object* l_Lean_Parser_Command_namedPrio_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_classTk___closed__1; static lean_object* l_Lean_Parser_Command_set__option___closed__7; static lean_object* l_Lean_Parser_Command_protected_parenthesizer___closed__3; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__4; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__30; LEAN_EXPORT lean_object* l_Lean_Parser_Command_quot; static lean_object* l_Lean_Parser_Command_partial___closed__8; static lean_object* l_Lean_Parser_Command_declId___closed__9; @@ -3095,7 +3116,6 @@ static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__4; static lean_object* l_Lean_Parser_Command_computedFields_formatter___closed__1; lean_object* l_Lean_Parser_Term_bracketedBinder_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_partial; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__33; static lean_object* l_Lean_Parser_Command_abbrev___closed__11; static lean_object* l_Lean_Parser_Command_printEqns_formatter___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_formatter__1___closed__1; @@ -3111,6 +3131,7 @@ static lean_object* l_Lean_Parser_Command_structCtor_formatter___closed__6; static lean_object* l_Lean_Parser_Command_optDeclSig___closed__1; static lean_object* l_Lean_Parser_Command_structCtor___closed__5; static lean_object* l_Lean_Parser_Command_mutual_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_version__1(lean_object*); static lean_object* l_Lean_Parser_Term_quot___closed__18; static lean_object* l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_namespace_docString__1(lean_object*); @@ -3144,6 +3165,7 @@ static lean_object* l_Lean_Parser_Command_extends_formatter___closed__4; static lean_object* l_Lean_Parser_Command_printEqns___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_eval_docString__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_openOnly_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__43; static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_parenthesizer__1___closed__1; static lean_object* l_Lean_Parser_Command_omit_formatter___closed__5; static lean_object* l_Lean_Parser_Command_check__failure___closed__3; @@ -3151,6 +3173,7 @@ static lean_object* l_Lean_Parser_Command_classTk___closed__4; static lean_object* l_Lean_Parser_Command_axiom___closed__5; static lean_object* l_Lean_Parser_Term_open_formatter___closed__5; static lean_object* l_Lean_Parser_Command_declModifiers___closed__1; +LEAN_EXPORT lean_object* l_Lean_Parser_Command_version_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_check_formatter__1(lean_object*); static lean_object* l_Lean_Parser_Command_printTacTags_formatter___closed__6; static lean_object* l_Lean_Parser_Command_openRenamingItem___closed__3; @@ -3287,9 +3310,9 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_declRange__1__ static lean_object* l_Lean_Parser_Command_import___closed__6; static lean_object* l_Lean_Parser_Command_abbrev_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Command_noncomputable___closed__8; +static lean_object* l_Lean_Parser_Command_version_formatter___closed__2; static lean_object* l_Lean_Parser_Command_opaque_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__3; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__29; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declaration_parenthesizer__1(lean_object*); static lean_object* l_Lean_Parser_Term_open_parenthesizer___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_end_docString__1(lean_object*); @@ -3300,6 +3323,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_open_docString__1(lea LEAN_EXPORT lean_object* l_Lean_Parser_Command_universe_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_incQuotDepth_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter__1(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__34; static lean_object* l_Lean_Parser_Command_definition_parenthesizer___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Term_quot_formatter__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_omit_formatter__1___closed__1; @@ -3324,6 +3348,7 @@ static lean_object* l_Lean_Parser_Command_printEqns_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_declBody___closed__7; static lean_object* l_Lean_Parser_Command_structureTk_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_derivingClasses___closed__1; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__19; LEAN_EXPORT lean_object* l_Lean_Parser_Command_check__failure_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_example_formatter___closed__3; static lean_object* l_Lean_Parser_Command_optionValue_parenthesizer___closed__2; @@ -3351,6 +3376,7 @@ static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_inductive_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_declModifiers_docString__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_declRange__1___closed__5; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__23; static lean_object* l_Lean_Parser_Command_ctor___closed__1; static lean_object* l_Lean_Parser_Command_declModifiers___closed__6; static lean_object* l_Lean_Parser_Command_eraseAttr___closed__8; @@ -3361,12 +3387,12 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiers_formatter(uint8_t, static lean_object* l___regBuiltin_Lean_Parser_Command_export_parenthesizer__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_optionValue; LEAN_EXPORT lean_object* l_Lean_Parser_Command_check; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__36; static lean_object* l_Lean_Parser_Command_structCtor___closed__8; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_mutual_declRange__1(lean_object*); static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_example_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structureTk_formatter__1(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__18; static lean_object* l_Lean_Parser_Command_addDocString___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Command_quot_parenthesizer__1___closed__1; static lean_object* l_Lean_Parser_Tactic_set__option___closed__3; @@ -3438,6 +3464,7 @@ static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_import___closed__7; static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__6; static lean_object* l_Lean_Parser_Command_declValEqns___closed__3; +static lean_object* l_Lean_Parser_Command_version_formatter___closed__1; static lean_object* l_Lean_Parser_Command_optDefDeriving___closed__11; static lean_object* l_Lean_Parser_Command_classInductive___closed__4; static lean_object* l_Lean_Parser_Command_noncomputable___closed__2; @@ -3518,14 +3545,12 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_unsafe_parenthesizer(lean_object* static lean_object* l_Lean_Parser_Command_tactic__extension___closed__6; static lean_object* l_Lean_Parser_Command_openSimple___closed__3; static lean_object* l_Lean_Parser_Command_eraseAttr_parenthesizer___closed__3; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__38; lean_object* l_Lean_Parser_sepBy1_parenthesizer(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_extends___closed__6; static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__11; static lean_object* l_Lean_Parser_Command_noncomputable___closed__1; static lean_object* l_Lean_Parser_Term_open_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_optDeriving_parenthesizer___closed__4; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__7; static lean_object* l_Lean_Parser_Command_register__tactic__tag_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_attribute_formatter___closed__12; static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_formatter__1___closed__1; @@ -3545,7 +3570,6 @@ static lean_object* l_Lean_Parser_Command_whereStructInst___closed__29; static lean_object* l_Lean_Parser_Command_quot___closed__6; static lean_object* l_Lean_Parser_Command_classInductive___closed__16; static lean_object* l_Lean_Parser_Command_computedFields_parenthesizer___closed__4; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__18; static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_docString__1___closed__1; static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__2; static lean_object* l_Lean_Parser_Command_declSig___closed__2; @@ -3597,10 +3621,10 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structImplicitBinder lean_object* l_Lean_Parser_Term_bracketedBinder(uint8_t); LEAN_EXPORT lean_object* l_Lean_Parser_Command_optDeriving; static lean_object* l_Lean_Parser_Command_declId_parenthesizer___closed__4; +static lean_object* l_Lean_Parser_Command_version_formatter___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_declRange__1___closed__1; static lean_object* l_Lean_Parser_Command_openOnly_formatter___closed__5; static lean_object* l_Lean_Parser_Tactic_open_formatter___closed__7; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__14; static lean_object* l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_attribute___closed__11; static lean_object* l_Lean_Parser_Command_section_parenthesizer___closed__1; @@ -3660,6 +3684,7 @@ static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_definition_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_computedField_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_structSimpleBinder___closed__9; +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_print_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_attribute_declRange__1___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_partial_parenthesizer__1(lean_object*); @@ -3744,6 +3769,7 @@ static lean_object* l_Lean_Parser_Command_printTacTags___closed__11; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer__1(lean_object*); static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_declValSimple_formatter__1___closed__1; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_mutual_declRange__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_declRange__1___closed__2; static lean_object* l_Lean_Parser_Command_in___closed__1; @@ -3770,13 +3796,12 @@ static lean_object* l_Lean_Parser_Command_evalBang_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_include___closed__1; static lean_object* l_Lean_Parser_Command_variable___closed__10; lean_object* l_Lean_Parser_ppGroup_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_version___closed__8; static lean_object* l_Lean_Parser_Command_attribute___closed__10; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__43; static lean_object* l_Lean_Parser_Command_inductive___closed__15; static lean_object* l_Lean_Parser_Command_set__option_formatter___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_include_formatter__1___closed__1; static lean_object* l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__13; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__39; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_initialize__1(lean_object*); static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__6; static lean_object* l_Lean_Parser_Command_whereStructInst_formatter___closed__10; @@ -3804,6 +3829,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_in__1(lean_object*); static lean_object* l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_initialize_formatter__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__1; static lean_object* l_Lean_Parser_Command_private___closed__6; static lean_object* l_Lean_Parser_Command_definition_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_exit___closed__2; @@ -31185,6 +31211,295 @@ x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } } +static lean_object* _init_l_Lean_Parser_Command_version___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("version", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean_Parser_Command_version___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_Parser_Term_quot___closed__1; +x_2 = l_Lean_Parser_Term_quot___closed__2; +x_3 = l_Lean_Parser_Command_quot___closed__1; +x_4 = l_Lean_Parser_Command_version___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_Parser_Command_version___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; +x_1 = l_Lean_Parser_Command_version___closed__1; +x_2 = l_Lean_Parser_Command_version___closed__2; +x_3 = 1; +x_4 = 0; +x_5 = l_Lean_Parser_mkAntiquot(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Parser_Command_version___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("#version", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_Parser_Command_version___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_version___closed__4; +x_2 = l_Lean_Parser_symbol(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_Command_version___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Parser_Command_version___closed__2; +x_2 = lean_unsigned_to_nat(1024u); +x_3 = l_Lean_Parser_Command_version___closed__5; +x_4 = l_Lean_Parser_leadingNode(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Parser_Command_version___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_version___closed__3; +x_2 = l_Lean_Parser_Command_version___closed__6; +x_3 = l_Lean_Parser_withAntiquot(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_version___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_version___closed__2; +x_2 = l_Lean_Parser_Command_version___closed__7; +x_3 = l_Lean_Parser_withCache(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_version() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Parser_Command_version___closed__8; +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_version__1(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; lean_object* x_7; +x_2 = l_Lean_Parser_Command_quot___closed__5; +x_3 = l_Lean_Parser_Command_version___closed__2; +x_4 = 1; +x_5 = l_Lean_Parser_Command_version; +x_6 = lean_unsigned_to_nat(1000u); +x_7 = l_Lean_Parser_addBuiltinParser(x_2, x_3, x_4, x_5, x_6, x_1); +return x_7; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_version_docString__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Shows the current Lean version. Prints `Lean.versionString`. ", 61, 61); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_version_docString__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_2 = l_Lean_Parser_Command_version___closed__2; +x_3 = l___regBuiltin_Lean_Parser_Command_version_docString__1___closed__1; +x_4 = l_Lean_addBuiltinDocString(x_2, x_3, x_1); +return x_4; +} +} +static lean_object* _init_l_Lean_Parser_Command_version_formatter___closed__1() { +_start: +{ +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; +x_1 = l_Lean_Parser_Command_version___closed__1; +x_2 = l_Lean_Parser_Command_version___closed__2; +x_3 = 1; +x_4 = 0; +x_5 = lean_box(x_3); +x_6 = lean_box(x_4); +x_7 = lean_alloc_closure((void*)(l_Lean_Parser_mkAntiquot_formatter___boxed), 9, 4); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +lean_closure_set(x_7, 2, x_5); +lean_closure_set(x_7, 3, x_6); +return x_7; +} +} +static lean_object* _init_l_Lean_Parser_Command_version_formatter___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_version___closed__4; +x_2 = lean_alloc_closure((void*)(l_Lean_Parser_symbol_formatter), 6, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_Command_version_formatter___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Parser_Command_version___closed__2; +x_2 = lean_unsigned_to_nat(1024u); +x_3 = l_Lean_Parser_Command_version_formatter___closed__2; +x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); +lean_closure_set(x_4, 0, x_1); +lean_closure_set(x_4, 1, x_2); +lean_closure_set(x_4, 2, x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Parser_Command_version_formatter(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; +x_6 = l_Lean_Parser_Command_version_formatter___closed__1; +x_7 = l_Lean_Parser_Command_version_formatter___closed__3; +x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); +return x_8; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_version_formatter__1___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; +x_1 = l_Lean_Parser_Term_quot___closed__1; +x_2 = l_Lean_Parser_Term_quot___closed__2; +x_3 = l_Lean_Parser_Command_quot___closed__1; +x_4 = l_Lean_Parser_Command_version___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_quot_formatter__1___closed__1; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_version_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_version_formatter__1(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___regBuiltin_Lean_Parser_Term_quot_formatter__1___closed__3; +x_3 = l_Lean_Parser_Command_version___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Command_version_parenthesizer___closed__1() { +_start: +{ +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; +x_1 = l_Lean_Parser_Command_version___closed__1; +x_2 = l_Lean_Parser_Command_version___closed__2; +x_3 = 1; +x_4 = 0; +x_5 = lean_box(x_3); +x_6 = lean_box(x_4); +x_7 = lean_alloc_closure((void*)(l_Lean_Parser_mkAntiquot_parenthesizer___boxed), 9, 4); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +lean_closure_set(x_7, 2, x_5); +lean_closure_set(x_7, 3, x_6); +return x_7; +} +} +static lean_object* _init_l_Lean_Parser_Command_version_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_version___closed__4; +x_2 = lean_alloc_closure((void*)(l_Lean_Parser_symbol_parenthesizer), 6, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_Command_version_parenthesizer___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Parser_Command_version___closed__2; +x_2 = lean_unsigned_to_nat(1024u); +x_3 = l_Lean_Parser_Command_version_parenthesizer___closed__2; +x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer), 8, 3); +lean_closure_set(x_4, 0, x_1); +lean_closure_set(x_4, 1, x_2); +lean_closure_set(x_4, 2, x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Parser_Command_version_parenthesizer(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; +x_6 = l_Lean_Parser_Command_version_parenthesizer___closed__1; +x_7 = l_Lean_Parser_Command_version_parenthesizer___closed__3; +x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); +return x_8; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___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; +x_1 = l_Lean_Parser_Term_quot___closed__1; +x_2 = l_Lean_Parser_Term_quot___closed__2; +x_3 = l_Lean_Parser_Command_quot___closed__1; +x_4 = l_Lean_Parser_Command_version___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer__1___closed__1; +x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_version_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1(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___regBuiltin_Lean_Parser_Term_quot_parenthesizer__1___closed__3; +x_3 = l_Lean_Parser_Command_version___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_init__quot___closed__1() { _start: { @@ -41753,7 +42068,7 @@ x_1 = l_Lean_Parser_Command_eoi___closed__5; return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3073_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3092_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -41814,7 +42129,7 @@ x_1 = l_Lean_Parser_Command_ctor___closed__8; return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__1() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -41824,7 +42139,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__2() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__2() { _start: { lean_object* x_1; @@ -41832,19 +42147,19 @@ x_1 = lean_mk_string_unchecked("declModifiersF", 14, 14); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__3() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____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_Parser_Term_quot___closed__1; x_2 = l_Lean_Parser_Term_quot___closed__2; x_3 = l_Lean_Parser_Command_quot___closed__1; -x_4 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__2; +x_4 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____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_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__4() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__4() { _start: { lean_object* x_1; lean_object* x_2; @@ -41854,7 +42169,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__5() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -41864,7 +42179,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__6() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__6() { _start: { lean_object* x_1; lean_object* x_2; @@ -41874,12 +42189,12 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__7() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__7() { _start: { lean_object* x_1; lean_object* x_2; uint8_t x_3; lean_object* x_4; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__6; +x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__6; x_3 = 1; x_4 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_4, 0, x_1); @@ -41888,7 +42203,7 @@ lean_ctor_set_uint8(x_4, sizeof(void*)*2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__8() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__8() { _start: { lean_object* x_1; @@ -41896,17 +42211,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declModifiersF_formatter) return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__9() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__8; +x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__8; 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_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__10() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__10() { _start: { lean_object* x_1; @@ -41914,7 +42229,7 @@ x_1 = l_Lean_PrettyPrinter_Formatter_formatterAliasesRef; return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__11() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__11() { _start: { lean_object* x_1; @@ -41922,17 +42237,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declModifiersF_parenthesi return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__12() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__11; +x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__11; 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_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__13() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__13() { _start: { lean_object* x_1; @@ -41940,7 +42255,7 @@ x_1 = l_Lean_PrettyPrinter_Parenthesizer_parenthesizerAliasesRef; return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__14() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__14() { _start: { lean_object* x_1; @@ -41948,17 +42263,17 @@ x_1 = lean_mk_string_unchecked("nestedDeclModifiers", 19, 19); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__15() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__14; +x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__14; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__16() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__16() { _start: { lean_object* x_1; @@ -41966,19 +42281,19 @@ x_1 = lean_mk_string_unchecked("declModifiersT", 14, 14); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__17() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____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_Parser_Term_quot___closed__1; x_2 = l_Lean_Parser_Term_quot___closed__2; x_3 = l_Lean_Parser_Command_quot___closed__1; -x_4 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__16; +x_4 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____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_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__18() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__18() { _start: { lean_object* x_1; lean_object* x_2; @@ -41988,7 +42303,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__19() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__19() { _start: { lean_object* x_1; @@ -41996,17 +42311,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declModifiersT_formatter) return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__20() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__20() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__19; +x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__19; 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_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__21() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__21() { _start: { lean_object* x_1; @@ -42014,17 +42329,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declModifiersT_parenthesi return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__22() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__22() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__21; +x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__21; 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_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__23() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__23() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -42034,7 +42349,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__24() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__24() { _start: { lean_object* x_1; lean_object* x_2; @@ -42044,7 +42359,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__25() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__25() { _start: { lean_object* x_1; lean_object* x_2; @@ -42054,7 +42369,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__26() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__26() { _start: { lean_object* x_1; lean_object* x_2; @@ -42064,7 +42379,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__27() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__27() { _start: { lean_object* x_1; lean_object* x_2; @@ -42074,7 +42389,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__28() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__28() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -42084,7 +42399,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__29() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__29() { _start: { lean_object* x_1; lean_object* x_2; @@ -42094,7 +42409,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__30() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__30() { _start: { lean_object* x_1; lean_object* x_2; @@ -42104,7 +42419,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__31() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__31() { _start: { lean_object* x_1; lean_object* x_2; @@ -42114,7 +42429,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__32() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__32() { _start: { lean_object* x_1; lean_object* x_2; @@ -42124,7 +42439,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__33() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__33() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -42134,7 +42449,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__34() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__34() { _start: { lean_object* x_1; lean_object* x_2; @@ -42144,7 +42459,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__35() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__35() { _start: { lean_object* x_1; lean_object* x_2; @@ -42154,7 +42469,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__36() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__36() { _start: { lean_object* x_1; lean_object* x_2; @@ -42164,7 +42479,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__37() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__37() { _start: { lean_object* x_1; lean_object* x_2; @@ -42174,7 +42489,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__38() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__38() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -42184,7 +42499,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__39() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__39() { _start: { lean_object* x_1; lean_object* x_2; @@ -42194,7 +42509,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__40() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__40() { _start: { lean_object* x_1; lean_object* x_2; @@ -42204,7 +42519,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__41() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__41() { _start: { lean_object* x_1; lean_object* x_2; @@ -42214,7 +42529,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__42() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__42() { _start: { lean_object* x_1; lean_object* x_2; @@ -42224,7 +42539,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__43() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__43() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -42234,7 +42549,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__44() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__44() { _start: { lean_object* x_1; lean_object* x_2; @@ -42244,7 +42559,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__45() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__45() { _start: { lean_object* x_1; lean_object* x_2; @@ -42254,7 +42569,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__46() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__46() { _start: { lean_object* x_1; lean_object* x_2; @@ -42264,7 +42579,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__47() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__47() { _start: { lean_object* x_1; lean_object* x_2; @@ -42274,7 +42589,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__48() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__48() { _start: { lean_object* x_1; @@ -42282,29 +42597,29 @@ x_1 = lean_mk_string_unchecked("docComment", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__49() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__49() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__48; +x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__48; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__50() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__50() { _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_Parser_Term_quot___closed__1; x_2 = l_Lean_Parser_Term_quot___closed__2; x_3 = l_Lean_Parser_Command_quot___closed__1; -x_4 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__48; +x_4 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__48; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__51() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__51() { _start: { lean_object* x_1; lean_object* x_2; @@ -42314,17 +42629,17 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__52() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__52() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__50; +x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__50; 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_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__53() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__53() { _start: { lean_object* x_1; lean_object* x_2; @@ -42334,7 +42649,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__54() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__54() { _start: { lean_object* x_1; lean_object* x_2; @@ -42344,15 +42659,15 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116_(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; -x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__1; -x_3 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__3; -x_4 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__4; -x_5 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__5; -x_6 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__7; +x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__1; +x_3 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__3; +x_4 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__4; +x_5 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__5; +x_6 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__7; x_7 = l_Lean_Parser_registerAlias(x_2, x_3, x_4, x_5, x_6, x_1); if (lean_obj_tag(x_7) == 0) { @@ -42360,8 +42675,8 @@ lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); lean_dec(x_7); -x_9 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__10; -x_10 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__9; +x_9 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__10; +x_10 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__9; x_11 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_2, x_10, x_8); if (lean_obj_tag(x_11) == 0) { @@ -42369,8 +42684,8 @@ lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; x_12 = lean_ctor_get(x_11, 1); lean_inc(x_12); lean_dec(x_11); -x_13 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__13; -x_14 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__12; +x_13 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__13; +x_14 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__12; x_15 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_2, x_14, x_12); if (lean_obj_tag(x_15) == 0) { @@ -42378,9 +42693,9 @@ lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean x_16 = lean_ctor_get(x_15, 1); lean_inc(x_16); lean_dec(x_15); -x_17 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__15; -x_18 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__17; -x_19 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__18; +x_17 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__15; +x_18 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__17; +x_19 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__18; x_20 = l_Lean_Parser_registerAlias(x_17, x_18, x_19, x_5, x_6, x_16); if (lean_obj_tag(x_20) == 0) { @@ -42388,7 +42703,7 @@ lean_object* x_21; lean_object* x_22; lean_object* x_23; x_21 = lean_ctor_get(x_20, 1); lean_inc(x_21); lean_dec(x_20); -x_22 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__20; +x_22 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__20; x_23 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_17, x_22, x_21); if (lean_obj_tag(x_23) == 0) { @@ -42396,7 +42711,7 @@ lean_object* x_24; lean_object* x_25; lean_object* x_26; x_24 = lean_ctor_get(x_23, 1); lean_inc(x_24); lean_dec(x_23); -x_25 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__22; +x_25 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__22; x_26 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_17, x_25, x_24); if (lean_obj_tag(x_26) == 0) { @@ -42404,10 +42719,10 @@ lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean x_27 = lean_ctor_get(x_26, 1); lean_inc(x_27); lean_dec(x_26); -x_28 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__23; +x_28 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__23; x_29 = l_Lean_Parser_Command_declId___closed__2; -x_30 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__24; -x_31 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__25; +x_30 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__24; +x_31 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__25; x_32 = l_Lean_Parser_registerAlias(x_28, x_29, x_30, x_31, x_6, x_27); if (lean_obj_tag(x_32) == 0) { @@ -42415,7 +42730,7 @@ 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 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__26; +x_34 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__26; x_35 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_28, x_34, x_33); if (lean_obj_tag(x_35) == 0) { @@ -42423,7 +42738,7 @@ lean_object* x_36; lean_object* x_37; lean_object* x_38; x_36 = lean_ctor_get(x_35, 1); lean_inc(x_36); lean_dec(x_35); -x_37 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__27; +x_37 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__27; x_38 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_28, x_37, x_36); if (lean_obj_tag(x_38) == 0) { @@ -42431,10 +42746,10 @@ lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean x_39 = lean_ctor_get(x_38, 1); lean_inc(x_39); lean_dec(x_38); -x_40 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__28; +x_40 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__28; x_41 = l_Lean_Parser_Command_declSig___closed__2; -x_42 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__29; -x_43 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__30; +x_42 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__29; +x_43 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__30; x_44 = l_Lean_Parser_registerAlias(x_40, x_41, x_42, x_43, x_6, x_39); if (lean_obj_tag(x_44) == 0) { @@ -42442,7 +42757,7 @@ lean_object* x_45; lean_object* x_46; lean_object* x_47; x_45 = lean_ctor_get(x_44, 1); lean_inc(x_45); lean_dec(x_44); -x_46 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__31; +x_46 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__31; x_47 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_40, x_46, x_45); if (lean_obj_tag(x_47) == 0) { @@ -42450,7 +42765,7 @@ lean_object* x_48; lean_object* x_49; lean_object* x_50; x_48 = lean_ctor_get(x_47, 1); lean_inc(x_48); lean_dec(x_47); -x_49 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__32; +x_49 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__32; x_50 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_40, x_49, x_48); if (lean_obj_tag(x_50) == 0) { @@ -42458,10 +42773,10 @@ lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean x_51 = lean_ctor_get(x_50, 1); lean_inc(x_51); lean_dec(x_50); -x_52 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__33; +x_52 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__33; x_53 = l___regBuiltin_Lean_Parser_Command_declVal_docString__1___closed__2; -x_54 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__34; -x_55 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__35; +x_54 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__34; +x_55 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__35; x_56 = l_Lean_Parser_registerAlias(x_52, x_53, x_54, x_55, x_6, x_51); if (lean_obj_tag(x_56) == 0) { @@ -42469,7 +42784,7 @@ lean_object* x_57; lean_object* x_58; lean_object* x_59; x_57 = lean_ctor_get(x_56, 1); lean_inc(x_57); lean_dec(x_56); -x_58 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__36; +x_58 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__36; x_59 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_52, x_58, x_57); if (lean_obj_tag(x_59) == 0) { @@ -42477,7 +42792,7 @@ lean_object* x_60; lean_object* x_61; lean_object* x_62; x_60 = lean_ctor_get(x_59, 1); lean_inc(x_60); lean_dec(x_59); -x_61 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__37; +x_61 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__37; x_62 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_52, x_61, x_60); if (lean_obj_tag(x_62) == 0) { @@ -42485,10 +42800,10 @@ lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean x_63 = lean_ctor_get(x_62, 1); lean_inc(x_63); lean_dec(x_62); -x_64 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__38; +x_64 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__38; x_65 = l_Lean_Parser_Command_optDeclSig___closed__2; -x_66 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__39; -x_67 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__40; +x_66 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__39; +x_67 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__40; x_68 = l_Lean_Parser_registerAlias(x_64, x_65, x_66, x_67, x_6, x_63); if (lean_obj_tag(x_68) == 0) { @@ -42496,7 +42811,7 @@ lean_object* x_69; lean_object* x_70; lean_object* x_71; x_69 = lean_ctor_get(x_68, 1); lean_inc(x_69); lean_dec(x_68); -x_70 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__41; +x_70 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__41; x_71 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_64, x_70, x_69); if (lean_obj_tag(x_71) == 0) { @@ -42504,7 +42819,7 @@ lean_object* x_72; lean_object* x_73; lean_object* x_74; x_72 = lean_ctor_get(x_71, 1); lean_inc(x_72); lean_dec(x_71); -x_73 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__42; +x_73 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__42; x_74 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_64, x_73, x_72); if (lean_obj_tag(x_74) == 0) { @@ -42512,10 +42827,10 @@ lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean x_75 = lean_ctor_get(x_74, 1); lean_inc(x_75); lean_dec(x_74); -x_76 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__43; +x_76 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__43; x_77 = l___regBuiltin_Lean_Parser_Command_openDecl_docString__1___closed__2; -x_78 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__44; -x_79 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__45; +x_78 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__44; +x_79 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__45; x_80 = l_Lean_Parser_registerAlias(x_76, x_77, x_78, x_79, x_6, x_75); if (lean_obj_tag(x_80) == 0) { @@ -42523,7 +42838,7 @@ lean_object* x_81; lean_object* x_82; lean_object* x_83; x_81 = lean_ctor_get(x_80, 1); lean_inc(x_81); lean_dec(x_80); -x_82 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__46; +x_82 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__46; x_83 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_76, x_82, x_81); if (lean_obj_tag(x_83) == 0) { @@ -42531,7 +42846,7 @@ lean_object* x_84; lean_object* x_85; lean_object* x_86; x_84 = lean_ctor_get(x_83, 1); lean_inc(x_84); lean_dec(x_83); -x_85 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__47; +x_85 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__47; x_86 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_76, x_85, x_84); if (lean_obj_tag(x_86) == 0) { @@ -42539,10 +42854,10 @@ lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean x_87 = lean_ctor_get(x_86, 1); lean_inc(x_87); lean_dec(x_86); -x_88 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__49; -x_89 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__50; -x_90 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__51; -x_91 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__52; +x_88 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__49; +x_89 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__50; +x_90 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__51; +x_91 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__52; x_92 = l_Lean_Parser_registerAlias(x_88, x_89, x_90, x_91, x_6, x_87); if (lean_obj_tag(x_92) == 0) { @@ -42550,7 +42865,7 @@ lean_object* x_93; lean_object* x_94; lean_object* x_95; x_93 = lean_ctor_get(x_92, 1); lean_inc(x_93); lean_dec(x_92); -x_94 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__53; +x_94 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__53; x_95 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_88, x_94, x_93); if (lean_obj_tag(x_95) == 0) { @@ -42558,7 +42873,7 @@ lean_object* x_96; lean_object* x_97; lean_object* x_98; x_96 = lean_ctor_get(x_95, 1); lean_inc(x_96); lean_dec(x_95); -x_97 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__54; +x_97 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__54; x_98 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_88, x_97, x_96); return x_98; } @@ -49867,6 +50182,58 @@ lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_printTacTags_parenthesiz if (builtin) {res = l___regBuiltin_Lean_Parser_Command_printTacTags_parenthesizer__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +}l_Lean_Parser_Command_version___closed__1 = _init_l_Lean_Parser_Command_version___closed__1(); +lean_mark_persistent(l_Lean_Parser_Command_version___closed__1); +l_Lean_Parser_Command_version___closed__2 = _init_l_Lean_Parser_Command_version___closed__2(); +lean_mark_persistent(l_Lean_Parser_Command_version___closed__2); +l_Lean_Parser_Command_version___closed__3 = _init_l_Lean_Parser_Command_version___closed__3(); +lean_mark_persistent(l_Lean_Parser_Command_version___closed__3); +l_Lean_Parser_Command_version___closed__4 = _init_l_Lean_Parser_Command_version___closed__4(); +lean_mark_persistent(l_Lean_Parser_Command_version___closed__4); +l_Lean_Parser_Command_version___closed__5 = _init_l_Lean_Parser_Command_version___closed__5(); +lean_mark_persistent(l_Lean_Parser_Command_version___closed__5); +l_Lean_Parser_Command_version___closed__6 = _init_l_Lean_Parser_Command_version___closed__6(); +lean_mark_persistent(l_Lean_Parser_Command_version___closed__6); +l_Lean_Parser_Command_version___closed__7 = _init_l_Lean_Parser_Command_version___closed__7(); +lean_mark_persistent(l_Lean_Parser_Command_version___closed__7); +l_Lean_Parser_Command_version___closed__8 = _init_l_Lean_Parser_Command_version___closed__8(); +lean_mark_persistent(l_Lean_Parser_Command_version___closed__8); +l_Lean_Parser_Command_version = _init_l_Lean_Parser_Command_version(); +lean_mark_persistent(l_Lean_Parser_Command_version); +if (builtin) {res = l___regBuiltin_Lean_Parser_Command_version__1(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l___regBuiltin_Lean_Parser_Command_version_docString__1___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_version_docString__1___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_version_docString__1___closed__1); +if (builtin) {res = l___regBuiltin_Lean_Parser_Command_version_docString__1(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_Parser_Command_version_formatter___closed__1 = _init_l_Lean_Parser_Command_version_formatter___closed__1(); +lean_mark_persistent(l_Lean_Parser_Command_version_formatter___closed__1); +l_Lean_Parser_Command_version_formatter___closed__2 = _init_l_Lean_Parser_Command_version_formatter___closed__2(); +lean_mark_persistent(l_Lean_Parser_Command_version_formatter___closed__2); +l_Lean_Parser_Command_version_formatter___closed__3 = _init_l_Lean_Parser_Command_version_formatter___closed__3(); +lean_mark_persistent(l_Lean_Parser_Command_version_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__1); +l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_version_formatter__1___closed__2); +if (builtin) {res = l___regBuiltin_Lean_Parser_Command_version_formatter__1(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_Parser_Command_version_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_version_parenthesizer___closed__1(); +lean_mark_persistent(l_Lean_Parser_Command_version_parenthesizer___closed__1); +l_Lean_Parser_Command_version_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_version_parenthesizer___closed__2(); +lean_mark_persistent(l_Lean_Parser_Command_version_parenthesizer___closed__2); +l_Lean_Parser_Command_version_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_version_parenthesizer___closed__3(); +lean_mark_persistent(l_Lean_Parser_Command_version_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__1); +l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1___closed__2); +if (builtin) {res = l___regBuiltin_Lean_Parser_Command_version_parenthesizer__1(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); }l_Lean_Parser_Command_init__quot___closed__1 = _init_l_Lean_Parser_Command_init__quot___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_init__quot___closed__1); l_Lean_Parser_Command_init__quot___closed__2 = _init_l_Lean_Parser_Command_init__quot___closed__2(); @@ -51713,122 +52080,122 @@ l_Lean_Parser_Command_eoi___closed__5 = _init_l_Lean_Parser_Command_eoi___closed lean_mark_persistent(l_Lean_Parser_Command_eoi___closed__5); l_Lean_Parser_Command_eoi = _init_l_Lean_Parser_Command_eoi(); lean_mark_persistent(l_Lean_Parser_Command_eoi); -if (builtin) {res = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3073_(lean_io_mk_world()); +if (builtin) {res = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3092_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Lean_Parser_Command_declModifiersF = _init_l_Lean_Parser_Command_declModifiersF(); lean_mark_persistent(l_Lean_Parser_Command_declModifiersF); l_Lean_Parser_Command_declModifiersT = _init_l_Lean_Parser_Command_declModifiersT(); lean_mark_persistent(l_Lean_Parser_Command_declModifiersT); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__1 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__1(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__1); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__2 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__2(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__2); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__3 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__3(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__3); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__4 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__4(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__4); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__5 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__5(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__5); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__6 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__6(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__6); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__7 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__7(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__7); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__8 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__8(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__8); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__9 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__9(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__9); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__10 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__10(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__10); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__11 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__11(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__11); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__12 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__12(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__12); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__13 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__13(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__13); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__14 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__14(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__14); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__15 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__15(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__15); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__16 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__16(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__16); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__17 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__17(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__17); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__18 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__18(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__18); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__19 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__19(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__19); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__20 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__20(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__20); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__21 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__21(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__21); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__22 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__22(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__22); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__23 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__23(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__23); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__24 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__24(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__24); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__25 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__25(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__25); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__26 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__26(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__26); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__27 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__27(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__27); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__28 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__28(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__28); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__29 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__29(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__29); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__30 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__30(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__30); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__31 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__31(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__31); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__32 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__32(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__32); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__33 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__33(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__33); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__34 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__34(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__34); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__35 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__35(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__35); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__36 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__36(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__36); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__37 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__37(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__37); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__38 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__38(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__38); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__39 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__39(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__39); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__40 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__40(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__40); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__41 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__41(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__41); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__42 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__42(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__42); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__43 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__43(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__43); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__44 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__44(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__44); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__45 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__45(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__45); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__46 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__46(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__46); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__47 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__47(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__47); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__48 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__48(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__48); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__49 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__49(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__49); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__50 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__50(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__50); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__51 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__51(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__51); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__52 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__52(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__52); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__53 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__53(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__53); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__54 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__54(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097____closed__54); -if (builtin) {res = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3097_(lean_io_mk_world()); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__1 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__1(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__1); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__2 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__2(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__2); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__3 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__3(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__3); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__4 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__4(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__4); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__5 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__5(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__5); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__6 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__6(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__6); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__7 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__7(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__7); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__8 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__8(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__8); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__9 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__9(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__9); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__10 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__10(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__10); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__11 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__11(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__11); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__12 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__12(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__12); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__13 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__13(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__13); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__14 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__14(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__14); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__15 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__15(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__15); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__16 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__16(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__16); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__17 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__17(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__17); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__18 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__18(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__18); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__19 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__19(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__19); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__20 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__20(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__20); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__21 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__21(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__21); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__22 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__22(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__22); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__23 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__23(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__23); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__24 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__24(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__24); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__25 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__25(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__25); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__26 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__26(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__26); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__27 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__27(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__27); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__28 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__28(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__28); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__29 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__29(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__29); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__30 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__30(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__30); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__31 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__31(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__31); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__32 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__32(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__32); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__33 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__33(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__33); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__34 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__34(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__34); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__35 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__35(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__35); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__36 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__36(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__36); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__37 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__37(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__37); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__38 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__38(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__38); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__39 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__39(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__39); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__40 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__40(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__40); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__41 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__41(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__41); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__42 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__42(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__42); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__43 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__43(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__43); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__44 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__44(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__44); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__45 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__45(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__45); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__46 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__46(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__46); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__47 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__47(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__47); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__48 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__48(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__48); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__49 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__49(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__49); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__50 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__50(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__50); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__51 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__51(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__51); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__52 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__52(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__52); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__53 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__53(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__53); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__54 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__54(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116____closed__54); +if (builtin) {res = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_3116_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Lean_Parser_Term_open___closed__1 = _init_l_Lean_Parser_Term_open___closed__1(); diff --git a/stage0/stdlib/Lean/Parser/Extra.c b/stage0/stdlib/Lean/Parser/Extra.c index 7b727c9e9a85..dd820afb91c8 100644 --- a/stage0/stdlib/Lean/Parser/Extra.c +++ b/stage0/stdlib/Lean/Parser/Extra.c @@ -19,12 +19,12 @@ LEAN_EXPORT lean_object* l_Lean_Parser_sepByIndent_parenthesizer___boxed(lean_ob LEAN_EXPORT lean_object* l_Lean_Parser_many1_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_setLhsPrec_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppHardSpace_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__20; lean_object* lean_string_utf8_extract(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__33; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__85; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__41; lean_object* l_Lean_Parser_checkColEq(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__63; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__86; LEAN_EXPORT lean_object* l_Lean_Parser_rawIdent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_many_formatter___closed__3; lean_object* l_Lean_Syntax_mkNameLit(lean_object*, lean_object*); @@ -34,9 +34,11 @@ LEAN_EXPORT lean_object* l_Lean_Parser_identWithPartialTrailingDot; LEAN_EXPORT lean_object* l_Lean_Parser_ppHardLineUnlessUngrouped; LEAN_EXPORT lean_object* l_Lean_Parser_optional_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__37; +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770_(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_ppDedent_docString__1(lean_object*); static lean_object* l_Lean_Parser_sepByIndent_parenthesizer___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__5; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__65; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__17; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__57; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__19; static lean_object* l___regBuiltin_Lean_Parser_ppSpace_docString__1___closed__1; @@ -44,28 +46,27 @@ LEAN_EXPORT lean_object* l_Lean_Parser_ppHardSpace_parenthesizer(lean_object*, l extern lean_object* l_Lean_Parser_pushNone; LEAN_EXPORT lean_object* l_Lean_Parser_rawIdent_formatter(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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__18; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__33; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__87; extern lean_object* l_Lean_Parser_nameLitNoAntiquot; static lean_object* l_Lean_Parser_identWithPartialTrailingDot_formatter___closed__6; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__53; lean_object* l_Lean_addBuiltinDocString(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___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_Parser_withCache_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppRealGroup_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__81; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__26; LEAN_EXPORT lean_object* l_Lean_Parser_adaptCacheableContext_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_manyIndent_docString__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_ppRealGroup___boxed(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__12; lean_object* l_Lean_PrettyPrinter_Formatter_orelse_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__48; static lean_object* l___regBuiltin_Lean_Parser_ppHardSpace_docString__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_withForbidden_parenthesizer___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__13; LEAN_EXPORT lean_object* l_Lean_ppLine_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_fill(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__74; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__70; lean_object* l_Lean_PrettyPrinter_Formatter_rawIdentNoAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Parser_sepByIndent_formatter___spec__2___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_ppHardSpace_docString__1(lean_object*); @@ -81,33 +82,35 @@ static lean_object* l___regBuiltin_Lean_Parser_strLit_docString__1___closed__1; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__50; uint8_t l_Lean_Exception_isInterrupt(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_charLit_docString__1___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__36; LEAN_EXPORT lean_object* l_Lean_Parser_ppRealFill___boxed(lean_object*); lean_object* l_Lean_TSyntax_getString(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__34; static lean_object* l_Lean_Parser_charLit___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_withCache_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__39; lean_object* l_Lean_PrettyPrinter_Formatter_checkPrec_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_identWithPartialTrailingDot___closed__8; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__38; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__11; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__75; static lean_object* l_Lean_ppDedent_formatter___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__83; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__94; LEAN_EXPORT lean_object* l_Lean_Parser_many_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_charLit_docString__1(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__70; lean_object* l_Lean_Syntax_getId(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__77; LEAN_EXPORT lean_object* l_Lean_Parser_dbgTraceState_parenthesizer___boxed(lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Parser_sepByIndent_formatter___spec__2___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_ppGroup_docString__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_ppSpace_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_sepByIndent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__43; static lean_object* l_Lean_Parser_strLit_formatter___closed__2; lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_group_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_ident_docString__1(lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_sepByNoAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__57; static lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___closed__5; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__57; LEAN_EXPORT lean_object* l_Lean_Parser_notSymbol(lean_object*); static lean_object* l_Lean_Parser_optional___closed__1; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__28; @@ -117,13 +120,15 @@ static lean_object* l_Lean_Parser_rawIdent___closed__1; static lean_object* l___regBuiltin_Lean_Parser_ppHardLineUnlessUngrouped_docString__1___closed__3; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__8; static lean_object* l___regBuiltin_Lean_Parser_ppIndent_docString__1___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__93; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__22; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__12; static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_ppSpace_parenthesizer___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_sepBy1Indent_parenthesizer___boxed(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_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_notSymbol_parenthesizer___rarg(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__24; LEAN_EXPORT lean_object* l_Lean_Parser_evalInsideQuot_parenthesizer___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ppHardLineUnlessUngrouped_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter__1___closed__2; @@ -138,6 +143,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_dbgTraceState_formatter___rarg(lean_objec LEAN_EXPORT lean_object* l_Lean_Parser_optional(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_termParser_formatter___boxed(lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__61; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__37; LEAN_EXPORT lean_object* l_Lean_Parser_nameLit_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__25; static lean_object* l_Lean_Parser_strLit___closed__2; @@ -146,8 +152,9 @@ lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* l_ReaderT_bind___at_Lean_PrettyPrinter_Formatter_categoryFormatterCore___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppDedent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29____________; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__38; LEAN_EXPORT lean_object* l_Lean_Parser_evalInsideQuot_parenthesizer___boxed(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__98; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__81; lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_mkAntiquotSplice_formatter___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_strLit; @@ -159,10 +166,10 @@ LEAN_EXPORT lean_object* l_Lean_Parser_withOpen_formatter(lean_object*, lean_obj lean_object* l_Lean_Parser_checkLinebreakBefore(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_withOpenDecl_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__30; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__88; lean_object* l_Lean_Macro_throwError___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__69; LEAN_EXPORT lean_object* l_Lean_Parser_withPositionAfterLinebreak_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__99; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__79; LEAN_EXPORT lean_object* l_Lean_Parser_incQuotDepth_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_scientificLit_parenthesizer___closed__1; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__18; @@ -173,15 +180,14 @@ static lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___closed__8; lean_object* l_Lean_PrettyPrinter_Formatter_checkNoWsBefore_formatter___boxed(lean_object*); lean_object* l_Lean_Parser_orelse(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_ppDedentIfGrouped_docString__1___closed__2; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__7; lean_object* l_Lean_mkIdentFrom(lean_object*, lean_object*, uint8_t); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__23; static lean_object* l_Lean_Parser_mkAntiquotSplice_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_ppDedent_docString__1___closed__1; static lean_object* l_Lean_Parser_ident_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_decQuotDepth_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_hygieneInfo; lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkColEq_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__52; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__14; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__55; static lean_object* l___regBuiltin_Lean_Parser_patternIgnore_docString__1___closed__2; @@ -191,6 +197,7 @@ lean_object* l_Lean_Syntax_node5(lean_object*, lean_object*, lean_object*, lean_ static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__4; static lean_object* l_Lean_Parser_antiquotExpr_formatter___closed__4; uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_withForbidden_formatter(lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__35; static lean_object* l_Lean_Parser_antiquotExpr_formatter___closed__3; @@ -199,12 +206,11 @@ static lean_object* l_Lean_Parser_group_formatter___closed__1; static lean_object* l_Lean_Parser_rawIdent_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_termParser_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_scientificLit_formatter___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__86; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__91; LEAN_EXPORT lean_object* l_Lean_Parser_ppAllowUngrouped_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_nameLit_docString__1___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__7; lean_object* l_Lean_PrettyPrinter_Formatter_tokenWithAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__21; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__30; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__56; static lean_object* l___regBuiltin_Lean_Parser_ppSpace_docString__1___closed__2; static lean_object* l_List_forIn_loop___at_Lean_Parser_sepByIndent_formatter___spec__2___closed__3; @@ -241,12 +247,11 @@ LEAN_EXPORT lean_object* l_Lean_Parser_sepByIndent_formatter___boxed(lean_object LEAN_EXPORT lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Parser_Basic_0__Lean_Parser_addQuotDepth_parenthesizer(lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__29; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__95; lean_object* l_Lean_PrettyPrinter_Parenthesizer_withAntiquotSuffixSplice_parenthesizer___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__6; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__97; LEAN_EXPORT lean_object* l_Lean_Parser_setExpected_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer__1___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__78; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__48; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_nameLit_docString__1(lean_object*); static lean_object* l_Lean_Parser_strLit_parenthesizer___closed__1; @@ -257,21 +262,23 @@ lean_object* l_Lean_PrettyPrinter_Formatter_withoutInfo_formatter(lean_object*, LEAN_EXPORT lean_object* l_Lean_Parser_setExpected_parenthesizer___rarg(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_Parser_sepByElemParser_formatter___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__33; LEAN_EXPORT lean_object* l_Lean_Parser_mkAntiquot_formatter___boxed(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_Parser_ppDedentIfGrouped_docString__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppAllowUngrouped_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_notSymbol_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__90; LEAN_EXPORT lean_object* l_Lean_Parser_ppGroup(lean_object*); size_t lean_usize_of_nat(lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkNoWsBefore_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_identWithPartialTrailingDot_formatter___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_strLit_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_charLit_formatter___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__95; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__64; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__46; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__15; LEAN_EXPORT lean_object* l_Lean_Parser_notSymbol_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Macro_resolveGlobalName(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__58; static lean_object* l_Lean_Parser_antiquotExpr_parenthesizer___closed__3; static lean_object* l_Lean_Parser_many1Indent_formatter___closed__1; static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__6; @@ -283,7 +290,6 @@ extern lean_object* l_Lean_Parser_hygieneInfoNoAntiquot; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__14; static lean_object* l_Lean_Parser_scientificLit_formatter___closed__4; lean_object* l_Lean_Parser_optionalNoAntiquot(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__94; static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__8; lean_object* lean_st_ref_take(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ident_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -292,17 +298,18 @@ static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Le static lean_object* l_Lean_ppHardSpace_formatter___closed__2; lean_object* l_Lean_Syntax_MonadTraverser_getCur___at_Lean_PrettyPrinter_Formatter_visitArgs___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__18; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__90; LEAN_EXPORT lean_object* l_Lean_Parser_setExpected_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_notSymbol_formatter___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_many1_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_commandParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__72; LEAN_EXPORT lean_object* l_Lean_Parser_commandParser_formatter(lean_object*); static lean_object* l_Lean_Parser_patternIgnore_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_withoutPosition_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_strLit___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__50; static lean_object* l_Lean_Parser_hygieneInfo_parenthesizer___closed__2; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__58; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__54; LEAN_EXPORT lean_object* l_Lean_Parser_ppRealFill_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Parser_charLitNoAntiquot; lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); @@ -315,21 +322,24 @@ static lean_object* l_Lean_Parser_identWithPartialTrailingDot_parenthesizer___cl LEAN_EXPORT lean_object* l_Lean_ppAllowUngrouped_formatter___boxed(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_ppHardLineUnlessUngrouped_docString__1___closed__2; lean_object* l_Lean_PrettyPrinter_Formatter_manyNoAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__87; LEAN_EXPORT lean_object* l_Lean_ppRealGroup_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__25; LEAN_EXPORT lean_object* l_Lean_Parser_sepByElemParser_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_ppLine_docString__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_numLit_docString__1___closed__3; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__62; LEAN_EXPORT lean_object* l_Lean_Parser_withOpen_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__9; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__61; lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkColGe_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__69; static lean_object* l_Lean_Parser_identWithPartialTrailingDot_formatter___closed__1; lean_object* l_List_range(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_nonReservedSymbol_parenthesizer___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_Extra___hyg_1770____closed__66; lean_object* l_Lean_PrettyPrinter_Parenthesizer_sepByNoAntiquot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_atomic_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__4; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__78; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__23; static lean_object* l_Lean_Parser_charLit_formatter___closed__4; static lean_object* l___regBuiltin_Lean_Parser_charLit_docString__1___closed__2; @@ -337,32 +347,29 @@ static lean_object* l___regBuiltin_Lean_Parser_ppLine_docString__1___closed__1; extern lean_object* l_Lean_PrettyPrinter_parenthesizerAttribute; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__43; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter__1(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__73; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__14; LEAN_EXPORT lean_object* l_Lean_Parser_identWithPartialTrailingDot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__52; static lean_object* l___regBuiltin_Lean_Parser_scientificLit_docString__1___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__74; LEAN_EXPORT lean_object* l_Lean_Parser_numLit_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_ppHardLineUnlessUngrouped_parenthesizer___rarg(lean_object*); extern lean_object* l_Lean_Parser_rawIdentNoAntiquot; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__59; static lean_object* l_Lean_Parser_sepByIndent_parenthesizer___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__42; static lean_object* l_Lean_Parser_identWithPartialTrailingDot_parenthesizer___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__64; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__12; LEAN_EXPORT lean_object* l_Lean_Parser_adaptCacheableContext_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_sepByElemParser_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_ppHardSpace_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__37; lean_object* l_Lean_quoteNameMk(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__68; static lean_object* l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__3; static lean_object* l_Lean_Parser_nameLit___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__31; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__40; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__96; static lean_object* l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__4; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__32; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__44; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__9; lean_object* lean_st_ref_get(lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__54; @@ -372,7 +379,6 @@ static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Le LEAN_EXPORT lean_object* l_Lean_ppLine_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__46; lean_object* l_Lean_PrettyPrinter_Formatter_concat___lambda__1___boxed(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__65; static lean_object* l_Lean_Parser_nameLit_parenthesizer___closed__1; lean_object* l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_nameLitNoAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -390,18 +396,16 @@ lean_object* l_Lean_Parser_notFollowedBy(lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__34; lean_object* l_Lean_PrettyPrinter_Formatter_pushWhitespace(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_identWithPartialTrailingDot_formatter___closed__7; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__1; lean_object* l_Lean_Parser_symbol(lean_object*); static lean_object* l_Lean_Parser_sepByIndent___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_sepBy1Indent_parenthesizer(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_withForbidden_parenthesizer___boxed(lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__25; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__37; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__74; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_ppHardLineUnlessUngrouped_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Parser_sepByIndent_formatter___spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ppDedentIfGrouped_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__14; lean_object* l_Lean_Syntax_node3(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_Lean_Parser_ppGroup___boxed(lean_object*); @@ -411,6 +415,7 @@ static lean_object* l_Lean_Parser_commandParser_formatter___rarg___closed__2; static lean_object* l_Lean_Parser_mkAntiquotSplice_formatter___closed__2; static lean_object* l_Lean_Parser_nameLit___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_symbol_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__24; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__17; static lean_object* l___regBuiltin_Lean_Parser_ppRealGroup_docString__1___closed__3; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__40; @@ -418,30 +423,32 @@ LEAN_EXPORT lean_object* l_Lean_Parser_withResetCache_parenthesizer(lean_object* lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkLinebreakBefore_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppSpace; lean_object* l_Lean_PrettyPrinter_Formatter_optionalNoAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__8; static lean_object* l_Lean_Parser_optional_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_nameLit_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_scientificLit_docString__1___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__97; LEAN_EXPORT lean_object* l_Lean_Parser_nameLit; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__19; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__8; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__10; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__59; LEAN_EXPORT lean_object* l_Lean_Parser_suppressInsideQuot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__33; lean_object* l_Lean_Parser_checkNoWsBefore(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__92; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__3; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Parser_sepByIndent_formatter___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_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__5; static lean_object* l_Lean_Parser_sepByIndent___closed__2; static lean_object* l_Lean_Parser_hygieneInfo_formatter___closed__4; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__80; static lean_object* l_Lean_Parser_scientificLit___closed__1; static lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___closed__9; static lean_object* l_Lean_Parser_strLit_formatter___closed__4; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__11; static lean_object* l_Lean_Parser_scientificLit_parenthesizer___closed__2; lean_object* l_Lean_Parser_withAntiquot(lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__23; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__13; static lean_object* l_Lean_Parser_sepByIndent___closed__3; lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_withPosition_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -457,12 +464,11 @@ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppAllowUngrouped; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__6; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__4; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__10; static lean_object* l_Lean_Parser_hygieneInfo_formatter___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__45; lean_object* l_Lean_PrettyPrinter_Parenthesizer_nonReservedSymbolNoAntiquot_parenthesizer___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_withForbidden_formatter___boxed(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__49; lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_ppHardSpace_docString__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_scientificLit_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -477,16 +483,17 @@ LEAN_EXPORT lean_object* l_Lean_Parser_withResetCache_formatter(lean_object*, le static lean_object* l_Lean_Parser_sepByElemParser_formatter___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Parser_Basic_0__Lean_Parser_addQuotDepth_parenthesizer___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_nonReservedSymbol_parenthesizer(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__80; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__28; LEAN_EXPORT lean_object* l_Lean_Parser_withAntiquotSpliceAndSuffix_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__39; uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__11; static lean_object* l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__2; static lean_object* l_Lean_Parser_nameLit_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_adaptCacheableContext_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer__1(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__51; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__16; static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter__1___closed__3; static lean_object* l_Lean_Parser_ident___closed__2; lean_object* l_Lean_Parser_many1NoAntiquot(lean_object*); @@ -510,9 +517,8 @@ static lean_object* l_Lean_Parser_identWithPartialTrailingDot___closed__4; static lean_object* l_Lean_Parser_charLit_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_ppRealFill_docString__1___closed__3; static lean_object* l_List_forIn_loop___at_Lean_Parser_sepByIndent_formatter___spec__2___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__53; LEAN_EXPORT lean_object* l_Lean_Parser_ppHardSpace_parenthesizer___rarg(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__3; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__7; static lean_object* l_Lean_Parser_identWithPartialTrailingDot___closed__5; static lean_object* l___regBuiltin_Lean_Parser_ppGroup_docString__1___closed__2; @@ -521,19 +527,20 @@ static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer_ static lean_object* l_Lean_Parser_rawIdent_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_commandParser_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_withForbidden_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__84; lean_object* l_Lean_Parser_andthen(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppHardSpace; lean_object* l_Lean_PrettyPrinter_Parenthesizer_manyNoAntiquot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_symbol_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__62; LEAN_EXPORT lean_object* l_Lean_Parser_withForbidden_parenthesizer(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__29; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__20; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_strLit_docString__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_setExpected_parenthesizer___boxed(lean_object*); lean_object* l_Lean_Parser_checkColGe(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__62; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__44; static lean_object* l___regBuiltin_Lean_Parser_many1Indent_docString__1___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__88; static lean_object* l_Lean_Parser_charLit_formatter___closed__3; static lean_object* l_Lean_Parser_optional_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_evalInsideQuot_parenthesizer(lean_object*); @@ -542,7 +549,6 @@ LEAN_EXPORT lean_object* l_Lean_Parser_ppSpace_parenthesizer___boxed(lean_object static lean_object* l___regBuiltin_Lean_Parser_ppRealGroup_docString__1___closed__2; lean_object* lean_int_sub(lean_object*, lean_object*); static lean_object* l_Lean_Parser_numLit_formatter___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__32; LEAN_EXPORT lean_object* l_Lean_Parser_ident_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_charLit; LEAN_EXPORT lean_object* l_Lean_Parser_sepBy_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -554,7 +560,6 @@ static lean_object* l_Lean_Parser_termParser_formatter___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_rawIdent; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__2; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__8; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__26; LEAN_EXPORT lean_object* l_Lean_Parser_evalInsideQuot_formatter(lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__27; extern lean_object* l_Lean_PrettyPrinter_Formatter_formatterAliasesRef; @@ -564,62 +569,58 @@ LEAN_EXPORT lean_object* l_Lean_Parser_commandParser_formatter___boxed(lean_obje LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_hygieneInfo_docString__1(lean_object*); static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__9; static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__34; LEAN_EXPORT lean_object* l_Lean_Parser_sepByIndent_formatter___lambda__1(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_Lean_Parser_scientificLit; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_many(lean_object*); LEAN_EXPORT lean_object* l_Lean_ppDedent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_numLit_parenthesizer___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__43; lean_object* l_Lean_PrettyPrinter_Parenthesizer_unicodeSymbolNoAntiquot_parenthesizer___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__44; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__73; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__45; static lean_object* l_Lean_Parser_many1Indent___closed__1; static lean_object* l_Lean_Parser_hygieneInfo___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__27; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__24; lean_object* l_Lean_PrettyPrinter_Formatter_pushNone_formatter___boxed(lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__51; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__16; LEAN_EXPORT lean_object* l_Lean_ppAllowUngrouped_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_many_formatter___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__35; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__18; static lean_object* l___regBuiltin_Lean_Parser_numLit_docString__1___closed__2; static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__2; static lean_object* l_Lean_Parser_scientificLit___closed__2; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Parser_sepByIndent_formatter___spec__3(lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Parser_sepBy1Indent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__67; static lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___closed__1; static lean_object* l_Lean_Parser_mkAntiquotSplice_formatter___closed__4; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__45; LEAN_EXPORT lean_object* l_Lean_Parser_ppLine; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__91; LEAN_EXPORT lean_object* l_Lean_ppSpace_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_antiquotNestedExpr_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_ppIndent_docString__1___closed__3; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__27; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__55; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_manyIndent_docString__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_sepBy1Indent_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__11; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__32; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__42; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__2; static lean_object* l_Lean_Parser_identWithPartialTrailingDot___closed__7; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__26; LEAN_EXPORT lean_object* l_Lean_Parser_withPosition_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_leadingNode_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_hygieneInfo_parenthesizer___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__56; lean_object* l_Lean_PrettyPrinter_Parenthesizer_withoutInfo_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_adaptCacheableContext_formatter___boxed(lean_object*); static lean_object* l_Lean_Parser_optional_formatter___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__29; LEAN_EXPORT lean_object* l___private_Lean_Parser_Basic_0__Lean_Parser_addQuotDepth_formatter___boxed(lean_object*); lean_object* l_Lean_Parser_registerAliasCore___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_patternIgnore_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_identWithPartialTrailingDot_parenthesizer___closed__4; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_termParser_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ident; LEAN_EXPORT lean_object* l_Lean_Parser_optional_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -634,26 +635,24 @@ lean_object* l_Lean_PrettyPrinter_Formatter_group(lean_object*, lean_object*, le static lean_object* l_Lean_Parser_scientificLit_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_manyIndent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__53; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__12; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_many1Indent_docString__1(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__35; static lean_object* l___regBuiltin_Lean_Parser_ppDedent_docString__1___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__93; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__82; static lean_object* l_Lean_Parser_strLit_formatter___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__71; static lean_object* l___regBuiltin_Lean_Parser_ppRealFill_docString__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_ppLine_parenthesizer___rarg(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__82; LEAN_EXPORT lean_object* l_Lean_Parser_withoutForbidden_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__55; lean_object* l_Lean_PrettyPrinter_Parenthesizer_scientificLitNoAntiquot_parenthesizer___boxed(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__48; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_visitArgs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__31; static lean_object* l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__6; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__13; LEAN_EXPORT lean_object* l_Lean_Parser_ppAllowUngrouped_parenthesizer___rarg(lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_fold(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_dbgTraceState_formatter___boxed(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__96; static lean_object* l___regBuiltin_Lean_Parser_many_docString__1___closed__2; static lean_object* l___regBuiltin_Lean_Parser_many1_docString__1___closed__3; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); @@ -662,17 +661,14 @@ lean_object* l_Substring_takeRightWhileAux___at_Substring_trimRight___spec__1(le LEAN_EXPORT lean_object* l_Lean_Parser_withCache_formatter___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_sepByElemParser_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_identWithPartialTrailingDot_parenthesizer___closed__6; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__17; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__2; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__39; LEAN_EXPORT lean_object* l_Lean_Parser_evalInsideQuot_formatter___boxed(lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_checkNoImmediateColon_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_atomic_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__22; static lean_object* l_Lean_Parser_ident_formatter___closed__3; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppGroup_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__10; static lean_object* l_Lean_Parser_identWithPartialTrailingDot_formatter___closed__4; extern lean_object* l_Lean_PrettyPrinter_Parenthesizer_parenthesizerAliasesRef; lean_object* l_Lean_Parser_withAntiquotSpliceAndSuffix(lean_object*, lean_object*, lean_object*); @@ -680,14 +676,12 @@ static lean_object* l_Lean_Parser_nameLit_formatter___closed__4; extern lean_object* l_Lean_Parser_skip; LEAN_EXPORT lean_object* l_Lean_Parser_decQuotDepth_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__24; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__18; static lean_object* l_Lean_Parser_charLit___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_ppIndent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ppHardLineUnlessUngrouped_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_withoutPosition_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__16; extern lean_object* l_Lean_Parser_scientificLitNoAntiquot; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__72; LEAN_EXPORT lean_object* l_Lean_Parser_unicodeSymbol_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_identWithPartialTrailingDot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__13; @@ -696,6 +690,8 @@ lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_ident_docString__1___closed__1; static lean_object* l_Lean_Parser_leadingNode_formatter___closed__2; lean_object* l_Lean_Parser_registerAlias(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__99; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__19; LEAN_EXPORT lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_group_docString__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_sepBy1Indent(lean_object*, lean_object*, lean_object*, uint8_t); @@ -712,10 +708,9 @@ LEAN_EXPORT lean_object* l_Lean_Parser_many1(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_nameLit_docString__1___closed__3; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__7; uint8_t l_Lean_Syntax_isNone(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__46; lean_object* l_Lean_PrettyPrinter_Formatter_withAntiquotSuffixSplice_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__61; static lean_object* l_Lean_Parser_group_formatter___closed__2; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__84; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__20; static lean_object* l_Lean_Parser_strLit_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_manyIndent_docString__1___closed__2; @@ -724,6 +719,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_antiquotExpr_formatter(lean_object*, lean static lean_object* l_Lean_Parser_charLit_parenthesizer___closed__1; static lean_object* l_Lean_Parser_commandParser_formatter___rarg___closed__1; lean_object* lean_nat_sub(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__63; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__21; lean_object* l_Std_Format_getIndent(lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__67; @@ -732,7 +728,6 @@ static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__13; static lean_object* l___regBuiltin_Lean_Parser_ppDedentIfGrouped_docString__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_mkAntiquotSplice_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_PrettyPrinter_backtrackExceptionId; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__40; LEAN_EXPORT lean_object* l_Lean_Parser_termParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Parser_Basic_0__Lean_Parser_addQuotDepth_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppRealGroup(lean_object*); @@ -747,40 +742,42 @@ static lean_object* l_Lean_Parser_numLit_formatter___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_numLit_docString__1(lean_object*); extern lean_object* l_Lean_Parser_maxPrec; static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter__1___closed__5; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__92; lean_object* l_Lean_Parser_sepBy(lean_object*, lean_object*, lean_object*, uint8_t); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__49; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__15; lean_object* l_Lean_PrettyPrinter_Formatter_strLitNoAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__52; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__21; extern lean_object* l_Lean_Parser_identNoAntiquot; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__66; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__60; static lean_object* l___regBuiltin_Lean_Parser_ppGroup_docString__1___closed__1; static lean_object* l_Lean_Parser_nameLit_parenthesizer___closed__2; lean_object* l_Lean_PrettyPrinter_Parenthesizer_charLitNoAntiquot_parenthesizer___boxed(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__36; static lean_object* l_Lean_Parser_antiquotExpr_parenthesizer___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__54; lean_object* l_List_reverse___rarg(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__30; LEAN_EXPORT lean_object* l_Lean_Parser_many1Indent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__35; static lean_object* l_Lean_Parser_identWithPartialTrailingDot___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_mkAntiquotSplice_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__60; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_ppAllowUngrouped_docString__1(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__8; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__1; lean_object* l_String_intercalate(lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__51; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__7; static lean_object* l___regBuiltin_Lean_Parser_ppSpace_docString__1___closed__3; static lean_object* l_Lean_Parser_identWithPartialTrailingDot___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_sepBy1_parenthesizer___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_Parser_many1Indent_docString__1___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__47; static lean_object* l___regBuiltin_Lean_Parser_ppIndent_docString__1___closed__2; lean_object* l_Lean_PrettyPrinter_Parenthesizer_tokenWithAntiquot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_identWithPartialTrailingDot_parenthesizer___closed__5; static lean_object* l_Lean_Parser_identWithPartialTrailingDot_formatter___closed__3; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__26; size_t lean_usize_add(size_t, size_t); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__89; LEAN_EXPORT lean_object* l_Lean_Parser_sepByIndent(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Parser_ppDedentIfGrouped(lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__6; @@ -794,11 +791,13 @@ static lean_object* l_Lean_Parser_many_formatter___closed__1; static lean_object* l_Lean_Parser_optional_formatter___closed__4; lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l_Lean_Parser_nodeWithAntiquot_formatter(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__56; static lean_object* l_Lean_Parser_numLit_formatter___closed__4; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__71; static lean_object* l___regBuiltin_Lean_Parser_ppHardSpace_docString__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_nodeWithAntiquot_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__28; LEAN_EXPORT lean_object* l_Lean_Parser_incQuotDepth_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__76; static lean_object* l_Lean_Parser_sepByIndent_formatter___closed__1; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_ident_docString__1___closed__2; @@ -818,29 +817,33 @@ static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___ static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__47; static lean_object* l_Lean_Parser_optional_formatter___closed__2; lean_object* l_Lean_PrettyPrinter_Parenthesizer_rawIdentNoAntiquot_parenthesizer___boxed(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__27; LEAN_EXPORT lean_object* l_Lean_Parser_sepBy_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__15; static lean_object* l___regBuiltin_Lean_Parser_optional_docString__1___closed__2; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__30; static lean_object* l___regBuiltin_Lean_Parser_scientificLit_docString__1___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__67; lean_object* lean_string_append(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__31; LEAN_EXPORT lean_object* l_Lean_Parser_nonReservedSymbol_formatter___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_Extra___hyg_1789____closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_group_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_numLit_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Parser_Basic_0__Lean_Parser_addQuotDepth_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_sepByIndent___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__16; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__50; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__49; lean_object* l_Lean_PrettyPrinter_Formatter_symbolNoAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_ppLine_docString__1(lean_object*); lean_object* lean_array_get_size(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_optional_docString__1___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_many_docString__1(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__47; static lean_object* l_Lean_Parser_mkAntiquotSplice_formatter___closed__3; static lean_object* l_Lean_Parser_numLit___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__60; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__42; static lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___closed__3; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__98; static lean_object* l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__5; lean_object* l_Lean_PrettyPrinter_Formatter_categoryParser_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_identWithPartialTrailingDot___closed__2; @@ -851,16 +854,15 @@ LEAN_EXPORT lean_object* l_Lean_Parser_sepBy1_parenthesizer(lean_object*, lean_o LEAN_EXPORT lean_object* l_Lean_Parser_notSymbol_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ppAllowUngrouped_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppDedentIfGrouped_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__79; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__4; static lean_object* l_Lean_Parser_identWithPartialTrailingDot_formatter___closed__2; static lean_object* l_Lean_ppDedentIfGrouped_formatter___closed__1; lean_object* l_Lean_PrettyPrinter_Formatter_unicodeSymbolNoAntiquot_formatter(lean_object*, lean_object*, 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_Parser_evalInsideQuot_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_mkAntiquotSplice_formatter___closed__6; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__75; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__73; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__31; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__68; uint8_t l_Lean_Exception_isRuntime(lean_object*); static lean_object* l_Lean_Parser_numLit_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_sepByIndent___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -873,10 +875,8 @@ static lean_object* l___regBuiltin_Lean_Parser_many1Indent_docString__1___closed static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__10; static lean_object* l_Lean_Parser_many1Indent_parenthesizer___closed__1; static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__10; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__41; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__34; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789_(lean_object*); lean_object* l_String_toSubstring_x27(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_many_docString__1___closed__1; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__20; @@ -884,14 +884,18 @@ LEAN_EXPORT lean_object* l_Lean_Parser_withoutForbidden_parenthesizer(lean_objec static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_dbgTraceState_formatter(lean_object*); static lean_object* l_Lean_Parser_sepByIndent___closed__5; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__76; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__1; static lean_object* l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__25; lean_object* l_Lean_PrettyPrinter_Parenthesizer_hygieneInfoNoAntiquot_parenthesizer___boxed(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__2; static lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___closed__6; static lean_object* l___regBuiltin_Lean_Parser_manyIndent_docString__1___closed__1; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__17; static lean_object* l_Lean_Parser_hygieneInfo_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_numLit_docString__1___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__77; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_patternIgnore_docString__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppDedentIfGrouped___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_adaptCacheableContext_parenthesizer___boxed(lean_object*); @@ -906,22 +910,18 @@ static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Le static lean_object* l_Lean_Parser_antiquotExpr_formatter___closed__1; static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_scientificLit_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__85; static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_ppRealGroup_docString__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_strLit_docString__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_ppGroup_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_node_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__19; LEAN_EXPORT lean_object* l_Lean_Parser_nonReservedSymbol_formatter(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_identWithPartialTrailingDot_parenthesizer___closed__2; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__89; lean_object* l_Lean_PrettyPrinter_Parenthesizer_nameLitNoAntiquot_parenthesizer___boxed(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_strLit_docString__1___closed__3; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__83; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__23; lean_object* l_Lean_PrettyPrinter_Parenthesizer_pushNone_parenthesizer___boxed(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__15; static lean_object* l_Lean_Parser_numLit_parenthesizer___closed__2; static lean_object* _init_l_Lean_Parser_leadingNode_formatter___closed__1() { _start: @@ -5012,88 +5012,86 @@ lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Parser_sepByIndent_formatter___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Parser_sepByIndent_formatter___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) { _start: { -lean_object* x_8; uint8_t x_9; -x_8 = lean_unsigned_to_nat(0u); -x_9 = lean_nat_dec_eq(x_4, x_8); -if (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; uint8_t x_16; lean_object* x_17; -x_10 = lean_unsigned_to_nat(1u); -x_11 = lean_nat_sub(x_4, x_10); -lean_dec(x_4); -x_12 = lean_array_fget(x_3, x_5); -x_13 = lean_array_get_size(x_2); -x_14 = lean_unsigned_to_nat(2u); -x_15 = lean_nat_mod(x_5, x_14); -x_16 = lean_nat_dec_eq(x_15, x_10); -lean_dec(x_15); -x_17 = lean_nat_add(x_5, x_10); -if (x_16 == 0) +lean_object* x_7; uint8_t x_8; +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_nat_dec_eq(x_3, x_7); +if (x_8 == 0) { -uint8_t x_18; lean_object* x_19; lean_object* x_20; +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; +x_9 = lean_unsigned_to_nat(1u); +x_10 = lean_nat_sub(x_3, x_9); +lean_dec(x_3); +x_11 = lean_array_fget(x_2, x_4); +x_12 = lean_unsigned_to_nat(2u); +x_13 = lean_nat_mod(x_4, x_12); +x_14 = lean_nat_dec_eq(x_13, x_9); lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_5); -x_18 = 0; -x_19 = lean_box(x_18); -x_20 = lean_array_push(x_7, x_19); -x_4 = x_11; -x_5 = x_17; -x_6 = lean_box(0); -x_7 = x_20; +x_15 = lean_nat_add(x_4, x_9); +if (x_14 == 0) +{ +uint8_t x_16; lean_object* x_17; lean_object* x_18; +lean_dec(x_11); +lean_dec(x_4); +x_16 = 0; +x_17 = lean_box(x_16); +x_18 = lean_array_push(x_6, x_17); +x_3 = x_10; +x_4 = x_15; +x_5 = lean_box(0); +x_6 = x_18; goto _start; } else { -uint8_t x_22; -x_22 = l_Lean_Syntax_matchesNull(x_12, x_8); -if (x_22 == 0) +uint8_t x_20; +x_20 = l_Lean_Syntax_matchesNull(x_11, x_7); +if (x_20 == 0) { -uint8_t x_23; lean_object* x_24; lean_object* x_25; -lean_dec(x_13); -lean_dec(x_5); -x_23 = 0; -x_24 = lean_box(x_23); -x_25 = lean_array_push(x_7, x_24); -x_4 = x_11; -x_5 = x_17; -x_6 = lean_box(0); -x_7 = x_25; +uint8_t x_21; lean_object* x_22; lean_object* x_23; +lean_dec(x_4); +x_21 = 0; +x_22 = lean_box(x_21); +x_23 = lean_array_push(x_6, x_22); +x_3 = x_10; +x_4 = x_15; +x_5 = lean_box(0); +x_6 = x_23; goto _start; } else { -lean_object* x_27; uint8_t x_28; -x_27 = lean_nat_sub(x_13, x_10); -lean_dec(x_13); -x_28 = lean_nat_dec_eq(x_5, x_27); -lean_dec(x_27); -lean_dec(x_5); -if (x_28 == 0) -{ -uint8_t x_29; lean_object* x_30; lean_object* x_31; -x_29 = 1; -x_30 = lean_box(x_29); -x_31 = lean_array_push(x_7, x_30); -x_4 = x_11; -x_5 = x_17; -x_6 = lean_box(0); -x_7 = x_31; +lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_25 = lean_array_get_size(x_1); +x_26 = lean_nat_sub(x_25, x_9); +lean_dec(x_25); +x_27 = lean_nat_dec_eq(x_4, x_26); +lean_dec(x_26); +lean_dec(x_4); +if (x_27 == 0) +{ +uint8_t x_28; lean_object* x_29; lean_object* x_30; +x_28 = 1; +x_29 = lean_box(x_28); +x_30 = lean_array_push(x_6, x_29); +x_3 = x_10; +x_4 = x_15; +x_5 = lean_box(0); +x_6 = x_30; goto _start; } else { -uint8_t x_33; lean_object* x_34; lean_object* x_35; -x_33 = 0; -x_34 = lean_box(x_33); -x_35 = lean_array_push(x_7, x_34); -x_4 = x_11; -x_5 = x_17; -x_6 = lean_box(0); -x_7 = x_35; +uint8_t x_32; lean_object* x_33; lean_object* x_34; +x_32 = 0; +x_33 = lean_box(x_32); +x_34 = lean_array_push(x_6, x_33); +x_3 = x_10; +x_4 = x_15; +x_5 = lean_box(0); +x_6 = x_34; goto _start; } } @@ -5101,9 +5099,9 @@ goto _start; } else { -lean_dec(x_5); lean_dec(x_4); -return x_7; +lean_dec(x_3); +return x_6; } } } @@ -5571,13 +5569,13 @@ x_11 = lean_ctor_get(x_9, 1); lean_inc(x_11); lean_dec(x_9); x_12 = l_Lean_Syntax_getArgs(x_10); +lean_dec(x_10); x_13 = lean_array_get_size(x_12); x_14 = lean_mk_empty_array_with_capacity(x_13); x_15 = lean_unsigned_to_nat(0u); lean_inc(x_13); -x_16 = l_Array_mapIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1(x_10, x_12, x_12, x_13, x_15, lean_box(0), x_14); +x_16 = l_Array_mapFinIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1(x_12, x_12, x_13, x_15, lean_box(0), x_14); lean_dec(x_12); -lean_dec(x_10); x_17 = lean_array_get_size(x_16); x_18 = lean_nat_dec_lt(x_15, x_17); lean_inc(x_13); @@ -5760,15 +5758,14 @@ return x_52; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Parser_sepByIndent_formatter___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Parser_sepByIndent_formatter___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) { _start: { -lean_object* x_8; -x_8 = l_Array_mapIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_3); +lean_object* x_7; +x_7 = l_Array_mapFinIdxM_map___at_Lean_Parser_sepByIndent_formatter___spec__1(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_2); lean_dec(x_1); -return x_8; +return x_7; } } LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Parser_sepByIndent_formatter___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) { @@ -9387,7 +9384,7 @@ lean_dec(x_1); return x_6; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__1() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__1() { _start: { lean_object* x_1; @@ -9395,17 +9392,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_patternIgnore), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__2() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__1; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__1; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__3() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__3() { _start: { lean_object* x_1; lean_object* x_2; @@ -9415,7 +9412,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__4() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__4() { _start: { lean_object* x_1; lean_object* x_2; @@ -9425,12 +9422,12 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__5() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__5() { _start: { lean_object* x_1; lean_object* x_2; uint8_t x_3; lean_object* x_4; x_1 = lean_box(0); -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__4; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__4; x_3 = 0; x_4 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_4, 0, x_1); @@ -9439,7 +9436,7 @@ lean_ctor_set_uint8(x_4, sizeof(void*)*2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__6() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__6() { _start: { lean_object* x_1; @@ -9447,17 +9444,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_patternIgnore_formatter), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__7() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__6; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__6; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__8() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__8() { _start: { lean_object* x_1; @@ -9465,7 +9462,7 @@ x_1 = l_Lean_PrettyPrinter_Formatter_formatterAliasesRef; return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__9() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__9() { _start: { lean_object* x_1; @@ -9473,17 +9470,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_patternIgnore_parenthesizer), 6, return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__10() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__9; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__9; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__11() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__11() { _start: { lean_object* x_1; @@ -9491,7 +9488,7 @@ x_1 = l_Lean_PrettyPrinter_Parenthesizer_parenthesizerAliasesRef; return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__12() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__12() { _start: { lean_object* x_1; @@ -9499,17 +9496,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_group), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__13() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__13() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__12; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__12; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__14() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__14() { _start: { lean_object* x_1; lean_object* x_2; @@ -9519,7 +9516,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__15() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__15() { _start: { lean_object* x_1; @@ -9527,17 +9524,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_group_formatter), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__16() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__16() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__15; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__15; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__17() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__17() { _start: { lean_object* x_1; @@ -9545,17 +9542,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_group_parenthesizer), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__18() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__18() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__17; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__17; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__19() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -9565,7 +9562,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__20() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__20() { _start: { lean_object* x_1; lean_object* x_2; @@ -9575,7 +9572,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__21() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__21() { _start: { lean_object* x_1; lean_object* x_2; @@ -9585,7 +9582,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__22() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__22() { _start: { lean_object* x_1; lean_object* x_2; @@ -9595,12 +9592,12 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__23() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__23() { _start: { lean_object* x_1; lean_object* x_2; uint8_t x_3; lean_object* x_4; x_1 = lean_box(0); -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__22; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__22; x_3 = 1; x_4 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_4, 0, x_1); @@ -9609,7 +9606,7 @@ lean_ctor_set_uint8(x_4, sizeof(void*)*2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__24() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__24() { _start: { lean_object* x_1; @@ -9617,17 +9614,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppHardSpace_formatter___boxed), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__25() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__25() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__24; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__24; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__26() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__26() { _start: { lean_object* x_1; @@ -9635,17 +9632,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppHardSpace_parenthesizer___boxed return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__27() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__27() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__26; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__26; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__28() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__28() { _start: { lean_object* x_1; lean_object* x_2; @@ -9655,7 +9652,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__29() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__29() { _start: { lean_object* x_1; @@ -9663,17 +9660,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppSpace_formatter___boxed), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__30() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__30() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__29; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__29; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__31() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__31() { _start: { lean_object* x_1; @@ -9681,17 +9678,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppSpace_parenthesizer___boxed), 4 return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__32() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__32() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__31; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__31; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__33() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__33() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -9701,7 +9698,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__34() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__34() { _start: { lean_object* x_1; lean_object* x_2; @@ -9711,7 +9708,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__35() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__35() { _start: { lean_object* x_1; @@ -9719,17 +9716,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppLine_formatter___boxed), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__36() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__36() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__35; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__35; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__37() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__37() { _start: { lean_object* x_1; @@ -9737,17 +9734,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppLine_parenthesizer___boxed), 4, return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__38() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__38() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__37; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__37; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__39() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__39() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -9757,7 +9754,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__40() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__40() { _start: { lean_object* x_1; @@ -9765,17 +9762,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppGroup___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__41() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__41() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__40; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__40; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__42() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__42() { _start: { lean_object* x_1; lean_object* x_2; @@ -9785,7 +9782,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__43() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__43() { _start: { lean_object* x_1; lean_object* x_2; uint8_t x_3; lean_object* x_4; @@ -9799,7 +9796,7 @@ lean_ctor_set_uint8(x_4, sizeof(void*)*2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__44() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__44() { _start: { lean_object* x_1; @@ -9807,17 +9804,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppGroup_formatter), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__45() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__45() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__44; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__44; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__46() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__46() { _start: { lean_object* x_1; @@ -9825,17 +9822,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppGroup_parenthesizer), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__47() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__47() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__46; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__46; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__48() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__48() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -9845,7 +9842,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__49() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__49() { _start: { lean_object* x_1; @@ -9853,17 +9850,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppRealGroup___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__50() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__50() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__49; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__49; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__51() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__51() { _start: { lean_object* x_1; lean_object* x_2; @@ -9873,7 +9870,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__52() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__52() { _start: { lean_object* x_1; @@ -9881,17 +9878,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppRealGroup_formatter), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__53() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__53() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__52; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__52; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__54() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__54() { _start: { lean_object* x_1; @@ -9899,17 +9896,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppRealGroup_parenthesizer), 6, 0) return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__55() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__55() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__54; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__54; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__56() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__56() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -9919,7 +9916,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__57() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__57() { _start: { lean_object* x_1; @@ -9927,17 +9924,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppRealFill___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__58() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__58() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__57; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__57; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__59() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__59() { _start: { lean_object* x_1; lean_object* x_2; @@ -9947,7 +9944,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__60() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__60() { _start: { lean_object* x_1; @@ -9955,17 +9952,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppRealFill_formatter), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__61() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__61() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__60; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__60; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__62() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__62() { _start: { lean_object* x_1; @@ -9973,17 +9970,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppRealFill_parenthesizer), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__63() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__63() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__62; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__62; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__64() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__64() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -9993,7 +9990,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__65() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__65() { _start: { lean_object* x_1; @@ -10001,17 +9998,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppIndent___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__66() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__66() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__65; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__65; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__67() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__67() { _start: { lean_object* x_1; lean_object* x_2; @@ -10021,7 +10018,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__68() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__68() { _start: { lean_object* x_1; @@ -10029,17 +10026,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppIndent_formatter), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__69() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__69() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__68; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__68; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__70() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__70() { _start: { lean_object* x_1; @@ -10047,17 +10044,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppIndent_parenthesizer), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__71() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__71() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__70; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__70; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__72() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__72() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -10067,7 +10064,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__73() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__73() { _start: { lean_object* x_1; @@ -10075,17 +10072,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppDedent___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__74() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__74() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__73; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__73; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__75() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__75() { _start: { lean_object* x_1; lean_object* x_2; @@ -10095,7 +10092,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__76() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__76() { _start: { lean_object* x_1; @@ -10103,17 +10100,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppDedent_formatter), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__77() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__77() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__76; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__76; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__78() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__78() { _start: { lean_object* x_1; @@ -10121,17 +10118,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppDedent_parenthesizer), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__79() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__79() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__78; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__78; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__80() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__80() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -10141,7 +10138,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__81() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__81() { _start: { lean_object* x_1; @@ -10149,17 +10146,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppDedentIfGrouped___boxed), 1, 0) return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__82() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__82() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__81; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__81; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__83() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__83() { _start: { lean_object* x_1; lean_object* x_2; @@ -10169,7 +10166,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__84() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__84() { _start: { lean_object* x_1; @@ -10177,17 +10174,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppDedentIfGrouped_formatter), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__85() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__85() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__84; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__84; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__86() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__86() { _start: { lean_object* x_1; @@ -10195,17 +10192,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppDedentIfGrouped_parenthesizer), return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__87() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__87() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__86; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__86; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__88() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__88() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -10215,7 +10212,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__89() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__89() { _start: { lean_object* x_1; lean_object* x_2; @@ -10225,7 +10222,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__90() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__90() { _start: { lean_object* x_1; @@ -10233,17 +10230,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppAllowUngrouped_formatter___boxed), 1, return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__91() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__91() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__90; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__90; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__92() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__92() { _start: { lean_object* x_1; @@ -10251,17 +10248,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppAllowUngrouped_parenthesizer___ return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__93() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__93() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__92; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__92; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__94() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__94() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -10271,7 +10268,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__95() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__95() { _start: { lean_object* x_1; lean_object* x_2; @@ -10281,7 +10278,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__96() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__96() { _start: { lean_object* x_1; @@ -10289,17 +10286,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppHardLineUnlessUngrouped_formatter___bo return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__97() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__97() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__96; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__96; 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_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__98() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__98() { _start: { lean_object* x_1; @@ -10307,25 +10304,25 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppHardLineUnlessUngrouped_parenth return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__99() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__99() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__98; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__98; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770_(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; x_2 = l_Lean_Parser_patternIgnore_formatter___closed__2; x_3 = l___regBuiltin_Lean_Parser_patternIgnore_docString__1___closed__1; -x_4 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__2; -x_5 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__3; -x_6 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__5; +x_4 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__2; +x_5 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__3; +x_6 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__5; x_7 = l_Lean_Parser_registerAlias(x_2, x_3, x_4, x_5, x_6, x_1); if (lean_obj_tag(x_7) == 0) { @@ -10333,8 +10330,8 @@ lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); lean_dec(x_7); -x_9 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__8; -x_10 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__7; +x_9 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__8; +x_10 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__7; x_11 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_2, x_10, x_8); if (lean_obj_tag(x_11) == 0) { @@ -10342,8 +10339,8 @@ lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; x_12 = lean_ctor_get(x_11, 1); lean_inc(x_12); lean_dec(x_11); -x_13 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__11; -x_14 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__10; +x_13 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__11; +x_14 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__10; x_15 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_2, x_14, x_12); if (lean_obj_tag(x_15) == 0) { @@ -10353,8 +10350,8 @@ lean_inc(x_16); lean_dec(x_15); x_17 = l_Lean_Parser_group_formatter___closed__2; x_18 = l___regBuiltin_Lean_Parser_group_docString__1___closed__1; -x_19 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__13; -x_20 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__14; +x_19 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__13; +x_20 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__14; x_21 = l_Lean_Parser_registerAlias(x_17, x_18, x_19, x_20, x_6, x_16); if (lean_obj_tag(x_21) == 0) { @@ -10362,7 +10359,7 @@ lean_object* x_22; lean_object* x_23; lean_object* x_24; x_22 = lean_ctor_get(x_21, 1); lean_inc(x_22); lean_dec(x_21); -x_23 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__16; +x_23 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__16; x_24 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_17, x_23, x_22); if (lean_obj_tag(x_24) == 0) { @@ -10370,7 +10367,7 @@ lean_object* x_25; lean_object* x_26; lean_object* x_27; x_25 = lean_ctor_get(x_24, 1); lean_inc(x_25); lean_dec(x_24); -x_26 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__18; +x_26 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__18; x_27 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_17, x_26, x_25); if (lean_obj_tag(x_27) == 0) { @@ -10378,11 +10375,11 @@ lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean x_28 = lean_ctor_get(x_27, 1); lean_inc(x_28); lean_dec(x_27); -x_29 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__19; +x_29 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__19; x_30 = l___regBuiltin_Lean_Parser_ppHardSpace_docString__1___closed__2; -x_31 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__20; -x_32 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__21; -x_33 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__23; +x_31 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__20; +x_32 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__21; +x_33 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__23; x_34 = l_Lean_Parser_registerAlias(x_29, x_30, x_31, x_32, x_33, x_28); if (lean_obj_tag(x_34) == 0) { @@ -10390,7 +10387,7 @@ lean_object* x_35; lean_object* x_36; lean_object* x_37; x_35 = lean_ctor_get(x_34, 1); lean_inc(x_35); lean_dec(x_34); -x_36 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__25; +x_36 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__25; x_37 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_29, x_36, x_35); if (lean_obj_tag(x_37) == 0) { @@ -10398,7 +10395,7 @@ lean_object* x_38; lean_object* x_39; lean_object* x_40; x_38 = lean_ctor_get(x_37, 1); lean_inc(x_38); lean_dec(x_37); -x_39 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__27; +x_39 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__27; x_40 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_29, x_39, x_38); if (lean_obj_tag(x_40) == 0) { @@ -10408,7 +10405,7 @@ lean_inc(x_41); lean_dec(x_40); x_42 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29_______________closed__23; x_43 = l___regBuiltin_Lean_Parser_ppSpace_docString__1___closed__2; -x_44 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__28; +x_44 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__28; x_45 = l_Lean_Parser_registerAlias(x_42, x_43, x_31, x_44, x_33, x_41); if (lean_obj_tag(x_45) == 0) { @@ -10416,7 +10413,7 @@ lean_object* x_46; lean_object* x_47; lean_object* x_48; x_46 = lean_ctor_get(x_45, 1); lean_inc(x_46); lean_dec(x_45); -x_47 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__30; +x_47 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__30; x_48 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_42, x_47, x_46); if (lean_obj_tag(x_48) == 0) { @@ -10424,7 +10421,7 @@ lean_object* x_49; lean_object* x_50; lean_object* x_51; x_49 = lean_ctor_get(x_48, 1); lean_inc(x_49); lean_dec(x_48); -x_50 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__32; +x_50 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__32; x_51 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_42, x_50, x_49); if (lean_obj_tag(x_51) == 0) { @@ -10432,9 +10429,9 @@ lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean x_52 = lean_ctor_get(x_51, 1); lean_inc(x_52); lean_dec(x_51); -x_53 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__33; +x_53 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__33; x_54 = l___regBuiltin_Lean_Parser_ppLine_docString__1___closed__2; -x_55 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__34; +x_55 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__34; x_56 = l_Lean_Parser_registerAlias(x_53, x_54, x_31, x_55, x_33, x_52); if (lean_obj_tag(x_56) == 0) { @@ -10442,7 +10439,7 @@ lean_object* x_57; lean_object* x_58; lean_object* x_59; x_57 = lean_ctor_get(x_56, 1); lean_inc(x_57); lean_dec(x_56); -x_58 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__36; +x_58 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__36; x_59 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_53, x_58, x_57); if (lean_obj_tag(x_59) == 0) { @@ -10450,7 +10447,7 @@ lean_object* x_60; lean_object* x_61; lean_object* x_62; x_60 = lean_ctor_get(x_59, 1); lean_inc(x_60); lean_dec(x_59); -x_61 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__38; +x_61 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__38; x_62 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_53, x_61, x_60); if (lean_obj_tag(x_62) == 0) { @@ -10458,11 +10455,11 @@ lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean x_63 = lean_ctor_get(x_62, 1); lean_inc(x_63); lean_dec(x_62); -x_64 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__39; +x_64 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__39; x_65 = l___regBuiltin_Lean_Parser_ppGroup_docString__1___closed__2; -x_66 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__41; -x_67 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__42; -x_68 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__43; +x_66 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__41; +x_67 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__42; +x_68 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__43; x_69 = l_Lean_Parser_registerAlias(x_64, x_65, x_66, x_67, x_68, x_63); if (lean_obj_tag(x_69) == 0) { @@ -10470,7 +10467,7 @@ lean_object* x_70; lean_object* x_71; lean_object* x_72; x_70 = lean_ctor_get(x_69, 1); lean_inc(x_70); lean_dec(x_69); -x_71 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__45; +x_71 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__45; x_72 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_64, x_71, x_70); if (lean_obj_tag(x_72) == 0) { @@ -10478,7 +10475,7 @@ lean_object* x_73; lean_object* x_74; lean_object* x_75; x_73 = lean_ctor_get(x_72, 1); lean_inc(x_73); lean_dec(x_72); -x_74 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__47; +x_74 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__47; x_75 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_64, x_74, x_73); if (lean_obj_tag(x_75) == 0) { @@ -10486,10 +10483,10 @@ lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean x_76 = lean_ctor_get(x_75, 1); lean_inc(x_76); lean_dec(x_75); -x_77 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__48; +x_77 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__48; x_78 = l___regBuiltin_Lean_Parser_ppRealGroup_docString__1___closed__2; -x_79 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__50; -x_80 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__51; +x_79 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__50; +x_80 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__51; x_81 = l_Lean_Parser_registerAlias(x_77, x_78, x_79, x_80, x_68, x_76); if (lean_obj_tag(x_81) == 0) { @@ -10497,7 +10494,7 @@ lean_object* x_82; lean_object* x_83; lean_object* x_84; x_82 = lean_ctor_get(x_81, 1); lean_inc(x_82); lean_dec(x_81); -x_83 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__53; +x_83 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__53; x_84 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_77, x_83, x_82); if (lean_obj_tag(x_84) == 0) { @@ -10505,7 +10502,7 @@ lean_object* x_85; lean_object* x_86; lean_object* x_87; x_85 = lean_ctor_get(x_84, 1); lean_inc(x_85); lean_dec(x_84); -x_86 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__55; +x_86 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__55; x_87 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_77, x_86, x_85); if (lean_obj_tag(x_87) == 0) { @@ -10513,10 +10510,10 @@ lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean x_88 = lean_ctor_get(x_87, 1); lean_inc(x_88); lean_dec(x_87); -x_89 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__56; +x_89 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__56; x_90 = l___regBuiltin_Lean_Parser_ppRealFill_docString__1___closed__2; -x_91 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__58; -x_92 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__59; +x_91 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__58; +x_92 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__59; x_93 = l_Lean_Parser_registerAlias(x_89, x_90, x_91, x_92, x_68, x_88); if (lean_obj_tag(x_93) == 0) { @@ -10524,7 +10521,7 @@ lean_object* x_94; lean_object* x_95; lean_object* x_96; x_94 = lean_ctor_get(x_93, 1); lean_inc(x_94); lean_dec(x_93); -x_95 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__61; +x_95 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__61; x_96 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_89, x_95, x_94); if (lean_obj_tag(x_96) == 0) { @@ -10532,7 +10529,7 @@ lean_object* x_97; lean_object* x_98; lean_object* x_99; x_97 = lean_ctor_get(x_96, 1); lean_inc(x_97); lean_dec(x_96); -x_98 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__63; +x_98 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__63; x_99 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_89, x_98, x_97); if (lean_obj_tag(x_99) == 0) { @@ -10540,10 +10537,10 @@ lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; x_100 = lean_ctor_get(x_99, 1); lean_inc(x_100); lean_dec(x_99); -x_101 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__64; +x_101 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__64; x_102 = l___regBuiltin_Lean_Parser_ppIndent_docString__1___closed__2; -x_103 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__66; -x_104 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__67; +x_103 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__66; +x_104 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__67; x_105 = l_Lean_Parser_registerAlias(x_101, x_102, x_103, x_104, x_68, x_100); if (lean_obj_tag(x_105) == 0) { @@ -10551,7 +10548,7 @@ lean_object* x_106; lean_object* x_107; lean_object* x_108; x_106 = lean_ctor_get(x_105, 1); lean_inc(x_106); lean_dec(x_105); -x_107 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__69; +x_107 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__69; x_108 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_101, x_107, x_106); if (lean_obj_tag(x_108) == 0) { @@ -10559,7 +10556,7 @@ lean_object* x_109; lean_object* x_110; lean_object* x_111; x_109 = lean_ctor_get(x_108, 1); lean_inc(x_109); lean_dec(x_108); -x_110 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__71; +x_110 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__71; x_111 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_101, x_110, x_109); if (lean_obj_tag(x_111) == 0) { @@ -10567,10 +10564,10 @@ lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; x_112 = lean_ctor_get(x_111, 1); lean_inc(x_112); lean_dec(x_111); -x_113 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__72; +x_113 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__72; x_114 = l___regBuiltin_Lean_Parser_ppDedent_docString__1___closed__2; -x_115 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__74; -x_116 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__75; +x_115 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__74; +x_116 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__75; x_117 = l_Lean_Parser_registerAlias(x_113, x_114, x_115, x_116, x_68, x_112); if (lean_obj_tag(x_117) == 0) { @@ -10578,7 +10575,7 @@ lean_object* x_118; lean_object* x_119; lean_object* x_120; x_118 = lean_ctor_get(x_117, 1); lean_inc(x_118); lean_dec(x_117); -x_119 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__77; +x_119 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__77; x_120 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_113, x_119, x_118); if (lean_obj_tag(x_120) == 0) { @@ -10586,7 +10583,7 @@ lean_object* x_121; lean_object* x_122; lean_object* x_123; x_121 = lean_ctor_get(x_120, 1); lean_inc(x_121); lean_dec(x_120); -x_122 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__79; +x_122 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__79; x_123 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_113, x_122, x_121); if (lean_obj_tag(x_123) == 0) { @@ -10594,10 +10591,10 @@ lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; x_124 = lean_ctor_get(x_123, 1); lean_inc(x_124); lean_dec(x_123); -x_125 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__80; +x_125 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__80; x_126 = l___regBuiltin_Lean_Parser_ppDedentIfGrouped_docString__1___closed__2; -x_127 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__82; -x_128 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__83; +x_127 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__82; +x_128 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__83; x_129 = l_Lean_Parser_registerAlias(x_125, x_126, x_127, x_128, x_68, x_124); if (lean_obj_tag(x_129) == 0) { @@ -10605,7 +10602,7 @@ lean_object* x_130; lean_object* x_131; lean_object* x_132; x_130 = lean_ctor_get(x_129, 1); lean_inc(x_130); lean_dec(x_129); -x_131 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__85; +x_131 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__85; x_132 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_125, x_131, x_130); if (lean_obj_tag(x_132) == 0) { @@ -10613,7 +10610,7 @@ lean_object* x_133; lean_object* x_134; lean_object* x_135; x_133 = lean_ctor_get(x_132, 1); lean_inc(x_133); lean_dec(x_132); -x_134 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__87; +x_134 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__87; x_135 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_125, x_134, x_133); if (lean_obj_tag(x_135) == 0) { @@ -10621,9 +10618,9 @@ lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; x_136 = lean_ctor_get(x_135, 1); lean_inc(x_136); lean_dec(x_135); -x_137 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__88; +x_137 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__88; x_138 = l___regBuiltin_Lean_Parser_ppAllowUngrouped_docString__1___closed__2; -x_139 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__89; +x_139 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__89; x_140 = l_Lean_Parser_registerAlias(x_137, x_138, x_31, x_139, x_33, x_136); if (lean_obj_tag(x_140) == 0) { @@ -10631,7 +10628,7 @@ lean_object* x_141; lean_object* x_142; lean_object* x_143; x_141 = lean_ctor_get(x_140, 1); lean_inc(x_141); lean_dec(x_140); -x_142 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__91; +x_142 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__91; x_143 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_137, x_142, x_141); if (lean_obj_tag(x_143) == 0) { @@ -10639,7 +10636,7 @@ lean_object* x_144; lean_object* x_145; lean_object* x_146; x_144 = lean_ctor_get(x_143, 1); lean_inc(x_144); lean_dec(x_143); -x_145 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__93; +x_145 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__93; x_146 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_137, x_145, x_144); if (lean_obj_tag(x_146) == 0) { @@ -10647,9 +10644,9 @@ lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; x_147 = lean_ctor_get(x_146, 1); lean_inc(x_147); lean_dec(x_146); -x_148 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__94; +x_148 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__94; x_149 = l___regBuiltin_Lean_Parser_ppHardLineUnlessUngrouped_docString__1___closed__2; -x_150 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__95; +x_150 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__95; x_151 = l_Lean_Parser_registerAlias(x_148, x_149, x_31, x_150, x_33, x_147); if (lean_obj_tag(x_151) == 0) { @@ -10657,7 +10654,7 @@ lean_object* x_152; lean_object* x_153; lean_object* x_154; x_152 = lean_ctor_get(x_151, 1); lean_inc(x_152); lean_dec(x_151); -x_153 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__97; +x_153 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__97; x_154 = l_Lean_Parser_registerAliasCore___rarg(x_9, x_148, x_153, x_152); if (lean_obj_tag(x_154) == 0) { @@ -10665,7 +10662,7 @@ lean_object* x_155; lean_object* x_156; lean_object* x_157; x_155 = lean_ctor_get(x_154, 1); lean_inc(x_155); lean_dec(x_154); -x_156 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__99; +x_156 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__99; x_157 = l_Lean_Parser_registerAliasCore___rarg(x_13, x_148, x_156, x_155); return x_157; } @@ -12424,205 +12421,205 @@ l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegi lean_mark_persistent(l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__74); l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__75 = _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__75(); lean_mark_persistent(l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29______________1___lambda__1___closed__75); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__1(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__1); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__2(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__2); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__3 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__3(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__3); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__4 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__4(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__4); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__5 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__5(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__5); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__6 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__6(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__6); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__7 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__7(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__7); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__8 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__8(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__8); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__9 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__9(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__9); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__10 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__10(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__10); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__11 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__11(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__11); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__12 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__12(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__12); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__13 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__13(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__13); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__14 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__14(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__14); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__15 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__15(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__15); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__16 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__16(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__16); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__17 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__17(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__17); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__18 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__18(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__18); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__19 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__19(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__19); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__20 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__20(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__20); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__21 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__21(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__21); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__22 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__22(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__22); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__23 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__23(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__23); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__24 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__24(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__24); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__25 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__25(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__25); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__26 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__26(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__26); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__27 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__27(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__27); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__28 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__28(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__28); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__29 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__29(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__29); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__30 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__30(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__30); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__31 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__31(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__31); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__32 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__32(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__32); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__33 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__33(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__33); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__34 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__34(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__34); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__35 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__35(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__35); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__36 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__36(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__36); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__37 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__37(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__37); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__38 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__38(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__38); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__39 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__39(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__39); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__40 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__40(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__40); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__41 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__41(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__41); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__42 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__42(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__42); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__43 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__43(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__43); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__44 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__44(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__44); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__45 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__45(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__45); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__46 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__46(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__46); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__47 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__47(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__47); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__48 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__48(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__48); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__49 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__49(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__49); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__50 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__50(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__50); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__51 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__51(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__51); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__52 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__52(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__52); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__53 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__53(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__53); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__54 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__54(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__54); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__55 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__55(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__55); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__56 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__56(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__56); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__57 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__57(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__57); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__58 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__58(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__58); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__59 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__59(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__59); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__60 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__60(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__60); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__61 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__61(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__61); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__62 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__62(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__62); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__63 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__63(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__63); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__64 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__64(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__64); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__65 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__65(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__65); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__66 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__66(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__66); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__67 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__67(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__67); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__68 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__68(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__68); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__69 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__69(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__69); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__70 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__70(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__70); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__71 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__71(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__71); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__72 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__72(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__72); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__73 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__73(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__73); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__74 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__74(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__74); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__75 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__75(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__75); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__76 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__76(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__76); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__77 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__77(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__77); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__78 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__78(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__78); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__79 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__79(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__79); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__80 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__80(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__80); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__81 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__81(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__81); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__82 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__82(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__82); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__83 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__83(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__83); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__84 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__84(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__84); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__85 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__85(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__85); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__86 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__86(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__86); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__87 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__87(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__87); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__88 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__88(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__88); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__89 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__89(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__89); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__90 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__90(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__90); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__91 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__91(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__91); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__92 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__92(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__92); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__93 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__93(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__93); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__94 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__94(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__94); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__95 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__95(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__95); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__96 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__96(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__96); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__97 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__97(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__97); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__98 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__98(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__98); -l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__99 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__99(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789____closed__99); -if (builtin) {res = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1789_(lean_io_mk_world()); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__1(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__1); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__2(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__2); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__3 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__3(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__3); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__4 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__4(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__4); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__5 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__5(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__5); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__6 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__6(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__6); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__7 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__7(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__7); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__8 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__8(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__8); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__9 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__9(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__9); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__10 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__10(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__10); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__11 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__11(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__11); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__12 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__12(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__12); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__13 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__13(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__13); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__14 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__14(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__14); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__15 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__15(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__15); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__16 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__16(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__16); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__17 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__17(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__17); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__18 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__18(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__18); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__19 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__19(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__19); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__20 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__20(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__20); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__21 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__21(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__21); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__22 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__22(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__22); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__23 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__23(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__23); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__24 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__24(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__24); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__25 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__25(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__25); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__26 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__26(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__26); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__27 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__27(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__27); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__28 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__28(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__28); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__29 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__29(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__29); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__30 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__30(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__30); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__31 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__31(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__31); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__32 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__32(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__32); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__33 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__33(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__33); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__34 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__34(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__34); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__35 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__35(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__35); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__36 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__36(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__36); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__37 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__37(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__37); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__38 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__38(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__38); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__39 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__39(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__39); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__40 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__40(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__40); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__41 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__41(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__41); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__42 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__42(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__42); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__43 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__43(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__43); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__44 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__44(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__44); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__45 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__45(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__45); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__46 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__46(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__46); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__47 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__47(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__47); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__48 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__48(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__48); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__49 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__49(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__49); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__50 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__50(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__50); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__51 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__51(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__51); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__52 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__52(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__52); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__53 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__53(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__53); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__54 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__54(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__54); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__55 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__55(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__55); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__56 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__56(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__56); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__57 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__57(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__57); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__58 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__58(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__58); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__59 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__59(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__59); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__60 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__60(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__60); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__61 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__61(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__61); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__62 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__62(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__62); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__63 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__63(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__63); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__64 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__64(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__64); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__65 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__65(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__65); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__66 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__66(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__66); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__67 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__67(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__67); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__68 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__68(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__68); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__69 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__69(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__69); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__70 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__70(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__70); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__71 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__71(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__71); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__72 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__72(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__72); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__73 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__73(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__73); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__74 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__74(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__74); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__75 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__75(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__75); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__76 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__76(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__76); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__77 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__77(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__77); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__78 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__78(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__78); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__79 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__79(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__79); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__80 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__80(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__80); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__81 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__81(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__81); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__82 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__82(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__82); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__83 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__83(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__83); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__84 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__84(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__84); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__85 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__85(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__85); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__86 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__86(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__86); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__87 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__87(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__87); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__88 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__88(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__88); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__89 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__89(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__89); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__90 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__90(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__90); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__91 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__91(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__91); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__92 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__92(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__92); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__93 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__93(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__93); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__94 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__94(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__94); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__95 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__95(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__95); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__96 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__96(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__96); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__97 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__97(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__97); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__98 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__98(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__98); +l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__99 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__99(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770____closed__99); +if (builtin) {res = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1770_(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/PrettyPrinter/Delaborator/Builtins.c b/stage0/stdlib/Lean/PrettyPrinter/Delaborator/Builtins.c index 96bfca56a8db..8338afc9eff5 100644 --- a/stage0/stdlib/Lean/PrettyPrinter/Delaborator/Builtins.c +++ b/stage0/stdlib/Lean/PrettyPrinter/Delaborator/Builtins.c @@ -30,6 +30,7 @@ static lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__3_ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParams___spec__2(lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_unresolveNameGlobal___at_Lean_PrettyPrinter_Delaborator_delabConst___spec__1___lambda__1___closed__1; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabCond__1___closed__1; +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__2; lean_object* lean_string_utf8_extract(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_withMDataOptions___spec__8___rarg(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_Lean_PrettyPrinter_Delaborator_withMDataOptions___spec__11(lean_object*); @@ -113,6 +114,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBod static lean_object* l_Lean_PrettyPrinter_Delaborator_delabDoElems___closed__5; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_PrettyPrinter_Delaborator_delabLam___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_pp_fullNames; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___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_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___lambda__15___closed__2; LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_delabProj___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_PrettyPrinter_Delaborator_delabLam___lambda__3___closed__2; @@ -124,7 +126,9 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_instInhabitedParamKind static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppMatch___lambda__6___closed__3; static lean_object* l_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___lambda__8___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___spec__13(lean_object*, lean_object*, size_t, size_t, lean_object*); +lean_object* l_Lean_Expr_name_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore_tryAppUnexpanders(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__2; lean_object* lean_whnf(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__3___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabDIte___lambda__1___closed__9; @@ -155,7 +159,6 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_declSigWi static lean_object* l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__8; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabConst___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_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___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_PrettyPrinter_Delaborator_reifyName___closed__1; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabFVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_unresolveNameGlobal___at_Lean_PrettyPrinter_Delaborator_delabConst___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_PrettyPrinter_Delaborator_delabAppImplicitCore___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -235,7 +238,6 @@ LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_delabProj__ static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabMData__1___closed__3; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBody_x27___at_Lean_PrettyPrinter_Delaborator_delabDIte_delabBranch___spec__2___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_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withAppFn___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDelayedAssignedMVar___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabApp___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppExplicitCore___closed__4; @@ -246,6 +248,7 @@ uint8_t l_Array_contains___at_Lean_findField_x3f___spec__1(lean_object*, lean_ob static lean_object* l_Lean_PrettyPrinter_Delaborator_delabLam___lambda__1___closed__2; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabLetE__1___closed__5; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore_mkArg___closed__1; +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__2; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDivRatCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_withMDatasOptions(lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); @@ -278,6 +281,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBoundedApp LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__21(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabLetE___closed__1; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabLetFun(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabConst___closed__13; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabLit__1___closed__3; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabConst___closed__9; @@ -424,7 +428,6 @@ static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabLam__1___ lean_object* l_Lean_getPPUniverses___boxed(lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabMData__1___closed__2; uint8_t l_Lean_Name_isPrefixOf(lean_object*, lean_object*); -static lean_object* l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___lambda__18(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_PrettyPrinter_Delaborator_unexpandStructureInstance___spec__1___closed__4; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore_tryAppUnexpanders_go___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -546,7 +549,6 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDoElems___lambda_ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_getConstInfo___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__2___closed__4; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabBVar__1___closed__5; -lean_object* l_Lean_Name_mkStr7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__8; lean_object* l_Lean_Meta_withLocalDecl___at_Lean_PrettyPrinter_Delaborator_withBindingBodyUnusedName___spec__3___rarg(lean_object*, uint8_t, 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_PrettyPrinter_Delaborator_delabLam___lambda__3___closed__3; @@ -665,7 +667,6 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabCond(lean_object* static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppMatch___lambda__6___closed__6; LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_withMDataOptions___spec__3(lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_maybeAddBlockImplicit___closed__3; -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__8; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabHDiv__1___closed__4; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDoElems___lambda__9(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_PrettyPrinter_Delaborator_delabSort___closed__7; @@ -756,7 +757,6 @@ uint8_t l_Lean_Expr_hasLooseBVars(lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___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_EXPORT lean_object* l___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_evalSyntaxConstantUnsafe___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabForall___lambda__2___closed__3; -lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabOfNat__1(lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppExplicitCore___lambda__8___closed__2; lean_object* l_Lean_Syntax_node3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -776,6 +776,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabMVarAux___lambda_ static lean_object* l_Std_Range_forIn_loop___at_Lean_PrettyPrinter_Delaborator_getParamKinds___spec__1___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__22(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_PrettyPrinter_Delaborator_annotateTermInfo___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDIte___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_descend___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_skippingBinders_loop_visitLambda___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -813,7 +814,6 @@ static lean_object* l_Lean_PrettyPrinter_Delaborator_delabSort___closed__4; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_declSigWithId_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_BinderInfo_isInstImplicit(uint8_t); -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__7; LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabLetFun__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabDIte___lambda__1___closed__2; @@ -844,6 +844,7 @@ static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabCond__1__ static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__5; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabPSigma__1___closed__3; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__2; +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__2; static lean_object* l_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___lambda__8___closed__3; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabPSigma__1___closed__2; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabForall___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*); @@ -902,6 +903,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delabora uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabLam__1(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabLam___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withMDataExpr___at_Lean_PrettyPrinter_Delaborator_withMDataOptions___spec__2___rarg___closed__3; LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_withMDataOptions___spec__10___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_PrettyPrinter_Delaborator_delabAppMatch_withDummyBinders___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*, lean_object*, lean_object*); @@ -918,7 +920,6 @@ static lean_object* l_Lean_PrettyPrinter_Delaborator_delabLam___lambda__1___clos extern lean_object* l_Lean_diagnostics; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDoElems(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isIdent(lean_object*); -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__12; lean_object* l_Lean_SubExpr_Pos_pushNaryArg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___lambda__3___closed__6; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; @@ -981,7 +982,6 @@ static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore_mkName LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_descend___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_skippingBinders_loop_visitLambda___spec__3(lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDo__1___closed__2; lean_object* l_Lean_MessageData_ofExpr(lean_object*); -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__3; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__3; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabMVarAux___closed__1; lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withType___at_Lean_PrettyPrinter_Delaborator_delab___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1018,12 +1018,10 @@ static lean_object* l___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_ lean_object* l_Lean_LocalDecl_userName(lean_object*); lean_object* l_Lean_getPPMVarsWithType___boxed(lean_object*); lean_object* l_Array_extract___rarg(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_object* l_Lean_Syntax_node4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabMProdMk__1(lean_object*); uint8_t l_Lean_Expr_isAutoParam(lean_object*); lean_object* l_Lean_getPPMVarsAnonymous___boxed(lean_object*); -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__2; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_declSigWithId_formatter__1___closed__2; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___lambda__12___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__2___closed__1; @@ -1040,7 +1038,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4(lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabProj__1___closed__4; static lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBody___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_skippingBinders_loop_visitLambda___spec__1___rarg___closed__1; -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__5; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParams___closed__6; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabHDiv(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1097,6 +1094,7 @@ lean_object* l_Lean_Name_appendCore(lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore_mkNamedArg___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabSigmaCore___lambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppExplicitCore___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*); +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__2; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabLam___lambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabPProdMk__1___closed__3; @@ -1108,6 +1106,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBod LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_PrettyPrinter_Delaborator_needsExplicit___spec__2(lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabSigmaCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabDo___closed__1; +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__5; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___at_Lean_PrettyPrinter_Delaborator_delabLetFun___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Delaborator_returnsPi___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1119,6 +1118,7 @@ static lean_object* l_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_del LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBody_x27___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_shouldGroupWithNext___spec__2___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*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabSort___closed__13; LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_withMDataOptions___spec__12___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__2; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_needsExplicit___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__9; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_declSigWithId_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1132,7 +1132,6 @@ uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_x27___s static lean_object* l_Lean_PrettyPrinter_Delaborator_delabCond___closed__1; lean_object* l_Lean_getPPPiBinderTypes___boxed(lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabLetFun___lambda__2___closed__4; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___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_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_coeDelaborator___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabSort___closed__12; @@ -1157,7 +1156,6 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDoElems_prependAn lean_object* l_Lean_PrettyPrinter_Delaborator_failure___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDIte_delabBranch___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_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_withoutParentProjections___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_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___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_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_PrettyPrinter_Delaborator_unexpandStructureInstance___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*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_delabProj___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_withCache(lean_object*, lean_object*); @@ -1197,10 +1195,9 @@ LEAN_EXPORT lean_object* l___private_Lean_PrettyPrinter_Delaborator_Builtins_0__ static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabAppMatch__1___closed__3; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_PrettyPrinter_Delaborator_needsExplicit___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabForall___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*); -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__11; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBody_x27___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_skippingBinders_loop_visitLambda___spec__2(lean_object*, lean_object*); -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__4; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore_mkArg___closed__2; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppExplicitCore___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabProj___closed__1; @@ -1318,7 +1315,6 @@ extern lean_object* l_Lean_Parser_maxPrec; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___spec__5(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBody_x27___at_Lean_PrettyPrinter_Delaborator_delabAppMatch_usingNames___spec__2___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*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabDivRatCore___closed__1; -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_stripParentProjections___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabDoElems___lambda__1___closed__2; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabLetE___closed__4; @@ -1327,7 +1323,6 @@ LEAN_EXPORT lean_object* l_Lean_unresolveNameGlobal_unresolveNameCore___at_Lean_ lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); lean_object* l_Array_ofSubarray___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___lambda__13(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_PrettyPrinter_Delaborator_reifyName___closed__6; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabSigmaCore___lambda__1___closed__1; uint8_t l_Lean_LocalDecl_binderInfo(lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabOfScientific___closed__3; @@ -1337,6 +1332,7 @@ static lean_object* l_Lean_PrettyPrinter_Delaborator_useAppExplicit___lambda__2_ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBody_x27___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_skippingBinders_loop_visitLambda___spec__8___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_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_delabMData___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_PrettyPrinter_Delaborator_delabNeg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__2; lean_object* lean_erase_macro_scopes(lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabOfScientific___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -1345,6 +1341,7 @@ lean_object* l_Array_back___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_delabMData___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___closed__2; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabChar__1___closed__4; +static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_delabMData___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_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParams___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBody_x27___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_skippingBinders_loop_visitLambda___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1358,6 +1355,7 @@ size_t lean_usize_sub(size_t, size_t); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabLam__1___closed__1; lean_object* lean_array_mk(lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabForall__1___closed__5; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___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_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___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_PrettyPrinter_Delaborator_delabAppMatch___lambda__3___closed__4; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabNegIntCore___closed__7; @@ -1379,7 +1377,6 @@ size_t lean_usize_add(size_t, size_t); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppMatch___closed__4; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_declSigWithId_parenthesizer__1___closed__2; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppCore___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_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabPProdMk__1___closed__4; LEAN_EXPORT uint8_t l_Lean_PrettyPrinter_Delaborator_delabAppImplicitCore___lambda__3(lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabApp___lambda__2(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1419,7 +1416,6 @@ extern lean_object* l_Lean_instInhabitedSyntax; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_useAppExplicit___closed__1; LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_withMDataOptions___spec__10(lean_object*); -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_delabBinders___closed__1; lean_object* l_Lean_SubExpr_Pos_pushNaryFn(lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Delaborator_addFieldInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1467,7 +1463,6 @@ LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_PrettyPrinter_Delabo static lean_object* l_Lean_PrettyPrinter_Delaborator_delabSort___closed__1; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_declSigWithId_parenthesizer__1___closed__4; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabForall___lambda__2___closed__1; -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__9; lean_object* l_Lean_PrettyPrinter_Delaborator_withBindingBodyUnusedName___rarg(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_PrettyPrinter_Delaborator_delabAppMatch___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1501,7 +1496,6 @@ uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_404_( LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_PrettyPrinter_Delaborator_getParamKinds___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNeg__1___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDIte__1(lean_object*); -static lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___closed__10; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabConst___spec__6(uint8_t, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabConst___spec__7(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_declSigWithId_formatter__1(lean_object*); @@ -1594,6 +1588,7 @@ static lean_object* l___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_ LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_withMDataOptions___spec__7___rarg(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_PrettyPrinter_Delaborator_delabConstWithSignature_delabParams___spec__1(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabAppMatch___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_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__2; lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingImp___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__6; @@ -1619,7 +1614,6 @@ static lean_object* l_Lean_PrettyPrinter_Delaborator_appFieldNotationCandidate_x static lean_object* l_Lean_PrettyPrinter_Delaborator_delabConst___closed__12; lean_object* l_Lean_Syntax_mkNumLit(lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabLam___lambda__1___closed__8; -lean_object* l_Lean_Name_mkStr8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_PrettyPrinter_Delaborator_delabConst___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_PrettyPrinter_Delaborator_SubExpr_withBindingBody___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_shouldGroupWithNext___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_throwError___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -24671,7 +24665,7 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___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; @@ -24728,7 +24722,7 @@ return x_20; } } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -24738,15 +24732,15 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2() { +static lean_object* _init_l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___lambda__1), 8, 0); +x_1 = lean_alloc_closure((void*)(l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___lambda__1), 8, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, 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_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, 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; @@ -24776,8 +24770,8 @@ x_24 = lean_ctor_get(x_1, 6); x_25 = lean_array_get_size(x_24); x_26 = lean_nat_dec_lt(x_6, x_25); lean_dec(x_25); -x_27 = l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1; -x_28 = l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2; +x_27 = l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1; +x_28 = l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2; x_29 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_SubExpr_withAppFnArgs___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__14), 9, 2); lean_closure_set(x_29, 0, x_27); lean_closure_set(x_29, 1, x_28); @@ -26640,7 +26634,7 @@ lean_dec(x_16); x_18 = lean_array_get_size(x_17); x_19 = lean_mk_empty_array_with_capacity(x_18); x_20 = lean_unsigned_to_nat(0u); -x_21 = l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18(x_1, x_14, x_17, x_17, x_18, x_20, lean_box(0), x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_21 = l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18(x_1, x_14, x_17, x_17, x_18, x_20, lean_box(0), x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_17); lean_dec(x_14); return x_21; @@ -28023,11 +28017,11 @@ lean_dec(x_4); return x_14; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__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, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__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, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { lean_object* x_16; -x_16 = l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18(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 = l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18(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_4); lean_dec(x_3); lean_dec(x_2); @@ -45078,3206 +45072,6 @@ x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } } -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Name", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("anonymous", 9, 9); -return x_1; -} -} -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("mkStr1", 6, 6); -return x_1; -} -} -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("str", 3, 3); -return x_1; -} -} -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("num", 3, 3); -return x_1; -} -} -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("mkStr2", 6, 6); -return x_1; -} -} -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("mkStr3", 6, 6); -return x_1; -} -} -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("mkStr4", 6, 6); -return x_1; -} -} -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__9() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("mkStr5", 6, 6); -return x_1; -} -} -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__10() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("mkStr6", 6, 6); -return x_1; -} -} -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__11() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("mkStr7", 6, 6); -return x_1; -} -} -static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__12() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("mkStr8", 6, 6); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName(lean_object* x_1, lean_object* x_2, 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: -{ -switch (lean_obj_tag(x_1)) { -case 4: -{ -lean_object* x_9; -x_9 = lean_ctor_get(x_1, 0); -lean_inc(x_9); -lean_dec(x_1); -if (lean_obj_tag(x_9) == 1) -{ -lean_object* x_10; -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -if (lean_obj_tag(x_10) == 1) -{ -lean_object* x_11; -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -if (lean_obj_tag(x_11) == 1) -{ -lean_object* x_12; -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -if (lean_obj_tag(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_9, 1); -lean_inc(x_13); -lean_dec(x_9); -x_14 = lean_ctor_get(x_10, 1); -lean_inc(x_14); -lean_dec(x_10); -x_15 = lean_ctor_get(x_11, 1); -lean_inc(x_15); -lean_dec(x_11); -x_16 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_17 = lean_string_dec_eq(x_15, x_16); -lean_dec(x_15); -if (x_17 == 0) -{ -lean_object* x_18; -lean_dec(x_14); -lean_dec(x_13); -x_18 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_18; -} -else -{ -lean_object* x_19; uint8_t x_20; -x_19 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_20 = lean_string_dec_eq(x_14, x_19); -lean_dec(x_14); -if (x_20 == 0) -{ -lean_object* x_21; -lean_dec(x_13); -x_21 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_21; -} -else -{ -lean_object* x_22; uint8_t x_23; -x_22 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__2; -x_23 = lean_string_dec_eq(x_13, x_22); -lean_dec(x_13); -if (x_23 == 0) -{ -lean_object* x_24; -x_24 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_24; -} -else -{ -lean_object* x_25; lean_object* x_26; -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_8); -return x_26; -} -} -} -} -else -{ -lean_object* x_27; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -x_27 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_27; -} -} -else -{ -lean_object* x_28; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -x_28 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_28; -} -} -else -{ -lean_object* x_29; -lean_dec(x_10); -lean_dec(x_9); -x_29 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_29; -} -} -else -{ -lean_object* x_30; -lean_dec(x_9); -x_30 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_30; -} -} -case 5: -{ -lean_object* x_31; -x_31 = lean_ctor_get(x_1, 0); -lean_inc(x_31); -switch (lean_obj_tag(x_31)) { -case 4: -{ -lean_object* x_32; -x_32 = lean_ctor_get(x_31, 0); -lean_inc(x_32); -lean_dec(x_31); -if (lean_obj_tag(x_32) == 1) -{ -lean_object* x_33; -x_33 = lean_ctor_get(x_32, 0); -lean_inc(x_33); -if (lean_obj_tag(x_33) == 1) -{ -lean_object* x_34; -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -if (lean_obj_tag(x_34) == 1) -{ -lean_object* x_35; -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -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; uint8_t x_41; -x_36 = lean_ctor_get(x_1, 1); -lean_inc(x_36); -lean_dec(x_1); -x_37 = lean_ctor_get(x_32, 1); -lean_inc(x_37); -lean_dec(x_32); -x_38 = lean_ctor_get(x_33, 1); -lean_inc(x_38); -lean_dec(x_33); -x_39 = lean_ctor_get(x_34, 1); -lean_inc(x_39); -lean_dec(x_34); -x_40 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_41 = lean_string_dec_eq(x_39, x_40); -lean_dec(x_39); -if (x_41 == 0) -{ -lean_object* x_42; -lean_dec(x_38); -lean_dec(x_37); -lean_dec(x_36); -x_42 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_42; -} -else -{ -lean_object* x_43; uint8_t x_44; -x_43 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_44 = lean_string_dec_eq(x_38, x_43); -lean_dec(x_38); -if (x_44 == 0) -{ -lean_object* x_45; -lean_dec(x_37); -lean_dec(x_36); -x_45 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_45; -} -else -{ -lean_object* x_46; uint8_t x_47; -x_46 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__3; -x_47 = lean_string_dec_eq(x_37, x_46); -lean_dec(x_37); -if (x_47 == 0) -{ -lean_object* x_48; -lean_dec(x_36); -x_48 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_48; -} -else -{ -if (lean_obj_tag(x_36) == 9) -{ -lean_object* x_49; -x_49 = lean_ctor_get(x_36, 0); -lean_inc(x_49); -lean_dec(x_36); -if (lean_obj_tag(x_49) == 0) -{ -lean_object* x_50; -lean_dec(x_49); -x_50 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_50; -} -else -{ -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_51 = lean_ctor_get(x_49, 0); -lean_inc(x_51); -lean_dec(x_49); -x_52 = lean_box(0); -x_53 = l_Lean_Name_str___override(x_52, x_51); -x_54 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_54, 0, x_53); -lean_ctor_set(x_54, 1, x_8); -return x_54; -} -} -else -{ -lean_object* x_55; -lean_dec(x_36); -x_55 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_55; -} -} -} -} -} -else -{ -lean_object* x_56; -lean_dec(x_35); -lean_dec(x_34); -lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_1); -x_56 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_56; -} -} -else -{ -lean_object* x_57; -lean_dec(x_34); -lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_1); -x_57 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_57; -} -} -else -{ -lean_object* x_58; -lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_1); -x_58 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_58; -} -} -else -{ -lean_object* x_59; -lean_dec(x_32); -lean_dec(x_1); -x_59 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_59; -} -} -case 5: -{ -lean_object* x_60; -x_60 = lean_ctor_get(x_31, 0); -lean_inc(x_60); -switch (lean_obj_tag(x_60)) { -case 4: -{ -lean_object* x_61; -x_61 = lean_ctor_get(x_60, 0); -lean_inc(x_61); -lean_dec(x_60); -if (lean_obj_tag(x_61) == 1) -{ -lean_object* x_62; -x_62 = lean_ctor_get(x_61, 0); -lean_inc(x_62); -if (lean_obj_tag(x_62) == 1) -{ -lean_object* x_63; -x_63 = lean_ctor_get(x_62, 0); -lean_inc(x_63); -if (lean_obj_tag(x_63) == 1) -{ -lean_object* x_64; -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; lean_object* x_68; lean_object* x_69; lean_object* x_70; uint8_t x_71; -x_65 = lean_ctor_get(x_1, 1); -lean_inc(x_65); -lean_dec(x_1); -x_66 = lean_ctor_get(x_31, 1); -lean_inc(x_66); -lean_dec(x_31); -x_67 = lean_ctor_get(x_61, 1); -lean_inc(x_67); -lean_dec(x_61); -x_68 = lean_ctor_get(x_62, 1); -lean_inc(x_68); -lean_dec(x_62); -x_69 = lean_ctor_get(x_63, 1); -lean_inc(x_69); -lean_dec(x_63); -x_70 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_71 = lean_string_dec_eq(x_69, x_70); -lean_dec(x_69); -if (x_71 == 0) -{ -lean_object* x_72; -lean_dec(x_68); -lean_dec(x_67); -lean_dec(x_66); -lean_dec(x_65); -x_72 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_72; -} -else -{ -lean_object* x_73; uint8_t x_74; -x_73 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_74 = lean_string_dec_eq(x_68, x_73); -lean_dec(x_68); -if (x_74 == 0) -{ -lean_object* x_75; -lean_dec(x_67); -lean_dec(x_66); -lean_dec(x_65); -x_75 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_75; -} -else -{ -lean_object* x_76; uint8_t x_77; -x_76 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__4; -x_77 = lean_string_dec_eq(x_67, x_76); -if (x_77 == 0) -{ -lean_object* x_78; uint8_t x_79; -x_78 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__5; -x_79 = lean_string_dec_eq(x_67, x_78); -if (x_79 == 0) -{ -lean_object* x_80; uint8_t x_81; -x_80 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__6; -x_81 = lean_string_dec_eq(x_67, x_80); -lean_dec(x_67); -if (x_81 == 0) -{ -lean_object* x_82; -lean_dec(x_66); -lean_dec(x_65); -x_82 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_82; -} -else -{ -if (lean_obj_tag(x_66) == 9) -{ -lean_object* x_83; -x_83 = lean_ctor_get(x_66, 0); -lean_inc(x_83); -lean_dec(x_66); -if (lean_obj_tag(x_83) == 0) -{ -lean_object* x_84; -lean_dec(x_83); -lean_dec(x_65); -x_84 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_84; -} -else -{ -if (lean_obj_tag(x_65) == 9) -{ -lean_object* x_85; -x_85 = lean_ctor_get(x_65, 0); -lean_inc(x_85); -lean_dec(x_65); -if (lean_obj_tag(x_85) == 0) -{ -lean_object* x_86; -lean_dec(x_85); -lean_dec(x_83); -x_86 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_86; -} -else -{ -lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; -x_87 = lean_ctor_get(x_83, 0); -lean_inc(x_87); -lean_dec(x_83); -x_88 = lean_ctor_get(x_85, 0); -lean_inc(x_88); -lean_dec(x_85); -x_89 = l_Lean_Name_mkStr2(x_87, 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_8); -return x_90; -} -} -else -{ -lean_object* x_91; -lean_dec(x_83); -lean_dec(x_65); -x_91 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_91; -} -} -} -else -{ -lean_object* x_92; -lean_dec(x_66); -lean_dec(x_65); -x_92 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_92; -} -} -} -else -{ -lean_dec(x_67); -if (lean_obj_tag(x_65) == 9) -{ -lean_object* x_93; -x_93 = lean_ctor_get(x_65, 0); -lean_inc(x_93); -lean_dec(x_65); -if (lean_obj_tag(x_93) == 0) -{ -lean_object* x_94; lean_object* x_95; -x_94 = lean_ctor_get(x_93, 0); -lean_inc(x_94); -lean_dec(x_93); -x_95 = l_Lean_PrettyPrinter_Delaborator_reifyName(x_66, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_95) == 0) -{ -uint8_t x_96; -x_96 = !lean_is_exclusive(x_95); -if (x_96 == 0) -{ -lean_object* x_97; lean_object* x_98; -x_97 = lean_ctor_get(x_95, 0); -x_98 = l_Lean_Name_num___override(x_97, x_94); -lean_ctor_set(x_95, 0, x_98); -return x_95; -} -else -{ -lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; -x_99 = lean_ctor_get(x_95, 0); -x_100 = lean_ctor_get(x_95, 1); -lean_inc(x_100); -lean_inc(x_99); -lean_dec(x_95); -x_101 = l_Lean_Name_num___override(x_99, x_94); -x_102 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_102, 0, x_101); -lean_ctor_set(x_102, 1, x_100); -return x_102; -} -} -else -{ -uint8_t x_103; -lean_dec(x_94); -x_103 = !lean_is_exclusive(x_95); -if (x_103 == 0) -{ -return x_95; -} -else -{ -lean_object* x_104; lean_object* x_105; lean_object* x_106; -x_104 = lean_ctor_get(x_95, 0); -x_105 = lean_ctor_get(x_95, 1); -lean_inc(x_105); -lean_inc(x_104); -lean_dec(x_95); -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_107; -lean_dec(x_93); -lean_dec(x_66); -x_107 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_107; -} -} -else -{ -lean_object* x_108; -lean_dec(x_66); -lean_dec(x_65); -x_108 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_108; -} -} -} -else -{ -lean_dec(x_67); -if (lean_obj_tag(x_65) == 9) -{ -lean_object* x_109; -x_109 = lean_ctor_get(x_65, 0); -lean_inc(x_109); -lean_dec(x_65); -if (lean_obj_tag(x_109) == 0) -{ -lean_object* x_110; -lean_dec(x_109); -lean_dec(x_66); -x_110 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_110; -} -else -{ -lean_object* x_111; lean_object* x_112; -x_111 = lean_ctor_get(x_109, 0); -lean_inc(x_111); -lean_dec(x_109); -x_112 = l_Lean_PrettyPrinter_Delaborator_reifyName(x_66, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_112) == 0) -{ -uint8_t x_113; -x_113 = !lean_is_exclusive(x_112); -if (x_113 == 0) -{ -lean_object* x_114; lean_object* x_115; -x_114 = lean_ctor_get(x_112, 0); -x_115 = l_Lean_Name_str___override(x_114, x_111); -lean_ctor_set(x_112, 0, x_115); -return x_112; -} -else -{ -lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; -x_116 = lean_ctor_get(x_112, 0); -x_117 = lean_ctor_get(x_112, 1); -lean_inc(x_117); -lean_inc(x_116); -lean_dec(x_112); -x_118 = l_Lean_Name_str___override(x_116, x_111); -x_119 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_119, 0, x_118); -lean_ctor_set(x_119, 1, x_117); -return x_119; -} -} -else -{ -uint8_t x_120; -lean_dec(x_111); -x_120 = !lean_is_exclusive(x_112); -if (x_120 == 0) -{ -return x_112; -} -else -{ -lean_object* x_121; lean_object* x_122; lean_object* x_123; -x_121 = lean_ctor_get(x_112, 0); -x_122 = lean_ctor_get(x_112, 1); -lean_inc(x_122); -lean_inc(x_121); -lean_dec(x_112); -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 -{ -lean_object* x_124; -lean_dec(x_66); -lean_dec(x_65); -x_124 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_124; -} -} -} -} -} -else -{ -lean_object* x_125; -lean_dec(x_64); -lean_dec(x_63); -lean_dec(x_62); -lean_dec(x_61); -lean_dec(x_31); -lean_dec(x_1); -x_125 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_125; -} -} -else -{ -lean_object* x_126; -lean_dec(x_63); -lean_dec(x_62); -lean_dec(x_61); -lean_dec(x_31); -lean_dec(x_1); -x_126 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_126; -} -} -else -{ -lean_object* x_127; -lean_dec(x_62); -lean_dec(x_61); -lean_dec(x_31); -lean_dec(x_1); -x_127 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_127; -} -} -else -{ -lean_object* x_128; -lean_dec(x_61); -lean_dec(x_31); -lean_dec(x_1); -x_128 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_128; -} -} -case 5: -{ -lean_object* x_129; -x_129 = lean_ctor_get(x_60, 0); -lean_inc(x_129); -switch (lean_obj_tag(x_129)) { -case 4: -{ -lean_object* x_130; -x_130 = lean_ctor_get(x_129, 0); -lean_inc(x_130); -lean_dec(x_129); -if (lean_obj_tag(x_130) == 1) -{ -lean_object* x_131; -x_131 = lean_ctor_get(x_130, 0); -lean_inc(x_131); -if (lean_obj_tag(x_131) == 1) -{ -lean_object* x_132; -x_132 = lean_ctor_get(x_131, 0); -lean_inc(x_132); -if (lean_obj_tag(x_132) == 1) -{ -lean_object* x_133; -x_133 = lean_ctor_get(x_132, 0); -lean_inc(x_133); -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; uint8_t x_141; -x_134 = lean_ctor_get(x_1, 1); -lean_inc(x_134); -lean_dec(x_1); -x_135 = lean_ctor_get(x_31, 1); -lean_inc(x_135); -lean_dec(x_31); -x_136 = lean_ctor_get(x_60, 1); -lean_inc(x_136); -lean_dec(x_60); -x_137 = lean_ctor_get(x_130, 1); -lean_inc(x_137); -lean_dec(x_130); -x_138 = lean_ctor_get(x_131, 1); -lean_inc(x_138); -lean_dec(x_131); -x_139 = lean_ctor_get(x_132, 1); -lean_inc(x_139); -lean_dec(x_132); -x_140 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_141 = lean_string_dec_eq(x_139, x_140); -lean_dec(x_139); -if (x_141 == 0) -{ -lean_object* x_142; -lean_dec(x_138); -lean_dec(x_137); -lean_dec(x_136); -lean_dec(x_135); -lean_dec(x_134); -x_142 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_142; -} -else -{ -lean_object* x_143; uint8_t x_144; -x_143 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_144 = lean_string_dec_eq(x_138, x_143); -lean_dec(x_138); -if (x_144 == 0) -{ -lean_object* x_145; -lean_dec(x_137); -lean_dec(x_136); -lean_dec(x_135); -lean_dec(x_134); -x_145 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_145; -} -else -{ -lean_object* x_146; uint8_t x_147; -x_146 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__7; -x_147 = lean_string_dec_eq(x_137, x_146); -lean_dec(x_137); -if (x_147 == 0) -{ -lean_object* x_148; -lean_dec(x_136); -lean_dec(x_135); -lean_dec(x_134); -x_148 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_148; -} -else -{ -if (lean_obj_tag(x_136) == 9) -{ -lean_object* x_149; -x_149 = lean_ctor_get(x_136, 0); -lean_inc(x_149); -lean_dec(x_136); -if (lean_obj_tag(x_149) == 0) -{ -lean_object* x_150; -lean_dec(x_149); -lean_dec(x_135); -lean_dec(x_134); -x_150 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_150; -} -else -{ -if (lean_obj_tag(x_135) == 9) -{ -lean_object* x_151; -x_151 = lean_ctor_get(x_135, 0); -lean_inc(x_151); -lean_dec(x_135); -if (lean_obj_tag(x_151) == 0) -{ -lean_object* x_152; -lean_dec(x_151); -lean_dec(x_149); -lean_dec(x_134); -x_152 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_152; -} -else -{ -if (lean_obj_tag(x_134) == 9) -{ -lean_object* x_153; -x_153 = lean_ctor_get(x_134, 0); -lean_inc(x_153); -lean_dec(x_134); -if (lean_obj_tag(x_153) == 0) -{ -lean_object* x_154; -lean_dec(x_153); -lean_dec(x_151); -lean_dec(x_149); -x_154 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_154; -} -else -{ -lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; -x_155 = lean_ctor_get(x_149, 0); -lean_inc(x_155); -lean_dec(x_149); -x_156 = lean_ctor_get(x_151, 0); -lean_inc(x_156); -lean_dec(x_151); -x_157 = lean_ctor_get(x_153, 0); -lean_inc(x_157); -lean_dec(x_153); -x_158 = l_Lean_Name_mkStr3(x_155, x_156, x_157); -x_159 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_159, 0, x_158); -lean_ctor_set(x_159, 1, x_8); -return x_159; -} -} -else -{ -lean_object* x_160; -lean_dec(x_151); -lean_dec(x_149); -lean_dec(x_134); -x_160 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_160; -} -} -} -else -{ -lean_object* x_161; -lean_dec(x_149); -lean_dec(x_135); -lean_dec(x_134); -x_161 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_161; -} -} -} -else -{ -lean_object* x_162; -lean_dec(x_136); -lean_dec(x_135); -lean_dec(x_134); -x_162 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_162; -} -} -} -} -} -else -{ -lean_object* x_163; -lean_dec(x_133); -lean_dec(x_132); -lean_dec(x_131); -lean_dec(x_130); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_163 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_163; -} -} -else -{ -lean_object* x_164; -lean_dec(x_132); -lean_dec(x_131); -lean_dec(x_130); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_164 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_164; -} -} -else -{ -lean_object* x_165; -lean_dec(x_131); -lean_dec(x_130); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_165 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_165; -} -} -else -{ -lean_object* x_166; -lean_dec(x_130); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_166 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_166; -} -} -case 5: -{ -lean_object* x_167; -x_167 = lean_ctor_get(x_129, 0); -lean_inc(x_167); -switch (lean_obj_tag(x_167)) { -case 4: -{ -lean_object* x_168; -x_168 = lean_ctor_get(x_167, 0); -lean_inc(x_168); -lean_dec(x_167); -if (lean_obj_tag(x_168) == 1) -{ -lean_object* x_169; -x_169 = lean_ctor_get(x_168, 0); -lean_inc(x_169); -if (lean_obj_tag(x_169) == 1) -{ -lean_object* x_170; -x_170 = lean_ctor_get(x_169, 0); -lean_inc(x_170); -if (lean_obj_tag(x_170) == 1) -{ -lean_object* x_171; -x_171 = lean_ctor_get(x_170, 0); -lean_inc(x_171); -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; uint8_t x_180; -x_172 = lean_ctor_get(x_1, 1); -lean_inc(x_172); -lean_dec(x_1); -x_173 = lean_ctor_get(x_31, 1); -lean_inc(x_173); -lean_dec(x_31); -x_174 = lean_ctor_get(x_60, 1); -lean_inc(x_174); -lean_dec(x_60); -x_175 = lean_ctor_get(x_129, 1); -lean_inc(x_175); -lean_dec(x_129); -x_176 = lean_ctor_get(x_168, 1); -lean_inc(x_176); -lean_dec(x_168); -x_177 = lean_ctor_get(x_169, 1); -lean_inc(x_177); -lean_dec(x_169); -x_178 = lean_ctor_get(x_170, 1); -lean_inc(x_178); -lean_dec(x_170); -x_179 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_180 = lean_string_dec_eq(x_178, x_179); -lean_dec(x_178); -if (x_180 == 0) -{ -lean_object* x_181; -lean_dec(x_177); -lean_dec(x_176); -lean_dec(x_175); -lean_dec(x_174); -lean_dec(x_173); -lean_dec(x_172); -x_181 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_181; -} -else -{ -lean_object* x_182; uint8_t x_183; -x_182 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_183 = lean_string_dec_eq(x_177, x_182); -lean_dec(x_177); -if (x_183 == 0) -{ -lean_object* x_184; -lean_dec(x_176); -lean_dec(x_175); -lean_dec(x_174); -lean_dec(x_173); -lean_dec(x_172); -x_184 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_184; -} -else -{ -lean_object* x_185; uint8_t x_186; -x_185 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__8; -x_186 = lean_string_dec_eq(x_176, x_185); -lean_dec(x_176); -if (x_186 == 0) -{ -lean_object* x_187; -lean_dec(x_175); -lean_dec(x_174); -lean_dec(x_173); -lean_dec(x_172); -x_187 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_187; -} -else -{ -if (lean_obj_tag(x_175) == 9) -{ -lean_object* x_188; -x_188 = lean_ctor_get(x_175, 0); -lean_inc(x_188); -lean_dec(x_175); -if (lean_obj_tag(x_188) == 0) -{ -lean_object* x_189; -lean_dec(x_188); -lean_dec(x_174); -lean_dec(x_173); -lean_dec(x_172); -x_189 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_189; -} -else -{ -if (lean_obj_tag(x_174) == 9) -{ -lean_object* x_190; -x_190 = lean_ctor_get(x_174, 0); -lean_inc(x_190); -lean_dec(x_174); -if (lean_obj_tag(x_190) == 0) -{ -lean_object* x_191; -lean_dec(x_190); -lean_dec(x_188); -lean_dec(x_173); -lean_dec(x_172); -x_191 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_191; -} -else -{ -if (lean_obj_tag(x_173) == 9) -{ -lean_object* x_192; -x_192 = lean_ctor_get(x_173, 0); -lean_inc(x_192); -lean_dec(x_173); -if (lean_obj_tag(x_192) == 0) -{ -lean_object* x_193; -lean_dec(x_192); -lean_dec(x_190); -lean_dec(x_188); -lean_dec(x_172); -x_193 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_193; -} -else -{ -if (lean_obj_tag(x_172) == 9) -{ -lean_object* x_194; -x_194 = lean_ctor_get(x_172, 0); -lean_inc(x_194); -lean_dec(x_172); -if (lean_obj_tag(x_194) == 0) -{ -lean_object* x_195; -lean_dec(x_194); -lean_dec(x_192); -lean_dec(x_190); -lean_dec(x_188); -x_195 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_195; -} -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; -x_196 = lean_ctor_get(x_188, 0); -lean_inc(x_196); -lean_dec(x_188); -x_197 = lean_ctor_get(x_190, 0); -lean_inc(x_197); -lean_dec(x_190); -x_198 = lean_ctor_get(x_192, 0); -lean_inc(x_198); -lean_dec(x_192); -x_199 = lean_ctor_get(x_194, 0); -lean_inc(x_199); -lean_dec(x_194); -x_200 = l_Lean_Name_mkStr4(x_196, x_197, x_198, x_199); -x_201 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_201, 0, x_200); -lean_ctor_set(x_201, 1, x_8); -return x_201; -} -} -else -{ -lean_object* x_202; -lean_dec(x_192); -lean_dec(x_190); -lean_dec(x_188); -lean_dec(x_172); -x_202 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_202; -} -} -} -else -{ -lean_object* x_203; -lean_dec(x_190); -lean_dec(x_188); -lean_dec(x_173); -lean_dec(x_172); -x_203 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_203; -} -} -} -else -{ -lean_object* x_204; -lean_dec(x_188); -lean_dec(x_174); -lean_dec(x_173); -lean_dec(x_172); -x_204 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_204; -} -} -} -else -{ -lean_object* x_205; -lean_dec(x_175); -lean_dec(x_174); -lean_dec(x_173); -lean_dec(x_172); -x_205 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_205; -} -} -} -} -} -else -{ -lean_object* x_206; -lean_dec(x_171); -lean_dec(x_170); -lean_dec(x_169); -lean_dec(x_168); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_206 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_206; -} -} -else -{ -lean_object* x_207; -lean_dec(x_170); -lean_dec(x_169); -lean_dec(x_168); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_207 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_207; -} -} -else -{ -lean_object* x_208; -lean_dec(x_169); -lean_dec(x_168); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_208 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_208; -} -} -else -{ -lean_object* x_209; -lean_dec(x_168); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_209 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_209; -} -} -case 5: -{ -lean_object* x_210; -x_210 = lean_ctor_get(x_167, 0); -lean_inc(x_210); -switch (lean_obj_tag(x_210)) { -case 4: -{ -lean_object* x_211; -x_211 = lean_ctor_get(x_210, 0); -lean_inc(x_211); -lean_dec(x_210); -if (lean_obj_tag(x_211) == 1) -{ -lean_object* x_212; -x_212 = lean_ctor_get(x_211, 0); -lean_inc(x_212); -if (lean_obj_tag(x_212) == 1) -{ -lean_object* x_213; -x_213 = lean_ctor_get(x_212, 0); -lean_inc(x_213); -if (lean_obj_tag(x_213) == 1) -{ -lean_object* x_214; -x_214 = lean_ctor_get(x_213, 0); -lean_inc(x_214); -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; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; uint8_t x_224; -x_215 = lean_ctor_get(x_1, 1); -lean_inc(x_215); -lean_dec(x_1); -x_216 = lean_ctor_get(x_31, 1); -lean_inc(x_216); -lean_dec(x_31); -x_217 = lean_ctor_get(x_60, 1); -lean_inc(x_217); -lean_dec(x_60); -x_218 = lean_ctor_get(x_129, 1); -lean_inc(x_218); -lean_dec(x_129); -x_219 = lean_ctor_get(x_167, 1); -lean_inc(x_219); -lean_dec(x_167); -x_220 = lean_ctor_get(x_211, 1); -lean_inc(x_220); -lean_dec(x_211); -x_221 = lean_ctor_get(x_212, 1); -lean_inc(x_221); -lean_dec(x_212); -x_222 = lean_ctor_get(x_213, 1); -lean_inc(x_222); -lean_dec(x_213); -x_223 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_224 = lean_string_dec_eq(x_222, x_223); -lean_dec(x_222); -if (x_224 == 0) -{ -lean_object* x_225; -lean_dec(x_221); -lean_dec(x_220); -lean_dec(x_219); -lean_dec(x_218); -lean_dec(x_217); -lean_dec(x_216); -lean_dec(x_215); -x_225 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_225; -} -else -{ -lean_object* x_226; uint8_t x_227; -x_226 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_227 = lean_string_dec_eq(x_221, x_226); -lean_dec(x_221); -if (x_227 == 0) -{ -lean_object* x_228; -lean_dec(x_220); -lean_dec(x_219); -lean_dec(x_218); -lean_dec(x_217); -lean_dec(x_216); -lean_dec(x_215); -x_228 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_228; -} -else -{ -lean_object* x_229; uint8_t x_230; -x_229 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__9; -x_230 = lean_string_dec_eq(x_220, x_229); -lean_dec(x_220); -if (x_230 == 0) -{ -lean_object* x_231; -lean_dec(x_219); -lean_dec(x_218); -lean_dec(x_217); -lean_dec(x_216); -lean_dec(x_215); -x_231 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_231; -} -else -{ -if (lean_obj_tag(x_219) == 9) -{ -lean_object* x_232; -x_232 = lean_ctor_get(x_219, 0); -lean_inc(x_232); -lean_dec(x_219); -if (lean_obj_tag(x_232) == 0) -{ -lean_object* x_233; -lean_dec(x_232); -lean_dec(x_218); -lean_dec(x_217); -lean_dec(x_216); -lean_dec(x_215); -x_233 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_233; -} -else -{ -if (lean_obj_tag(x_218) == 9) -{ -lean_object* x_234; -x_234 = lean_ctor_get(x_218, 0); -lean_inc(x_234); -lean_dec(x_218); -if (lean_obj_tag(x_234) == 0) -{ -lean_object* x_235; -lean_dec(x_234); -lean_dec(x_232); -lean_dec(x_217); -lean_dec(x_216); -lean_dec(x_215); -x_235 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_235; -} -else -{ -if (lean_obj_tag(x_217) == 9) -{ -lean_object* x_236; -x_236 = lean_ctor_get(x_217, 0); -lean_inc(x_236); -lean_dec(x_217); -if (lean_obj_tag(x_236) == 0) -{ -lean_object* x_237; -lean_dec(x_236); -lean_dec(x_234); -lean_dec(x_232); -lean_dec(x_216); -lean_dec(x_215); -x_237 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_237; -} -else -{ -if (lean_obj_tag(x_216) == 9) -{ -lean_object* x_238; -x_238 = lean_ctor_get(x_216, 0); -lean_inc(x_238); -lean_dec(x_216); -if (lean_obj_tag(x_238) == 0) -{ -lean_object* x_239; -lean_dec(x_238); -lean_dec(x_236); -lean_dec(x_234); -lean_dec(x_232); -lean_dec(x_215); -x_239 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_239; -} -else -{ -if (lean_obj_tag(x_215) == 9) -{ -lean_object* x_240; -x_240 = lean_ctor_get(x_215, 0); -lean_inc(x_240); -lean_dec(x_215); -if (lean_obj_tag(x_240) == 0) -{ -lean_object* x_241; -lean_dec(x_240); -lean_dec(x_238); -lean_dec(x_236); -lean_dec(x_234); -lean_dec(x_232); -x_241 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_241; -} -else -{ -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; -x_242 = lean_ctor_get(x_232, 0); -lean_inc(x_242); -lean_dec(x_232); -x_243 = lean_ctor_get(x_234, 0); -lean_inc(x_243); -lean_dec(x_234); -x_244 = lean_ctor_get(x_236, 0); -lean_inc(x_244); -lean_dec(x_236); -x_245 = lean_ctor_get(x_238, 0); -lean_inc(x_245); -lean_dec(x_238); -x_246 = lean_ctor_get(x_240, 0); -lean_inc(x_246); -lean_dec(x_240); -x_247 = l_Lean_Name_mkStr5(x_242, x_243, x_244, x_245, x_246); -x_248 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_248, 0, x_247); -lean_ctor_set(x_248, 1, x_8); -return x_248; -} -} -else -{ -lean_object* x_249; -lean_dec(x_238); -lean_dec(x_236); -lean_dec(x_234); -lean_dec(x_232); -lean_dec(x_215); -x_249 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_249; -} -} -} -else -{ -lean_object* x_250; -lean_dec(x_236); -lean_dec(x_234); -lean_dec(x_232); -lean_dec(x_216); -lean_dec(x_215); -x_250 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_250; -} -} -} -else -{ -lean_object* x_251; -lean_dec(x_234); -lean_dec(x_232); -lean_dec(x_217); -lean_dec(x_216); -lean_dec(x_215); -x_251 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_251; -} -} -} -else -{ -lean_object* x_252; -lean_dec(x_232); -lean_dec(x_218); -lean_dec(x_217); -lean_dec(x_216); -lean_dec(x_215); -x_252 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_252; -} -} -} -else -{ -lean_object* x_253; -lean_dec(x_219); -lean_dec(x_218); -lean_dec(x_217); -lean_dec(x_216); -lean_dec(x_215); -x_253 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_253; -} -} -} -} -} -else -{ -lean_object* x_254; -lean_dec(x_214); -lean_dec(x_213); -lean_dec(x_212); -lean_dec(x_211); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_254 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_254; -} -} -else -{ -lean_object* x_255; -lean_dec(x_213); -lean_dec(x_212); -lean_dec(x_211); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_255 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_255; -} -} -else -{ -lean_object* x_256; -lean_dec(x_212); -lean_dec(x_211); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_256 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_256; -} -} -else -{ -lean_object* x_257; -lean_dec(x_211); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_257 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_257; -} -} -case 5: -{ -lean_object* x_258; -x_258 = lean_ctor_get(x_210, 0); -lean_inc(x_258); -switch (lean_obj_tag(x_258)) { -case 4: -{ -lean_object* x_259; -x_259 = lean_ctor_get(x_258, 0); -lean_inc(x_259); -lean_dec(x_258); -if (lean_obj_tag(x_259) == 1) -{ -lean_object* x_260; -x_260 = lean_ctor_get(x_259, 0); -lean_inc(x_260); -if (lean_obj_tag(x_260) == 1) -{ -lean_object* x_261; -x_261 = lean_ctor_get(x_260, 0); -lean_inc(x_261); -if (lean_obj_tag(x_261) == 1) -{ -lean_object* x_262; -x_262 = lean_ctor_get(x_261, 0); -lean_inc(x_262); -if (lean_obj_tag(x_262) == 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; lean_object* x_270; lean_object* x_271; lean_object* x_272; uint8_t x_273; -x_263 = lean_ctor_get(x_1, 1); -lean_inc(x_263); -lean_dec(x_1); -x_264 = lean_ctor_get(x_31, 1); -lean_inc(x_264); -lean_dec(x_31); -x_265 = lean_ctor_get(x_60, 1); -lean_inc(x_265); -lean_dec(x_60); -x_266 = lean_ctor_get(x_129, 1); -lean_inc(x_266); -lean_dec(x_129); -x_267 = lean_ctor_get(x_167, 1); -lean_inc(x_267); -lean_dec(x_167); -x_268 = lean_ctor_get(x_210, 1); -lean_inc(x_268); -lean_dec(x_210); -x_269 = lean_ctor_get(x_259, 1); -lean_inc(x_269); -lean_dec(x_259); -x_270 = lean_ctor_get(x_260, 1); -lean_inc(x_270); -lean_dec(x_260); -x_271 = lean_ctor_get(x_261, 1); -lean_inc(x_271); -lean_dec(x_261); -x_272 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_273 = lean_string_dec_eq(x_271, x_272); -lean_dec(x_271); -if (x_273 == 0) -{ -lean_object* x_274; -lean_dec(x_270); -lean_dec(x_269); -lean_dec(x_268); -lean_dec(x_267); -lean_dec(x_266); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_274 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_274; -} -else -{ -lean_object* x_275; uint8_t x_276; -x_275 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_276 = lean_string_dec_eq(x_270, x_275); -lean_dec(x_270); -if (x_276 == 0) -{ -lean_object* x_277; -lean_dec(x_269); -lean_dec(x_268); -lean_dec(x_267); -lean_dec(x_266); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_277 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_277; -} -else -{ -lean_object* x_278; uint8_t x_279; -x_278 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__10; -x_279 = lean_string_dec_eq(x_269, x_278); -lean_dec(x_269); -if (x_279 == 0) -{ -lean_object* x_280; -lean_dec(x_268); -lean_dec(x_267); -lean_dec(x_266); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_280 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_280; -} -else -{ -if (lean_obj_tag(x_268) == 9) -{ -lean_object* x_281; -x_281 = lean_ctor_get(x_268, 0); -lean_inc(x_281); -lean_dec(x_268); -if (lean_obj_tag(x_281) == 0) -{ -lean_object* x_282; -lean_dec(x_281); -lean_dec(x_267); -lean_dec(x_266); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_282 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_282; -} -else -{ -if (lean_obj_tag(x_267) == 9) -{ -lean_object* x_283; -x_283 = lean_ctor_get(x_267, 0); -lean_inc(x_283); -lean_dec(x_267); -if (lean_obj_tag(x_283) == 0) -{ -lean_object* x_284; -lean_dec(x_283); -lean_dec(x_281); -lean_dec(x_266); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_284 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_284; -} -else -{ -if (lean_obj_tag(x_266) == 9) -{ -lean_object* x_285; -x_285 = lean_ctor_get(x_266, 0); -lean_inc(x_285); -lean_dec(x_266); -if (lean_obj_tag(x_285) == 0) -{ -lean_object* x_286; -lean_dec(x_285); -lean_dec(x_283); -lean_dec(x_281); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_286 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_286; -} -else -{ -if (lean_obj_tag(x_265) == 9) -{ -lean_object* x_287; -x_287 = lean_ctor_get(x_265, 0); -lean_inc(x_287); -lean_dec(x_265); -if (lean_obj_tag(x_287) == 0) -{ -lean_object* x_288; -lean_dec(x_287); -lean_dec(x_285); -lean_dec(x_283); -lean_dec(x_281); -lean_dec(x_264); -lean_dec(x_263); -x_288 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_288; -} -else -{ -if (lean_obj_tag(x_264) == 9) -{ -lean_object* x_289; -x_289 = lean_ctor_get(x_264, 0); -lean_inc(x_289); -lean_dec(x_264); -if (lean_obj_tag(x_289) == 0) -{ -lean_object* x_290; -lean_dec(x_289); -lean_dec(x_287); -lean_dec(x_285); -lean_dec(x_283); -lean_dec(x_281); -lean_dec(x_263); -x_290 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_290; -} -else -{ -if (lean_obj_tag(x_263) == 9) -{ -lean_object* x_291; -x_291 = lean_ctor_get(x_263, 0); -lean_inc(x_291); -lean_dec(x_263); -if (lean_obj_tag(x_291) == 0) -{ -lean_object* x_292; -lean_dec(x_291); -lean_dec(x_289); -lean_dec(x_287); -lean_dec(x_285); -lean_dec(x_283); -lean_dec(x_281); -x_292 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_292; -} -else -{ -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; -x_293 = lean_ctor_get(x_281, 0); -lean_inc(x_293); -lean_dec(x_281); -x_294 = lean_ctor_get(x_283, 0); -lean_inc(x_294); -lean_dec(x_283); -x_295 = lean_ctor_get(x_285, 0); -lean_inc(x_295); -lean_dec(x_285); -x_296 = lean_ctor_get(x_287, 0); -lean_inc(x_296); -lean_dec(x_287); -x_297 = lean_ctor_get(x_289, 0); -lean_inc(x_297); -lean_dec(x_289); -x_298 = lean_ctor_get(x_291, 0); -lean_inc(x_298); -lean_dec(x_291); -x_299 = l_Lean_Name_mkStr6(x_293, x_294, x_295, x_296, x_297, x_298); -x_300 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_300, 0, x_299); -lean_ctor_set(x_300, 1, x_8); -return x_300; -} -} -else -{ -lean_object* x_301; -lean_dec(x_289); -lean_dec(x_287); -lean_dec(x_285); -lean_dec(x_283); -lean_dec(x_281); -lean_dec(x_263); -x_301 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_301; -} -} -} -else -{ -lean_object* x_302; -lean_dec(x_287); -lean_dec(x_285); -lean_dec(x_283); -lean_dec(x_281); -lean_dec(x_264); -lean_dec(x_263); -x_302 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_302; -} -} -} -else -{ -lean_object* x_303; -lean_dec(x_285); -lean_dec(x_283); -lean_dec(x_281); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_303 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_303; -} -} -} -else -{ -lean_object* x_304; -lean_dec(x_283); -lean_dec(x_281); -lean_dec(x_266); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_304 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_304; -} -} -} -else -{ -lean_object* x_305; -lean_dec(x_281); -lean_dec(x_267); -lean_dec(x_266); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_305 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_305; -} -} -} -else -{ -lean_object* x_306; -lean_dec(x_268); -lean_dec(x_267); -lean_dec(x_266); -lean_dec(x_265); -lean_dec(x_264); -lean_dec(x_263); -x_306 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_306; -} -} -} -} -} -else -{ -lean_object* x_307; -lean_dec(x_262); -lean_dec(x_261); -lean_dec(x_260); -lean_dec(x_259); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_307 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_307; -} -} -else -{ -lean_object* x_308; -lean_dec(x_261); -lean_dec(x_260); -lean_dec(x_259); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_308 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_308; -} -} -else -{ -lean_object* x_309; -lean_dec(x_260); -lean_dec(x_259); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_309 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_309; -} -} -else -{ -lean_object* x_310; -lean_dec(x_259); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_310 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_310; -} -} -case 5: -{ -lean_object* x_311; -x_311 = lean_ctor_get(x_258, 0); -lean_inc(x_311); -switch (lean_obj_tag(x_311)) { -case 4: -{ -lean_object* x_312; -x_312 = lean_ctor_get(x_311, 0); -lean_inc(x_312); -lean_dec(x_311); -if (lean_obj_tag(x_312) == 1) -{ -lean_object* x_313; -x_313 = lean_ctor_get(x_312, 0); -lean_inc(x_313); -if (lean_obj_tag(x_313) == 1) -{ -lean_object* x_314; -x_314 = lean_ctor_get(x_313, 0); -lean_inc(x_314); -if (lean_obj_tag(x_314) == 1) -{ -lean_object* x_315; -x_315 = lean_ctor_get(x_314, 0); -lean_inc(x_315); -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; lean_object* x_326; uint8_t x_327; -x_316 = lean_ctor_get(x_1, 1); -lean_inc(x_316); -lean_dec(x_1); -x_317 = lean_ctor_get(x_31, 1); -lean_inc(x_317); -lean_dec(x_31); -x_318 = lean_ctor_get(x_60, 1); -lean_inc(x_318); -lean_dec(x_60); -x_319 = lean_ctor_get(x_129, 1); -lean_inc(x_319); -lean_dec(x_129); -x_320 = lean_ctor_get(x_167, 1); -lean_inc(x_320); -lean_dec(x_167); -x_321 = lean_ctor_get(x_210, 1); -lean_inc(x_321); -lean_dec(x_210); -x_322 = lean_ctor_get(x_258, 1); -lean_inc(x_322); -lean_dec(x_258); -x_323 = lean_ctor_get(x_312, 1); -lean_inc(x_323); -lean_dec(x_312); -x_324 = lean_ctor_get(x_313, 1); -lean_inc(x_324); -lean_dec(x_313); -x_325 = lean_ctor_get(x_314, 1); -lean_inc(x_325); -lean_dec(x_314); -x_326 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_327 = lean_string_dec_eq(x_325, x_326); -lean_dec(x_325); -if (x_327 == 0) -{ -lean_object* x_328; -lean_dec(x_324); -lean_dec(x_323); -lean_dec(x_322); -lean_dec(x_321); -lean_dec(x_320); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_328 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_328; -} -else -{ -lean_object* x_329; uint8_t x_330; -x_329 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_330 = lean_string_dec_eq(x_324, x_329); -lean_dec(x_324); -if (x_330 == 0) -{ -lean_object* x_331; -lean_dec(x_323); -lean_dec(x_322); -lean_dec(x_321); -lean_dec(x_320); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_331 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_331; -} -else -{ -lean_object* x_332; uint8_t x_333; -x_332 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__11; -x_333 = lean_string_dec_eq(x_323, x_332); -lean_dec(x_323); -if (x_333 == 0) -{ -lean_object* x_334; -lean_dec(x_322); -lean_dec(x_321); -lean_dec(x_320); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_334 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_334; -} -else -{ -if (lean_obj_tag(x_322) == 9) -{ -lean_object* x_335; -x_335 = lean_ctor_get(x_322, 0); -lean_inc(x_335); -lean_dec(x_322); -if (lean_obj_tag(x_335) == 0) -{ -lean_object* x_336; -lean_dec(x_335); -lean_dec(x_321); -lean_dec(x_320); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_336 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_336; -} -else -{ -if (lean_obj_tag(x_321) == 9) -{ -lean_object* x_337; -x_337 = lean_ctor_get(x_321, 0); -lean_inc(x_337); -lean_dec(x_321); -if (lean_obj_tag(x_337) == 0) -{ -lean_object* x_338; -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_320); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_338 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_338; -} -else -{ -if (lean_obj_tag(x_320) == 9) -{ -lean_object* x_339; -x_339 = lean_ctor_get(x_320, 0); -lean_inc(x_339); -lean_dec(x_320); -if (lean_obj_tag(x_339) == 0) -{ -lean_object* x_340; -lean_dec(x_339); -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_340 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_340; -} -else -{ -if (lean_obj_tag(x_319) == 9) -{ -lean_object* x_341; -x_341 = lean_ctor_get(x_319, 0); -lean_inc(x_341); -lean_dec(x_319); -if (lean_obj_tag(x_341) == 0) -{ -lean_object* x_342; -lean_dec(x_341); -lean_dec(x_339); -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_342 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_342; -} -else -{ -if (lean_obj_tag(x_318) == 9) -{ -lean_object* x_343; -x_343 = lean_ctor_get(x_318, 0); -lean_inc(x_343); -lean_dec(x_318); -if (lean_obj_tag(x_343) == 0) -{ -lean_object* x_344; -lean_dec(x_343); -lean_dec(x_341); -lean_dec(x_339); -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_317); -lean_dec(x_316); -x_344 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_344; -} -else -{ -if (lean_obj_tag(x_317) == 9) -{ -lean_object* x_345; -x_345 = lean_ctor_get(x_317, 0); -lean_inc(x_345); -lean_dec(x_317); -if (lean_obj_tag(x_345) == 0) -{ -lean_object* x_346; -lean_dec(x_345); -lean_dec(x_343); -lean_dec(x_341); -lean_dec(x_339); -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_316); -x_346 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_346; -} -else -{ -if (lean_obj_tag(x_316) == 9) -{ -lean_object* x_347; -x_347 = lean_ctor_get(x_316, 0); -lean_inc(x_347); -lean_dec(x_316); -if (lean_obj_tag(x_347) == 0) -{ -lean_object* x_348; -lean_dec(x_347); -lean_dec(x_345); -lean_dec(x_343); -lean_dec(x_341); -lean_dec(x_339); -lean_dec(x_337); -lean_dec(x_335); -x_348 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_348; -} -else -{ -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; -x_349 = lean_ctor_get(x_335, 0); -lean_inc(x_349); -lean_dec(x_335); -x_350 = lean_ctor_get(x_337, 0); -lean_inc(x_350); -lean_dec(x_337); -x_351 = lean_ctor_get(x_339, 0); -lean_inc(x_351); -lean_dec(x_339); -x_352 = lean_ctor_get(x_341, 0); -lean_inc(x_352); -lean_dec(x_341); -x_353 = lean_ctor_get(x_343, 0); -lean_inc(x_353); -lean_dec(x_343); -x_354 = lean_ctor_get(x_345, 0); -lean_inc(x_354); -lean_dec(x_345); -x_355 = lean_ctor_get(x_347, 0); -lean_inc(x_355); -lean_dec(x_347); -x_356 = l_Lean_Name_mkStr7(x_349, x_350, x_351, x_352, x_353, x_354, x_355); -x_357 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_357, 0, x_356); -lean_ctor_set(x_357, 1, x_8); -return x_357; -} -} -else -{ -lean_object* x_358; -lean_dec(x_345); -lean_dec(x_343); -lean_dec(x_341); -lean_dec(x_339); -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_316); -x_358 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_358; -} -} -} -else -{ -lean_object* x_359; -lean_dec(x_343); -lean_dec(x_341); -lean_dec(x_339); -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_317); -lean_dec(x_316); -x_359 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_359; -} -} -} -else -{ -lean_object* x_360; -lean_dec(x_341); -lean_dec(x_339); -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_360 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_360; -} -} -} -else -{ -lean_object* x_361; -lean_dec(x_339); -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_361 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_361; -} -} -} -else -{ -lean_object* x_362; -lean_dec(x_337); -lean_dec(x_335); -lean_dec(x_320); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_362 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_362; -} -} -} -else -{ -lean_object* x_363; -lean_dec(x_335); -lean_dec(x_321); -lean_dec(x_320); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_363 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_363; -} -} -} -else -{ -lean_object* x_364; -lean_dec(x_322); -lean_dec(x_321); -lean_dec(x_320); -lean_dec(x_319); -lean_dec(x_318); -lean_dec(x_317); -lean_dec(x_316); -x_364 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_364; -} -} -} -} -} -else -{ -lean_object* x_365; -lean_dec(x_315); -lean_dec(x_314); -lean_dec(x_313); -lean_dec(x_312); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_365 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_365; -} -} -else -{ -lean_object* x_366; -lean_dec(x_314); -lean_dec(x_313); -lean_dec(x_312); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_366 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_366; -} -} -else -{ -lean_object* x_367; -lean_dec(x_313); -lean_dec(x_312); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_367 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_367; -} -} -else -{ -lean_object* x_368; -lean_dec(x_312); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_368 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_368; -} -} -case 5: -{ -lean_object* x_369; -x_369 = lean_ctor_get(x_311, 0); -lean_inc(x_369); -if (lean_obj_tag(x_369) == 4) -{ -lean_object* x_370; -x_370 = lean_ctor_get(x_369, 0); -lean_inc(x_370); -lean_dec(x_369); -if (lean_obj_tag(x_370) == 1) -{ -lean_object* x_371; -x_371 = lean_ctor_get(x_370, 0); -lean_inc(x_371); -if (lean_obj_tag(x_371) == 1) -{ -lean_object* x_372; -x_372 = lean_ctor_get(x_371, 0); -lean_inc(x_372); -if (lean_obj_tag(x_372) == 1) -{ -lean_object* x_373; -x_373 = lean_ctor_get(x_372, 0); -lean_inc(x_373); -if (lean_obj_tag(x_373) == 0) -{ -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; uint8_t x_386; -x_374 = lean_ctor_get(x_1, 1); -lean_inc(x_374); -lean_dec(x_1); -x_375 = lean_ctor_get(x_31, 1); -lean_inc(x_375); -lean_dec(x_31); -x_376 = lean_ctor_get(x_60, 1); -lean_inc(x_376); -lean_dec(x_60); -x_377 = lean_ctor_get(x_129, 1); -lean_inc(x_377); -lean_dec(x_129); -x_378 = lean_ctor_get(x_167, 1); -lean_inc(x_378); -lean_dec(x_167); -x_379 = lean_ctor_get(x_210, 1); -lean_inc(x_379); -lean_dec(x_210); -x_380 = lean_ctor_get(x_258, 1); -lean_inc(x_380); -lean_dec(x_258); -x_381 = lean_ctor_get(x_311, 1); -lean_inc(x_381); -lean_dec(x_311); -x_382 = lean_ctor_get(x_370, 1); -lean_inc(x_382); -lean_dec(x_370); -x_383 = lean_ctor_get(x_371, 1); -lean_inc(x_383); -lean_dec(x_371); -x_384 = lean_ctor_get(x_372, 1); -lean_inc(x_384); -lean_dec(x_372); -x_385 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_386 = lean_string_dec_eq(x_384, x_385); -lean_dec(x_384); -if (x_386 == 0) -{ -lean_object* x_387; -lean_dec(x_383); -lean_dec(x_382); -lean_dec(x_381); -lean_dec(x_380); -lean_dec(x_379); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_387 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_387; -} -else -{ -lean_object* x_388; uint8_t x_389; -x_388 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_389 = lean_string_dec_eq(x_383, x_388); -lean_dec(x_383); -if (x_389 == 0) -{ -lean_object* x_390; -lean_dec(x_382); -lean_dec(x_381); -lean_dec(x_380); -lean_dec(x_379); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_390 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_390; -} -else -{ -lean_object* x_391; uint8_t x_392; -x_391 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__12; -x_392 = lean_string_dec_eq(x_382, x_391); -lean_dec(x_382); -if (x_392 == 0) -{ -lean_object* x_393; -lean_dec(x_381); -lean_dec(x_380); -lean_dec(x_379); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_393 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_393; -} -else -{ -if (lean_obj_tag(x_381) == 9) -{ -lean_object* x_394; -x_394 = lean_ctor_get(x_381, 0); -lean_inc(x_394); -lean_dec(x_381); -if (lean_obj_tag(x_394) == 0) -{ -lean_object* x_395; -lean_dec(x_394); -lean_dec(x_380); -lean_dec(x_379); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_395 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_395; -} -else -{ -if (lean_obj_tag(x_380) == 9) -{ -lean_object* x_396; -x_396 = lean_ctor_get(x_380, 0); -lean_inc(x_396); -lean_dec(x_380); -if (lean_obj_tag(x_396) == 0) -{ -lean_object* x_397; -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_379); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_397 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_397; -} -else -{ -if (lean_obj_tag(x_379) == 9) -{ -lean_object* x_398; -x_398 = lean_ctor_get(x_379, 0); -lean_inc(x_398); -lean_dec(x_379); -if (lean_obj_tag(x_398) == 0) -{ -lean_object* x_399; -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_399 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_399; -} -else -{ -if (lean_obj_tag(x_378) == 9) -{ -lean_object* x_400; -x_400 = lean_ctor_get(x_378, 0); -lean_inc(x_400); -lean_dec(x_378); -if (lean_obj_tag(x_400) == 0) -{ -lean_object* x_401; -lean_dec(x_400); -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_401 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_401; -} -else -{ -if (lean_obj_tag(x_377) == 9) -{ -lean_object* x_402; -x_402 = lean_ctor_get(x_377, 0); -lean_inc(x_402); -lean_dec(x_377); -if (lean_obj_tag(x_402) == 0) -{ -lean_object* x_403; -lean_dec(x_402); -lean_dec(x_400); -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_403 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_403; -} -else -{ -if (lean_obj_tag(x_376) == 9) -{ -lean_object* x_404; -x_404 = lean_ctor_get(x_376, 0); -lean_inc(x_404); -lean_dec(x_376); -if (lean_obj_tag(x_404) == 0) -{ -lean_object* x_405; -lean_dec(x_404); -lean_dec(x_402); -lean_dec(x_400); -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_375); -lean_dec(x_374); -x_405 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_405; -} -else -{ -if (lean_obj_tag(x_375) == 9) -{ -lean_object* x_406; -x_406 = lean_ctor_get(x_375, 0); -lean_inc(x_406); -lean_dec(x_375); -if (lean_obj_tag(x_406) == 0) -{ -lean_object* x_407; -lean_dec(x_406); -lean_dec(x_404); -lean_dec(x_402); -lean_dec(x_400); -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_374); -x_407 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_407; -} -else -{ -if (lean_obj_tag(x_374) == 9) -{ -lean_object* x_408; -x_408 = lean_ctor_get(x_374, 0); -lean_inc(x_408); -lean_dec(x_374); -if (lean_obj_tag(x_408) == 0) -{ -lean_object* x_409; -lean_dec(x_408); -lean_dec(x_406); -lean_dec(x_404); -lean_dec(x_402); -lean_dec(x_400); -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -x_409 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_409; -} -else -{ -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; -x_410 = lean_ctor_get(x_394, 0); -lean_inc(x_410); -lean_dec(x_394); -x_411 = lean_ctor_get(x_396, 0); -lean_inc(x_411); -lean_dec(x_396); -x_412 = lean_ctor_get(x_398, 0); -lean_inc(x_412); -lean_dec(x_398); -x_413 = lean_ctor_get(x_400, 0); -lean_inc(x_413); -lean_dec(x_400); -x_414 = lean_ctor_get(x_402, 0); -lean_inc(x_414); -lean_dec(x_402); -x_415 = lean_ctor_get(x_404, 0); -lean_inc(x_415); -lean_dec(x_404); -x_416 = lean_ctor_get(x_406, 0); -lean_inc(x_416); -lean_dec(x_406); -x_417 = lean_ctor_get(x_408, 0); -lean_inc(x_417); -lean_dec(x_408); -x_418 = l_Lean_Name_mkStr8(x_410, x_411, x_412, x_413, x_414, x_415, x_416, x_417); -x_419 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_419, 0, x_418); -lean_ctor_set(x_419, 1, x_8); -return x_419; -} -} -else -{ -lean_object* x_420; -lean_dec(x_406); -lean_dec(x_404); -lean_dec(x_402); -lean_dec(x_400); -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_374); -x_420 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_420; -} -} -} -else -{ -lean_object* x_421; -lean_dec(x_404); -lean_dec(x_402); -lean_dec(x_400); -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_375); -lean_dec(x_374); -x_421 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_421; -} -} -} -else -{ -lean_object* x_422; -lean_dec(x_402); -lean_dec(x_400); -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_422 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_422; -} -} -} -else -{ -lean_object* x_423; -lean_dec(x_400); -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_423 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_423; -} -} -} -else -{ -lean_object* x_424; -lean_dec(x_398); -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_424 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_424; -} -} -} -else -{ -lean_object* x_425; -lean_dec(x_396); -lean_dec(x_394); -lean_dec(x_379); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_425 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_425; -} -} -} -else -{ -lean_object* x_426; -lean_dec(x_394); -lean_dec(x_380); -lean_dec(x_379); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_426 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_426; -} -} -} -else -{ -lean_object* x_427; -lean_dec(x_381); -lean_dec(x_380); -lean_dec(x_379); -lean_dec(x_378); -lean_dec(x_377); -lean_dec(x_376); -lean_dec(x_375); -lean_dec(x_374); -x_427 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_427; -} -} -} -} -} -else -{ -lean_object* x_428; -lean_dec(x_373); -lean_dec(x_372); -lean_dec(x_371); -lean_dec(x_370); -lean_dec(x_311); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_428 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_428; -} -} -else -{ -lean_object* x_429; -lean_dec(x_372); -lean_dec(x_371); -lean_dec(x_370); -lean_dec(x_311); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_429 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_429; -} -} -else -{ -lean_object* x_430; -lean_dec(x_371); -lean_dec(x_370); -lean_dec(x_311); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_430 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_430; -} -} -else -{ -lean_object* x_431; -lean_dec(x_370); -lean_dec(x_311); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_431 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_431; -} -} -else -{ -lean_object* x_432; -lean_dec(x_369); -lean_dec(x_311); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_432 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_432; -} -} -default: -{ -lean_object* x_433; -lean_dec(x_311); -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_433 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_433; -} -} -} -default: -{ -lean_object* x_434; -lean_dec(x_258); -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_434 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_434; -} -} -} -default: -{ -lean_object* x_435; -lean_dec(x_210); -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_435 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_435; -} -} -} -default: -{ -lean_object* x_436; -lean_dec(x_167); -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_436 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_436; -} -} -} -default: -{ -lean_object* x_437; -lean_dec(x_129); -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_437 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_437; -} -} -} -default: -{ -lean_object* x_438; -lean_dec(x_60); -lean_dec(x_31); -lean_dec(x_1); -x_438 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_438; -} -} -} -default: -{ -lean_object* x_439; -lean_dec(x_31); -lean_dec(x_1); -x_439 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_439; -} -} -} -default: -{ -lean_object* x_440; -lean_dec(x_1); -x_440 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); -return x_440; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_reifyName___boxed(lean_object* x_1, lean_object* x_2, 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_PrettyPrinter_Delaborator_reifyName(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 uint8_t l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__1(lean_object* x_1) { _start: { @@ -48326,15 +45120,19 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambd _start: { lean_object* x_9; -x_9 = l_Lean_PrettyPrinter_Delaborator_reifyName(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Expr_name_x3f(x_1); 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_10; +x_10 = l_Lean_PrettyPrinter_Delaborator_failure___rarg(x_8); +return x_10; +} +else { -lean_object* 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; lean_object* x_23; lean_object* x_24; lean_object* x_25; +lean_object* 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; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +lean_dec(x_9); x_12 = 1; x_13 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__3; x_14 = l_Lean_Name_toString(x_11, x_12, x_13); @@ -48355,64 +45153,10 @@ x_25 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_25, 0, x_19); lean_ctor_set(x_25, 1, x_24); lean_ctor_set(x_25, 2, x_23); -lean_ctor_set(x_9, 0, x_25); -return x_9; -} -else -{ -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; -x_26 = lean_ctor_get(x_9, 0); -x_27 = lean_ctor_get(x_9, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_9); -x_28 = 1; -x_29 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__3; -x_30 = l_Lean_Name_toString(x_26, x_28, x_29); -x_31 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__4; -x_32 = lean_string_append(x_31, x_30); -lean_dec(x_30); -x_33 = l_Lean_PrettyPrinter_Delaborator_delabOfScientific___lambda__1___closed__2; -x_34 = lean_string_append(x_32, x_33); -x_35 = lean_box(2); -x_36 = l_Lean_Syntax_mkNameLit(x_34, x_35); -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 = l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__2; -x_41 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_41, 0, x_35); -lean_ctor_set(x_41, 1, x_40); -lean_ctor_set(x_41, 2, 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_27); -return x_42; -} -} -else -{ -uint8_t x_43; -x_43 = !lean_is_exclusive(x_9); -if (x_43 == 0) -{ -return x_9; -} -else -{ -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_9, 0); -x_45 = lean_ctor_get(x_9, 1); -lean_inc(x_45); -lean_inc(x_44); -lean_dec(x_9); -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; -} +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_8); +return x_26; } } } @@ -48473,16 +45217,32 @@ return x_9; static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Name", 4, 4); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("str", 3, 3); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__4; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__2; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4() { _start: { lean_object* x_1; @@ -48490,19 +45250,19 @@ x_1 = lean_mk_string_unchecked("delabNameMkStr", 14, 14); return x_1; } } -static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3() { +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__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_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__3; x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__4; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4() { +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6() { _start: { lean_object* x_1; @@ -48515,9 +45275,9 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabName { 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_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } @@ -48525,11 +45285,19 @@ return x_6; static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__1() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr1", 6, 6); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__3; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -48539,9 +45307,9 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabName { 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_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } @@ -48549,11 +45317,19 @@ return x_6; static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__1() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr2", 6, 6); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__6; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -48563,9 +45339,9 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabName { 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_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } @@ -48573,11 +45349,19 @@ return x_6; static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__1() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr3", 6, 6); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__7; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -48587,9 +45371,9 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabName { 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_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } @@ -48597,11 +45381,19 @@ return x_6; static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__1() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr4", 6, 6); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__8; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -48611,9 +45403,9 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabName { 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_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } @@ -48621,11 +45413,19 @@ return x_6; static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__1() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr5", 6, 6); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__9; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -48635,9 +45435,9 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabName { 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_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } @@ -48645,11 +45445,19 @@ return x_6; static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__1() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr6", 6, 6); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__10; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -48659,9 +45467,9 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabName { 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_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } @@ -48669,11 +45477,19 @@ return x_6; static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__1() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr7", 6, 6); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__11; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -48683,9 +45499,9 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabName { 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_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } @@ -48693,11 +45509,19 @@ return x_6; static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__1() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr8", 6, 6); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__12; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -48707,9 +45531,9 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabName { 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_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6; x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } @@ -48725,16 +45549,24 @@ return x_8; static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__1() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("num", 3, 3); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabApp__1___closed__1; x_2 = l_Lean_PrettyPrinter_Delaborator_withTypeAscription___closed__2; -x_3 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1; -x_4 = l_Lean_PrettyPrinter_Delaborator_reifyName___closed__5; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__1; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__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___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__3() { _start: { lean_object* x_1; @@ -48742,19 +45574,19 @@ x_1 = lean_mk_string_unchecked("delabNameMkNum", 14, 14); return x_1; } } -static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__3() { +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___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_PrettyPrinter_Delaborator_withTypeAscription___closed__2; x_2 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__3; x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabFVar__1___closed__4; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__3; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__4() { +static lean_object* _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__5() { _start: { lean_object* x_1; @@ -48767,9 +45599,9 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabName { 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_PrettyPrinter_Delaborator_delabFVar__1___closed__7; -x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__1; -x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__3; -x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__4; +x_3 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__2; +x_4 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__4; +x_5 = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__5; x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } @@ -51792,7 +48624,7 @@ static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_delabConstWithSignatu 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_PrettyPrinter_Delaborator_delabFVar___closed__1; x_2 = l_Lean_PrettyPrinter_Delaborator_delabConstWithSignature_delabParamsAux___closed__1; -x_3 = lean_unsigned_to_nat(1307u); +x_3 = lean_unsigned_to_nat(1286u); x_4 = lean_unsigned_to_nat(42u); x_5 = l_Lean_PrettyPrinter_Delaborator_delabFVar___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -54450,10 +51282,10 @@ l_Lean_getConstInfo___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__2_ lean_mark_persistent(l_Lean_getConstInfo___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__2___closed__3); l_Lean_getConstInfo___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__2___closed__4 = _init_l_Lean_getConstInfo___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__2___closed__4(); lean_mark_persistent(l_Lean_getConstInfo___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__2___closed__4); -l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1 = _init_l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1); -l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2 = _init_l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2(); -lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2); +l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1 = _init_l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__1); +l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2 = _init_l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2(); +lean_mark_persistent(l_Array_mapFinIdxM_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__18___closed__2); l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__19___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__19___closed__1(); lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__19___closed__1); l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__19___closed__2 = _init_l_Array_mapMUnsafe_map___at_Lean_PrettyPrinter_Delaborator_delabAppMatch___spec__19___closed__2(); @@ -55150,31 +51982,7 @@ lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDo__1___ if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabDo__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__1); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__2 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__2(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__2); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__3 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__3(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__3); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__4 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__4(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__4); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__5 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__5(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__5); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__6 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__6(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__6); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__7 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__7(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__7); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__8 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__8(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__8); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__9 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__9(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__9); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__10 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__10(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__10); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__11 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__11(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__11); -l_Lean_PrettyPrinter_Delaborator_reifyName___closed__12 = _init_l_Lean_PrettyPrinter_Delaborator_reifyName___closed__12(); -lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_reifyName___closed__12); -l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__1 = _init_l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__1(); +}l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__1 = _init_l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__1(); lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__1); l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__2 = _init_l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__2(); lean_mark_persistent(l_Lean_PrettyPrinter_Delaborator_delabNameMkStr___lambda__2___closed__2); @@ -55194,46 +52002,66 @@ l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3 = _i lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__3); l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__4); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__5); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1___closed__6); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__1); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2___closed__2); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__2(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__1); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3___closed__2); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__3(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__1); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4___closed__2); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__4(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__1); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5___closed__2); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__5(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__1); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6___closed__2); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__6(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__1); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7___closed__2); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__7(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__1); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8___closed__2); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__8(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__1 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__1); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__2 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9___closed__2); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkStr__9(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); @@ -55245,6 +52073,8 @@ l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__3 = _i lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__3); l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__4 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__4(); lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__4); +l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__5 = _init_l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__5(); +lean_mark_persistent(l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1___closed__5); if (builtin) {res = l___regBuiltin_Lean_PrettyPrinter_Delaborator_delabNameMkNum__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Lean/Server/CodeActions/Basic.c b/stage0/stdlib/Lean/Server/CodeActions/Basic.c index 091aef5554c0..a388116a38a6 100644 --- a/stage0/stdlib/Lean/Server/CodeActions/Basic.c +++ b/stage0/stdlib/Lean/Server/CodeActions/Basic.c @@ -92,6 +92,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Serve extern lean_object* l_Lean_Server_requestHandlers; lean_object* l_Lean_stringToMessageData(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_handleCodeActionResolve(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_fromJsonCodeAction____x40_Lean_Data_Lsp_CodeActions___hyg_1204_(lean_object*); static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____lambda__2___closed__6; LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_1540____spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); @@ -113,12 +114,12 @@ LEAN_EXPORT lean_object* l_Lean_Server_instFileSourceCodeAction(lean_object*); static lean_object* l_Lean_Server_CodeAction_getFileSource_x21___closed__4; size_t lean_usize_of_nat(lean_object*); extern lean_object* l_Lean_Server_instInhabitedRequestError; +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9(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_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____closed__25; static lean_object* l___private_Lean_Server_CodeActions_Basic_0__Lean_Server_fromJsonCodeActionResolveData____x40_Lean_Server_CodeActions_Basic___hyg_125____closed__1; static lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_1209____spec__2___closed__2; LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_1209____spec__3___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FileMap_lspPosToUtf8Pos(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9(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_registerLspRequestHandler___at_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_1540____spec__1___lambda__2___closed__1; static lean_object* l_Lean_Server_instFromJsonCodeActionResolveData___closed__1; lean_object* lean_st_ref_take(lean_object*, lean_object*); @@ -162,6 +163,7 @@ lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_454____closed__4; LEAN_EXPORT lean_object* l_Lean_Server_handleCodeAction(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____closed__3; +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____closed__26; static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____closed__8; static lean_object* l___private_Lean_Server_CodeActions_Basic_0__Lean_Server_fromJsonCodeActionResolveData____x40_Lean_Server_CodeActions_Basic___hyg_125____closed__7; @@ -189,7 +191,6 @@ lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_ lean_object* l_Lean_registerSimplePersistentEnvExtension___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_handleCodeAction___spec__10(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ofExcept___at_Lean_Server_handleCodeAction___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); lean_object* l_Pi_instInhabited___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_codeActionProviderExt; static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____lambda__3___closed__2; @@ -208,6 +209,7 @@ lean_object* l_Array_append___rarg(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__18; LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____lambda__3(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeActionParams____x40_Lean_Data_Lsp_CodeActions___hyg_612_(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____lambda__5___closed__1; static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_454____closed__1; static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____lambda__2___closed__4; @@ -255,7 +257,6 @@ static lean_object* l___private_Lean_Server_CodeActions_Basic_0__Lean_Server_fro lean_object* l_Lean_registerBuiltinAttribute(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, 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__12; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Attributes_0__Lean_beqAttributeKind____x40_Lean_Attributes___hyg_162_(uint8_t, uint8_t); lean_object* l___private_Lean_ToExpr_0__Lean_Name_toExprAux(lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_revFold___at_Lean_Server_handleCodeAction___spec__7(lean_object*, lean_object*); @@ -277,17 +278,16 @@ LEAN_EXPORT lean_object* l_Lean_Server_handleCodeActionResolve___lambda__3(lean_ LEAN_EXPORT lean_object* l_Lean_Server_CodeAction_getFileSource_x21(lean_object*); static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_1209____spec__1___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Server_handleCodeAction___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_CodeActions_0__Lean_Lsp_toJsonCodeAction____x40_Lean_Data_Lsp_CodeActions___hyg_1130_(lean_object*); uint8_t l_Lean_PersistentHashMap_contains___at_Lean_Server_registerLspRequestHandler___spec__6(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_1209_(lean_object*); LEAN_EXPORT lean_object* l_Lean_RBMap_toList___at_Lean_Server_handleCodeAction___spec__6(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__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_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_454____lambda__3(lean_object*); static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9___boxed(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*); uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_513____lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -424,7 +424,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_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_24, x_25); +x_26 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_24, x_25); x_27 = l_Lean_Json_mkObj(x_26); return x_27; } @@ -2588,7 +2588,7 @@ x_3 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Server_handleCodeActio return x_3; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9___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_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9___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; lean_object* x_10; uint8_t x_11; @@ -2656,7 +2656,7 @@ return x_26; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___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, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___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, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; uint8_t x_12; @@ -2694,7 +2694,7 @@ x_21 = lean_box(0); lean_inc(x_6); lean_inc(x_2); lean_inc(x_1); -x_22 = l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1(x_1, x_2, x_6, x_15, x_21, x_9, x_10); +x_22 = l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1(x_1, x_2, x_6, x_15, x_21, x_9, x_10); x_23 = lean_ctor_get(x_22, 0); lean_inc(x_23); x_24 = lean_ctor_get(x_22, 1); @@ -2755,7 +2755,7 @@ x_16 = lean_array_get_size(x_14); x_17 = lean_mk_empty_array_with_capacity(x_16); x_18 = lean_unsigned_to_nat(0u); lean_inc(x_1); -x_19 = l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9(x_1, x_11, x_14, x_14, x_16, x_18, lean_box(0), x_17, x_7, x_15); +x_19 = l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9(x_1, x_11, x_14, x_14, x_16, x_18, lean_box(0), x_17, x_7, x_15); lean_dec(x_14); x_20 = lean_ctor_get(x_19, 0); lean_inc(x_20); @@ -3288,21 +3288,21 @@ lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9___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_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9___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_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__9___lambda__1(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; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___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) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___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: { lean_object* x_11; -x_11 = l_Array_mapIdxM_map___at_Lean_Server_handleCodeAction___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Array_mapFinIdxM_map___at_Lean_Server_handleCodeAction___spec__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_4); lean_dec(x_3); diff --git a/stage0/stdlib/Lean/Server/Completion.c b/stage0/stdlib/Lean/Server/Completion.c index 6c70fea7af8d..fc258ad8e42c 100644 --- a/stage0/stdlib/Lean/Server/Completion.c +++ b/stage0/stdlib/Lean/Server/Completion.c @@ -23,7 +23,6 @@ lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___spec__24(lean_object*, 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_Server_Completion_completeNamespaces___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_string_utf8_extract(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_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_Lean_Lsp_CompletionItem_resolve___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Completion_completeNamespaces___spec__9(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* l_Lean_Meta_ppExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -45,6 +44,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_toJsonCo LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_matchDecl_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_Server_Completion_0__Lean_Server_Completion_isDefEqToAppOf___lambda__1___boxed(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___private_Lean_Server_Completion_0__Lean_Server_Completion_addUnresolvedCompletionItem(lean_object*, lean_object*, uint8_t, double, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotIdCompletion___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_PersistentHashMap_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_forEligibleDeclsM___spec__3(lean_object*); @@ -62,11 +62,11 @@ LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Compl LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotIdCompletion___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_Lean_PersistentHashMap_foldlMAux_traverse___at_Lean_Server_Completion_completeNamespaces___spec__8___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_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_isSyntheticTacticCompletion_isCompletionOnTacticBlockIndentation(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__3; static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136____lambda__3___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_addNamespaceCompletionItem___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_private_to_user_name(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_fieldIdCompletion___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findCompletionInfoAt_x3f_choose___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_Server_Completion_0__Lean_Server_Completion_getIndentationAmount___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Json_mkObj(lean_object*); @@ -141,11 +141,11 @@ LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Compl LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotCompletion___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ConstantInfo_name(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___spec__23(lean_object*, 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_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__1; static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findSyntheticIdentifierCompletion_x3f___lambda__3___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_isDefEqToAppOf___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_getDotCompletionTypeNames_visit___spec__3(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl(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*); @@ -153,7 +153,7 @@ uint8_t lean_float_decLt(double, double); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f_choose___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_addUnresolvedCompletionItem___lambda__2___closed__1; static lean_object* l_Lean_Server_Completion_getEligibleHeaderDecls___closed__2; -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__4; +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_forEligibleDeclsM___spec__4(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findSyntheticIdentifierCompletion_x3f___lambda__2___boxed(lean_object*); static lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Server_Completion_0__Lean_Server_Completion_isSyntheticTacticCompletion_isCompletionAfterSemicolon___spec__1___closed__1; @@ -165,7 +165,7 @@ LEAN_EXPORT lean_object* l_Lean_isEnumType___at___private_Lean_Server_Completion LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_toJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_270_(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeMAux___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findOutermostContextInfo_x3f_go___spec__2___boxed(lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_addKeywordCompletionItem___closed__3; -LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___lambda__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_InfoTree_foldInfo___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Completion_completeNamespaces___lambda__2(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_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136_(lean_object*); @@ -175,7 +175,6 @@ extern lean_object* l_Lean_instInhabitedJson; static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136____lambda__1___closed__2; uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_optionCompletion___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___boxed(lean_object*, lean_object*, 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_Lean_Expr_cleanupAnnotations(lean_object*); @@ -210,12 +209,10 @@ LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Compl static double l___private_Lean_Server_Completion_0__Lean_Server_Completion_matchAtomic___closed__1; static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotCompletion___lambda__6___closed__2; extern lean_object* l_instInhabitedNat; -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1(lean_object*); lean_object* l_Lean_Parser_getTokenTable(lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Server_Completion_completeNamespaces___spec__1___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___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_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___lambda__3___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2(lean_object*); lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_CompletionItemData_0__Lean_Lsp_fromJsonCompletionItemData____x40_Lean_Server_CompletionItemData___hyg_15____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_insert___at___private_Lean_Server_Completion_0__Lean_Server_Completion_getDotCompletionTypeNames_visit___spec__1(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_projectionFnInfoExt; @@ -227,7 +224,6 @@ LEAN_EXPORT lean_object* l_Lean_RBNode_ins___at___private_Lean_Server_Completion LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findOutermostContextInfo_x3f_go___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotIdCompletion___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_Server_Completion_0__Lean_Lsp_fromJsonCompletionItemDataWithId____x40_Lean_Server_Completion___hyg_366____closed__2; -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_truncate_go(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_getDotCompletionTypeNames(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_allowCompletion(lean_object*, lean_object*, lean_object*); @@ -255,7 +251,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Compl LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___spec__17___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 uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_isSyntheticTacticCompletion_isEmpty(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_isDotCompletionMethod___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_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlMAux_traverse___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___spec__15(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonCompletionItemDataWithId; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_forEligibleDeclsM___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -319,6 +314,7 @@ lean_object* l_Lean_Name_getPrefix(lean_object*); lean_object* l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at___private_Lean_Server_Completion_0__Lean_Server_Completion_dotCompletion___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_ConstantInfo_isCtor(lean_object*); +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2(lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___closed__5; static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136____closed__6; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_addKeywordCompletionItem___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -346,6 +342,7 @@ LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonCompletionIdentifier; static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionItemDataWithId____x40_Lean_Server_Completion___hyg_366____closed__11; LEAN_EXPORT lean_object* l_Lean_Lsp_CompletionItem_resolve___lambda__1___boxed(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_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*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_forEligibleDeclsM___spec__4___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore(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_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___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*, lean_object*, lean_object*, lean_object*); @@ -373,6 +370,7 @@ lean_object* l_Lean_Name_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f_choose___spec__1___rarg(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getTrailingSize(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts(lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); uint8_t lean_string_utf8_at_end(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionItemDataWithId____x40_Lean_Server_Completion___hyg_366____closed__15; static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_addNamespaceCompletionItem___closed__3; @@ -426,13 +424,11 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlMAux_traverse___at_Lean_S LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotCompletion___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_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136____lambda__3___closed__5; LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_findSyntheticIdentifierCompletion_x3f___lambda__2(lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_normPrivateName_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_addNamespaceCompletionItem(lean_object*, double, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_CompletionItem_resolve(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___spec__1___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*); uint8_t l_Lean_Syntax_isIdent(lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_isSyntheticTacticCompletion_isCompletionAfterSemicolon(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_fvarId(lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136____lambda__3___closed__8; @@ -461,7 +457,6 @@ extern lean_object* l_Lean_instInhabitedProjectionFunctionInfo; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_truncate(lean_object*, lean_object*); uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_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*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f_choose___spec__1(lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_isSyntheticTacticCompletion_isEmptyTacticBlock___closed__1; @@ -482,7 +477,6 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlMAux_traverse___at___priv static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_isSyntheticTacticCompletion_getTacticsNode_x3f___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___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 lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_isSyntheticTacticCompletion_go___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4(lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136____lambda__3___closed__9; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotCompletion___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_Server_Completion_completeNamespaces(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -509,6 +503,7 @@ static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionItemDataWithId____x40_Lean_Server_Completion___hyg_366____closed__7; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotIdCompletion___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_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136____lambda__1(lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__3; LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_findClosestInfoWithLocalContextAt_x3f_isBetter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___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_Server_Completion_0__Lean_Server_Completion_isDotIdCompletionMethod___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -556,8 +551,6 @@ static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_getDotCompletionTypeNames_visit___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___private_Lean_Server_Completion_0__Lean_Server_Completion_findSyntheticIdentifierCompletion_x3f___lambda__5___closed__1; lean_object* l_Lean_ParametricAttribute_getParam_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4___rarg___boxed(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_findBest_x3f___spec__3(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findOutermostContextInfo_x3f_go___spec__5(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findSyntheticIdentifierCompletion_x3f___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___spec__16(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -607,6 +600,7 @@ uint8_t l_Lean_Expr_isProp(lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Server_Completion_0__Lean_Server_Completion_getCompletionKindForDecl___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_fieldIdCompletion___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_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_getDotCompletionTypeNames_visit___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotCompletion___lambda__6___closed__1; lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); @@ -644,7 +638,6 @@ lean_object* l_Lean_instantiateMVarsCore(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_isDotCompletionMethod___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_truncate_go___closed__2; lean_object* l_List_dropWhile___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__2; lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__2___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_getIndentationAmount___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_optionCompletion___closed__4; @@ -711,6 +704,7 @@ static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___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___private_Lean_Server_Completion_0__Lean_Server_Completion_isSyntheticTacticCompletion_go___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_findSomeM_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findOutermostContextInfo_x3f_go___spec__1___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotIdCompletion___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_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); @@ -751,7 +745,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Compl uint8_t l_Lean_Name_isInternal(lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Server_Completion_0__Lean_Lsp_toJsonCompletionItemDataWithId____x40_Lean_Server_Completion___hyg_472____spec__1(lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonCompletionIdentifier; uint8_t lean_local_ctx_is_empty(lean_object*); lean_object* lean_expr_instantiate1(lean_object*, lean_object*); @@ -759,21 +752,23 @@ lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Completion_getEligibleHeaderDecls___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_CompletionItem_resolve___closed__2; lean_object* l_Lean_Elab_ContextInfo_runMetaM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg(lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_addUnresolvedCompletionItem___lambda__2___closed__3; static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_dotCompletion___lambda__6___closed__3; LEAN_EXPORT lean_object* l_Lean_Server_Completion_completeNamespaces___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_Server_Completion_0__Lean_Server_Completion_allowCompletion___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___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*); -static lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_SMap_forM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_idCompletionCore___spec__9(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_Server_Completion_0__Lean_Server_Completion_forEligibleDeclsM___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg(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_Server_Completion_0__Lean_Server_Completion_findSyntheticIdentifierCompletion_x3f___lambda__3___boxed(lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Lsp_fromJsonCompletionIdentifier____x40_Lean_Server_Completion___hyg_136____closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1(lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_fieldIdCompletion___closed__1; static lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Server_Completion_0__Lean_Server_Completion_optionCompletion___spec__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findClosestInfoWithLocalContextAt_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_matchDecl_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findSyntheticIdentifierCompletion_x3f___lambda__5___closed__3; lean_object* lean_data_value_to_string(lean_object*); @@ -2215,7 +2210,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_Completion_0__Lean_Lsp_toJsonCompletionItemDataWithId____x40_Lean_Server_Completion___hyg_472____closed__1; -x_14 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -25133,7 +25128,7 @@ x_2 = lean_alloc_closure((void*)(l___private_Lean_Server_Completion_0__Lean_Serv return x_2; } } -static lean_object* _init_l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg___closed__1() { +static lean_object* _init_l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -25143,24 +25138,24 @@ x_3 = l_instInhabitedOfMonad___rarg(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg(lean_object* x_1) { +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg___closed__1; +x_2 = l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1; x_3 = lean_panic_fn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3(lean_object* x_1) { +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg), 1, 0); +x_2 = lean_alloc_closure((void*)(l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg), 1, 0); return x_2; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4___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_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___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_4) == 0) @@ -25168,6 +25163,7 @@ if (lean_obj_tag(x_4) == 0) lean_object* x_6; lean_dec(x_3); lean_dec(x_2); +lean_dec(x_1); x_6 = l_List_reverse___rarg(x_5); return x_6; } @@ -25182,7 +25178,8 @@ x_8 = lean_ctor_get(x_4, 0); x_9 = lean_ctor_get(x_4, 1); lean_inc(x_3); lean_inc(x_2); -x_10 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg(x_1, x_2, x_3, x_8); +lean_inc(x_1); +x_10 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg(x_1, x_2, x_3, x_8); lean_ctor_set(x_4, 1, x_5); lean_ctor_set(x_4, 0, x_10); { @@ -25203,7 +25200,8 @@ lean_inc(x_12); lean_dec(x_4); lean_inc(x_3); lean_inc(x_2); -x_14 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg(x_1, x_2, x_3, x_12); +lean_inc(x_1); +x_14 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg(x_1, x_2, x_3, 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_5); @@ -25214,15 +25212,15 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4(lean_object* x_1) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4___rarg___boxed), 5, 0); +x_2 = lean_alloc_closure((void*)(l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg), 5, 0); return x_2; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__1() { _start: { lean_object* x_1; @@ -25230,7 +25228,7 @@ x_1 = lean_mk_string_unchecked("Lean.Server.InfoUtils", 21, 21); return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__2() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__2() { _start: { lean_object* x_1; @@ -25238,7 +25236,7 @@ x_1 = lean_mk_string_unchecked("Lean.Elab.InfoTree.visitM.go", 28, 28); return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__3() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__3() { _start: { lean_object* x_1; @@ -25246,20 +25244,20 @@ x_1 = lean_mk_string_unchecked("unexpected context-free info tree node", 38, 38) return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__4() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___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_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1; -x_2 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__2; -x_3 = lean_unsigned_to_nat(56u); +x_1 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__1; +x_2 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__2; +x_3 = lean_unsigned_to_nat(62u); x_4 = lean_unsigned_to_nat(21u); -x_5 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__3; +x_5 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___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_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_3) == 0) @@ -25283,8 +25281,9 @@ case 1: lean_object* x_9; lean_object* x_10; lean_dec(x_4); lean_dec(x_2); -x_9 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__4; -x_10 = l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg(x_9); +lean_dec(x_1); +x_9 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__4; +x_10 = l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg(x_9); return x_10; } default: @@ -25292,6 +25291,7 @@ return x_10; lean_object* x_11; lean_dec(x_4); lean_dec(x_2); +lean_dec(x_1); x_11 = lean_box(0); return x_11; } @@ -25319,92 +25319,117 @@ uint8_t x_16; x_16 = !lean_is_exclusive(x_3); 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_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; x_17 = lean_ctor_get(x_3, 0); x_18 = lean_ctor_get(x_4, 0); lean_inc(x_18); x_19 = lean_ctor_get(x_4, 1); lean_inc(x_19); lean_dec(x_4); +lean_inc(x_1); +lean_inc(x_19); +lean_inc(x_18); lean_inc(x_17); -x_20 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_18); -x_21 = l_Lean_PersistentArray_toList___rarg(x_19); +x_20 = lean_apply_3(x_1, x_17, x_18, x_19); +x_21 = lean_unbox(x_20); +lean_dec(x_20); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; +lean_dec(x_1); x_22 = lean_box(0); +x_23 = lean_apply_4(x_2, x_17, x_18, x_19, x_22); +lean_ctor_set(x_3, 0, x_23); +return x_3; +} +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_inc(x_17); +x_24 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_18); +x_25 = l_Lean_PersistentArray_toList___rarg(x_19); +x_26 = lean_box(0); lean_inc(x_2); -x_23 = l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4___rarg(x_1, x_2, x_20, x_21, x_22); -x_24 = lean_apply_4(x_2, x_17, x_18, x_19, x_23); -x_25 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +x_27 = l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg(x_1, x_2, x_24, x_25, x_26); +x_28 = lean_apply_4(x_2, x_17, x_18, x_19, x_27); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_28); +return x_29; +} } 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; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_26 = lean_ctor_get(x_3, 0); -lean_inc(x_26); +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_30 = lean_ctor_get(x_3, 0); +lean_inc(x_30); lean_dec(x_3); -x_27 = lean_ctor_get(x_4, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_4, 1); -lean_inc(x_28); +x_31 = lean_ctor_get(x_4, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_4, 1); +lean_inc(x_32); lean_dec(x_4); -lean_inc(x_26); -x_29 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_29, 0, x_26); -x_30 = l_Lean_Elab_Info_updateContext_x3f(x_29, x_27); -x_31 = l_Lean_PersistentArray_toList___rarg(x_28); -x_32 = lean_box(0); +lean_inc(x_1); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +x_33 = lean_apply_3(x_1, x_30, x_31, x_32); +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_dec(x_1); +x_35 = lean_box(0); +x_36 = lean_apply_4(x_2, x_30, x_31, x_32, x_35); +x_37 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_37, 0, x_36); +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; lean_object* x_44; +lean_inc(x_30); +x_38 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_38, 0, x_30); +x_39 = l_Lean_Elab_Info_updateContext_x3f(x_38, x_31); +x_40 = l_Lean_PersistentArray_toList___rarg(x_32); +x_41 = lean_box(0); lean_inc(x_2); -x_33 = l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4___rarg(x_1, x_2, x_30, x_31, x_32); -x_34 = lean_apply_4(x_2, x_26, x_27, x_28, x_33); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_34); -return x_35; +x_42 = l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg(x_1, x_2, x_39, x_40, x_41); +x_43 = lean_apply_4(x_2, x_30, x_31, x_32, x_42); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +return x_44; +} } } default: { -lean_object* x_36; +lean_object* x_45; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_36 = lean_box(0); -return x_36; -} -} -} -} +lean_dec(x_1); +x_45 = lean_box(0); +return x_45; } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___boxed), 4, 0); -return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg(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_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg(x_1, x_2, x_4, x_3); -return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___boxed), 3, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg), 4, 0); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; -x_4 = lean_box(0); +uint8_t x_4; +x_4 = 1; return x_4; } } @@ -25419,25 +25444,26 @@ return x_1; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg(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_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_4 = lean_alloc_closure((void*)(l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f_choose___rarg), 6, 2); lean_closure_set(x_4, 0, x_2); lean_closure_set(x_4, 1, x_3); -x_5 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___closed__1; -x_6 = l_Lean_Elab_InfoTree_visitM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg(x_5, x_4, x_1); -if (lean_obj_tag(x_6) == 0) +x_5 = lean_box(0); +x_6 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___closed__1; +x_7 = l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg(x_6, x_4, x_5, x_1); +if (lean_obj_tag(x_7) == 0) { -lean_object* x_7; -x_7 = lean_box(0); -return x_7; +lean_object* x_8; +x_8 = lean_box(0); +return x_8; } else { -lean_object* x_8; -x_8 = lean_ctor_get(x_6, 0); -lean_inc(x_8); -lean_dec(x_6); -return x_8; +lean_object* x_9; +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +return x_9; } } } @@ -25449,42 +25475,16 @@ x_2 = lean_alloc_closure((void*)(l___private_Lean_Server_Completion_0__Lean_Serv return x_2; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4___rarg___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_List_mapM_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__4___rarg(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_1); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___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_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg(x_1, x_2, x_3, x_4); -lean_dec(x_1); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_Elab_InfoTree_visitM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg(x_1, x_2, x_3); -lean_dec(x_1); -return x_4; -} -} LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; +uint8_t x_4; lean_object* x_5; x_4 = l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -return x_4; +x_5 = lean_box(x_4); +return x_5; } } LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_0__Lean_Server_Completion_findClosestInfoWithLocalContextAt_x3f_isBetter(lean_object* x_1, lean_object* x_2) { @@ -29447,7 +29447,7 @@ return x_53; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___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) { _start: { lean_object* x_7; uint8_t x_8; @@ -29729,24 +29729,24 @@ uint8_t x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_3 = lean_ctor_get_uint8(x_1, sizeof(void*)*1); x_4 = lean_ctor_get(x_1, 0); lean_inc(x_4); -x_5 = lean_array_get_size(x_4); -x_6 = lean_mk_empty_array_with_capacity(x_5); -x_7 = lean_unsigned_to_nat(0u); -x_8 = l_Array_mapIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__1(x_1, x_4, x_5, x_7, lean_box(0), x_6); -lean_dec(x_4); if (lean_is_exclusive(x_1)) { lean_ctor_release(x_1, 0); - x_9 = x_1; + x_5 = x_1; } else { lean_dec_ref(x_1); - x_9 = lean_box(0); + x_5 = lean_box(0); } -x_10 = lean_array_get_size(x_8); +x_6 = lean_array_get_size(x_4); +x_7 = lean_mk_empty_array_with_capacity(x_6); +x_8 = lean_unsigned_to_nat(0u); +x_9 = l_Array_mapFinIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__1(x_4, x_4, x_6, x_8, lean_box(0), x_7); +lean_dec(x_4); +x_10 = lean_array_get_size(x_9); x_11 = lean_unsigned_to_nat(1u); x_12 = lean_nat_sub(x_10, x_11); x_13 = lean_nat_dec_lt(x_12, x_10); lean_dec(x_10); -x_14 = lean_array_size(x_8); +x_14 = lean_array_size(x_9); x_15 = 0; if (x_13 == 0) { @@ -29778,7 +29778,7 @@ goto block_20; else { lean_object* x_27; lean_object* x_28; -x_27 = lean_array_fget(x_8, x_12); +x_27 = lean_array_fget(x_9, x_12); lean_dec(x_12); x_28 = lean_ctor_get(x_27, 5); lean_inc(x_28); @@ -29806,12 +29806,12 @@ goto block_20; lean_object* x_17; lean_object* x_18; lean_object* x_19; x_17 = lean_string_length(x_16); lean_dec(x_16); -x_18 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__2(x_17, x_14, x_15, x_8); +x_18 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__2(x_17, x_14, x_15, x_9); lean_dec(x_17); -if (lean_is_scalar(x_9)) { +if (lean_is_scalar(x_5)) { x_19 = lean_alloc_ctor(0, 1, 1); } else { - x_19 = x_9; + x_19 = x_5; } lean_ctor_set(x_19, 0, x_18); lean_ctor_set_uint8(x_19, sizeof(void*)*1, x_3); @@ -29840,11 +29840,11 @@ return x_1; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___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) { _start: { lean_object* x_7; -x_7 = l_Array_mapIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__1(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Array_mapFinIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__1(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_2); lean_dec(x_1); return x_7; @@ -30976,16 +30976,16 @@ l___private_Lean_Server_Completion_0__Lean_Server_Completion_optionCompletion___ lean_mark_persistent(l___private_Lean_Server_Completion_0__Lean_Server_Completion_optionCompletion___closed__6); l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_tacticCompletion___spec__1___boxed__const__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_tacticCompletion___spec__1___boxed__const__1(); lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_tacticCompletion___spec__1___boxed__const__1); -l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg___closed__1 = _init_l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg___closed__1(); -lean_mark_persistent(l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__3___rarg___closed__1); -l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1); -l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__2(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__2); -l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__3(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__3); -l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__4(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__4); +l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1 = _init_l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1(); +lean_mark_persistent(l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__2___rarg___closed__1); +l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__1(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__1); +l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__2(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__2); +l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__3(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__3); +l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__4(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___spec__1___rarg___closed__4); l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___closed__1 = _init_l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___closed__1(); lean_mark_persistent(l___private_Lean_Server_Completion_0__Lean_Server_Completion_findBest_x3f___rarg___closed__1); l___private_Lean_Server_Completion_0__Lean_Server_Completion_findClosestInfoWithLocalContextAt_x3f___closed__1 = _init_l___private_Lean_Server_Completion_0__Lean_Server_Completion_findClosestInfoWithLocalContextAt_x3f___closed__1(); diff --git a/stage0/stdlib/Lean/Server/CompletionItemData.c b/stage0/stdlib/Lean/Server/CompletionItemData.c index 0ee0daac90c9..76668c813afe 100644 --- a/stage0/stdlib/Lean/Server/CompletionItemData.c +++ b/stage0/stdlib/Lean/Server/CompletionItemData.c @@ -23,6 +23,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Server_CompletionItemData_0__Lean_Lsp_ static lean_object* l___private_Lean_Server_CompletionItemData_0__Lean_Lsp_fromJsonCompletionItemData____x40_Lean_Server_CompletionItemData___hyg_15____closed__12; static lean_object* l___private_Lean_Server_CompletionItemData_0__Lean_Lsp_fromJsonCompletionItemData____x40_Lean_Server_CompletionItemData___hyg_15____closed__10; static lean_object* l___private_Lean_Server_CompletionItemData_0__Lean_Lsp_fromJsonCompletionItemData____x40_Lean_Server_CompletionItemData___hyg_15____closed__13; +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Lsp_CompletionItem_getFileSource_x21___closed__2; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_CompletionItemData_0__Lean_Lsp_fromJsonCompletionItemData____x40_Lean_Server_CompletionItemData___hyg_15____spec__1(lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); @@ -40,7 +41,6 @@ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2476_(lean_object*); static lean_object* l___private_Lean_Server_CompletionItemData_0__Lean_Lsp_fromJsonCompletionItemData____x40_Lean_Server_CompletionItemData___hyg_15____closed__5; -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_CompletionItemData_0__Lean_Lsp_toJsonCompletionItemData____x40_Lean_Server_CompletionItemData___hyg_82_(lean_object*); static lean_object* l_Lean_Lsp_CompletionItem_getFileSource_x21___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Server_CompletionItemData_0__Lean_Lsp_fromJsonCompletionItemData____x40_Lean_Server_CompletionItemData___hyg_15_(lean_object*); @@ -321,7 +321,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___private_Lean_Server_CompletionItemData_0__Lean_Lsp_toJsonCompletionItemData____x40_Lean_Server_CompletionItemData___hyg_82____closed__1; -x_9 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } diff --git a/stage0/stdlib/Lean/Server/FileWorker/RequestHandling.c b/stage0/stdlib/Lean/Server/FileWorker/RequestHandling.c index a36ad45017a6..552945b4b3aa 100644 --- a/stage0/stdlib/Lean/Server/FileWorker/RequestHandling.c +++ b/stage0/stdlib/Lean/Server/FileWorker/RequestHandling.c @@ -403,6 +403,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileW LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getTrailingSize(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12731____spec__7___lambda__1(lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___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*); extern lean_object* l_Lean_levelZero; @@ -493,7 +494,6 @@ 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_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12731_(lean_object*); static lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__8___closed__11; -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12731____spec__37___lambda__1(lean_object*); static lean_object* l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_fromJsonAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8744____closed__11; static lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12731____spec__2___closed__1; @@ -19925,7 +19925,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_handleCompletion___lambda__1___closed__1; -x_22 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); +x_22 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_20, x_21); x_23 = l_Lean_Json_mkObj(x_22); return x_23; } diff --git a/stage0/stdlib/Lean/Server/FileWorker/WidgetRequests.c b/stage0/stdlib/Lean/Server/FileWorker/WidgetRequests.c index c37c057dd348..128d1eb8ff7d 100644 --- a/stage0/stdlib/Lean/Server/FileWorker/WidgetRequests.c +++ b/stage0/stdlib/Lean/Server/FileWorker/WidgetRequests.c @@ -154,6 +154,7 @@ lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1387____spec__2___closed__1; static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1387____closed__2; LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1387____spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); extern lean_object* l_Lean_Lsp_instFromJsonLocationLink; static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_520____closed__6; extern lean_object* l_Lean_Widget_instRpcEncodableInteractiveTermGoal; @@ -179,7 +180,6 @@ LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodableInfoPopup_enc____x40_Lean static lean_object* l_Lean_Widget_instRpcEncodableGetGoToLocationParams___closed__2; static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_58____closed__33; lean_object* l_Lean_Server_instRpcEncodableWithRpcRefOfTypeName_rpcEncode___rarg(lean_object*, lean_object*, lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1450____spec__1___closed__1; static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_58____closed__26; static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_58____closed__12; @@ -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_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(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_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(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_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -4338,7 +4338,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_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -4573,7 +4573,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_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -4607,7 +4607,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_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } diff --git a/stage0/stdlib/Lean/Server/InfoUtils.c b/stage0/stdlib/Lean/Server/InfoUtils.c index 5977b9022882..01e0c6c57405 100644 --- a/stage0/stdlib/Lean/Server/InfoUtils.c +++ b/stage0/stdlib/Lean/Server/InfoUtils.c @@ -15,36 +15,31 @@ extern "C" { #endif LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); -LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__6___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_Meta_ppExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterMapTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_goalsAt_x3f(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtModule_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_InfoTree_goalsAt_x3f_isEmptyBy(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__11___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__1___boxed(lean_object*); -LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__7(lean_object*); static lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__21___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_PrettyPrinter_ppSignature(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__16___boxed(lean_object*, lean_object*, 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_Elab_InfoTree_visitM_go___rarg___closed__3; +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___spec__3(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlFromMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__15(lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_visitM_go___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__24___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); size_t lean_usize_shift_right(size_t, size_t); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__39___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_foldlM___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__17(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_smallestInfo_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__21___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__17___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12; LEAN_EXPORT lean_object* l_Lean_Elab_Info_isTerm___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_occursInside_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_docString_x3f___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -56,29 +51,27 @@ LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_ uint8_t l_List_all___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtModule_x3f___closed__5; LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__26___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_visitM_x27___spec__2___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___closed__1; +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__28___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_goalsAt_x3f___spec__8___boxed(lean_object*, lean_object*); uint8_t l_Lean_Exception_isInterrupt(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__38___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9; -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlFromMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_foldlM___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__14___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__49(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_foldInfo_go(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_getCompletionInfos(lean_object*); static lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__7___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__7___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__2(lean_object*); @@ -89,18 +82,17 @@ LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___lamb lean_object* l_Lean_findDocString_x3f(lean_object*, lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isApp(lean_object*); -LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__13___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); +LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12(lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapTR_loop___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__1___closed__4; +LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__53(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_foldInfo_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__12___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_foldlM___at_Lean_Elab_InfoTree_foldInfo_go___spec__14___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__37(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -123,11 +115,14 @@ LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f_h LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__22___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); static lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg___closed__2; +LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__17(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__22___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_List_mapTR_loop___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__1___closed__3; static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__1___closed__5; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__22(lean_object*); +LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__14(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__27___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_deepestNodes(lean_object*); @@ -143,7 +138,7 @@ extern lean_object* l_Lean_LocalContext_empty; LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__11(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__26___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__13___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__7___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__41(lean_object*, lean_object*, lean_object*); @@ -151,6 +146,7 @@ LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_ lean_object* l_Lean_instInhabitedPersistentArrayNode(lean_object*); lean_object* l_Lean_PersistentArray_toList___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__30(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___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_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__8___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__23___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_docString_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -160,7 +156,6 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldI LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_occursInOrOnBoundary___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__9(lean_object*); -LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlFromMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__15(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_docString_x3f___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -170,6 +165,7 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldI lean_object* l_Lean_Elab_CompletionInfo_stx(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__2(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_InfoTree_foldInfoTree_go___spec__11(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_smallestInfo_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__46(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__1___boxed(lean_object*, lean_object*, lean_object*); @@ -179,19 +175,17 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__18___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__4___closed__2; LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4(lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27(lean_object*); -LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__16___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f_isAtomicFormat___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_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_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__21(lean_object*); -static lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__19___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__19___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f(lean_object*, lean_object*, lean_object*); @@ -205,6 +199,7 @@ size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__9(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__7___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_deepestNodes___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__52(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__11(lean_object*); LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_goalsAt_x3f___spec__7(lean_object*); @@ -231,6 +226,7 @@ LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_goa LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__23___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Info_docString_x3f___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_PersistentArray_foldlM___at_Lean_Elab_InfoTree_foldInfo_go___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__1___closed__8; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__21___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_goalsAt_x3f___spec__8(lean_object*, lean_object*); @@ -238,16 +234,15 @@ static lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__2 LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__25(lean_object*); LEAN_EXPORT lean_object* l_List_filterMapTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__7(lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_visitM_x27___spec__2(lean_object*); LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__10(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__13(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__13(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__14(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_range_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__4(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__23___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Info_updateContext_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__1___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_go___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__11___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_type_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -267,17 +262,17 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldI lean_object* l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__13(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__18___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__17___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__20(lean_object*); +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__30___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getKind(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_isSmaller___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_goalsAt_x3f___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_CompletionInfo_lctx(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__10(lean_object*); -LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__54(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__7___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__23(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__17___boxed(lean_object*, lean_object*, lean_object*); @@ -317,6 +312,7 @@ static lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArra LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__42___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__8___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__6(lean_object*); +static lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlFromMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__15___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_InfoTree_getCompletionInfos___closed__1; LEAN_EXPORT lean_object* l_Array_getMax_x3f___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__2(lean_object*); @@ -326,7 +322,7 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldI lean_object* l_Lean_Expr_constName_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__22(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__19(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapTR_loop___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__1___closed__1; static lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__4___closed__6; LEAN_EXPORT lean_object* l_Lean_PersistentArray_foldlM___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__14(lean_object*); @@ -334,13 +330,14 @@ static lean_object* l_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___closed__2 LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___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_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__26___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__48(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__16(lean_object*); static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtModule_x3f___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__3___boxed(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_InfoTree_foldInfoTree_go___spec__4(lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); -static lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__24(lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__7___closed__1; @@ -352,8 +349,8 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldI LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__17___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f___lambda__4___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_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__1___closed__6; +LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__1(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_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__50___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__50(lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -369,45 +366,50 @@ uint8_t l_Lean_Syntax_isIdent(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__19___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__1(lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8; +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__23(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__18___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__10___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__51(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11; +LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__7___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__4___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__3(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_usize_to_nat(size_t); LEAN_EXPORT lean_object* l_Lean_Elab_Info_pos_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_docString_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__33___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__35___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassApp_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__2(lean_object*); +LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__43___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__4___closed__3; +LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_userName(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__23(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__13___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_foldlM___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__14___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__40(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5(lean_object*); lean_object* l_panic___at_Lean_Parser_ParserState_mkUnexpectedTokenErrors___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_smallestInfo_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__2; +static lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Info_docString_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__47(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__33(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17___boxed(lean_object*, lean_object*); uint8_t l_Lean_Syntax_isToken(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_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_365____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__22___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -415,7 +417,6 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry uint8_t l_Lean_Name_hasMacroScopes(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__26___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_visitM_x27___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__16___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_lexOrd___elambda__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_termGoalAt_x3f(lean_object*, lean_object*); @@ -423,10 +424,12 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldI uint8_t l_String_Range_contains(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__44(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg___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_InfoTree_visitM_go___rarg___closed__4; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__28(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__6(lean_object*, lean_object*, lean_object*); +static lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__2; LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__26(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__8(lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -435,7 +438,6 @@ static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtModule_x3f___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__19___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__10___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_go___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__35(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_deepestNodes___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -447,8 +449,8 @@ lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__38(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__34___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_goalsAt_x3f_isEmptyBy___boxed(lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__10___rarg___boxed(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_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__9___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__43(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -463,14 +465,16 @@ LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_Persisten LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__2(lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3(lean_object*); +LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__11___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__6___rarg___boxed(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_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__7(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__6(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlFromMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__15___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6(lean_object*); uint8_t l_instDecidableRelLe___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__12___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__46___boxed(lean_object*, lean_object*, lean_object*); @@ -482,12 +486,12 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldI LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__25(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_goalsAt_x3f___lambda__1___boxed(lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_int_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__12___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_getCompletionInfos___lambda__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6___rarg___boxed(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_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__24(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__36___boxed(lean_object*, lean_object*, lean_object*); @@ -500,22 +504,19 @@ lean_object* l_Lean_Elab_TermInfo_runMetaM___rarg(lean_object*, lean_object*, le LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__6___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__55(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__2(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_range_x3f(lean_object*); static lean_object* l_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__14(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_deepestNodes___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlFromMAux___at_Lean_Elab_InfoTree_foldInfo_go___spec__2___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_List_foldl___at_Array_appendList___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Info_fmtHover_x3f_fmtModule_x3f___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__7(lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__13___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_Environment_getModuleIdxFor_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__18(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_InfoTree_goalsAt_x3f___spec__6(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_visitM_go___spec__1(lean_object*, lean_object*); @@ -527,7 +528,7 @@ uint8_t l_Lean_Syntax_structEq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_foldlM___at_Lean_Elab_InfoTree_foldInfo_go___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_InfoTree_goalsAt_x3f___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__21___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Elab_InfoTree_goalsAt_x3f___spec__9___boxed(lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); @@ -550,7 +551,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Info_lctx(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__25___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_getMax_x3f___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__2___boxed(lean_object*); -LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__20___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_goalsAt_x3f_hasNestedTactic___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -564,9 +564,10 @@ 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_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__39(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_foldInfoTree___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__1___closed__3; +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__22___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__18(lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -585,12 +586,12 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry lean_object* l_Lean_RBNode_find___at_Lean_NameMap_find_x3f___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__7(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__12(lean_object*); -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_PersistentArray_0__Lean_PersistentArray_foldlFromMAux___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__2___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__24(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_goalsAt_x3f___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); static lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__1___closed__4; +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__2___boxed(lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Elab_InfoTree_hasSorry_go___spec__42(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t); @@ -621,10 +622,8 @@ uint8_t l_Lean_Expr_isSyntheticSorry(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalContext_findFVar_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfoTree_go___spec__25___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_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_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__2___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_stx___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__26___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__34(lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -632,7 +631,6 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyM___at_Lean_Elab_InfoTree_hasSorry_go___spec__36(lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_foldInfo(lean_object*); -LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__20(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__5(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTermAndModule_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Info_contains(lean_object*, lean_object*, uint8_t); @@ -750,29 +748,43 @@ x_10 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_8, x_9); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg___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_Lean_Elab_InfoTree_visitM_go___rarg___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, uint8_t 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; +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_dec(x_7); +x_9 = lean_box(0); +x_10 = lean_apply_4(x_1, x_2, x_3, x_4, x_9); +x_11 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__1), 2, 1); +lean_closure_set(x_11, 0, x_5); +x_12 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_10, x_11); +return x_12; +} +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; +lean_inc(x_2); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_2); +x_14 = l_Lean_Elab_Info_updateContext_x3f(x_13, x_3); +x_15 = l_Lean_PersistentArray_toList___rarg(x_4); +x_16 = lean_box(0); lean_inc(x_1); -x_9 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_9, 0, x_1); -x_10 = l_Lean_Elab_Info_updateContext_x3f(x_9, x_2); -x_11 = l_Lean_PersistentArray_toList___rarg(x_3); -x_12 = lean_box(0); +lean_inc(x_5); +x_17 = l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_go___spec__2___rarg(x_5, x_7, x_1, x_14, x_15, x_16); lean_inc(x_6); -lean_inc(x_4); -x_13 = l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_go___spec__2___rarg(x_4, x_5, x_6, x_10, x_11, x_12); -lean_inc(x_7); -x_14 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__2), 7, 6); -lean_closure_set(x_14, 0, x_6); -lean_closure_set(x_14, 1, x_1); -lean_closure_set(x_14, 2, x_2); -lean_closure_set(x_14, 3, x_3); -lean_closure_set(x_14, 4, x_4); -lean_closure_set(x_14, 5, x_7); -x_15 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_13, x_14); -return x_15; +x_18 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__2), 7, 6); +lean_closure_set(x_18, 0, x_1); +lean_closure_set(x_18, 1, x_2); +lean_closure_set(x_18, 2, x_3); +lean_closure_set(x_18, 3, x_4); +lean_closure_set(x_18, 4, x_5); +lean_closure_set(x_18, 5, x_6); +x_19 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_17, x_18); +return x_19; +} } } static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___rarg___closed__1() { @@ -805,7 +817,7 @@ static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___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_Lean_Elab_InfoTree_visitM_go___rarg___closed__1; x_2 = l_Lean_Elab_InfoTree_visitM_go___rarg___closed__2; -x_3 = lean_unsigned_to_nat(56u); +x_3 = lean_unsigned_to_nat(62u); x_4 = lean_unsigned_to_nat(21u); x_5 = l_Lean_Elab_InfoTree_visitM_go___rarg___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -895,13 +907,13 @@ lean_inc(x_20); x_24 = lean_apply_3(x_2, x_20, x_21, x_22); lean_inc(x_23); x_25 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__3___boxed), 8, 7); -lean_closure_set(x_25, 0, x_20); -lean_closure_set(x_25, 1, x_21); -lean_closure_set(x_25, 2, x_22); -lean_closure_set(x_25, 3, x_1); -lean_closure_set(x_25, 4, x_2); -lean_closure_set(x_25, 5, x_3); -lean_closure_set(x_25, 6, x_23); +lean_closure_set(x_25, 0, x_3); +lean_closure_set(x_25, 1, x_20); +lean_closure_set(x_25, 2, x_21); +lean_closure_set(x_25, 3, x_22); +lean_closure_set(x_25, 4, x_1); +lean_closure_set(x_25, 5, x_23); +lean_closure_set(x_25, 6, x_2); x_26 = lean_apply_4(x_23, lean_box(0), lean_box(0), x_24, x_25); return x_26; } @@ -937,18 +949,18 @@ return x_3; LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___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) { _start: { -lean_object* x_9; -x_9 = l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_8); lean_dec(x_8); -return x_9; +x_10 = l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9); +return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___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_5; lean_object* x_6; -x_5 = lean_box(0); -x_6 = l_Lean_Elab_InfoTree_visitM_go___rarg(x_1, x_2, x_3, x_5, x_4); +lean_object* x_6; +x_6 = l_Lean_Elab_InfoTree_visitM_go___rarg(x_1, x_2, x_3, x_4, x_5); return x_6; } } @@ -956,24 +968,251 @@ LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM(lean_object* x_1, lean_obje _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM___rarg), 4, 0); +x_3 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM___rarg), 5, 0); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_visitM_x27___spec__2___rarg(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_5; lean_object* x_6; -x_5 = lean_box(0); -x_6 = l_Lean_Elab_InfoTree_visitM_go___rarg(x_1, x_2, x_3, x_5, x_4); -return x_6; +lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_3 = lean_box(0); +x_4 = l_instInhabitedOfMonad___rarg(x_1, x_3); +x_5 = lean_panic_fn(x_4, x_2); +return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_visitM_x27___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_visitM_x27___spec__2(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg), 4, 0); +x_2 = lean_alloc_closure((void*)(l_panic___at_Lean_Elab_InfoTree_visitM_x27___spec__2___rarg), 2, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___spec__3___rarg___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; +x_8 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_1); +x_9 = l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___spec__3___rarg(x_2, x_3, x_4, x_5, x_6, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___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) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = l_List_reverse___rarg(x_6); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +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_5, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_5, 1); +lean_inc(x_12); +lean_dec(x_5); +x_13 = lean_ctor_get(x_1, 1); +lean_inc(x_13); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg(x_1, x_2, x_3, x_4, x_11); +x_15 = lean_alloc_closure((void*)(l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___spec__3___rarg___lambda__1), 7, 6); +lean_closure_set(x_15, 0, x_6); +lean_closure_set(x_15, 1, x_1); +lean_closure_set(x_15, 2, x_2); +lean_closure_set(x_15, 3, x_3); +lean_closure_set(x_15, 4, x_4); +lean_closure_set(x_15, 5, x_12); +x_16 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_14, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___spec__3(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___spec__3___rarg), 6, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg___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, uint8_t x_8) { +_start: +{ +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_dec(x_7); +x_9 = lean_box(0); +x_10 = lean_apply_4(x_1, x_2, x_3, x_4, x_9); +x_11 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__1), 2, 1); +lean_closure_set(x_11, 0, x_5); +x_12 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_10, x_11); +return x_12; +} +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; +lean_inc(x_2); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_2); +x_14 = l_Lean_Elab_Info_updateContext_x3f(x_13, x_3); +x_15 = l_Lean_PersistentArray_toList___rarg(x_4); +x_16 = lean_box(0); +lean_inc(x_1); +lean_inc(x_5); +x_17 = l_List_mapM_loop___at_Lean_Elab_InfoTree_visitM_x27___spec__3___rarg(x_5, x_7, x_1, x_14, x_15, x_16); +lean_inc(x_6); +x_18 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___rarg___lambda__2), 7, 6); +lean_closure_set(x_18, 0, x_1); +lean_closure_set(x_18, 1, x_2); +lean_closure_set(x_18, 2, x_3); +lean_closure_set(x_18, 3, x_4); +lean_closure_set(x_18, 4, x_5); +lean_closure_set(x_18, 5, x_6); +x_19 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_17, x_18); +return x_19; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___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_4) == 0) +{ +switch (lean_obj_tag(x_5)) { +case 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_PartialContextInfo_mergeIntoOuter_x3f(x_6, x_4); +x_4 = x_8; +x_5 = x_7; +goto _start; +} +case 1: +{ +lean_object* x_10; lean_object* x_11; +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +x_10 = l_Lean_Elab_InfoTree_visitM_go___rarg___closed__4; +x_11 = l_panic___at_Lean_Elab_InfoTree_visitM_x27___spec__2___rarg(x_1, x_10); +return x_11; +} +default: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +lean_dec(x_1); +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_box(0); +x_15 = lean_apply_2(x_13, lean_box(0), x_14); +return x_15; +} +} +} +else +{ +switch (lean_obj_tag(x_5)) { +case 0: +{ +lean_object* x_16; lean_object* x_17; lean_object* 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 = l_Lean_Elab_PartialContextInfo_mergeIntoOuter_x3f(x_16, x_4); +x_4 = x_18; +x_5 = x_17; +goto _start; +} +case 1: +{ +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_4, 0); +lean_inc(x_20); +lean_dec(x_4); +x_21 = lean_ctor_get(x_5, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_5, 1); +lean_inc(x_22); +lean_dec(x_5); +x_23 = lean_ctor_get(x_1, 1); +lean_inc(x_23); +lean_inc(x_2); +lean_inc(x_22); +lean_inc(x_21); +lean_inc(x_20); +x_24 = lean_apply_3(x_2, x_20, x_21, x_22); +lean_inc(x_23); +x_25 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg___lambda__1___boxed), 8, 7); +lean_closure_set(x_25, 0, x_3); +lean_closure_set(x_25, 1, x_20); +lean_closure_set(x_25, 2, x_21); +lean_closure_set(x_25, 3, x_22); +lean_closure_set(x_25, 4, x_1); +lean_closure_set(x_25, 5, x_23); +lean_closure_set(x_25, 6, x_2); +x_26 = lean_apply_4(x_23, lean_box(0), lean_box(0), x_24, x_25); +return x_26; +} +default: +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_27 = lean_ctor_get(x_1, 0); +lean_inc(x_27); +lean_dec(x_1); +x_28 = lean_ctor_get(x_27, 1); +lean_inc(x_28); +lean_dec(x_27); +x_29 = lean_box(0); +x_30 = lean_apply_2(x_28, lean_box(0), x_29); +return x_30; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg), 5, 0); return x_2; } } @@ -985,34 +1224,44 @@ x_6 = lean_apply_3(x_1, x_2, x_3, x_4); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___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_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_5 = lean_ctor_get(x_1, 0); -lean_inc(x_5); -x_6 = lean_ctor_get(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; +x_6 = lean_ctor_get(x_1, 0); lean_inc(x_6); -lean_dec(x_5); -x_7 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___rarg___lambda__1___boxed), 5, 1); -lean_closure_set(x_7, 0, x_3); -x_8 = l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg(x_1, x_2, x_7, x_4); -x_9 = lean_ctor_get(x_6, 1); -lean_inc(x_9); +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); lean_dec(x_6); -x_10 = lean_box(0); -x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_10, x_8); -return x_11; +x_8 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___rarg___lambda__1___boxed), 5, 1); +lean_closure_set(x_8, 0, x_3); +x_9 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg(x_1, x_2, x_8, x_4, x_5); +x_10 = lean_ctor_get(x_7, 1); +lean_inc(x_10); +lean_dec(x_7); +x_11 = lean_box(0); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_11, x_9); +return x_12; } } LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___rarg), 4, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___rarg), 5, 0); return x_2; } } +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___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: +{ +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_8); +lean_dec(x_8); +x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_visitM_x27___spec__1___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9); +return x_10; +} +} LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -1070,7 +1319,7 @@ x_2 = lean_alloc_closure((void*)(l_List_filterMapTR_go___at_Lean_Elab_InfoTree_c return x_2; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2___rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2___rarg(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -1094,15 +1343,15 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_List_bindTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2___rarg), 2, 0); +x_2 = lean_alloc_closure((void*)(l_List_flatMapTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2___rarg), 2, 0); return x_2; } } -static lean_object* _init_l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg___closed__1() { +static lean_object* _init_l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -1112,24 +1361,24 @@ x_3 = l_instInhabitedOfMonad___rarg(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg(lean_object* x_1) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg___closed__1; +x_2 = l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___closed__1; x_3 = lean_panic_fn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5(lean_object* x_1) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg), 1, 0); +x_2 = lean_alloc_closure((void*)(l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg), 1, 0); return x_2; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6___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_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___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_4) == 0) @@ -1137,6 +1386,7 @@ if (lean_obj_tag(x_4) == 0) lean_object* x_6; lean_dec(x_3); lean_dec(x_2); +lean_dec(x_1); x_6 = l_List_reverse___rarg(x_5); return x_6; } @@ -1151,7 +1401,8 @@ x_8 = lean_ctor_get(x_4, 0); x_9 = lean_ctor_get(x_4, 1); lean_inc(x_3); lean_inc(x_2); -x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg(x_1, x_2, x_3, x_8); +lean_inc(x_1); +x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg(x_1, x_2, x_3, x_8); lean_ctor_set(x_4, 1, x_5); lean_ctor_set(x_4, 0, x_10); { @@ -1172,7 +1423,8 @@ lean_inc(x_12); lean_dec(x_4); lean_inc(x_3); lean_inc(x_2); -x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg(x_1, x_2, x_3, x_12); +lean_inc(x_1); +x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg(x_1, x_2, x_3, 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_5); @@ -1183,15 +1435,15 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6(lean_object* x_1) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6___rarg___boxed), 5, 0); +x_2 = lean_alloc_closure((void*)(l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_3) == 0) @@ -1215,8 +1467,9 @@ case 1: lean_object* x_9; lean_object* x_10; lean_dec(x_4); lean_dec(x_2); +lean_dec(x_1); x_9 = l_Lean_Elab_InfoTree_visitM_go___rarg___closed__4; -x_10 = l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg(x_9); +x_10 = l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg(x_9); return x_10; } default: @@ -1224,6 +1477,7 @@ return x_10; lean_object* x_11; lean_dec(x_4); lean_dec(x_2); +lean_dec(x_1); x_11 = lean_box(0); return x_11; } @@ -1251,92 +1505,117 @@ uint8_t x_16; x_16 = !lean_is_exclusive(x_3); 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_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; x_17 = lean_ctor_get(x_3, 0); x_18 = lean_ctor_get(x_4, 0); lean_inc(x_18); x_19 = lean_ctor_get(x_4, 1); lean_inc(x_19); lean_dec(x_4); +lean_inc(x_1); +lean_inc(x_19); +lean_inc(x_18); lean_inc(x_17); -x_20 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_18); -x_21 = l_Lean_PersistentArray_toList___rarg(x_19); +x_20 = lean_apply_3(x_1, x_17, x_18, x_19); +x_21 = lean_unbox(x_20); +lean_dec(x_20); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; +lean_dec(x_1); x_22 = lean_box(0); +x_23 = lean_apply_4(x_2, x_17, x_18, x_19, x_22); +lean_ctor_set(x_3, 0, x_23); +return x_3; +} +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_inc(x_17); +x_24 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_18); +x_25 = l_Lean_PersistentArray_toList___rarg(x_19); +x_26 = lean_box(0); lean_inc(x_2); -x_23 = l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6___rarg(x_1, x_2, x_20, x_21, x_22); -x_24 = lean_apply_4(x_2, x_17, x_18, x_19, x_23); -x_25 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +x_27 = l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg(x_1, x_2, x_24, x_25, x_26); +x_28 = lean_apply_4(x_2, x_17, x_18, x_19, x_27); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_28); +return x_29; +} } 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; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_26 = lean_ctor_get(x_3, 0); -lean_inc(x_26); +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_30 = lean_ctor_get(x_3, 0); +lean_inc(x_30); lean_dec(x_3); -x_27 = lean_ctor_get(x_4, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_4, 1); -lean_inc(x_28); +x_31 = lean_ctor_get(x_4, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_4, 1); +lean_inc(x_32); lean_dec(x_4); -lean_inc(x_26); -x_29 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_29, 0, x_26); -x_30 = l_Lean_Elab_Info_updateContext_x3f(x_29, x_27); -x_31 = l_Lean_PersistentArray_toList___rarg(x_28); -x_32 = lean_box(0); +lean_inc(x_1); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +x_33 = lean_apply_3(x_1, x_30, x_31, x_32); +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_dec(x_1); +x_35 = lean_box(0); +x_36 = lean_apply_4(x_2, x_30, x_31, x_32, x_35); +x_37 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_37, 0, x_36); +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; lean_object* x_44; +lean_inc(x_30); +x_38 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_38, 0, x_30); +x_39 = l_Lean_Elab_Info_updateContext_x3f(x_38, x_31); +x_40 = l_Lean_PersistentArray_toList___rarg(x_32); +x_41 = lean_box(0); lean_inc(x_2); -x_33 = l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6___rarg(x_1, x_2, x_30, x_31, x_32); -x_34 = lean_apply_4(x_2, x_26, x_27, x_28, x_33); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_34); -return x_35; +x_42 = l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg(x_1, x_2, x_39, x_40, x_41); +x_43 = lean_apply_4(x_2, x_30, x_31, x_32, x_42); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +return x_44; +} } } default: { -lean_object* x_36; +lean_object* x_45; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_36 = lean_box(0); -return x_36; +lean_dec(x_1); +x_45 = lean_box(0); +return x_45; } } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___boxed), 4, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg), 4, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___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_box(0); -x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg(x_1, x_2, x_4, x_3); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg___boxed), 3, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = lean_box(0); +uint8_t x_4; +x_4 = 1; return x_4; } } @@ -1355,7 +1634,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lamb lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; x_6 = l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__2___closed__1; x_7 = l_List_filterMapTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__1___rarg(x_5, x_6); -x_8 = l_List_bindTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2___rarg(x_7, x_6); +x_8 = l_List_flatMapTR_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__2___rarg(x_7, x_6); x_9 = lean_apply_4(x_1, x_2, x_3, x_4, x_8); return x_9; } @@ -1371,24 +1650,25 @@ return x_1; LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___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_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_3 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__2), 5, 1); lean_closure_set(x_3, 0, x_1); -x_4 = l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___closed__1; -x_5 = l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg(x_4, x_3, x_2); -if (lean_obj_tag(x_5) == 0) +x_4 = lean_box(0); +x_5 = l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___closed__1; +x_6 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg(x_5, x_3, x_4, x_2); +if (lean_obj_tag(x_6) == 0) { -lean_object* x_6; -x_6 = lean_box(0); -return x_6; +lean_object* x_7; +x_7 = lean_box(0); +return x_7; } else { -lean_object* x_7; -x_7 = lean_ctor_get(x_5, 0); -lean_inc(x_7); -lean_dec(x_5); -return x_7; +lean_object* x_8; +x_8 = lean_ctor_get(x_6, 0); +lean_inc(x_8); +lean_dec(x_6); +return x_8; } } } @@ -1400,42 +1680,16 @@ x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_collectNodesBottomUp___rar return x_2; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6___rarg___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_List_mapM_loop___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__6___rarg(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_1); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___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_InfoTree_visitM_go___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg(x_1, x_2, x_3, x_4); -lean_dec(x_1); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__3___rarg(x_1, x_2, x_3); -lean_dec(x_1); -return x_4; -} -} LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; +uint8_t x_4; lean_object* x_5; x_4 = l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__1(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -return x_4; +x_5 = lean_box(x_4); +return x_5; } } LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_deepestNodes___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { @@ -6510,7 +6764,7 @@ lean_dec(x_4); return x_5; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -6730,16 +6984,16 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__7(lean_object* x_1) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg___closed__1; +x_2 = l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___closed__1; x_3 = lean_panic_fn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8(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_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__7(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_4) == 0) @@ -6747,6 +7001,7 @@ if (lean_obj_tag(x_4) == 0) lean_object* x_6; lean_dec(x_3); lean_dec(x_2); +lean_dec(x_1); x_6 = l_List_reverse___rarg(x_5); return x_6; } @@ -6761,7 +7016,8 @@ x_8 = lean_ctor_get(x_4, 0); x_9 = lean_ctor_get(x_4, 1); lean_inc(x_3); lean_inc(x_2); -x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6(x_1, x_2, x_3, x_8); +lean_inc(x_1); +x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5(x_1, x_2, x_3, x_8); lean_ctor_set(x_4, 1, x_5); lean_ctor_set(x_4, 0, x_10); { @@ -6782,7 +7038,8 @@ lean_inc(x_12); lean_dec(x_4); lean_inc(x_3); lean_inc(x_2); -x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6(x_1, x_2, x_3, x_12); +lean_inc(x_1); +x_14 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5(x_1, x_2, x_3, 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_5); @@ -6793,7 +7050,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_3) == 0) @@ -6817,8 +7074,9 @@ case 1: lean_object* x_9; lean_object* x_10; lean_dec(x_4); lean_dec(x_2); +lean_dec(x_1); x_9 = l_Lean_Elab_InfoTree_visitM_go___rarg___closed__4; -x_10 = l_panic___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__7(x_9); +x_10 = l_panic___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6(x_9); return x_10; } default: @@ -6826,6 +7084,7 @@ return x_10; lean_object* x_11; lean_dec(x_4); lean_dec(x_2); +lean_dec(x_1); x_11 = lean_box(0); return x_11; } @@ -6853,72 +7112,105 @@ uint8_t x_16; x_16 = !lean_is_exclusive(x_3); 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_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; x_17 = lean_ctor_get(x_3, 0); x_18 = lean_ctor_get(x_4, 0); lean_inc(x_18); x_19 = lean_ctor_get(x_4, 1); lean_inc(x_19); lean_dec(x_4); +lean_inc(x_1); +lean_inc(x_19); +lean_inc(x_18); lean_inc(x_17); -x_20 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_18); -x_21 = l_Lean_PersistentArray_toList___rarg(x_19); +x_20 = lean_apply_3(x_1, x_17, x_18, x_19); +x_21 = lean_unbox(x_20); +lean_dec(x_20); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; +lean_dec(x_1); x_22 = lean_box(0); +x_23 = lean_apply_4(x_2, x_17, x_18, x_19, x_22); +lean_ctor_set(x_3, 0, x_23); +return x_3; +} +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_inc(x_17); +x_24 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_18); +x_25 = l_Lean_PersistentArray_toList___rarg(x_19); +x_26 = lean_box(0); lean_inc(x_2); -x_23 = l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8(x_1, x_2, x_20, x_21, x_22); -x_24 = lean_apply_4(x_2, x_17, x_18, x_19, x_23); -x_25 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +x_27 = l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__7(x_1, x_2, x_24, x_25, x_26); +x_28 = lean_apply_4(x_2, x_17, x_18, x_19, x_27); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_28); +return x_29; +} } 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; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_26 = lean_ctor_get(x_3, 0); -lean_inc(x_26); +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_30 = lean_ctor_get(x_3, 0); +lean_inc(x_30); lean_dec(x_3); -x_27 = lean_ctor_get(x_4, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_4, 1); -lean_inc(x_28); +x_31 = lean_ctor_get(x_4, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_4, 1); +lean_inc(x_32); lean_dec(x_4); -lean_inc(x_26); -x_29 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_29, 0, x_26); -x_30 = l_Lean_Elab_Info_updateContext_x3f(x_29, x_27); -x_31 = l_Lean_PersistentArray_toList___rarg(x_28); -x_32 = lean_box(0); +lean_inc(x_1); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +x_33 = lean_apply_3(x_1, x_30, x_31, x_32); +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_dec(x_1); +x_35 = lean_box(0); +x_36 = lean_apply_4(x_2, x_30, x_31, x_32, x_35); +x_37 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_37, 0, x_36); +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; lean_object* x_44; +lean_inc(x_30); +x_38 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_38, 0, x_30); +x_39 = l_Lean_Elab_Info_updateContext_x3f(x_38, x_31); +x_40 = l_Lean_PersistentArray_toList___rarg(x_32); +x_41 = lean_box(0); lean_inc(x_2); -x_33 = l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8(x_1, x_2, x_30, x_31, x_32); -x_34 = lean_apply_4(x_2, x_26, x_27, x_28, x_33); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_34); -return x_35; +x_42 = l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__7(x_1, x_2, x_39, x_40, x_41); +x_43 = lean_apply_4(x_2, x_30, x_31, x_32, x_42); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +return x_44; +} } } default: { -lean_object* x_36; +lean_object* x_45; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_36 = lean_box(0); -return x_36; -} -} +lean_dec(x_1); +x_45 = lean_box(0); +return x_45; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5(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_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6(x_1, x_2, x_4, x_3); -return x_5; } } -LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9(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; @@ -6955,7 +7247,7 @@ return x_10; } } } -LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__10(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; @@ -6992,7 +7284,7 @@ return x_10; } } } -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__1(lean_object* x_1) { _start: { lean_object* x_2; @@ -7001,7 +7293,7 @@ lean_inc(x_2); return x_2; } } -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__2(lean_object* x_1) { _start: { lean_object* x_2; @@ -7010,31 +7302,31 @@ lean_inc(x_2); return x_2; } } -static lean_object* _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__1() { +static lean_object* _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__1___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__1___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__2() { +static lean_object* _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__2___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__2___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9() { +static lean_object* _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__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_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__1; -x_2 = lean_alloc_closure((void*)(l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__10___boxed), 3, 1); +x_1 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__1; +x_2 = lean_alloc_closure((void*)(l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___boxed), 3, 1); lean_closure_set(x_2, 0, x_1); -x_3 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__2; -x_4 = lean_alloc_closure((void*)(l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11___boxed), 3, 1); +x_3 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__2; +x_4 = lean_alloc_closure((void*)(l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__10___boxed), 3, 1); lean_closure_set(x_4, 0, x_3); x_5 = lean_alloc_closure((void*)(l_lexOrd___elambda__1___rarg), 4, 2); lean_closure_set(x_5, 0, x_2); @@ -7042,7 +7334,7 @@ lean_closure_set(x_5, 1, x_4); return x_5; } } -LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__13(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12(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; @@ -7079,27 +7371,27 @@ return x_10; } } } -LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__14(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__13(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_inc(x_1); x_4 = lean_apply_1(x_1, x_2); x_5 = lean_apply_1(x_1, x_3); -x_6 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9; +x_6 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8; x_7 = lean_apply_2(x_6, x_4, x_5); return x_7; } } -static lean_object* _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12() { +static lean_object* _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__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_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__1; -x_2 = lean_alloc_closure((void*)(l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__13___boxed), 3, 1); +x_1 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__1; +x_2 = lean_alloc_closure((void*)(l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12___boxed), 3, 1); lean_closure_set(x_2, 0, x_1); -x_3 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__2; -x_4 = lean_alloc_closure((void*)(l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__14), 3, 1); +x_3 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__2; +x_4 = lean_alloc_closure((void*)(l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__13), 3, 1); lean_closure_set(x_4, 0, x_3); x_5 = lean_alloc_closure((void*)(l_lexOrd___elambda__1___rarg), 4, 2); lean_closure_set(x_5, 0, x_2); @@ -7107,7 +7399,7 @@ lean_closure_set(x_5, 1, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__14(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -7159,7 +7451,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_4) == 0) @@ -7195,7 +7487,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) @@ -7213,14 +7505,14 @@ lean_inc(x_5); x_6 = lean_ctor_get(x_3, 1); lean_inc(x_6); lean_dec(x_3); -x_7 = l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17(x_1, x_2, x_5, x_6); +x_7 = l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16(x_1, x_2, x_5, x_6); x_8 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_8, 0, x_7); return x_8; } } } -LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -7287,7 +7579,7 @@ return x_20; } } } -LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__20(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_4) == 0) @@ -7323,7 +7615,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) @@ -7341,7 +7633,7 @@ lean_inc(x_5); x_6 = lean_ctor_get(x_3, 1); lean_inc(x_6); lean_dec(x_3); -x_7 = l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__20(x_1, x_2, x_5, x_6); +x_7 = l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19(x_1, x_2, x_5, x_6); x_8 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_8, 0, x_7); return x_8; @@ -7827,7 +8119,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__7(le lean_object* x_9; lean_object* x_10; lean_object* x_11; x_9 = lean_box(0); x_10 = l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__2___closed__1; -x_11 = l_List_bindTR_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__1(x_8, x_10); +x_11 = l_List_flatMapTR_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__1(x_8, x_10); if (x_4 == 0) { lean_object* x_12; lean_object* x_13; @@ -7885,7 +8177,7 @@ x_3 = lean_ctor_get(x_2, 0); lean_inc(x_3); x_4 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_4, 0, x_3); -x_5 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18(x_4, x_1); +x_5 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17(x_4, x_1); lean_dec(x_4); return x_5; } @@ -7893,7 +8185,7 @@ return x_5; LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, uint8_t x_5) { _start: { -lean_object* x_6; 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_6; 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_14 = lean_box(x_3); x_15 = lean_box(x_5); x_16 = lean_box(x_4); @@ -7902,47 +8194,46 @@ lean_closure_set(x_17, 0, x_2); lean_closure_set(x_17, 1, x_14); lean_closure_set(x_17, 2, x_15); lean_closure_set(x_17, 3, x_16); -x_18 = l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___closed__1; -x_19 = l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5(x_18, x_17, x_1); -x_20 = lean_box(0); +x_18 = lean_box(0); +x_19 = l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___closed__1; +x_20 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5(x_19, x_17, x_18, x_1); x_21 = lean_box(0); -if (lean_obj_tag(x_19) == 0) +x_22 = lean_box(0); +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 = l_List_mapTR_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15(x_21, x_21); -x_23 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12; -x_24 = l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16(x_23, x_20, x_22); -x_25 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__8___boxed), 2, 1); -lean_closure_set(x_25, 0, x_24); -x_26 = l_List_find_x3f___rarg(x_25, x_21); -if (lean_obj_tag(x_26) == 0) +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_23 = l_List_mapTR_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__14(x_22, x_22); +x_24 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11; +x_25 = l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15(x_24, x_21, x_23); +x_26 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__8___boxed), 2, 1); +lean_closure_set(x_26, 0, x_25); +x_27 = l_List_find_x3f___rarg(x_26, x_22); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_27; -x_27 = lean_box(0); -x_6 = x_27; +x_6 = x_18; goto block_13; } else { uint8_t x_28; -x_28 = !lean_is_exclusive(x_26); +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_26, 0); +x_29 = lean_ctor_get(x_27, 0); x_30 = lean_ctor_get(x_29, 1); lean_inc(x_30); lean_dec(x_29); -lean_ctor_set(x_26, 0, x_30); -x_6 = x_26; +lean_ctor_set(x_27, 0, x_30); +x_6 = x_27; goto block_13; } else { lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_26, 0); +x_31 = lean_ctor_get(x_27, 0); lean_inc(x_31); -lean_dec(x_26); +lean_dec(x_27); x_32 = lean_ctor_get(x_31, 1); lean_inc(x_32); lean_dec(x_31); @@ -7956,50 +8247,48 @@ goto block_13; 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_19, 0); +x_34 = lean_ctor_get(x_20, 0); lean_inc(x_34); -lean_dec(x_19); +lean_dec(x_20); lean_inc(x_34); -x_35 = l_List_mapTR_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15(x_34, x_21); -x_36 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12; -x_37 = l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19(x_36, x_20, x_35); +x_35 = l_List_mapTR_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__14(x_34, x_22); +x_36 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11; +x_37 = l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18(x_36, x_21, x_35); x_38 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__8___boxed), 2, 1); lean_closure_set(x_38, 0, x_37); x_39 = l_List_find_x3f___rarg(x_38, x_34); if (lean_obj_tag(x_39) == 0) { -lean_object* x_40; -x_40 = lean_box(0); -x_6 = x_40; +x_6 = x_18; goto block_13; } else { -uint8_t x_41; -x_41 = !lean_is_exclusive(x_39); -if (x_41 == 0) +uint8_t x_40; +x_40 = !lean_is_exclusive(x_39); +if (x_40 == 0) { -lean_object* x_42; lean_object* x_43; -x_42 = lean_ctor_get(x_39, 0); -x_43 = lean_ctor_get(x_42, 1); -lean_inc(x_43); -lean_dec(x_42); -lean_ctor_set(x_39, 0, x_43); +lean_object* x_41; lean_object* x_42; +x_41 = lean_ctor_get(x_39, 0); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +lean_ctor_set(x_39, 0, x_42); x_6 = x_39; goto block_13; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_39, 0); -lean_inc(x_44); +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_39, 0); +lean_inc(x_43); lean_dec(x_39); -x_45 = lean_ctor_get(x_44, 1); -lean_inc(x_45); -lean_dec(x_44); -x_46 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_46, 0, x_45); -x_6 = 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_6 = x_45; goto block_13; } } @@ -8050,121 +8339,94 @@ return x_6; } } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___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_List_mapM_loop___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_1); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6___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_InfoTree_visitM_go___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__6(x_1, x_2, x_3, x_4); -lean_dec(x_1); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_Elab_InfoTree_visitM___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__5(x_1, x_2, x_3); -lean_dec(x_1); -return x_4; -} -} -LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__10(x_1, x_2, x_3); +x_4 = l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9(x_1, x_2, x_3); x_5 = lean_box(x_4); return x_5; } } -LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11(x_1, x_2, x_3); +x_4 = l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__10(x_1, x_2, x_3); x_5 = lean_box(x_4); return x_5; } } -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__1___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__1___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__1(x_1); +x_2 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__1(x_1); lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__2___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__2___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___lambda__2(x_1); +x_2 = l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___lambda__2(x_1); lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; -x_4 = l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__13(x_1, x_2, x_3); +x_4 = l_compareOn___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12(x_1, x_2, x_3); x_5 = lean_box(x_4); return x_5; } } -LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16___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_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17(x_1, x_2, x_3, x_4); +x_5 = l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16(x_1, x_2, x_3, x_4); lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__16(x_1, x_2, x_3); +x_4 = l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__15(x_1, x_2, x_3); lean_dec(x_2); return x_4; } } -LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18(x_1, x_2); +x_3 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__17(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_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19___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_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__20(x_1, x_2, x_3, x_4); +x_5 = l_List_foldl___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19(x_1, x_2, x_3, x_4); lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__19(x_1, x_2, x_3); +x_4 = l_List_max_x3f___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__18(x_1, x_2, x_3); lean_dec(x_2); return x_4; } @@ -19514,8 +19776,8 @@ l_Lean_Elab_InfoTree_visitM_go___rarg___closed__3 = _init_l_Lean_Elab_InfoTree_v lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___rarg___closed__3); l_Lean_Elab_InfoTree_visitM_go___rarg___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___rarg___closed__4(); lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___rarg___closed__4); -l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg___closed__1 = _init_l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg___closed__1(); -lean_mark_persistent(l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__5___rarg___closed__1); +l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___closed__1 = _init_l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___closed__1(); +lean_mark_persistent(l_panic___at_Lean_Elab_InfoTree_collectNodesBottomUp___spec__4___rarg___closed__1); l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__2___closed__1 = _init_l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___lambda__2___closed__1); l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___closed__1 = _init_l_Lean_Elab_InfoTree_collectNodesBottomUp___rarg___closed__1(); @@ -19532,14 +19794,14 @@ l_List_mapTR_loop___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__1___closed__3 lean_mark_persistent(l_List_mapTR_loop___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__1___closed__3); l_List_mapTR_loop___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__1___closed__4 = _init_l_List_mapTR_loop___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__1___closed__4(); lean_mark_persistent(l_List_mapTR_loop___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__1___closed__4); -l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__1 = _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__1(); -lean_mark_persistent(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__1); -l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__2 = _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__2(); -lean_mark_persistent(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9___closed__2); -l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9 = _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9(); -lean_mark_persistent(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__9); -l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12 = _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12(); -lean_mark_persistent(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__12); +l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__1 = _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__1(); +lean_mark_persistent(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__1); +l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__2 = _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__2(); +lean_mark_persistent(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8___closed__2); +l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8 = _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8(); +lean_mark_persistent(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__8); +l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11 = _init_l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11(); +lean_mark_persistent(l_lexOrd___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__11); l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__4___closed__1 = _init_l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__4___closed__1(); lean_mark_persistent(l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__4___closed__1); l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__4___closed__2 = _init_l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__4___closed__2(); diff --git a/stage0/stdlib/Lean/Server/References.c b/stage0/stdlib/Lean/Server/References.c index e74881e3b117..eace061f0f84 100644 --- a/stage0/stdlib/Lean/Server/References.c +++ b/stage0/stdlib/Lean/Server/References.c @@ -20,13 +20,11 @@ lean_object* l_Lean_JsonNumber_fromNat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_findDeclarationRanges_x3f___at_Lean_Server_RefInfo_toLspRefInfo___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Lsp_RefIdent_toJson(lean_object*); -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Server_combineIdents_buildIdMap___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_definitionsMatching___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Server_References_removeIlean___spec__3(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_2012____spec__1(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_References_allRefsFor___spec__3___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_useConstRepresentatives___spec__26(size_t, lean_object*, lean_object*, size_t, size_t, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_RefInfo_empty; lean_object* l_instBEqOfDecidableEq___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_References_allRefs___spec__6___boxed(lean_object*, lean_object*); @@ -35,6 +33,7 @@ lean_object* l_Lean_Json_compress(lean_object*); static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_References_addIlean___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isRec___at_Lean_Server_RefInfo_toLspRefInfo___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_IO_throwServerError___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_findAt(lean_object*, lean_object*, lean_object*, uint8_t); uint8_t l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_beqRange____x40_Lean_Data_Lsp_Basic___hyg_627_(lean_object*, lean_object*); @@ -43,6 +42,7 @@ uint64_t l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_hashRefIdent____x40_Lean LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_allRefs___spec__10(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_allRefsFor___spec__5(lean_object*, size_t, size_t, lean_object*); static lean_object* l_List_mapTR_loop___at___private_Lean_Server_References_0__Lean_Server_toJsonIlean____x40_Lean_Server_References___hyg_1478____spec__2___closed__3; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_References_allRefs___spec__3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_dedupReferences___closed__2; static lean_object* l_Lean_Server_findModuleRefs___closed__2; @@ -50,14 +50,15 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Ser LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_useConstRepresentatives___spec__24(size_t, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_References_removeWorkerRefs___spec__1___boxed(lean_object*, lean_object*); lean_object* l_Lean_Json_mkObj(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_declRangeExt; static lean_object* l_Lean_Server_dedupReferences___closed__11; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_useConstRepresentatives___spec__23(size_t, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_dedupReferences(lean_object*, uint8_t); static lean_object* l_Lean_Server_dedupReferences___closed__10; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_definitionsMatching___spec__5(lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_Syntax_getHeadInfo(lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_ModuleRefs_addRef___spec__6(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_allRefs___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_References_updateWorkerRefs___spec__6(lean_object*, lean_object*, lean_object*); @@ -91,7 +92,6 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Ser lean_object* l_Array_qpartition___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_References_definitionOf_x3f___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_References_allRefsFor___spec__7___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Server_combineIdents_buildIdMap___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_RefInfo_toLspRefInfo___spec__6___closed__3; lean_object* lean_mk_array(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_combineIdents_buildIdMap___spec__1___boxed(lean_object*, lean_object*); @@ -107,20 +107,19 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_findModuleRe static lean_object* l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__10___closed__1; static lean_object* l_Lean_Server_dedupReferences___closed__6; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_RefInfo_toLspRefInfo___spec__6(size_t, size_t, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_panic___at_Lean_Server_combineIdents_buildIdMap___spec__6(lean_object*, lean_object*); extern lean_object* l_Lean_Lsp_instOrdPosition; 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_List_forIn_loop___at_Lean_Server_References_definitionsMatching___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_combineIdents___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_removeIlean___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__5; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__10(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_combineIdents_useConstRepresentatives___spec__12(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_combineIdents_useConstRepresentatives___spec__6(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_dedupReferences___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___boxed(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_References_allRefs___spec__6(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_allRefs___spec__11(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Lsp_ModuleRefs_findRange_x3f___spec__3(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); @@ -129,19 +128,20 @@ lean_object* l_System_Uri_pathToUri(lean_object*); LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Server_ModuleRefs_toLspModuleRefs___spec__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_combineIdents_useConstRepresentatives___spec__9(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Lsp_ModuleRefs_findAt___spec__2(lean_object*, uint8_t, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_useConstRepresentatives___spec__21(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_combineIdents_useConstRepresentatives___spec__18(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_findRange_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Lsp_ModuleRefs_findRange_x3f___spec__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_References_0__Lean_Server_toJsonIlean____x40_Lean_Server_References___hyg_1478____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_References_allRefsFor___spec__4___boxed(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_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_combineIdents_buildIdMap___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_combineIdents_buildIdMap___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_instDecidableRelLt___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_ModuleRefs_findRange_x3f___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Server_References_removeIlean___spec__4(lean_object*, lean_object*); static lean_object* l_Lean_Lsp_RefInfo_findReferenceLocation_x3f___lambda__2___closed__1; +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__14; lean_object* l_EStateM_instMonad(lean_object*, lean_object*); lean_object* l_Lean_PersistentArray_toList___rarg(lean_object*); @@ -175,19 +175,19 @@ LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_References_definitio lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__6; LEAN_EXPORT lean_object* l_Lean_Server_findModuleRefs(lean_object*, lean_object*, uint8_t, uint8_t); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__2(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_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__1; LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__10___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_References_definitionsMatching___spec__6___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_instToJsonIlean___closed__1; size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_findModuleRefs___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Server_combineIdents_buildIdMap___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_TagDeclarationExtension_isTagged(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_findModuleRefs___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_findAt___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Lsp_ModuleRefs_findAt___spec__4(lean_object*, size_t, size_t, lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_ModuleRefs_findAt(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_useConstRepresentatives___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_RefInfo_findReferenceLocation_x3f(lean_object*, lean_object*, uint8_t); @@ -195,18 +195,19 @@ LEAN_EXPORT lean_object* l_Lean_Lsp_RefInfo_contains___boxed(lean_object*, lean_ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_combineIdents_useConstRepresentatives___spec__12___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_definitionsMatching(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Lsp_ModuleRefs_findRange_x3f___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Server_combineIdents_findCanonicalRepresentative___spec__3(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_findDeclarationRangesCore_x3f___at_Lean_Server_RefInfo_toLspRefInfo___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_empty; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__17; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_References_allRefsFor___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_panic___at_Lean_Server_findReferences___spec__4___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_buildIdMap___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Server_References_0__Lean_Server_toJsonIlean____x40_Lean_Server_References___hyg_1478____spec__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_finalizeWorkerRefs___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Server_References_updateWorkerRefs___spec__9___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_panic___at_Lean_Server_findReferences___spec__3___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_removeIlean___spec__7(lean_object*, size_t, size_t, lean_object*); uint64_t lean_uint64_shift_right(uint64_t, uint64_t); static uint64_t l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_dedupReferences___spec__4___at_Lean_Server_dedupReferences___spec__5___closed__2; @@ -260,6 +261,7 @@ lean_object* l_instDecidableEqBool___boxed(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_References_allRefs___spec__1(lean_object*, lean_object*); static lean_object* l_List_mapTR_loop___at___private_Lean_Server_References_0__Lean_Server_toJsonIlean____x40_Lean_Server_References___hyg_1478____spec__2___closed__2; static lean_object* l_Lean_Server_dedupReferences___closed__4; +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__4; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_References_definitionsMatching___spec__3(lean_object*); static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__16; LEAN_EXPORT lean_object* l_Lean_Server_combineIdents_findCanonicalRepresentative(lean_object*, lean_object*); @@ -283,7 +285,9 @@ static lean_object* l_Lean_Server_ModuleRefs_toLspModuleRefs___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_useConstRepresentatives___spec__26___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_References_definitionOf_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_References_allRefsFor___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7(lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_updateWorkerRefs___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*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__2; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Lsp_ModuleRefs_findRange_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_ModuleRefs_toLspModuleRefs___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_ModuleRefs_toLspModuleRefs___spec__1(lean_object*, lean_object*); @@ -299,7 +303,6 @@ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Server_Ilean_load___closed__2; lean_object* l_Lean_MapDeclarationExtension_find_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_RefInfo_addRef(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_panic___at_Lean_Server_findReferences___spec__4(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_findReferences___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_References_allRefs___spec__5(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_References_allRefs___spec__4(lean_object*, lean_object*); @@ -309,6 +312,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_Ilean_load(lean_object*, lean_object*); extern lean_object* l_instMonadBaseIO; static size_t l_Lean_Server_References_allRefsFor___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Server_combineIdents_buildIdMap___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_forInStep_go___at_Lean_Server_combineIdents_useConstRepresentatives___spec__14(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_Lean_Lsp_RefInfo_empty___closed__1; @@ -321,7 +325,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_References_re LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Server_References_removeIlean___spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_combineIdents_buildIdMap___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Server_ModuleRefs_addRef___spec__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Server_findReferences___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_References_allRefsFor___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_forInStep_go___at_Lean_Server_combineIdents_useConstRepresentatives___spec__20(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_References_addIlean___spec__2(lean_object*); @@ -341,15 +344,14 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get___at_Lean_Server_ LEAN_EXPORT lean_object* l_Lean_Server_ModuleRefs_toLspModuleRefs(lean_object*, lean_object*); extern lean_object* l_Lean_Lsp_instHashableRefIdent; static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__21; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_getModuleContainingDecl_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_References_allRefs___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Server_References_removeIlean___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_allRefs(lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_RefInfo_toLspRefInfo___spec__6___closed__2; lean_object* l_IO_FS_readFile(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_References_addIlean___spec__4(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8(lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_ModuleRefs_toLspModuleRefs___spec__4(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_References_0__Lean_Server_toJsonIlean____x40_Lean_Server_References___hyg_1478_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_definitionOf_x3f(lean_object*, lean_object*, lean_object*, lean_object*); @@ -359,11 +361,9 @@ LEAN_EXPORT lean_object* l_Lean_findDeclarationRanges_x3f___at_Lean_Server_RefIn static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__4; LEAN_EXPORT lean_object* l_Lean_Server_combineIdents_useConstRepresentatives(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_combineIdents_buildIdMap(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_References_findAt___lambda__1___boxed(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*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_definitionsMatching___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_panic___at_Lean_Server_findReferences___spec__4___closed__2; lean_object* l_StateT_instMonad___rarg(lean_object*); lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodableArray___spec__2(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_combineIdents_findCanonicalRepresentative___boxed(lean_object*, lean_object*); @@ -378,6 +378,7 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdent LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_ModuleRefs_toLspModuleRefs___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_combineIdents_findCanonicalRepresentative___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Server_combineIdents_findCanonicalRepresentative___spec__3___boxed(lean_object*, lean_object*); +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_useConstRepresentatives___spec__27___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_combineIdents_useConstRepresentatives___spec__1___boxed(lean_object*, lean_object*); lean_object* l_Std_Internal_Parsec_String_Parser_run___rarg(lean_object*, lean_object*); @@ -388,6 +389,7 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Ser LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_References_allRefsFor___spec__7(lean_object*, lean_object*); static lean_object* l_Lean_Server_References_findAt___closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_dedupReferences___spec__7(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__18; uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_PrettyPrinter_delabCore___spec__3(lean_object*, lean_object*); @@ -424,7 +426,6 @@ static lean_object* l_Lean_Server_dedupReferences___closed__1; extern lean_object* l_Lean_Lsp_instBEqRefIdent; lean_object* lean_panic_fn(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_dedupReferences___spec__4(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__2___boxed(lean_object*, 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_AssocList_foldlM___at_Lean_Lsp_ModuleRefs_findAt___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_References_definitionsMatching___spec__1___boxed(lean_object*, lean_object*); @@ -432,11 +433,8 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_a lean_object* lean_nat_mul(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_RefInfo_findReferenceLocation_x3f___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__22; -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__2; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Server_combineIdents_useConstRepresentatives___spec__2(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_ModuleRefs_toLspModuleRefs___closed__3; -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__3; -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Server_findReferences___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_ModuleRefs_addRef___spec__3(lean_object*); lean_object* l_Lean_Elab_Info_range_x3f(lean_object*); lean_object* l_Lean_Json_Parser_any(lean_object*); @@ -452,12 +450,15 @@ lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Position_0__Le lean_object* l_List_reverse___rarg(lean_object*); lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Lsp_instFromJsonModuleRefs___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_useConstRepresentatives___spec__15(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Server_findReferences___spec__4(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_Lean_Server_combineIdents_useConstRepresentatives___spec__5(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_References_definitionsMatching___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Server_References_removeIlean___spec__6(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_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__3; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___at_Lean_Server_References_updateWorkerRefs___spec__2___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Server_findReferences___spec__3(lean_object*, lean_object*); extern lean_object* l_Lean_noConfusionExt; uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Lsp_instFromJsonModuleRefs___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_useConstRepresentatives___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -465,13 +466,11 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_RefInfo_toLspRe static lean_object* l_Lean_Server_ModuleRefs_toLspModuleRefs___closed__2; static lean_object* l_Lean_Server_Ilean_load___closed__1; size_t lean_usize_add(size_t, size_t); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Server_RefInfo_toLspRefInfo___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_References_updateWorkerRefs___spec__4___boxed(lean_object*, lean_object*); static lean_object* l_List_mapTR_loop___at___private_Lean_Server_References_0__Lean_Server_toJsonIlean____x40_Lean_Server_References___hyg_1478____spec__2___closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_combineIdents___spec__4(lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_array_size(lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Server_References_removeIlean___spec__6___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__15; @@ -498,7 +497,6 @@ LEAN_EXPORT lean_object* l_Lean_Server_References_finalizeWorkerRefs(lean_object LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_References_addIlean___spec__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents_useConstRepresentatives___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); -static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__4; LEAN_EXPORT lean_object* l_Lean_Lsp_RefInfo_findReferenceLocation_x3f___lambda__2(lean_object*, lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_References_allRefsFor___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_ModuleRefs_addRef___spec__2___boxed(lean_object*, lean_object*); @@ -519,15 +517,14 @@ LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_ LEAN_EXPORT lean_object* l_Lean_Server_References_allRefs___boxed(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_RefInfo_toLspRefInfo___spec__6___closed__5; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineIdents___spec__7(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_Server_References_removeIlean___spec__8___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_References_updateWorkerRefs___spec__3(uint64_t, uint64_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_combineIdents___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instToJsonIlean; static lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_1333____closed__12; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_combineIdents_useConstRepresentatives___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_References_allRefs___spec__7(lean_object*, lean_object*); +static lean_object* l_panic___at_Lean_Server_findReferences___spec__3___closed__2; LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_References_addIlean___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_References_definitionsMatching___spec__4___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_Server_References_updateWorkerRefs___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, uint64_t, uint64_t, size_t, lean_object*); @@ -543,6 +540,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_ModuleRefs_toLspModuleRefs___boxed(lean_o LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_combineIdents_useConstRepresentatives___spec__10(lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Server_combineIdents(lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___closed__1; lean_object* l_Array_get_x3f___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Server_dedupReferences___closed__5; static lean_object* _init_l_Lean_Server_RefInfo_empty___closed__1() { @@ -10832,7 +10830,7 @@ x_29 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_29, 0, x_8); lean_ctor_set(x_29, 1, x_28); x_30 = l_Lean_Server_RefInfo_empty___closed__1; -x_31 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_29, x_30); +x_31 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_29, x_30); x_32 = l_Lean_Json_mkObj(x_31); return x_32; } @@ -10864,7 +10862,7 @@ x_41 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_41, 0, x_8); lean_ctor_set(x_41, 1, x_40); x_42 = l_Lean_Server_RefInfo_empty___closed__1; -x_43 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_41, x_42); +x_43 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_41, x_42); x_44 = l_Lean_Json_mkObj(x_43); return x_44; } @@ -10895,7 +10893,7 @@ x_55 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_55, 0, x_8); lean_ctor_set(x_55, 1, x_54); x_56 = l_Lean_Server_RefInfo_empty___closed__1; -x_57 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_55, x_56); +x_57 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_55, x_56); x_58 = l_Lean_Json_mkObj(x_57); return x_58; } @@ -11596,7 +11594,7 @@ return x_130; } } } -static lean_object* _init_l_panic___at_Lean_Server_findReferences___spec__4___closed__1() { +static lean_object* _init_l_panic___at_Lean_Server_findReferences___spec__3___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -11605,27 +11603,27 @@ x_2 = l_StateT_instMonad___rarg(x_1); return x_2; } } -static lean_object* _init_l_panic___at_Lean_Server_findReferences___spec__4___closed__2() { +static lean_object* _init_l_panic___at_Lean_Server_findReferences___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_panic___at_Lean_Server_findReferences___spec__4___closed__1; +x_2 = l_panic___at_Lean_Server_findReferences___spec__3___closed__1; x_3 = l_instInhabitedOfMonad___rarg(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_panic___at_Lean_Server_findReferences___spec__4(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Server_findReferences___spec__3(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_3 = l_panic___at_Lean_Server_findReferences___spec__4___closed__2; +x_3 = l_panic___at_Lean_Server_findReferences___spec__3___closed__2; x_4 = lean_panic_fn(x_3, x_1); x_5 = lean_apply_1(x_4, x_2); return x_5; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Server_findReferences___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_EXPORT lean_object* l_List_mapM_loop___at_Lean_Server_findReferences___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: { if (lean_obj_tag(x_4) == 0) @@ -11652,7 +11650,7 @@ x_11 = lean_ctor_get(x_4, 1); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3(x_1, x_2, x_3, x_10, x_6); +x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2(x_1, x_2, x_3, x_10, x_6); x_13 = lean_ctor_get(x_12, 0); lean_inc(x_13); x_14 = lean_ctor_get(x_12, 1); @@ -11681,7 +11679,7 @@ lean_dec(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_18 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3(x_1, x_2, x_3, x_16, x_6); +x_18 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2(x_1, x_2, x_3, x_16, x_6); x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); x_20 = lean_ctor_get(x_18, 1); @@ -11698,7 +11696,7 @@ goto _start; } } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__1() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__1() { _start: { lean_object* x_1; @@ -11706,7 +11704,7 @@ x_1 = lean_mk_string_unchecked("Lean.Server.InfoUtils", 21, 21); return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__2() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__2() { _start: { lean_object* x_1; @@ -11714,7 +11712,7 @@ x_1 = lean_mk_string_unchecked("Lean.Elab.InfoTree.visitM.go", 28, 28); return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__3() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__3() { _start: { lean_object* x_1; @@ -11722,20 +11720,20 @@ x_1 = lean_mk_string_unchecked("unexpected context-free info tree node", 38, 38) return x_1; } } -static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__4() { +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__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_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__1; -x_2 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__2; -x_3 = lean_unsigned_to_nat(56u); +x_1 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__1; +x_2 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__2; +x_3 = lean_unsigned_to_nat(62u); x_4 = lean_unsigned_to_nat(21u); -x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__3; +x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___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_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3(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_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2(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_3) == 0) @@ -11760,8 +11758,8 @@ lean_object* x_10; lean_object* x_11; lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__4; -x_11 = l_panic___at_Lean_Server_findReferences___spec__4(x_10, x_5); +x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__4; +x_11 = l_panic___at_Lean_Server_findReferences___spec__3(x_10, x_5); return x_11; } default: @@ -11800,7 +11798,7 @@ uint8_t x_18; x_18 = !lean_is_exclusive(x_3); 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; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; x_19 = lean_ctor_get(x_3, 0); x_20 = lean_ctor_get(x_4, 0); lean_inc(x_20); @@ -11812,128 +11810,200 @@ lean_inc(x_21); lean_inc(x_20); lean_inc(x_19); x_22 = lean_apply_4(x_1, x_19, x_20, x_21, x_5); -x_23 = lean_ctor_get(x_22, 1); +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; uint8_t x_28; +lean_dec(x_1); +x_25 = lean_ctor_get(x_22, 1); +lean_inc(x_25); lean_dec(x_22); -lean_inc(x_19); -x_24 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_20); -x_25 = l_Lean_PersistentArray_toList___rarg(x_21); x_26 = lean_box(0); -lean_inc(x_2); -x_27 = l_List_mapM_loop___at_Lean_Server_findReferences___spec__5(x_1, x_2, x_24, x_25, x_26, x_23); -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_5(x_2, x_19, x_20, x_21, x_28, x_29); -x_31 = !lean_is_exclusive(x_30); -if (x_31 == 0) +x_27 = lean_apply_5(x_2, x_19, x_20, x_21, x_26, x_25); +x_28 = !lean_is_exclusive(x_27); +if (x_28 == 0) { -lean_object* x_32; lean_object* x_33; -x_32 = lean_ctor_get(x_30, 0); -x_33 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_30, 0, x_33); -return x_30; +lean_object* x_29; +x_29 = lean_ctor_get(x_27, 0); +lean_ctor_set(x_3, 0, x_29); +lean_ctor_set(x_27, 0, x_3); +return x_27; } 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_alloc_ctor(1, 1, 0); -lean_ctor_set(x_36, 0, 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; +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_27, 0); +x_31 = lean_ctor_get(x_27, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_27); +lean_ctor_set(x_3, 0, x_30); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_3); +lean_ctor_set(x_32, 1, x_31); +return x_32; } } 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; 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_38 = lean_ctor_get(x_3, 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; uint8_t x_41; +x_33 = lean_ctor_get(x_22, 1); +lean_inc(x_33); +lean_dec(x_22); +lean_inc(x_19); +x_34 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_20); +x_35 = l_Lean_PersistentArray_toList___rarg(x_21); +x_36 = lean_box(0); +lean_inc(x_2); +x_37 = l_List_mapM_loop___at_Lean_Server_findReferences___spec__4(x_1, x_2, x_34, x_35, x_36, x_33); +x_38 = lean_ctor_get(x_37, 0); lean_inc(x_38); -lean_dec(x_3); -x_39 = lean_ctor_get(x_4, 0); -lean_inc(x_39); -x_40 = lean_ctor_get(x_4, 1); -lean_inc(x_40); -lean_dec(x_4); -lean_inc(x_1); -lean_inc(x_40); +x_39 = lean_ctor_get(x_37, 1); lean_inc(x_39); -lean_inc(x_38); -x_41 = lean_apply_4(x_1, x_38, x_39, x_40, x_5); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); -lean_inc(x_38); +lean_dec(x_37); +x_40 = lean_apply_5(x_2, x_19, x_20, x_21, x_38, x_39); +x_41 = !lean_is_exclusive(x_40); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; +x_42 = lean_ctor_get(x_40, 0); x_43 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_43, 0, x_38); -x_44 = l_Lean_Elab_Info_updateContext_x3f(x_43, x_39); -x_45 = l_Lean_PersistentArray_toList___rarg(x_40); -x_46 = lean_box(0); -lean_inc(x_2); -x_47 = l_List_mapM_loop___at_Lean_Server_findReferences___spec__5(x_1, x_2, x_44, x_45, x_46, x_42); -x_48 = lean_ctor_get(x_47, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_40, 0, x_43); +return x_40; +} +else +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_44 = lean_ctor_get(x_40, 0); +x_45 = lean_ctor_get(x_40, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_40); +x_46 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_46, 0, x_44); +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 +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; +x_48 = lean_ctor_get(x_3, 0); lean_inc(x_48); -x_49 = lean_ctor_get(x_47, 1); +lean_dec(x_3); +x_49 = lean_ctor_get(x_4, 0); lean_inc(x_49); -lean_dec(x_47); -x_50 = lean_apply_5(x_2, x_38, x_39, x_40, x_48, x_49); -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_50, 1); +x_50 = lean_ctor_get(x_4, 1); +lean_inc(x_50); +lean_dec(x_4); +lean_inc(x_1); +lean_inc(x_50); +lean_inc(x_49); +lean_inc(x_48); +x_51 = lean_apply_4(x_1, x_48, x_49, x_50, x_5); +x_52 = lean_ctor_get(x_51, 0); 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; +x_53 = lean_unbox(x_52); +lean_dec(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_dec(x_1); +x_54 = lean_ctor_get(x_51, 1); +lean_inc(x_54); +lean_dec(x_51); +x_55 = lean_box(0); +x_56 = lean_apply_5(x_2, x_48, x_49, x_50, x_55, x_54); +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_50); - x_53 = lean_box(0); + lean_dec_ref(x_56); + x_59 = lean_box(0); } -x_54 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_54, 0, x_51); -if (lean_is_scalar(x_53)) { - x_55 = lean_alloc_ctor(0, 2, 0); +x_60 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_60, 0, x_57); +if (lean_is_scalar(x_59)) { + x_61 = lean_alloc_ctor(0, 2, 0); } else { - x_55 = x_53; + x_61 = x_59; +} +lean_ctor_set(x_61, 0, x_60); +lean_ctor_set(x_61, 1, x_58); +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; lean_object* x_75; +x_62 = lean_ctor_get(x_51, 1); +lean_inc(x_62); +lean_dec(x_51); +lean_inc(x_48); +x_63 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_63, 0, x_48); +x_64 = l_Lean_Elab_Info_updateContext_x3f(x_63, x_49); +x_65 = l_Lean_PersistentArray_toList___rarg(x_50); +x_66 = lean_box(0); +lean_inc(x_2); +x_67 = l_List_mapM_loop___at_Lean_Server_findReferences___spec__4(x_1, x_2, x_64, x_65, x_66, x_62); +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_5(x_2, x_48, x_49, x_50, x_68, x_69); +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +if (lean_is_exclusive(x_70)) { + lean_ctor_release(x_70, 0); + lean_ctor_release(x_70, 1); + x_73 = x_70; +} else { + lean_dec_ref(x_70); + x_73 = lean_box(0); +} +x_74 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_74, 0, x_71); +if (lean_is_scalar(x_73)) { + x_75 = lean_alloc_ctor(0, 2, 0); +} else { + x_75 = x_73; +} +lean_ctor_set(x_75, 0, x_74); +lean_ctor_set(x_75, 1, x_72); +return x_75; } -lean_ctor_set(x_55, 0, x_54); -lean_ctor_set(x_55, 1, x_52); -return x_55; } } default: { -lean_object* x_56; lean_object* x_57; +lean_object* x_76; lean_object* x_77; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -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_5); -return x_57; -} -} +x_76 = lean_box(0); +x_77 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_77, 0, x_76); +lean_ctor_set(x_77, 1, x_5); +return x_77; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Server_findReferences___spec__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 = lean_box(0); -x_6 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3(x_1, x_2, x_5, x_3, x_4); -return x_6; } } LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___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) { @@ -11944,49 +12014,50 @@ x_7 = lean_apply_4(x_1, x_2, x_3, x_4, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__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_5; lean_object* x_6; uint8_t x_7; -x_5 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1___lambda__1___boxed), 6, 1); -lean_closure_set(x_5, 0, x_2); -x_6 = l_Lean_Elab_InfoTree_visitM___at_Lean_Server_findReferences___spec__2(x_1, x_5, x_3, x_4); -x_7 = !lean_is_exclusive(x_6); -if (x_7 == 0) +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1___lambda__1___boxed), 6, 1); +lean_closure_set(x_6, 0, x_2); +x_7 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2(x_1, x_6, x_3, x_4, x_5); +x_8 = !lean_is_exclusive(x_7); +if (x_8 == 0) { -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_6, 0); -lean_dec(x_8); -x_9 = lean_box(0); -lean_ctor_set(x_6, 0, x_9); -return x_6; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_7, 0); +lean_dec(x_9); +x_10 = lean_box(0); +lean_ctor_set(x_7, 0, x_10); +return x_7; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_ctor_get(x_6, 1); -lean_inc(x_10); -lean_dec(x_6); -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; +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_7, 1); +lean_inc(x_11); +lean_dec(x_7); +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; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__1(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 = lean_box(0); -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_5); -lean_ctor_set(x_6, 1, x_4); -return x_6; +uint8_t x_5; lean_object* x_6; lean_object* x_7; +x_5 = 1; +x_6 = lean_box(x_5); +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_4); +return x_7; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___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_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__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; @@ -12157,15 +12228,15 @@ return x_41; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__1___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__1___boxed), 4, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6(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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; @@ -12181,23 +12252,24 @@ return x_8; } else { -lean_object* x_9; 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_9; 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; lean_dec(x_5); x_9 = lean_array_uget(x_2, x_4); lean_inc(x_1); -x_10 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__2___boxed), 5, 1); +x_10 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__2___boxed), 5, 1); lean_closure_set(x_10, 0, x_1); -x_11 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___closed__1; -x_12 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1(x_11, x_10, x_9, x_6); -x_13 = lean_ctor_get(x_12, 1); -lean_inc(x_13); -lean_dec(x_12); -x_14 = 1; -x_15 = lean_usize_add(x_4, x_14); -x_16 = lean_box(0); -x_4 = x_15; -x_5 = x_16; -x_6 = x_13; +x_11 = lean_box(0); +x_12 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___closed__1; +x_13 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1(x_12, x_10, x_11, x_9, x_6); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = 1; +x_16 = lean_usize_add(x_4, x_15); +x_17 = lean_box(0); +x_4 = x_16; +x_5 = x_17; +x_6 = x_14; goto _start; } } @@ -12210,7 +12282,7 @@ x_3 = lean_array_size(x_2); x_4 = 0; x_5 = lean_box(0); x_6 = l_Lean_Server_RefInfo_empty___closed__1; -x_7 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5(x_1, x_2, x_3, x_4, x_5, x_6); x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); lean_dec(x_7); @@ -12226,27 +12298,27 @@ lean_dec(x_5); return x_7; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__1___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_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); return x_5; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__2___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_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__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_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___lambda__2(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___lambda__2(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); return x_6; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___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_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___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; @@ -12254,7 +12326,7 @@ x_7 = lean_unbox_usize(x_3); lean_dec(x_3); x_8 = lean_unbox_usize(x_4); lean_dec(x_4); -x_9 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6(x_1, x_2, x_7, x_8, x_5, x_6); +x_9 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5(x_1, x_2, x_7, x_8, x_5, x_6); lean_dec(x_2); return x_9; } @@ -15523,17 +15595,17 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_panic___at_Lean_Server_combineIdents_buildIdMap___spec__6(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Server_combineIdents_buildIdMap___spec__5(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_3 = l_panic___at_Lean_Server_findReferences___spec__4___closed__2; +x_3 = l_panic___at_Lean_Server_findReferences___spec__3___closed__2; x_4 = lean_panic_fn(x_3, x_1); x_5 = lean_apply_1(x_4, x_2); return x_5; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Server_combineIdents_buildIdMap___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_EXPORT lean_object* l_List_mapM_loop___at_Lean_Server_combineIdents_buildIdMap___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) { _start: { if (lean_obj_tag(x_4) == 0) @@ -15560,7 +15632,7 @@ x_11 = lean_ctor_get(x_4, 1); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__5(x_1, x_2, x_3, x_10, x_6); +x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__4(x_1, x_2, x_3, x_10, x_6); x_13 = lean_ctor_get(x_12, 0); lean_inc(x_13); x_14 = lean_ctor_get(x_12, 1); @@ -15589,7 +15661,7 @@ lean_dec(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_18 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__5(x_1, x_2, x_3, x_16, x_6); +x_18 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__4(x_1, x_2, x_3, x_16, x_6); x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); x_20 = lean_ctor_get(x_18, 1); @@ -15606,7 +15678,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__5(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_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__4(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_3) == 0) @@ -15631,8 +15703,8 @@ lean_object* x_10; lean_object* x_11; lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__4; -x_11 = l_panic___at_Lean_Server_combineIdents_buildIdMap___spec__6(x_10, x_5); +x_10 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__4; +x_11 = l_panic___at_Lean_Server_combineIdents_buildIdMap___spec__5(x_10, x_5); return x_11; } default: @@ -15671,7 +15743,7 @@ uint8_t x_18; x_18 = !lean_is_exclusive(x_3); 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; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; x_19 = lean_ctor_get(x_3, 0); x_20 = lean_ctor_get(x_4, 0); lean_inc(x_20); @@ -15683,162 +15755,234 @@ lean_inc(x_21); lean_inc(x_20); lean_inc(x_19); x_22 = lean_apply_4(x_1, x_19, x_20, x_21, x_5); -x_23 = lean_ctor_get(x_22, 1); +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; uint8_t x_28; +lean_dec(x_1); +x_25 = lean_ctor_get(x_22, 1); +lean_inc(x_25); lean_dec(x_22); -lean_inc(x_19); -x_24 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_20); -x_25 = l_Lean_PersistentArray_toList___rarg(x_21); x_26 = lean_box(0); -lean_inc(x_2); -x_27 = l_List_mapM_loop___at_Lean_Server_combineIdents_buildIdMap___spec__7(x_1, x_2, x_24, x_25, x_26, x_23); -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_5(x_2, x_19, x_20, x_21, x_28, x_29); -x_31 = !lean_is_exclusive(x_30); -if (x_31 == 0) +x_27 = lean_apply_5(x_2, x_19, x_20, x_21, x_26, x_25); +x_28 = !lean_is_exclusive(x_27); +if (x_28 == 0) { -lean_object* x_32; lean_object* x_33; -x_32 = lean_ctor_get(x_30, 0); -x_33 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_30, 0, x_33); -return x_30; +lean_object* x_29; +x_29 = lean_ctor_get(x_27, 0); +lean_ctor_set(x_3, 0, x_29); +lean_ctor_set(x_27, 0, x_3); +return x_27; } 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_alloc_ctor(1, 1, 0); -lean_ctor_set(x_36, 0, 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; +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_27, 0); +x_31 = lean_ctor_get(x_27, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_27); +lean_ctor_set(x_3, 0, x_30); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_3); +lean_ctor_set(x_32, 1, x_31); +return x_32; } } 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; 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_38 = lean_ctor_get(x_3, 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; uint8_t x_41; +x_33 = lean_ctor_get(x_22, 1); +lean_inc(x_33); +lean_dec(x_22); +lean_inc(x_19); +x_34 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_20); +x_35 = l_Lean_PersistentArray_toList___rarg(x_21); +x_36 = lean_box(0); +lean_inc(x_2); +x_37 = l_List_mapM_loop___at_Lean_Server_combineIdents_buildIdMap___spec__6(x_1, x_2, x_34, x_35, x_36, x_33); +x_38 = lean_ctor_get(x_37, 0); lean_inc(x_38); -lean_dec(x_3); -x_39 = lean_ctor_get(x_4, 0); -lean_inc(x_39); -x_40 = lean_ctor_get(x_4, 1); -lean_inc(x_40); -lean_dec(x_4); -lean_inc(x_1); -lean_inc(x_40); +x_39 = lean_ctor_get(x_37, 1); lean_inc(x_39); -lean_inc(x_38); -x_41 = lean_apply_4(x_1, x_38, x_39, x_40, x_5); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); -lean_inc(x_38); +lean_dec(x_37); +x_40 = lean_apply_5(x_2, x_19, x_20, x_21, x_38, x_39); +x_41 = !lean_is_exclusive(x_40); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; +x_42 = lean_ctor_get(x_40, 0); x_43 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_43, 0, x_38); -x_44 = l_Lean_Elab_Info_updateContext_x3f(x_43, x_39); -x_45 = l_Lean_PersistentArray_toList___rarg(x_40); -x_46 = lean_box(0); -lean_inc(x_2); -x_47 = l_List_mapM_loop___at_Lean_Server_combineIdents_buildIdMap___spec__7(x_1, x_2, x_44, x_45, x_46, x_42); -x_48 = lean_ctor_get(x_47, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_40, 0, x_43); +return x_40; +} +else +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_44 = lean_ctor_get(x_40, 0); +x_45 = lean_ctor_get(x_40, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_40); +x_46 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_46, 0, x_44); +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 +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; +x_48 = lean_ctor_get(x_3, 0); lean_inc(x_48); -x_49 = lean_ctor_get(x_47, 1); +lean_dec(x_3); +x_49 = lean_ctor_get(x_4, 0); lean_inc(x_49); -lean_dec(x_47); -x_50 = lean_apply_5(x_2, x_38, x_39, x_40, x_48, x_49); -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_50, 1); +x_50 = lean_ctor_get(x_4, 1); +lean_inc(x_50); +lean_dec(x_4); +lean_inc(x_1); +lean_inc(x_50); +lean_inc(x_49); +lean_inc(x_48); +x_51 = lean_apply_4(x_1, x_48, x_49, x_50, x_5); +x_52 = lean_ctor_get(x_51, 0); 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; +x_53 = lean_unbox(x_52); +lean_dec(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_dec(x_1); +x_54 = lean_ctor_get(x_51, 1); +lean_inc(x_54); +lean_dec(x_51); +x_55 = lean_box(0); +x_56 = lean_apply_5(x_2, x_48, x_49, x_50, x_55, x_54); +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_50); - x_53 = lean_box(0); + lean_dec_ref(x_56); + x_59 = lean_box(0); } -x_54 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_54, 0, x_51); -if (lean_is_scalar(x_53)) { - x_55 = lean_alloc_ctor(0, 2, 0); +x_60 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_60, 0, x_57); +if (lean_is_scalar(x_59)) { + x_61 = lean_alloc_ctor(0, 2, 0); } else { - x_55 = x_53; + x_61 = x_59; +} +lean_ctor_set(x_61, 0, x_60); +lean_ctor_set(x_61, 1, x_58); +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; lean_object* x_75; +x_62 = lean_ctor_get(x_51, 1); +lean_inc(x_62); +lean_dec(x_51); +lean_inc(x_48); +x_63 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_63, 0, x_48); +x_64 = l_Lean_Elab_Info_updateContext_x3f(x_63, x_49); +x_65 = l_Lean_PersistentArray_toList___rarg(x_50); +x_66 = lean_box(0); +lean_inc(x_2); +x_67 = l_List_mapM_loop___at_Lean_Server_combineIdents_buildIdMap___spec__6(x_1, x_2, x_64, x_65, x_66, x_62); +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_5(x_2, x_48, x_49, x_50, x_68, x_69); +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +if (lean_is_exclusive(x_70)) { + lean_ctor_release(x_70, 0); + lean_ctor_release(x_70, 1); + x_73 = x_70; +} else { + lean_dec_ref(x_70); + x_73 = lean_box(0); +} +x_74 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_74, 0, x_71); +if (lean_is_scalar(x_73)) { + x_75 = lean_alloc_ctor(0, 2, 0); +} else { + x_75 = x_73; +} +lean_ctor_set(x_75, 0, x_74); +lean_ctor_set(x_75, 1, x_72); +return x_75; } -lean_ctor_set(x_55, 0, x_54); -lean_ctor_set(x_55, 1, x_52); -return x_55; } } default: { -lean_object* x_56; lean_object* x_57; +lean_object* x_76; lean_object* x_77; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -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_5); -return x_57; -} +x_76 = lean_box(0); +x_77 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_77, 0, x_76); +lean_ctor_set(x_77, 1, x_5); +return x_77; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Server_combineIdents_buildIdMap___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; -x_5 = lean_box(0); -x_6 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__5(x_1, x_2, x_5, x_3, x_4); -return x_6; -} } -LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_combineIdents_buildIdMap___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_combineIdents_buildIdMap___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_5; lean_object* x_6; uint8_t x_7; -x_5 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1___lambda__1___boxed), 6, 1); -lean_closure_set(x_5, 0, x_2); -x_6 = l_Lean_Elab_InfoTree_visitM___at_Lean_Server_combineIdents_buildIdMap___spec__4(x_1, x_5, x_3, x_4); -x_7 = !lean_is_exclusive(x_6); -if (x_7 == 0) +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_findReferences___spec__1___lambda__1___boxed), 6, 1); +lean_closure_set(x_6, 0, x_2); +x_7 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_combineIdents_buildIdMap___spec__4(x_1, x_6, x_3, x_4, x_5); +x_8 = !lean_is_exclusive(x_7); +if (x_8 == 0) { -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_6, 0); -lean_dec(x_8); -x_9 = lean_box(0); -lean_ctor_set(x_6, 0, x_9); -return x_6; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_7, 0); +lean_dec(x_9); +x_10 = lean_box(0); +lean_ctor_set(x_7, 0, x_10); +return x_7; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_ctor_get(x_6, 1); -lean_inc(x_10); -lean_dec(x_6); -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; +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_7, 1); +lean_inc(x_11); +lean_dec(x_7); +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; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___lambda__1(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_combineIdents_buildIdMap___spec__7___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_2) == 9) @@ -15892,46 +16036,47 @@ return x_21; } } } -static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___closed__1() { +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___lambda__1___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___lambda__1___boxed), 4, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { _start: { uint8_t x_6; x_6 = lean_usize_dec_eq(x_2, x_3); if (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; size_t x_13; size_t x_14; +lean_object* x_7; lean_object* x_8; lean_object* x_9; 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_dec(x_4); x_7 = lean_array_uget(x_1, x_2); -x_8 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___closed__1; -x_9 = l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___closed__1; -x_10 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_combineIdents_buildIdMap___spec__3(x_8, x_9, x_7, x_5); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); +x_8 = lean_box(0); +x_9 = l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___closed__1; +x_10 = l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___closed__1; +x_11 = l_Lean_Elab_InfoTree_visitM_x27___at_Lean_Server_combineIdents_buildIdMap___spec__3(x_9, x_10, x_8, x_7, x_5); +x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); -lean_dec(x_10); -x_13 = 1; -x_14 = lean_usize_add(x_2, x_13); -x_2 = x_14; -x_4 = x_11; -x_5 = x_12; +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = 1; +x_15 = lean_usize_add(x_2, x_14); +x_2 = x_15; +x_4 = x_12; +x_5 = x_13; goto _start; } else { -lean_object* x_16; -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_4); -lean_ctor_set(x_16, 1, x_5); -return x_16; +lean_object* x_17; +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_4); +lean_ctor_set(x_17, 1, x_5); +return x_17; } } } @@ -15969,7 +16114,7 @@ else size_t x_14; lean_object* x_15; lean_object* x_16; x_14 = lean_usize_of_nat(x_10); lean_dec(x_10); -x_15 = l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8(x_1, x_5, x_14, x_6, x_9); +x_15 = l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7(x_1, x_5, x_14, x_6, x_9); x_16 = lean_ctor_get(x_15, 1); lean_inc(x_16); lean_dec(x_15); @@ -16002,16 +16147,16 @@ lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___lambda__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_Server_combineIdents_buildIdMap___spec__7___lambda__1___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_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___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_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___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; @@ -16019,7 +16164,7 @@ 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_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8(x_1, x_6, x_7, x_4, x_5); +x_8 = l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7(x_1, x_6, x_7, x_4, x_5); lean_dec(x_1); return x_8; } @@ -28052,22 +28197,22 @@ l_Lean_Server_Ilean_load___closed__2 = _init_l_Lean_Server_Ilean_load___closed__ lean_mark_persistent(l_Lean_Server_Ilean_load___closed__2); l_Lean_Server_Ilean_load___closed__3 = _init_l_Lean_Server_Ilean_load___closed__3(); lean_mark_persistent(l_Lean_Server_Ilean_load___closed__3); -l_panic___at_Lean_Server_findReferences___spec__4___closed__1 = _init_l_panic___at_Lean_Server_findReferences___spec__4___closed__1(); -lean_mark_persistent(l_panic___at_Lean_Server_findReferences___spec__4___closed__1); -l_panic___at_Lean_Server_findReferences___spec__4___closed__2 = _init_l_panic___at_Lean_Server_findReferences___spec__4___closed__2(); -lean_mark_persistent(l_panic___at_Lean_Server_findReferences___spec__4___closed__2); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__1(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__1); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__2(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__2); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__3(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__3); -l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__4(); -lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__3___closed__4); -l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__6___closed__1); -l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___closed__1 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___closed__1(); -lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__8___closed__1); +l_panic___at_Lean_Server_findReferences___spec__3___closed__1 = _init_l_panic___at_Lean_Server_findReferences___spec__3___closed__1(); +lean_mark_persistent(l_panic___at_Lean_Server_findReferences___spec__3___closed__1); +l_panic___at_Lean_Server_findReferences___spec__3___closed__2 = _init_l_panic___at_Lean_Server_findReferences___spec__3___closed__2(); +lean_mark_persistent(l_panic___at_Lean_Server_findReferences___spec__3___closed__2); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__1); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__2(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__2); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__3(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__3); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__4(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Server_findReferences___spec__2___closed__4); +l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__5___closed__1); +l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___closed__1 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___closed__1(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Server_combineIdents_buildIdMap___spec__7___closed__1); l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_dedupReferences___spec__4___at_Lean_Server_dedupReferences___spec__5___closed__1 = _init_l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_dedupReferences___spec__4___at_Lean_Server_dedupReferences___spec__5___closed__1(); l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_dedupReferences___spec__4___at_Lean_Server_dedupReferences___spec__5___closed__2 = _init_l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_dedupReferences___spec__4___at_Lean_Server_dedupReferences___spec__5___closed__2(); l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__10___closed__1 = _init_l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__10___closed__1(); diff --git a/stage0/stdlib/Lean/Server/Rpc/Basic.c b/stage0/stdlib/Lean/Server/Rpc/Basic.c index d514e6e87185..f56e0cceeaae 100644 --- a/stage0/stdlib/Lean/Server/Rpc/Basic.c +++ b/stage0/stdlib/Lean/Server/Rpc/Basic.c @@ -49,6 +49,7 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Server_rpc LEAN_EXPORT uint64_t l___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_hashRpcRef____x40_Lean_Server_Rpc_Basic___hyg_74_(size_t); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Server_rpcGetRef___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Server_instRpcEncodableOfFromJsonOfToJson___spec__1___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Server_rpcGetRef___spec__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_fromJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_106____closed__2; static lean_object* l_Lean_Server_instRpcEncodableOption___rarg___lambda__2___closed__1; @@ -116,7 +117,6 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_erase___at_Lean_Server_rpcRele LEAN_EXPORT uint8_t l___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_beqRpcRef____x40_Lean_Server_Rpc_Basic___hyg_16_(size_t, size_t); static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_fromJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_106____spec__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodableOfFromJsonOfToJson(lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_fromJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_106____closed__13; static lean_object* l_Lean_Lsp_instToJsonRpcRef___closed__1; static lean_object* l___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_fromJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_106____closed__5; @@ -592,7 +592,7 @@ x_1 = l_Lean_Lsp_instFromJsonRpcRef___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -643,7 +643,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); x_9 = l___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____closed__1; -x_10 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_8, x_9); +x_10 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_8, x_9); x_11 = l_Lean_Json_mkObj(x_10); return x_11; } diff --git a/stage0/stdlib/Lean/Server/Watchdog.c b/stage0/stdlib/Lean/Server/Watchdog.c index 9cc1b58faf67..6792c7c72dfe 100644 --- a/stage0/stdlib/Lean/Server/Watchdog.c +++ b/stage0/stdlib/Lean/Server/Watchdog.c @@ -200,6 +200,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Server_Watchdog_0__Lean_Server_Watchdo lean_object* l_Lean_Json_opt___at_Lean_JsonRpc_instToJsonMessage___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_Watchdog_findDefinitions___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_RBNode_balRight___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_groupByKey___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_IO_FS_Stream_writeLspResponse___at_Lean_Server_Watchdog_mainLoop___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleRename___spec__5(lean_object*); @@ -515,7 +516,6 @@ static lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_Watchdog_handleDid LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_mainLoop___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Server_References_allRefs(lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__4; -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleRequest___spec__7___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_mkLeanServerCapabilities___closed__15; LEAN_EXPORT lean_object* l_Lean_RBNode_erase___at_Lean_Server_Watchdog_ImportData_update___spec__5___boxed(lean_object*, lean_object*); @@ -17257,7 +17257,7 @@ x_18 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_18, 0, x_10); lean_ctor_set(x_18, 1, x_17); x_19 = l_Lean_Server_Watchdog_FileWorker_queuedMsgs___closed__1; -x_20 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_18, x_19); +x_20 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_18, x_19); x_21 = l_Lean_Json_mkObj(x_20); return x_21; } diff --git a/stage0/stdlib/Lean/SubExpr.c b/stage0/stdlib/Lean/SubExpr.c index 8a1d0ca291ed..eb3e1dbd20a2 100644 --- a/stage0/stdlib/Lean/SubExpr.c +++ b/stage0/stdlib/Lean/SubExpr.c @@ -61,6 +61,7 @@ LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_foldr(lean_object*); extern lean_object* l_Lean_instInhabitedJson; static lean_object* l_Lean_SubExpr_instFromJsonGoalLocation___closed__1; LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_pushBindingBody___boxed(lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_SubExpr_instToJsonFVarId___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_tail___boxed(lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); @@ -154,7 +155,6 @@ LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_pushAppFn___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_push(lean_object*, lean_object*); static lean_object* l___private_Lean_SubExpr_0__Lean_SubExpr_fromJsonGoalsLocation____x40_Lean_SubExpr___hyg_1812____closed__2; LEAN_EXPORT lean_object* l___private_Lean_SubExpr_0__Lean_SubExpr_fromJsonGoalLocation____x40_Lean_SubExpr___hyg_1411____lambda__3___boxed(lean_object*, lean_object*, lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_SubExpr_0__Lean_SubExpr_fromJsonGoalsLocation____x40_Lean_SubExpr___hyg_1812_(lean_object*); LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_asNat(lean_object*); static lean_object* l_Lean_SubExpr_Pos_typeCoord___closed__1; @@ -4783,7 +4783,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_10); lean_ctor_set(x_17, 1, x_16); x_18 = l_Lean_SubExpr_Pos_toArray___closed__2; -x_19 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } diff --git a/stage0/stdlib/Lean/Util/FileSetupInfo.c b/stage0/stdlib/Lean/Util/FileSetupInfo.c index bdf8c3d2ab91..d1c943478d7c 100644 --- a/stage0/stdlib/Lean/Util/FileSetupInfo.c +++ b/stage0/stdlib/Lean/Util/FileSetupInfo.c @@ -42,12 +42,12 @@ LEAN_EXPORT lean_object* l_Lean_instToJsonFileSetupInfo; static lean_object* l___private_Lean_Util_FileSetupInfo_0__Lean_fromJsonFileSetupInfo____x40_Lean_Util_FileSetupInfo___hyg_26____closed__7; static lean_object* l___private_Lean_Util_FileSetupInfo_0__Lean_fromJsonFileSetupInfo____x40_Lean_Util_FileSetupInfo___hyg_26____closed__9; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_FileSetupInfo_0__Lean_fromJsonFileSetupInfo____x40_Lean_Util_FileSetupInfo___hyg_26____spec__2___boxed(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_Util_FileSetupInfo_0__Lean_toJsonFileSetupInfo____x40_Lean_Util_FileSetupInfo___hyg_132____closed__1; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_FileSetupInfo_0__Lean_fromJsonFileSetupInfo____x40_Lean_Util_FileSetupInfo___hyg_26____spec__1(lean_object*, lean_object*); lean_object* l___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40_(lean_object*); lean_object* l_Lean_RBNode_fold___at_Lean_instToJsonLeanOptions___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); -lean_object* l_List_bindTR_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_Util_FileSetupInfo_0__Lean_fromJsonFileSetupInfo____x40_Lean_Util_FileSetupInfo___hyg_26____closed__16; static lean_object* l___private_Lean_Util_FileSetupInfo_0__Lean_fromJsonFileSetupInfo____x40_Lean_Util_FileSetupInfo___hyg_26____closed__15; static lean_object* l___private_Lean_Util_FileSetupInfo_0__Lean_fromJsonFileSetupInfo____x40_Lean_Util_FileSetupInfo___hyg_26____closed__18; @@ -516,7 +516,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_7); lean_ctor_set(x_16, 1, x_15); x_17 = l___private_Lean_Util_FileSetupInfo_0__Lean_toJsonFileSetupInfo____x40_Lean_Util_FileSetupInfo___hyg_132____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } diff --git a/stage0/stdlib/Lean/Util/Paths.c b/stage0/stdlib/Lean/Util/Paths.c index 74cc605db6c5..c0633e6c3e92 100644 --- a/stage0/stdlib/Lean/Util/Paths.c +++ b/stage0/stdlib/Lean/Util/Paths.c @@ -52,6 +52,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Util_Paths_0__Lean_fromJsonLeanPaths__ static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Paths_0__Lean_fromJsonLeanPaths____x40_Lean_Util_Paths___hyg_106____spec__1___closed__1; LEAN_EXPORT uint8_t l___private_Lean_Util_Paths_0__Lean_fromJsonLeanPaths____x40_Lean_Util_Paths___hyg_106____lambda__1(lean_object*); static lean_object* l_Lean_initSrcSearchPath___closed__4; +LEAN_EXPORT 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_Util_Paths_0__Lean_fromJsonLeanPaths____x40_Lean_Util_Paths___hyg_106____closed__12; LEAN_EXPORT lean_object* l_Lean_instToJsonLeanPaths; static lean_object* l___private_Lean_Util_Paths_0__Lean_fromJsonLeanPaths____x40_Lean_Util_Paths___hyg_106____closed__15; @@ -60,7 +61,6 @@ static lean_object* l___private_Lean_Util_Paths_0__Lean_fromJsonLeanPaths____x40 LEAN_EXPORT lean_object* l___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40_(lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____closed__2; -LEAN_EXPORT lean_object* l_List_bindTR_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_Util_Paths_0__Lean_fromJsonLeanPaths____x40_Lean_Util_Paths___hyg_106____closed__18; static lean_object* l___private_Lean_Util_Paths_0__Lean_fromJsonLeanPaths____x40_Lean_Util_Paths___hyg_106____closed__17; static lean_object* l___private_Lean_Util_Paths_0__Lean_fromJsonLeanPaths____x40_Lean_Util_Paths___hyg_106____closed__9; @@ -109,7 +109,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -224,7 +224,7 @@ x_29 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_29, 0, x_13); lean_ctor_set(x_29, 1, x_28); x_30 = l___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____closed__4; -x_31 = l_List_bindTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_29, x_30); +x_31 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_29, x_30); x_32 = l_Lean_Json_mkObj(x_31); return x_32; } diff --git a/stage0/stdlib/Lean/Util/Profiler.c b/stage0/stdlib/Lean/Util/Profiler.c index f4befe5f2bb0..5e9b5cad6ba3 100644 --- a/stage0/stdlib/Lean/Util/Profiler.c +++ b/stage0/stdlib/Lean/Util/Profiler.c @@ -161,6 +161,7 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStack LEAN_EXPORT lean_object* l_Lean_Firefox_instFromJsonThread; static lean_object* l_Lean_Firefox_instFromJsonCategory___closed__1; LEAN_EXPORT lean_object* l_Lean_Firefox_Profile_collide(lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfile____x40_Lean_Util_Profiler___hyg_3535____closed__14; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1172____closed__3; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfile____x40_Lean_Util_Profiler___hyg_3535____spec__2___boxed(lean_object*, lean_object*); @@ -403,7 +404,6 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncT LEAN_EXPORT uint8_t l___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Firefox_instFromJsonProfile; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_1585____closed__1; -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonProfileMeta____x40_Lean_Util_Profiler___hyg_634_(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonRawMarkerTable____x40_Lean_Util_Profiler___hyg_2419_(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__30(uint8_t, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); @@ -1323,7 +1323,7 @@ x_23 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_23, 0, x_9); lean_ctor_set(x_23, 1, x_22); x_24 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_25 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_23, x_24); +x_25 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_23, x_24); x_26 = l_Lean_Json_mkObj(x_25); return x_26; } @@ -2751,7 +2751,7 @@ x_53 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_53, 0, x_47); lean_ctor_set(x_53, 1, x_52); x_54 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_55 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_53, x_54); +x_55 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_53, x_54); x_56 = l_Lean_Json_mkObj(x_55); return x_56; } @@ -2777,7 +2777,7 @@ x_63 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_63, 0, x_47); lean_ctor_set(x_63, 1, x_62); x_64 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_65 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_63, x_64); +x_65 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_63, x_64); x_66 = l_Lean_Json_mkObj(x_65); return x_66; } @@ -2804,7 +2804,7 @@ x_72 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_72, 0, x_47); lean_ctor_set(x_72, 1, x_71); x_73 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_74 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_72, x_73); +x_74 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_72, x_73); x_75 = l_Lean_Json_mkObj(x_74); return x_75; } @@ -2830,7 +2830,7 @@ x_82 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_82, 0, x_47); lean_ctor_set(x_82, 1, x_81); x_83 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_84 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_82, x_83); +x_84 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_82, x_83); x_85 = l_Lean_Json_mkObj(x_84); return x_85; } @@ -2884,7 +2884,7 @@ x_98 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_98, 0, x_90); lean_ctor_set(x_98, 1, x_97); x_99 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_100 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_98, x_99); +x_100 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_98, x_99); x_101 = l_Lean_Json_mkObj(x_100); return x_101; } @@ -2921,7 +2921,7 @@ x_109 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_109, 0, x_90); lean_ctor_set(x_109, 1, x_108); x_110 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_111 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_109, x_110); +x_111 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_109, x_110); x_112 = l_Lean_Json_mkObj(x_111); return x_112; } @@ -2964,7 +2964,7 @@ x_122 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_122, 0, x_116); lean_ctor_set(x_122, 1, x_121); x_123 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_124 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_122, x_123); +x_124 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_122, x_123); x_125 = l_Lean_Json_mkObj(x_124); return x_125; } @@ -2990,7 +2990,7 @@ x_132 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_132, 0, x_116); lean_ctor_set(x_132, 1, x_131); x_133 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_134 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_132, x_133); +x_134 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_132, x_133); x_135 = l_Lean_Json_mkObj(x_134); return x_135; } @@ -3017,7 +3017,7 @@ x_141 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_141, 0, x_116); lean_ctor_set(x_141, 1, x_140); x_142 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_143 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_141, x_142); +x_143 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_141, x_142); x_144 = l_Lean_Json_mkObj(x_143); return x_144; } @@ -3043,7 +3043,7 @@ x_151 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_151, 0, x_116); lean_ctor_set(x_151, 1, x_150); x_152 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_153 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_151, x_152); +x_153 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_151, x_152); x_154 = l_Lean_Json_mkObj(x_153); return x_154; } @@ -3097,7 +3097,7 @@ x_167 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_167, 0, x_159); lean_ctor_set(x_167, 1, x_166); x_168 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_169 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_167, x_168); +x_169 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_167, x_168); x_170 = l_Lean_Json_mkObj(x_169); return x_170; } @@ -3134,7 +3134,7 @@ x_178 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_178, 0, x_159); lean_ctor_set(x_178, 1, x_177); x_179 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_180 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_178, x_179); +x_180 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_178, x_179); x_181 = l_Lean_Json_mkObj(x_180); return x_181; } @@ -4301,7 +4301,7 @@ x_42 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_42, 0, x_10); lean_ctor_set(x_42, 1, x_41); x_43 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_44 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_42, x_43); +x_44 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_42, x_43); x_45 = l_Lean_Json_mkObj(x_44); return x_45; } @@ -5224,7 +5224,7 @@ x_40 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_40, 0, x_10); lean_ctor_set(x_40, 1, x_39); x_41 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_42 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_40, x_41); +x_42 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_40, x_41); x_43 = l_Lean_Json_mkObj(x_42); return x_43; } @@ -6347,7 +6347,7 @@ x_66 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_66, 0, x_10); lean_ctor_set(x_66, 1, x_65); x_67 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_68 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_66, x_67); +x_68 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_66, x_67); x_69 = l_Lean_Json_mkObj(x_68); return x_69; } @@ -6865,7 +6865,7 @@ x_34 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_34, 0, x_10); lean_ctor_set(x_34, 1, x_33); x_35 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_36 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_34, x_35); +x_36 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_34, x_35); x_37 = l_Lean_Json_mkObj(x_36); return x_37; } @@ -7233,7 +7233,7 @@ x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_10); lean_ctor_set(x_26, 1, x_25); x_27 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_28 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } @@ -7522,7 +7522,7 @@ x_18 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_18, 0, x_10); lean_ctor_set(x_18, 1, x_17); x_19 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_20 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_18, x_19); +x_20 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_18, x_19); x_21 = l_Lean_Json_mkObj(x_20); return x_21; } @@ -8762,7 +8762,7 @@ x_65 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_65, 0, x_16); lean_ctor_set(x_65, 1, x_64); x_66 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_67 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_65, x_66); +x_67 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_65, x_66); x_68 = l_Lean_Json_mkObj(x_67); return x_68; } @@ -9388,7 +9388,7 @@ x_25 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_25, 0, x_7); lean_ctor_set(x_25, 1, x_24); x_26 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_189____closed__1; -x_27 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_25, x_26); +x_27 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_25, x_26); x_28 = l_Lean_Json_mkObj(x_27); return x_28; } diff --git a/stage0/stdlib/Lean/Util/Recognizers.c b/stage0/stdlib/Lean/Util/Recognizers.c index 98c038c5e35c..06b430b9fbf2 100644 --- a/stage0/stdlib/Lean/Util/Recognizers.c +++ b/stage0/stdlib/Lean/Util/Recognizers.c @@ -13,22 +13,29 @@ #ifdef __cplusplus extern "C" { #endif +lean_object* l_Lean_Expr_rawNatLit_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_and_x3f(lean_object*); static lean_object* l_Lean_Expr_natAdd_x3f___closed__2; +static lean_object* l_Lean_Expr_name_x3f___closed__1; static lean_object* l_Lean_Expr_heq_x3f___closed__2; static lean_object* l_Lean_Expr_listLit_x3f_loop___closed__1; LEAN_EXPORT uint8_t l_Lean_Expr_isDIte(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_arrow_x3f___boxed(lean_object*); static lean_object* l_Lean_Expr_not_x3f___closed__2; +static lean_object* l_Lean_Expr_name_x3f___closed__6; static lean_object* l_Lean_Expr_eq_x3f___closed__1; +LEAN_EXPORT lean_object* l_Lean_Expr_name_x3f(lean_object*); static lean_object* l_Lean_Expr_arrayLit_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_isHEq___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_app1_x3f(lean_object*, lean_object*); uint8_t l_Lean_Expr_isAppOfArity(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_natAdd_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_not_x3f___boxed(lean_object*); +static lean_object* l_Lean_Expr_name_x3f___closed__10; +static lean_object* l_Lean_Expr_name_x3f___closed__11; LEAN_EXPORT lean_object* l_Lean_Expr_eq_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_notNot_x3f(lean_object*); +static lean_object* l_Lean_Expr_name_x3f___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_not_x3f(lean_object*); static lean_object* l_Lean_Expr_isIte___closed__2; static lean_object* l_Lean_Expr_prod_x3f___closed__1; @@ -38,24 +45,33 @@ LEAN_EXPORT lean_object* l_Lean_Expr_arrayLit_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ne_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_app3_x3f(lean_object*, lean_object*); static lean_object* l_Lean_Expr_and_x3f___closed__2; +lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_appFn_x21_x27(lean_object*); +uint8_t lean_string_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ne_x3f___boxed(lean_object*); lean_object* l_Lean_Expr_appArg_x21(lean_object*); static lean_object* l_Lean_Expr_arrayLit_x3f___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_app4_x3f___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Expr_name_x3f___closed__7; +lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_natAdd_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_eqOrIff_x3f(lean_object*); +static lean_object* l_Lean_Expr_name_x3f___closed__3; uint8_t l_Lean_Expr_isAppOfArity_x27(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_const_x3f(lean_object*); +lean_object* l_Lean_Name_mkStr7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_and_x3f___boxed(lean_object*); static lean_object* l_Lean_Expr_heq_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_iff_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_isEq___boxed(lean_object*); static lean_object* l_Lean_Expr_listLit_x3f_loop___closed__2; LEAN_EXPORT uint8_t l_Lean_Expr_isEq(lean_object*); +static lean_object* l_Lean_Expr_name_x3f___closed__8; LEAN_EXPORT lean_object* l_Lean_Expr_arrow_x3f(lean_object*); +static lean_object* l_Lean_Expr_name_x3f___closed__5; uint8_t l_Lean_Expr_hasLooseBVars(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_listLit_x3f(lean_object*); +lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_prod_x3f(lean_object*); static lean_object* l_Lean_Expr_and_x3f___closed__1; static lean_object* l_Lean_Expr_natAdd_x3f___closed__1; @@ -64,16 +80,20 @@ LEAN_EXPORT lean_object* l_Lean_Expr_listLit_x3f_loop(lean_object*, lean_object* static lean_object* l_Lean_Expr_ne_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_isDIte___boxed(lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +static lean_object* l_Lean_Expr_name_x3f___closed__12; static lean_object* l_Lean_Expr_isDIte___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_app2_x3f(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_isIte(lean_object*); static lean_object* l_Lean_Expr_listLit_x3f_loop___closed__3; lean_object* l_Lean_Expr_appFn_x21(lean_object*); +static lean_object* l_Lean_Expr_name_x3f___closed__14; LEAN_EXPORT lean_object* l_Lean_Expr_eqOrIff_x3f___boxed(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_Expr_isDIte___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_arrayLit_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_app1_x3f___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Expr_natAdd_x3f___closed__3; +static lean_object* l_Lean_Expr_name_x3f___closed__9; static lean_object* l_Lean_Expr_iff_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_eq_x3f(lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); @@ -82,6 +102,7 @@ LEAN_EXPORT uint8_t l_Lean_Expr_isHEq(lean_object*); static lean_object* l_Lean_Expr_listLit_x3f_loop___closed__4; LEAN_EXPORT lean_object* l_Lean_Expr_app4_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_iff_x3f___boxed(lean_object*); +static lean_object* l_Lean_Expr_name_x3f___closed__4; LEAN_EXPORT lean_object* l_Lean_Expr_heq_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_prod_x3f___boxed(lean_object*); lean_object* l_List_reverse___rarg(lean_object*); @@ -89,12 +110,16 @@ LEAN_EXPORT lean_object* l_Lean_Expr_isIte___boxed(lean_object*); lean_object* l_Lean_Expr_appArg_x21_x27(lean_object*); static lean_object* l_Lean_Expr_iff_x3f___closed__2; static lean_object* l_Lean_Expr_prod_x3f___closed__2; +lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_heq_x3f(lean_object*); static lean_object* l_Lean_Expr_eq_x3f___closed__2; +static lean_object* l_Lean_Expr_name_x3f___closed__13; LEAN_EXPORT lean_object* l_Lean_Expr_notNot_x3f___boxed(lean_object*); +lean_object* l_Lean_Expr_nat_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_app3_x3f___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Expr_isIte___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_app2_x3f___boxed(lean_object*, lean_object*); +lean_object* l_Lean_Name_mkStr8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_const_x3f(lean_object* x_1) { _start: { @@ -1187,6 +1212,3298 @@ lean_dec(x_1); return x_2; } } +static lean_object* _init_l_Lean_Expr_name_x3f___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_Expr_name_x3f___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Name", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("anonymous", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__4() { +_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; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr1", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("str", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("num", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr2", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr3", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__10() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr4", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__11() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr5", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__12() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr6", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__13() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr7", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Expr_name_x3f___closed__14() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("mkStr8", 6, 6); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Expr_name_x3f(lean_object* x_1) { +_start: +{ +switch (lean_obj_tag(x_1)) { +case 4: +{ +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) == 1) +{ +lean_object* x_3; +x_3 = lean_ctor_get(x_2, 0); +lean_inc(x_3); +if (lean_obj_tag(x_3) == 1) +{ +lean_object* x_4; +x_4 = lean_ctor_get(x_3, 0); +lean_inc(x_4); +if (lean_obj_tag(x_4) == 1) +{ +lean_object* x_5; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; +x_6 = lean_ctor_get(x_2, 1); +lean_inc(x_6); +lean_dec(x_2); +x_7 = lean_ctor_get(x_3, 1); +lean_inc(x_7); +lean_dec(x_3); +x_8 = lean_ctor_get(x_4, 1); +lean_inc(x_8); +lean_dec(x_4); +x_9 = l_Lean_Expr_name_x3f___closed__1; +x_10 = lean_string_dec_eq(x_8, x_9); +lean_dec(x_8); +if (x_10 == 0) +{ +lean_object* x_11; +lean_dec(x_7); +lean_dec(x_6); +x_11 = lean_box(0); +return x_11; +} +else +{ +lean_object* x_12; uint8_t x_13; +x_12 = l_Lean_Expr_name_x3f___closed__2; +x_13 = lean_string_dec_eq(x_7, x_12); +lean_dec(x_7); +if (x_13 == 0) +{ +lean_object* x_14; +lean_dec(x_6); +x_14 = lean_box(0); +return x_14; +} +else +{ +lean_object* x_15; uint8_t x_16; +x_15 = l_Lean_Expr_name_x3f___closed__3; +x_16 = lean_string_dec_eq(x_6, x_15); +lean_dec(x_6); +if (x_16 == 0) +{ +lean_object* x_17; +x_17 = lean_box(0); +return x_17; +} +else +{ +lean_object* x_18; +x_18 = l_Lean_Expr_name_x3f___closed__4; +return x_18; +} +} +} +} +else +{ +lean_object* x_19; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_19 = lean_box(0); +return x_19; +} +} +else +{ +lean_object* x_20; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_20 = lean_box(0); +return x_20; +} +} +else +{ +lean_object* x_21; +lean_dec(x_3); +lean_dec(x_2); +x_21 = lean_box(0); +return x_21; +} +} +else +{ +lean_object* x_22; +lean_dec(x_2); +x_22 = lean_box(0); +return x_22; +} +} +case 5: +{ +lean_object* x_23; +x_23 = lean_ctor_get(x_1, 0); +lean_inc(x_23); +switch (lean_obj_tag(x_23)) { +case 4: +{ +lean_object* x_24; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +lean_dec(x_23); +if (lean_obj_tag(x_24) == 1) +{ +lean_object* x_25; +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +if (lean_obj_tag(x_25) == 1) +{ +lean_object* x_26; +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +if (lean_obj_tag(x_26) == 1) +{ +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; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +lean_dec(x_1); +x_29 = lean_ctor_get(x_24, 1); +lean_inc(x_29); +lean_dec(x_24); +x_30 = lean_ctor_get(x_25, 1); +lean_inc(x_30); +lean_dec(x_25); +x_31 = lean_ctor_get(x_26, 1); +lean_inc(x_31); +lean_dec(x_26); +x_32 = l_Lean_Expr_name_x3f___closed__1; +x_33 = lean_string_dec_eq(x_31, x_32); +lean_dec(x_31); +if (x_33 == 0) +{ +lean_object* x_34; +lean_dec(x_30); +lean_dec(x_29); +lean_dec(x_28); +x_34 = lean_box(0); +return x_34; +} +else +{ +lean_object* x_35; uint8_t x_36; +x_35 = l_Lean_Expr_name_x3f___closed__2; +x_36 = lean_string_dec_eq(x_30, x_35); +lean_dec(x_30); +if (x_36 == 0) +{ +lean_object* x_37; +lean_dec(x_29); +lean_dec(x_28); +x_37 = lean_box(0); +return x_37; +} +else +{ +lean_object* x_38; uint8_t x_39; +x_38 = l_Lean_Expr_name_x3f___closed__5; +x_39 = lean_string_dec_eq(x_29, x_38); +lean_dec(x_29); +if (x_39 == 0) +{ +lean_object* x_40; +lean_dec(x_28); +x_40 = lean_box(0); +return x_40; +} +else +{ +if (lean_obj_tag(x_28) == 9) +{ +lean_object* x_41; +x_41 = lean_ctor_get(x_28, 0); +lean_inc(x_41); +lean_dec(x_28); +if (lean_obj_tag(x_41) == 0) +{ +lean_object* x_42; +lean_dec(x_41); +x_42 = lean_box(0); +return x_42; +} +else +{ +uint8_t x_43; +x_43 = !lean_is_exclusive(x_41); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_41, 0); +x_45 = lean_box(0); +x_46 = l_Lean_Name_str___override(x_45, x_44); +lean_ctor_set(x_41, 0, x_46); +return x_41; +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_47 = lean_ctor_get(x_41, 0); +lean_inc(x_47); +lean_dec(x_41); +x_48 = lean_box(0); +x_49 = l_Lean_Name_str___override(x_48, x_47); +x_50 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_50, 0, x_49); +return x_50; +} +} +} +else +{ +lean_object* x_51; +lean_dec(x_28); +x_51 = lean_box(0); +return x_51; +} +} +} +} +} +else +{ +lean_object* x_52; +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_24); +lean_dec(x_1); +x_52 = lean_box(0); +return x_52; +} +} +else +{ +lean_object* x_53; +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_24); +lean_dec(x_1); +x_53 = lean_box(0); +return x_53; +} +} +else +{ +lean_object* x_54; +lean_dec(x_25); +lean_dec(x_24); +lean_dec(x_1); +x_54 = lean_box(0); +return x_54; +} +} +else +{ +lean_object* x_55; +lean_dec(x_24); +lean_dec(x_1); +x_55 = lean_box(0); +return x_55; +} +} +case 5: +{ +lean_object* x_56; +x_56 = lean_ctor_get(x_23, 0); +lean_inc(x_56); +switch (lean_obj_tag(x_56)) { +case 4: +{ +lean_object* x_57; +x_57 = lean_ctor_get(x_56, 0); +lean_inc(x_57); +lean_dec(x_56); +if (lean_obj_tag(x_57) == 1) +{ +lean_object* x_58; +x_58 = lean_ctor_get(x_57, 0); +lean_inc(x_58); +if (lean_obj_tag(x_58) == 1) +{ +lean_object* x_59; +x_59 = lean_ctor_get(x_58, 0); +lean_inc(x_59); +if (lean_obj_tag(x_59) == 1) +{ +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; lean_object* x_65; lean_object* x_66; uint8_t x_67; +x_61 = lean_ctor_get(x_1, 1); +lean_inc(x_61); +lean_dec(x_1); +x_62 = lean_ctor_get(x_23, 1); +lean_inc(x_62); +lean_dec(x_23); +x_63 = lean_ctor_get(x_57, 1); +lean_inc(x_63); +lean_dec(x_57); +x_64 = lean_ctor_get(x_58, 1); +lean_inc(x_64); +lean_dec(x_58); +x_65 = lean_ctor_get(x_59, 1); +lean_inc(x_65); +lean_dec(x_59); +x_66 = l_Lean_Expr_name_x3f___closed__1; +x_67 = lean_string_dec_eq(x_65, x_66); +lean_dec(x_65); +if (x_67 == 0) +{ +lean_object* x_68; +lean_dec(x_64); +lean_dec(x_63); +lean_dec(x_62); +lean_dec(x_61); +x_68 = lean_box(0); +return x_68; +} +else +{ +lean_object* x_69; uint8_t x_70; +x_69 = l_Lean_Expr_name_x3f___closed__2; +x_70 = lean_string_dec_eq(x_64, x_69); +lean_dec(x_64); +if (x_70 == 0) +{ +lean_object* x_71; +lean_dec(x_63); +lean_dec(x_62); +lean_dec(x_61); +x_71 = lean_box(0); +return x_71; +} +else +{ +lean_object* x_72; uint8_t x_73; +x_72 = l_Lean_Expr_name_x3f___closed__6; +x_73 = lean_string_dec_eq(x_63, x_72); +if (x_73 == 0) +{ +lean_object* x_74; uint8_t x_75; +x_74 = l_Lean_Expr_name_x3f___closed__7; +x_75 = lean_string_dec_eq(x_63, x_74); +if (x_75 == 0) +{ +lean_object* x_76; uint8_t x_77; +x_76 = l_Lean_Expr_name_x3f___closed__8; +x_77 = lean_string_dec_eq(x_63, x_76); +lean_dec(x_63); +if (x_77 == 0) +{ +lean_object* x_78; +lean_dec(x_62); +lean_dec(x_61); +x_78 = lean_box(0); +return x_78; +} +else +{ +if (lean_obj_tag(x_62) == 9) +{ +lean_object* x_79; +x_79 = lean_ctor_get(x_62, 0); +lean_inc(x_79); +lean_dec(x_62); +if (lean_obj_tag(x_79) == 0) +{ +lean_object* x_80; +lean_dec(x_79); +lean_dec(x_61); +x_80 = lean_box(0); +return x_80; +} +else +{ +if (lean_obj_tag(x_61) == 9) +{ +lean_object* x_81; +x_81 = lean_ctor_get(x_61, 0); +lean_inc(x_81); +lean_dec(x_61); +if (lean_obj_tag(x_81) == 0) +{ +lean_object* x_82; +lean_dec(x_81); +lean_dec(x_79); +x_82 = lean_box(0); +return x_82; +} +else +{ +lean_object* x_83; uint8_t x_84; +x_83 = lean_ctor_get(x_79, 0); +lean_inc(x_83); +lean_dec(x_79); +x_84 = !lean_is_exclusive(x_81); +if (x_84 == 0) +{ +lean_object* x_85; lean_object* x_86; +x_85 = lean_ctor_get(x_81, 0); +x_86 = l_Lean_Name_mkStr2(x_83, x_85); +lean_ctor_set(x_81, 0, x_86); +return x_81; +} +else +{ +lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_87 = lean_ctor_get(x_81, 0); +lean_inc(x_87); +lean_dec(x_81); +x_88 = l_Lean_Name_mkStr2(x_83, x_87); +x_89 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_89, 0, x_88); +return x_89; +} +} +} +else +{ +lean_object* x_90; +lean_dec(x_79); +lean_dec(x_61); +x_90 = lean_box(0); +return x_90; +} +} +} +else +{ +lean_object* x_91; +lean_dec(x_62); +lean_dec(x_61); +x_91 = lean_box(0); +return x_91; +} +} +} +else +{ +lean_object* x_92; +lean_dec(x_63); +lean_inc(x_61); +x_92 = l_Lean_Expr_rawNatLit_x3f(x_61); +if (lean_obj_tag(x_92) == 0) +{ +lean_object* x_93; +x_93 = l_Lean_Expr_nat_x3f(x_61); +if (lean_obj_tag(x_93) == 0) +{ +lean_object* x_94; +lean_dec(x_62); +x_94 = lean_box(0); +return x_94; +} +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 = l_Lean_Expr_name_x3f(x_62); +if (lean_obj_tag(x_96) == 0) +{ +lean_object* x_97; +lean_dec(x_95); +x_97 = lean_box(0); +return x_97; +} +else +{ +uint8_t x_98; +x_98 = !lean_is_exclusive(x_96); +if (x_98 == 0) +{ +lean_object* x_99; lean_object* x_100; +x_99 = lean_ctor_get(x_96, 0); +x_100 = l_Lean_Name_num___override(x_99, x_95); +lean_ctor_set(x_96, 0, x_100); +return x_96; +} +else +{ +lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_101 = lean_ctor_get(x_96, 0); +lean_inc(x_101); +lean_dec(x_96); +x_102 = l_Lean_Name_num___override(x_101, x_95); +x_103 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_103, 0, x_102); +return x_103; +} +} +} +} +else +{ +lean_object* x_104; lean_object* x_105; +lean_dec(x_61); +x_104 = lean_ctor_get(x_92, 0); +lean_inc(x_104); +lean_dec(x_92); +x_105 = l_Lean_Expr_name_x3f(x_62); +if (lean_obj_tag(x_105) == 0) +{ +lean_object* x_106; +lean_dec(x_104); +x_106 = lean_box(0); +return x_106; +} +else +{ +uint8_t x_107; +x_107 = !lean_is_exclusive(x_105); +if (x_107 == 0) +{ +lean_object* x_108; lean_object* x_109; +x_108 = lean_ctor_get(x_105, 0); +x_109 = l_Lean_Name_num___override(x_108, x_104); +lean_ctor_set(x_105, 0, x_109); +return x_105; +} +else +{ +lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_110 = lean_ctor_get(x_105, 0); +lean_inc(x_110); +lean_dec(x_105); +x_111 = l_Lean_Name_num___override(x_110, x_104); +x_112 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_112, 0, x_111); +return x_112; +} +} +} +} +} +else +{ +lean_dec(x_63); +if (lean_obj_tag(x_61) == 9) +{ +lean_object* x_113; +x_113 = lean_ctor_get(x_61, 0); +lean_inc(x_113); +lean_dec(x_61); +if (lean_obj_tag(x_113) == 0) +{ +lean_object* x_114; +lean_dec(x_113); +lean_dec(x_62); +x_114 = lean_box(0); +return x_114; +} +else +{ +lean_object* x_115; lean_object* x_116; +x_115 = lean_ctor_get(x_113, 0); +lean_inc(x_115); +lean_dec(x_113); +x_116 = l_Lean_Expr_name_x3f(x_62); +if (lean_obj_tag(x_116) == 0) +{ +lean_object* x_117; +lean_dec(x_115); +x_117 = lean_box(0); +return x_117; +} +else +{ +uint8_t x_118; +x_118 = !lean_is_exclusive(x_116); +if (x_118 == 0) +{ +lean_object* x_119; lean_object* x_120; +x_119 = lean_ctor_get(x_116, 0); +x_120 = l_Lean_Name_str___override(x_119, x_115); +lean_ctor_set(x_116, 0, x_120); +return x_116; +} +else +{ +lean_object* x_121; lean_object* x_122; lean_object* x_123; +x_121 = lean_ctor_get(x_116, 0); +lean_inc(x_121); +lean_dec(x_116); +x_122 = l_Lean_Name_str___override(x_121, x_115); +x_123 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_123, 0, x_122); +return x_123; +} +} +} +} +else +{ +lean_object* x_124; +lean_dec(x_62); +lean_dec(x_61); +x_124 = lean_box(0); +return x_124; +} +} +} +} +} +else +{ +lean_object* x_125; +lean_dec(x_60); +lean_dec(x_59); +lean_dec(x_58); +lean_dec(x_57); +lean_dec(x_23); +lean_dec(x_1); +x_125 = lean_box(0); +return x_125; +} +} +else +{ +lean_object* x_126; +lean_dec(x_59); +lean_dec(x_58); +lean_dec(x_57); +lean_dec(x_23); +lean_dec(x_1); +x_126 = lean_box(0); +return x_126; +} +} +else +{ +lean_object* x_127; +lean_dec(x_58); +lean_dec(x_57); +lean_dec(x_23); +lean_dec(x_1); +x_127 = lean_box(0); +return x_127; +} +} +else +{ +lean_object* x_128; +lean_dec(x_57); +lean_dec(x_23); +lean_dec(x_1); +x_128 = lean_box(0); +return x_128; +} +} +case 5: +{ +lean_object* x_129; +x_129 = lean_ctor_get(x_56, 0); +lean_inc(x_129); +switch (lean_obj_tag(x_129)) { +case 4: +{ +lean_object* x_130; +x_130 = lean_ctor_get(x_129, 0); +lean_inc(x_130); +lean_dec(x_129); +if (lean_obj_tag(x_130) == 1) +{ +lean_object* x_131; +x_131 = lean_ctor_get(x_130, 0); +lean_inc(x_131); +if (lean_obj_tag(x_131) == 1) +{ +lean_object* x_132; +x_132 = lean_ctor_get(x_131, 0); +lean_inc(x_132); +if (lean_obj_tag(x_132) == 1) +{ +lean_object* x_133; +x_133 = lean_ctor_get(x_132, 0); +lean_inc(x_133); +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; uint8_t x_141; +x_134 = lean_ctor_get(x_1, 1); +lean_inc(x_134); +lean_dec(x_1); +x_135 = lean_ctor_get(x_23, 1); +lean_inc(x_135); +lean_dec(x_23); +x_136 = lean_ctor_get(x_56, 1); +lean_inc(x_136); +lean_dec(x_56); +x_137 = lean_ctor_get(x_130, 1); +lean_inc(x_137); +lean_dec(x_130); +x_138 = lean_ctor_get(x_131, 1); +lean_inc(x_138); +lean_dec(x_131); +x_139 = lean_ctor_get(x_132, 1); +lean_inc(x_139); +lean_dec(x_132); +x_140 = l_Lean_Expr_name_x3f___closed__1; +x_141 = lean_string_dec_eq(x_139, x_140); +lean_dec(x_139); +if (x_141 == 0) +{ +lean_object* x_142; +lean_dec(x_138); +lean_dec(x_137); +lean_dec(x_136); +lean_dec(x_135); +lean_dec(x_134); +x_142 = lean_box(0); +return x_142; +} +else +{ +lean_object* x_143; uint8_t x_144; +x_143 = l_Lean_Expr_name_x3f___closed__2; +x_144 = lean_string_dec_eq(x_138, x_143); +lean_dec(x_138); +if (x_144 == 0) +{ +lean_object* x_145; +lean_dec(x_137); +lean_dec(x_136); +lean_dec(x_135); +lean_dec(x_134); +x_145 = lean_box(0); +return x_145; +} +else +{ +lean_object* x_146; uint8_t x_147; +x_146 = l_Lean_Expr_name_x3f___closed__9; +x_147 = lean_string_dec_eq(x_137, x_146); +lean_dec(x_137); +if (x_147 == 0) +{ +lean_object* x_148; +lean_dec(x_136); +lean_dec(x_135); +lean_dec(x_134); +x_148 = lean_box(0); +return x_148; +} +else +{ +if (lean_obj_tag(x_136) == 9) +{ +lean_object* x_149; +x_149 = lean_ctor_get(x_136, 0); +lean_inc(x_149); +lean_dec(x_136); +if (lean_obj_tag(x_149) == 0) +{ +lean_object* x_150; +lean_dec(x_149); +lean_dec(x_135); +lean_dec(x_134); +x_150 = lean_box(0); +return x_150; +} +else +{ +if (lean_obj_tag(x_135) == 9) +{ +lean_object* x_151; +x_151 = lean_ctor_get(x_135, 0); +lean_inc(x_151); +lean_dec(x_135); +if (lean_obj_tag(x_151) == 0) +{ +lean_object* x_152; +lean_dec(x_151); +lean_dec(x_149); +lean_dec(x_134); +x_152 = lean_box(0); +return x_152; +} +else +{ +if (lean_obj_tag(x_134) == 9) +{ +lean_object* x_153; +x_153 = lean_ctor_get(x_134, 0); +lean_inc(x_153); +lean_dec(x_134); +if (lean_obj_tag(x_153) == 0) +{ +lean_object* x_154; +lean_dec(x_153); +lean_dec(x_151); +lean_dec(x_149); +x_154 = lean_box(0); +return x_154; +} +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 = lean_ctor_get(x_151, 0); +lean_inc(x_156); +lean_dec(x_151); +x_157 = !lean_is_exclusive(x_153); +if (x_157 == 0) +{ +lean_object* x_158; lean_object* x_159; +x_158 = lean_ctor_get(x_153, 0); +x_159 = l_Lean_Name_mkStr3(x_155, x_156, x_158); +lean_ctor_set(x_153, 0, x_159); +return x_153; +} +else +{ +lean_object* x_160; lean_object* x_161; lean_object* x_162; +x_160 = lean_ctor_get(x_153, 0); +lean_inc(x_160); +lean_dec(x_153); +x_161 = l_Lean_Name_mkStr3(x_155, x_156, x_160); +x_162 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_162, 0, x_161); +return x_162; +} +} +} +else +{ +lean_object* x_163; +lean_dec(x_151); +lean_dec(x_149); +lean_dec(x_134); +x_163 = lean_box(0); +return x_163; +} +} +} +else +{ +lean_object* x_164; +lean_dec(x_149); +lean_dec(x_135); +lean_dec(x_134); +x_164 = lean_box(0); +return x_164; +} +} +} +else +{ +lean_object* x_165; +lean_dec(x_136); +lean_dec(x_135); +lean_dec(x_134); +x_165 = lean_box(0); +return x_165; +} +} +} +} +} +else +{ +lean_object* x_166; +lean_dec(x_133); +lean_dec(x_132); +lean_dec(x_131); +lean_dec(x_130); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_166 = lean_box(0); +return x_166; +} +} +else +{ +lean_object* x_167; +lean_dec(x_132); +lean_dec(x_131); +lean_dec(x_130); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_167 = lean_box(0); +return x_167; +} +} +else +{ +lean_object* x_168; +lean_dec(x_131); +lean_dec(x_130); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_168 = lean_box(0); +return x_168; +} +} +else +{ +lean_object* x_169; +lean_dec(x_130); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_169 = lean_box(0); +return x_169; +} +} +case 5: +{ +lean_object* x_170; +x_170 = lean_ctor_get(x_129, 0); +lean_inc(x_170); +switch (lean_obj_tag(x_170)) { +case 4: +{ +lean_object* x_171; +x_171 = lean_ctor_get(x_170, 0); +lean_inc(x_171); +lean_dec(x_170); +if (lean_obj_tag(x_171) == 1) +{ +lean_object* x_172; +x_172 = lean_ctor_get(x_171, 0); +lean_inc(x_172); +if (lean_obj_tag(x_172) == 1) +{ +lean_object* x_173; +x_173 = lean_ctor_get(x_172, 0); +lean_inc(x_173); +if (lean_obj_tag(x_173) == 1) +{ +lean_object* x_174; +x_174 = lean_ctor_get(x_173, 0); +lean_inc(x_174); +if (lean_obj_tag(x_174) == 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; lean_object* x_182; uint8_t x_183; +x_175 = lean_ctor_get(x_1, 1); +lean_inc(x_175); +lean_dec(x_1); +x_176 = lean_ctor_get(x_23, 1); +lean_inc(x_176); +lean_dec(x_23); +x_177 = lean_ctor_get(x_56, 1); +lean_inc(x_177); +lean_dec(x_56); +x_178 = lean_ctor_get(x_129, 1); +lean_inc(x_178); +lean_dec(x_129); +x_179 = lean_ctor_get(x_171, 1); +lean_inc(x_179); +lean_dec(x_171); +x_180 = lean_ctor_get(x_172, 1); +lean_inc(x_180); +lean_dec(x_172); +x_181 = lean_ctor_get(x_173, 1); +lean_inc(x_181); +lean_dec(x_173); +x_182 = l_Lean_Expr_name_x3f___closed__1; +x_183 = lean_string_dec_eq(x_181, x_182); +lean_dec(x_181); +if (x_183 == 0) +{ +lean_object* x_184; +lean_dec(x_180); +lean_dec(x_179); +lean_dec(x_178); +lean_dec(x_177); +lean_dec(x_176); +lean_dec(x_175); +x_184 = lean_box(0); +return x_184; +} +else +{ +lean_object* x_185; uint8_t x_186; +x_185 = l_Lean_Expr_name_x3f___closed__2; +x_186 = lean_string_dec_eq(x_180, x_185); +lean_dec(x_180); +if (x_186 == 0) +{ +lean_object* x_187; +lean_dec(x_179); +lean_dec(x_178); +lean_dec(x_177); +lean_dec(x_176); +lean_dec(x_175); +x_187 = lean_box(0); +return x_187; +} +else +{ +lean_object* x_188; uint8_t x_189; +x_188 = l_Lean_Expr_name_x3f___closed__10; +x_189 = lean_string_dec_eq(x_179, x_188); +lean_dec(x_179); +if (x_189 == 0) +{ +lean_object* x_190; +lean_dec(x_178); +lean_dec(x_177); +lean_dec(x_176); +lean_dec(x_175); +x_190 = lean_box(0); +return x_190; +} +else +{ +if (lean_obj_tag(x_178) == 9) +{ +lean_object* x_191; +x_191 = lean_ctor_get(x_178, 0); +lean_inc(x_191); +lean_dec(x_178); +if (lean_obj_tag(x_191) == 0) +{ +lean_object* x_192; +lean_dec(x_191); +lean_dec(x_177); +lean_dec(x_176); +lean_dec(x_175); +x_192 = lean_box(0); +return x_192; +} +else +{ +if (lean_obj_tag(x_177) == 9) +{ +lean_object* x_193; +x_193 = lean_ctor_get(x_177, 0); +lean_inc(x_193); +lean_dec(x_177); +if (lean_obj_tag(x_193) == 0) +{ +lean_object* x_194; +lean_dec(x_193); +lean_dec(x_191); +lean_dec(x_176); +lean_dec(x_175); +x_194 = lean_box(0); +return x_194; +} +else +{ +if (lean_obj_tag(x_176) == 9) +{ +lean_object* x_195; +x_195 = lean_ctor_get(x_176, 0); +lean_inc(x_195); +lean_dec(x_176); +if (lean_obj_tag(x_195) == 0) +{ +lean_object* x_196; +lean_dec(x_195); +lean_dec(x_193); +lean_dec(x_191); +lean_dec(x_175); +x_196 = lean_box(0); +return x_196; +} +else +{ +if (lean_obj_tag(x_175) == 9) +{ +lean_object* x_197; +x_197 = lean_ctor_get(x_175, 0); +lean_inc(x_197); +lean_dec(x_175); +if (lean_obj_tag(x_197) == 0) +{ +lean_object* x_198; +lean_dec(x_197); +lean_dec(x_195); +lean_dec(x_193); +lean_dec(x_191); +x_198 = lean_box(0); +return x_198; +} +else +{ +lean_object* x_199; lean_object* x_200; lean_object* x_201; uint8_t x_202; +x_199 = lean_ctor_get(x_191, 0); +lean_inc(x_199); +lean_dec(x_191); +x_200 = lean_ctor_get(x_193, 0); +lean_inc(x_200); +lean_dec(x_193); +x_201 = lean_ctor_get(x_195, 0); +lean_inc(x_201); +lean_dec(x_195); +x_202 = !lean_is_exclusive(x_197); +if (x_202 == 0) +{ +lean_object* x_203; lean_object* x_204; +x_203 = lean_ctor_get(x_197, 0); +x_204 = l_Lean_Name_mkStr4(x_199, x_200, x_201, x_203); +lean_ctor_set(x_197, 0, x_204); +return x_197; +} +else +{ +lean_object* x_205; lean_object* x_206; lean_object* x_207; +x_205 = lean_ctor_get(x_197, 0); +lean_inc(x_205); +lean_dec(x_197); +x_206 = l_Lean_Name_mkStr4(x_199, x_200, x_201, x_205); +x_207 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_207, 0, x_206); +return x_207; +} +} +} +else +{ +lean_object* x_208; +lean_dec(x_195); +lean_dec(x_193); +lean_dec(x_191); +lean_dec(x_175); +x_208 = lean_box(0); +return x_208; +} +} +} +else +{ +lean_object* x_209; +lean_dec(x_193); +lean_dec(x_191); +lean_dec(x_176); +lean_dec(x_175); +x_209 = lean_box(0); +return x_209; +} +} +} +else +{ +lean_object* x_210; +lean_dec(x_191); +lean_dec(x_177); +lean_dec(x_176); +lean_dec(x_175); +x_210 = lean_box(0); +return x_210; +} +} +} +else +{ +lean_object* x_211; +lean_dec(x_178); +lean_dec(x_177); +lean_dec(x_176); +lean_dec(x_175); +x_211 = lean_box(0); +return x_211; +} +} +} +} +} +else +{ +lean_object* x_212; +lean_dec(x_174); +lean_dec(x_173); +lean_dec(x_172); +lean_dec(x_171); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_212 = lean_box(0); +return x_212; +} +} +else +{ +lean_object* x_213; +lean_dec(x_173); +lean_dec(x_172); +lean_dec(x_171); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_213 = lean_box(0); +return x_213; +} +} +else +{ +lean_object* x_214; +lean_dec(x_172); +lean_dec(x_171); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_214 = lean_box(0); +return x_214; +} +} +else +{ +lean_object* x_215; +lean_dec(x_171); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_215 = lean_box(0); +return x_215; +} +} +case 5: +{ +lean_object* x_216; +x_216 = lean_ctor_get(x_170, 0); +lean_inc(x_216); +switch (lean_obj_tag(x_216)) { +case 4: +{ +lean_object* x_217; +x_217 = lean_ctor_get(x_216, 0); +lean_inc(x_217); +lean_dec(x_216); +if (lean_obj_tag(x_217) == 1) +{ +lean_object* x_218; +x_218 = lean_ctor_get(x_217, 0); +lean_inc(x_218); +if (lean_obj_tag(x_218) == 1) +{ +lean_object* x_219; +x_219 = lean_ctor_get(x_218, 0); +lean_inc(x_219); +if (lean_obj_tag(x_219) == 1) +{ +lean_object* x_220; +x_220 = lean_ctor_get(x_219, 0); +lean_inc(x_220); +if (lean_obj_tag(x_220) == 0) +{ +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; uint8_t x_230; +x_221 = lean_ctor_get(x_1, 1); +lean_inc(x_221); +lean_dec(x_1); +x_222 = lean_ctor_get(x_23, 1); +lean_inc(x_222); +lean_dec(x_23); +x_223 = lean_ctor_get(x_56, 1); +lean_inc(x_223); +lean_dec(x_56); +x_224 = lean_ctor_get(x_129, 1); +lean_inc(x_224); +lean_dec(x_129); +x_225 = lean_ctor_get(x_170, 1); +lean_inc(x_225); +lean_dec(x_170); +x_226 = lean_ctor_get(x_217, 1); +lean_inc(x_226); +lean_dec(x_217); +x_227 = lean_ctor_get(x_218, 1); +lean_inc(x_227); +lean_dec(x_218); +x_228 = lean_ctor_get(x_219, 1); +lean_inc(x_228); +lean_dec(x_219); +x_229 = l_Lean_Expr_name_x3f___closed__1; +x_230 = lean_string_dec_eq(x_228, x_229); +lean_dec(x_228); +if (x_230 == 0) +{ +lean_object* x_231; +lean_dec(x_227); +lean_dec(x_226); +lean_dec(x_225); +lean_dec(x_224); +lean_dec(x_223); +lean_dec(x_222); +lean_dec(x_221); +x_231 = lean_box(0); +return x_231; +} +else +{ +lean_object* x_232; uint8_t x_233; +x_232 = l_Lean_Expr_name_x3f___closed__2; +x_233 = lean_string_dec_eq(x_227, x_232); +lean_dec(x_227); +if (x_233 == 0) +{ +lean_object* x_234; +lean_dec(x_226); +lean_dec(x_225); +lean_dec(x_224); +lean_dec(x_223); +lean_dec(x_222); +lean_dec(x_221); +x_234 = lean_box(0); +return x_234; +} +else +{ +lean_object* x_235; uint8_t x_236; +x_235 = l_Lean_Expr_name_x3f___closed__11; +x_236 = lean_string_dec_eq(x_226, x_235); +lean_dec(x_226); +if (x_236 == 0) +{ +lean_object* x_237; +lean_dec(x_225); +lean_dec(x_224); +lean_dec(x_223); +lean_dec(x_222); +lean_dec(x_221); +x_237 = lean_box(0); +return x_237; +} +else +{ +if (lean_obj_tag(x_225) == 9) +{ +lean_object* x_238; +x_238 = lean_ctor_get(x_225, 0); +lean_inc(x_238); +lean_dec(x_225); +if (lean_obj_tag(x_238) == 0) +{ +lean_object* x_239; +lean_dec(x_238); +lean_dec(x_224); +lean_dec(x_223); +lean_dec(x_222); +lean_dec(x_221); +x_239 = lean_box(0); +return x_239; +} +else +{ +if (lean_obj_tag(x_224) == 9) +{ +lean_object* x_240; +x_240 = lean_ctor_get(x_224, 0); +lean_inc(x_240); +lean_dec(x_224); +if (lean_obj_tag(x_240) == 0) +{ +lean_object* x_241; +lean_dec(x_240); +lean_dec(x_238); +lean_dec(x_223); +lean_dec(x_222); +lean_dec(x_221); +x_241 = lean_box(0); +return x_241; +} +else +{ +if (lean_obj_tag(x_223) == 9) +{ +lean_object* x_242; +x_242 = lean_ctor_get(x_223, 0); +lean_inc(x_242); +lean_dec(x_223); +if (lean_obj_tag(x_242) == 0) +{ +lean_object* x_243; +lean_dec(x_242); +lean_dec(x_240); +lean_dec(x_238); +lean_dec(x_222); +lean_dec(x_221); +x_243 = lean_box(0); +return x_243; +} +else +{ +if (lean_obj_tag(x_222) == 9) +{ +lean_object* x_244; +x_244 = lean_ctor_get(x_222, 0); +lean_inc(x_244); +lean_dec(x_222); +if (lean_obj_tag(x_244) == 0) +{ +lean_object* x_245; +lean_dec(x_244); +lean_dec(x_242); +lean_dec(x_240); +lean_dec(x_238); +lean_dec(x_221); +x_245 = lean_box(0); +return x_245; +} +else +{ +if (lean_obj_tag(x_221) == 9) +{ +lean_object* x_246; +x_246 = lean_ctor_get(x_221, 0); +lean_inc(x_246); +lean_dec(x_221); +if (lean_obj_tag(x_246) == 0) +{ +lean_object* x_247; +lean_dec(x_246); +lean_dec(x_244); +lean_dec(x_242); +lean_dec(x_240); +lean_dec(x_238); +x_247 = lean_box(0); +return x_247; +} +else +{ +lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; uint8_t x_252; +x_248 = lean_ctor_get(x_238, 0); +lean_inc(x_248); +lean_dec(x_238); +x_249 = lean_ctor_get(x_240, 0); +lean_inc(x_249); +lean_dec(x_240); +x_250 = lean_ctor_get(x_242, 0); +lean_inc(x_250); +lean_dec(x_242); +x_251 = lean_ctor_get(x_244, 0); +lean_inc(x_251); +lean_dec(x_244); +x_252 = !lean_is_exclusive(x_246); +if (x_252 == 0) +{ +lean_object* x_253; lean_object* x_254; +x_253 = lean_ctor_get(x_246, 0); +x_254 = l_Lean_Name_mkStr5(x_248, x_249, x_250, x_251, x_253); +lean_ctor_set(x_246, 0, x_254); +return x_246; +} +else +{ +lean_object* x_255; lean_object* x_256; lean_object* x_257; +x_255 = lean_ctor_get(x_246, 0); +lean_inc(x_255); +lean_dec(x_246); +x_256 = l_Lean_Name_mkStr5(x_248, x_249, x_250, x_251, x_255); +x_257 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_257, 0, x_256); +return x_257; +} +} +} +else +{ +lean_object* x_258; +lean_dec(x_244); +lean_dec(x_242); +lean_dec(x_240); +lean_dec(x_238); +lean_dec(x_221); +x_258 = lean_box(0); +return x_258; +} +} +} +else +{ +lean_object* x_259; +lean_dec(x_242); +lean_dec(x_240); +lean_dec(x_238); +lean_dec(x_222); +lean_dec(x_221); +x_259 = lean_box(0); +return x_259; +} +} +} +else +{ +lean_object* x_260; +lean_dec(x_240); +lean_dec(x_238); +lean_dec(x_223); +lean_dec(x_222); +lean_dec(x_221); +x_260 = lean_box(0); +return x_260; +} +} +} +else +{ +lean_object* x_261; +lean_dec(x_238); +lean_dec(x_224); +lean_dec(x_223); +lean_dec(x_222); +lean_dec(x_221); +x_261 = lean_box(0); +return x_261; +} +} +} +else +{ +lean_object* x_262; +lean_dec(x_225); +lean_dec(x_224); +lean_dec(x_223); +lean_dec(x_222); +lean_dec(x_221); +x_262 = lean_box(0); +return x_262; +} +} +} +} +} +else +{ +lean_object* x_263; +lean_dec(x_220); +lean_dec(x_219); +lean_dec(x_218); +lean_dec(x_217); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_263 = lean_box(0); +return x_263; +} +} +else +{ +lean_object* x_264; +lean_dec(x_219); +lean_dec(x_218); +lean_dec(x_217); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_264 = lean_box(0); +return x_264; +} +} +else +{ +lean_object* x_265; +lean_dec(x_218); +lean_dec(x_217); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_265 = lean_box(0); +return x_265; +} +} +else +{ +lean_object* x_266; +lean_dec(x_217); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_266 = lean_box(0); +return x_266; +} +} +case 5: +{ +lean_object* x_267; +x_267 = lean_ctor_get(x_216, 0); +lean_inc(x_267); +switch (lean_obj_tag(x_267)) { +case 4: +{ +lean_object* x_268; +x_268 = lean_ctor_get(x_267, 0); +lean_inc(x_268); +lean_dec(x_267); +if (lean_obj_tag(x_268) == 1) +{ +lean_object* x_269; +x_269 = lean_ctor_get(x_268, 0); +lean_inc(x_269); +if (lean_obj_tag(x_269) == 1) +{ +lean_object* x_270; +x_270 = lean_ctor_get(x_269, 0); +lean_inc(x_270); +if (lean_obj_tag(x_270) == 1) +{ +lean_object* x_271; +x_271 = lean_ctor_get(x_270, 0); +lean_inc(x_271); +if (lean_obj_tag(x_271) == 0) +{ +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; uint8_t x_282; +x_272 = lean_ctor_get(x_1, 1); +lean_inc(x_272); +lean_dec(x_1); +x_273 = lean_ctor_get(x_23, 1); +lean_inc(x_273); +lean_dec(x_23); +x_274 = lean_ctor_get(x_56, 1); +lean_inc(x_274); +lean_dec(x_56); +x_275 = lean_ctor_get(x_129, 1); +lean_inc(x_275); +lean_dec(x_129); +x_276 = lean_ctor_get(x_170, 1); +lean_inc(x_276); +lean_dec(x_170); +x_277 = lean_ctor_get(x_216, 1); +lean_inc(x_277); +lean_dec(x_216); +x_278 = lean_ctor_get(x_268, 1); +lean_inc(x_278); +lean_dec(x_268); +x_279 = lean_ctor_get(x_269, 1); +lean_inc(x_279); +lean_dec(x_269); +x_280 = lean_ctor_get(x_270, 1); +lean_inc(x_280); +lean_dec(x_270); +x_281 = l_Lean_Expr_name_x3f___closed__1; +x_282 = lean_string_dec_eq(x_280, x_281); +lean_dec(x_280); +if (x_282 == 0) +{ +lean_object* x_283; +lean_dec(x_279); +lean_dec(x_278); +lean_dec(x_277); +lean_dec(x_276); +lean_dec(x_275); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_283 = lean_box(0); +return x_283; +} +else +{ +lean_object* x_284; uint8_t x_285; +x_284 = l_Lean_Expr_name_x3f___closed__2; +x_285 = lean_string_dec_eq(x_279, x_284); +lean_dec(x_279); +if (x_285 == 0) +{ +lean_object* x_286; +lean_dec(x_278); +lean_dec(x_277); +lean_dec(x_276); +lean_dec(x_275); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_286 = lean_box(0); +return x_286; +} +else +{ +lean_object* x_287; uint8_t x_288; +x_287 = l_Lean_Expr_name_x3f___closed__12; +x_288 = lean_string_dec_eq(x_278, x_287); +lean_dec(x_278); +if (x_288 == 0) +{ +lean_object* x_289; +lean_dec(x_277); +lean_dec(x_276); +lean_dec(x_275); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_289 = lean_box(0); +return x_289; +} +else +{ +if (lean_obj_tag(x_277) == 9) +{ +lean_object* x_290; +x_290 = lean_ctor_get(x_277, 0); +lean_inc(x_290); +lean_dec(x_277); +if (lean_obj_tag(x_290) == 0) +{ +lean_object* x_291; +lean_dec(x_290); +lean_dec(x_276); +lean_dec(x_275); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_291 = lean_box(0); +return x_291; +} +else +{ +if (lean_obj_tag(x_276) == 9) +{ +lean_object* x_292; +x_292 = lean_ctor_get(x_276, 0); +lean_inc(x_292); +lean_dec(x_276); +if (lean_obj_tag(x_292) == 0) +{ +lean_object* x_293; +lean_dec(x_292); +lean_dec(x_290); +lean_dec(x_275); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_293 = lean_box(0); +return x_293; +} +else +{ +if (lean_obj_tag(x_275) == 9) +{ +lean_object* x_294; +x_294 = lean_ctor_get(x_275, 0); +lean_inc(x_294); +lean_dec(x_275); +if (lean_obj_tag(x_294) == 0) +{ +lean_object* x_295; +lean_dec(x_294); +lean_dec(x_292); +lean_dec(x_290); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_295 = lean_box(0); +return x_295; +} +else +{ +if (lean_obj_tag(x_274) == 9) +{ +lean_object* x_296; +x_296 = lean_ctor_get(x_274, 0); +lean_inc(x_296); +lean_dec(x_274); +if (lean_obj_tag(x_296) == 0) +{ +lean_object* x_297; +lean_dec(x_296); +lean_dec(x_294); +lean_dec(x_292); +lean_dec(x_290); +lean_dec(x_273); +lean_dec(x_272); +x_297 = lean_box(0); +return x_297; +} +else +{ +if (lean_obj_tag(x_273) == 9) +{ +lean_object* x_298; +x_298 = lean_ctor_get(x_273, 0); +lean_inc(x_298); +lean_dec(x_273); +if (lean_obj_tag(x_298) == 0) +{ +lean_object* x_299; +lean_dec(x_298); +lean_dec(x_296); +lean_dec(x_294); +lean_dec(x_292); +lean_dec(x_290); +lean_dec(x_272); +x_299 = lean_box(0); +return x_299; +} +else +{ +if (lean_obj_tag(x_272) == 9) +{ +lean_object* x_300; +x_300 = lean_ctor_get(x_272, 0); +lean_inc(x_300); +lean_dec(x_272); +if (lean_obj_tag(x_300) == 0) +{ +lean_object* x_301; +lean_dec(x_300); +lean_dec(x_298); +lean_dec(x_296); +lean_dec(x_294); +lean_dec(x_292); +lean_dec(x_290); +x_301 = lean_box(0); +return x_301; +} +else +{ +lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; uint8_t x_307; +x_302 = lean_ctor_get(x_290, 0); +lean_inc(x_302); +lean_dec(x_290); +x_303 = lean_ctor_get(x_292, 0); +lean_inc(x_303); +lean_dec(x_292); +x_304 = lean_ctor_get(x_294, 0); +lean_inc(x_304); +lean_dec(x_294); +x_305 = lean_ctor_get(x_296, 0); +lean_inc(x_305); +lean_dec(x_296); +x_306 = lean_ctor_get(x_298, 0); +lean_inc(x_306); +lean_dec(x_298); +x_307 = !lean_is_exclusive(x_300); +if (x_307 == 0) +{ +lean_object* x_308; lean_object* x_309; +x_308 = lean_ctor_get(x_300, 0); +x_309 = l_Lean_Name_mkStr6(x_302, x_303, x_304, x_305, x_306, x_308); +lean_ctor_set(x_300, 0, x_309); +return x_300; +} +else +{ +lean_object* x_310; lean_object* x_311; lean_object* x_312; +x_310 = lean_ctor_get(x_300, 0); +lean_inc(x_310); +lean_dec(x_300); +x_311 = l_Lean_Name_mkStr6(x_302, x_303, x_304, x_305, x_306, x_310); +x_312 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_312, 0, x_311); +return x_312; +} +} +} +else +{ +lean_object* x_313; +lean_dec(x_298); +lean_dec(x_296); +lean_dec(x_294); +lean_dec(x_292); +lean_dec(x_290); +lean_dec(x_272); +x_313 = lean_box(0); +return x_313; +} +} +} +else +{ +lean_object* x_314; +lean_dec(x_296); +lean_dec(x_294); +lean_dec(x_292); +lean_dec(x_290); +lean_dec(x_273); +lean_dec(x_272); +x_314 = lean_box(0); +return x_314; +} +} +} +else +{ +lean_object* x_315; +lean_dec(x_294); +lean_dec(x_292); +lean_dec(x_290); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_315 = lean_box(0); +return x_315; +} +} +} +else +{ +lean_object* x_316; +lean_dec(x_292); +lean_dec(x_290); +lean_dec(x_275); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_316 = lean_box(0); +return x_316; +} +} +} +else +{ +lean_object* x_317; +lean_dec(x_290); +lean_dec(x_276); +lean_dec(x_275); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_317 = lean_box(0); +return x_317; +} +} +} +else +{ +lean_object* x_318; +lean_dec(x_277); +lean_dec(x_276); +lean_dec(x_275); +lean_dec(x_274); +lean_dec(x_273); +lean_dec(x_272); +x_318 = lean_box(0); +return x_318; +} +} +} +} +} +else +{ +lean_object* x_319; +lean_dec(x_271); +lean_dec(x_270); +lean_dec(x_269); +lean_dec(x_268); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_319 = lean_box(0); +return x_319; +} +} +else +{ +lean_object* x_320; +lean_dec(x_270); +lean_dec(x_269); +lean_dec(x_268); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_320 = lean_box(0); +return x_320; +} +} +else +{ +lean_object* x_321; +lean_dec(x_269); +lean_dec(x_268); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_321 = lean_box(0); +return x_321; +} +} +else +{ +lean_object* x_322; +lean_dec(x_268); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_322 = lean_box(0); +return x_322; +} +} +case 5: +{ +lean_object* x_323; +x_323 = lean_ctor_get(x_267, 0); +lean_inc(x_323); +switch (lean_obj_tag(x_323)) { +case 4: +{ +lean_object* x_324; +x_324 = lean_ctor_get(x_323, 0); +lean_inc(x_324); +lean_dec(x_323); +if (lean_obj_tag(x_324) == 1) +{ +lean_object* x_325; +x_325 = lean_ctor_get(x_324, 0); +lean_inc(x_325); +if (lean_obj_tag(x_325) == 1) +{ +lean_object* x_326; +x_326 = lean_ctor_get(x_325, 0); +lean_inc(x_326); +if (lean_obj_tag(x_326) == 1) +{ +lean_object* x_327; +x_327 = lean_ctor_get(x_326, 0); +lean_inc(x_327); +if (lean_obj_tag(x_327) == 0) +{ +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; uint8_t x_339; +x_328 = lean_ctor_get(x_1, 1); +lean_inc(x_328); +lean_dec(x_1); +x_329 = lean_ctor_get(x_23, 1); +lean_inc(x_329); +lean_dec(x_23); +x_330 = lean_ctor_get(x_56, 1); +lean_inc(x_330); +lean_dec(x_56); +x_331 = lean_ctor_get(x_129, 1); +lean_inc(x_331); +lean_dec(x_129); +x_332 = lean_ctor_get(x_170, 1); +lean_inc(x_332); +lean_dec(x_170); +x_333 = lean_ctor_get(x_216, 1); +lean_inc(x_333); +lean_dec(x_216); +x_334 = lean_ctor_get(x_267, 1); +lean_inc(x_334); +lean_dec(x_267); +x_335 = lean_ctor_get(x_324, 1); +lean_inc(x_335); +lean_dec(x_324); +x_336 = lean_ctor_get(x_325, 1); +lean_inc(x_336); +lean_dec(x_325); +x_337 = lean_ctor_get(x_326, 1); +lean_inc(x_337); +lean_dec(x_326); +x_338 = l_Lean_Expr_name_x3f___closed__1; +x_339 = lean_string_dec_eq(x_337, x_338); +lean_dec(x_337); +if (x_339 == 0) +{ +lean_object* x_340; +lean_dec(x_336); +lean_dec(x_335); +lean_dec(x_334); +lean_dec(x_333); +lean_dec(x_332); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_340 = lean_box(0); +return x_340; +} +else +{ +lean_object* x_341; uint8_t x_342; +x_341 = l_Lean_Expr_name_x3f___closed__2; +x_342 = lean_string_dec_eq(x_336, x_341); +lean_dec(x_336); +if (x_342 == 0) +{ +lean_object* x_343; +lean_dec(x_335); +lean_dec(x_334); +lean_dec(x_333); +lean_dec(x_332); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_343 = lean_box(0); +return x_343; +} +else +{ +lean_object* x_344; uint8_t x_345; +x_344 = l_Lean_Expr_name_x3f___closed__13; +x_345 = lean_string_dec_eq(x_335, x_344); +lean_dec(x_335); +if (x_345 == 0) +{ +lean_object* x_346; +lean_dec(x_334); +lean_dec(x_333); +lean_dec(x_332); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_346 = lean_box(0); +return x_346; +} +else +{ +if (lean_obj_tag(x_334) == 9) +{ +lean_object* x_347; +x_347 = lean_ctor_get(x_334, 0); +lean_inc(x_347); +lean_dec(x_334); +if (lean_obj_tag(x_347) == 0) +{ +lean_object* x_348; +lean_dec(x_347); +lean_dec(x_333); +lean_dec(x_332); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_348 = lean_box(0); +return x_348; +} +else +{ +if (lean_obj_tag(x_333) == 9) +{ +lean_object* x_349; +x_349 = lean_ctor_get(x_333, 0); +lean_inc(x_349); +lean_dec(x_333); +if (lean_obj_tag(x_349) == 0) +{ +lean_object* x_350; +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_332); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_350 = lean_box(0); +return x_350; +} +else +{ +if (lean_obj_tag(x_332) == 9) +{ +lean_object* x_351; +x_351 = lean_ctor_get(x_332, 0); +lean_inc(x_351); +lean_dec(x_332); +if (lean_obj_tag(x_351) == 0) +{ +lean_object* x_352; +lean_dec(x_351); +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_352 = lean_box(0); +return x_352; +} +else +{ +if (lean_obj_tag(x_331) == 9) +{ +lean_object* x_353; +x_353 = lean_ctor_get(x_331, 0); +lean_inc(x_353); +lean_dec(x_331); +if (lean_obj_tag(x_353) == 0) +{ +lean_object* x_354; +lean_dec(x_353); +lean_dec(x_351); +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_354 = lean_box(0); +return x_354; +} +else +{ +if (lean_obj_tag(x_330) == 9) +{ +lean_object* x_355; +x_355 = lean_ctor_get(x_330, 0); +lean_inc(x_355); +lean_dec(x_330); +if (lean_obj_tag(x_355) == 0) +{ +lean_object* x_356; +lean_dec(x_355); +lean_dec(x_353); +lean_dec(x_351); +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_329); +lean_dec(x_328); +x_356 = lean_box(0); +return x_356; +} +else +{ +if (lean_obj_tag(x_329) == 9) +{ +lean_object* x_357; +x_357 = lean_ctor_get(x_329, 0); +lean_inc(x_357); +lean_dec(x_329); +if (lean_obj_tag(x_357) == 0) +{ +lean_object* x_358; +lean_dec(x_357); +lean_dec(x_355); +lean_dec(x_353); +lean_dec(x_351); +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_328); +x_358 = lean_box(0); +return x_358; +} +else +{ +if (lean_obj_tag(x_328) == 9) +{ +lean_object* x_359; +x_359 = lean_ctor_get(x_328, 0); +lean_inc(x_359); +lean_dec(x_328); +if (lean_obj_tag(x_359) == 0) +{ +lean_object* x_360; +lean_dec(x_359); +lean_dec(x_357); +lean_dec(x_355); +lean_dec(x_353); +lean_dec(x_351); +lean_dec(x_349); +lean_dec(x_347); +x_360 = lean_box(0); +return x_360; +} +else +{ +lean_object* x_361; lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; uint8_t x_367; +x_361 = lean_ctor_get(x_347, 0); +lean_inc(x_361); +lean_dec(x_347); +x_362 = lean_ctor_get(x_349, 0); +lean_inc(x_362); +lean_dec(x_349); +x_363 = lean_ctor_get(x_351, 0); +lean_inc(x_363); +lean_dec(x_351); +x_364 = lean_ctor_get(x_353, 0); +lean_inc(x_364); +lean_dec(x_353); +x_365 = lean_ctor_get(x_355, 0); +lean_inc(x_365); +lean_dec(x_355); +x_366 = lean_ctor_get(x_357, 0); +lean_inc(x_366); +lean_dec(x_357); +x_367 = !lean_is_exclusive(x_359); +if (x_367 == 0) +{ +lean_object* x_368; lean_object* x_369; +x_368 = lean_ctor_get(x_359, 0); +x_369 = l_Lean_Name_mkStr7(x_361, x_362, x_363, x_364, x_365, x_366, x_368); +lean_ctor_set(x_359, 0, x_369); +return x_359; +} +else +{ +lean_object* x_370; lean_object* x_371; lean_object* x_372; +x_370 = lean_ctor_get(x_359, 0); +lean_inc(x_370); +lean_dec(x_359); +x_371 = l_Lean_Name_mkStr7(x_361, x_362, x_363, x_364, x_365, x_366, x_370); +x_372 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_372, 0, x_371); +return x_372; +} +} +} +else +{ +lean_object* x_373; +lean_dec(x_357); +lean_dec(x_355); +lean_dec(x_353); +lean_dec(x_351); +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_328); +x_373 = lean_box(0); +return x_373; +} +} +} +else +{ +lean_object* x_374; +lean_dec(x_355); +lean_dec(x_353); +lean_dec(x_351); +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_329); +lean_dec(x_328); +x_374 = lean_box(0); +return x_374; +} +} +} +else +{ +lean_object* x_375; +lean_dec(x_353); +lean_dec(x_351); +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_375 = lean_box(0); +return x_375; +} +} +} +else +{ +lean_object* x_376; +lean_dec(x_351); +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_376 = lean_box(0); +return x_376; +} +} +} +else +{ +lean_object* x_377; +lean_dec(x_349); +lean_dec(x_347); +lean_dec(x_332); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_377 = lean_box(0); +return x_377; +} +} +} +else +{ +lean_object* x_378; +lean_dec(x_347); +lean_dec(x_333); +lean_dec(x_332); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_378 = lean_box(0); +return x_378; +} +} +} +else +{ +lean_object* x_379; +lean_dec(x_334); +lean_dec(x_333); +lean_dec(x_332); +lean_dec(x_331); +lean_dec(x_330); +lean_dec(x_329); +lean_dec(x_328); +x_379 = lean_box(0); +return x_379; +} +} +} +} +} +else +{ +lean_object* x_380; +lean_dec(x_327); +lean_dec(x_326); +lean_dec(x_325); +lean_dec(x_324); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_380 = lean_box(0); +return x_380; +} +} +else +{ +lean_object* x_381; +lean_dec(x_326); +lean_dec(x_325); +lean_dec(x_324); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_381 = lean_box(0); +return x_381; +} +} +else +{ +lean_object* x_382; +lean_dec(x_325); +lean_dec(x_324); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_382 = lean_box(0); +return x_382; +} +} +else +{ +lean_object* x_383; +lean_dec(x_324); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_383 = lean_box(0); +return x_383; +} +} +case 5: +{ +lean_object* x_384; +x_384 = lean_ctor_get(x_323, 0); +lean_inc(x_384); +if (lean_obj_tag(x_384) == 4) +{ +lean_object* x_385; +x_385 = lean_ctor_get(x_384, 0); +lean_inc(x_385); +lean_dec(x_384); +if (lean_obj_tag(x_385) == 1) +{ +lean_object* x_386; +x_386 = lean_ctor_get(x_385, 0); +lean_inc(x_386); +if (lean_obj_tag(x_386) == 1) +{ +lean_object* x_387; +x_387 = lean_ctor_get(x_386, 0); +lean_inc(x_387); +if (lean_obj_tag(x_387) == 1) +{ +lean_object* x_388; +x_388 = lean_ctor_get(x_387, 0); +lean_inc(x_388); +if (lean_obj_tag(x_388) == 0) +{ +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; uint8_t x_401; +x_389 = lean_ctor_get(x_1, 1); +lean_inc(x_389); +lean_dec(x_1); +x_390 = lean_ctor_get(x_23, 1); +lean_inc(x_390); +lean_dec(x_23); +x_391 = lean_ctor_get(x_56, 1); +lean_inc(x_391); +lean_dec(x_56); +x_392 = lean_ctor_get(x_129, 1); +lean_inc(x_392); +lean_dec(x_129); +x_393 = lean_ctor_get(x_170, 1); +lean_inc(x_393); +lean_dec(x_170); +x_394 = lean_ctor_get(x_216, 1); +lean_inc(x_394); +lean_dec(x_216); +x_395 = lean_ctor_get(x_267, 1); +lean_inc(x_395); +lean_dec(x_267); +x_396 = lean_ctor_get(x_323, 1); +lean_inc(x_396); +lean_dec(x_323); +x_397 = lean_ctor_get(x_385, 1); +lean_inc(x_397); +lean_dec(x_385); +x_398 = lean_ctor_get(x_386, 1); +lean_inc(x_398); +lean_dec(x_386); +x_399 = lean_ctor_get(x_387, 1); +lean_inc(x_399); +lean_dec(x_387); +x_400 = l_Lean_Expr_name_x3f___closed__1; +x_401 = lean_string_dec_eq(x_399, x_400); +lean_dec(x_399); +if (x_401 == 0) +{ +lean_object* x_402; +lean_dec(x_398); +lean_dec(x_397); +lean_dec(x_396); +lean_dec(x_395); +lean_dec(x_394); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_402 = lean_box(0); +return x_402; +} +else +{ +lean_object* x_403; uint8_t x_404; +x_403 = l_Lean_Expr_name_x3f___closed__2; +x_404 = lean_string_dec_eq(x_398, x_403); +lean_dec(x_398); +if (x_404 == 0) +{ +lean_object* x_405; +lean_dec(x_397); +lean_dec(x_396); +lean_dec(x_395); +lean_dec(x_394); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_405 = lean_box(0); +return x_405; +} +else +{ +lean_object* x_406; uint8_t x_407; +x_406 = l_Lean_Expr_name_x3f___closed__14; +x_407 = lean_string_dec_eq(x_397, x_406); +lean_dec(x_397); +if (x_407 == 0) +{ +lean_object* x_408; +lean_dec(x_396); +lean_dec(x_395); +lean_dec(x_394); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_408 = lean_box(0); +return x_408; +} +else +{ +if (lean_obj_tag(x_396) == 9) +{ +lean_object* x_409; +x_409 = lean_ctor_get(x_396, 0); +lean_inc(x_409); +lean_dec(x_396); +if (lean_obj_tag(x_409) == 0) +{ +lean_object* x_410; +lean_dec(x_409); +lean_dec(x_395); +lean_dec(x_394); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_410 = lean_box(0); +return x_410; +} +else +{ +if (lean_obj_tag(x_395) == 9) +{ +lean_object* x_411; +x_411 = lean_ctor_get(x_395, 0); +lean_inc(x_411); +lean_dec(x_395); +if (lean_obj_tag(x_411) == 0) +{ +lean_object* x_412; +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_394); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_412 = lean_box(0); +return x_412; +} +else +{ +if (lean_obj_tag(x_394) == 9) +{ +lean_object* x_413; +x_413 = lean_ctor_get(x_394, 0); +lean_inc(x_413); +lean_dec(x_394); +if (lean_obj_tag(x_413) == 0) +{ +lean_object* x_414; +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_414 = lean_box(0); +return x_414; +} +else +{ +if (lean_obj_tag(x_393) == 9) +{ +lean_object* x_415; +x_415 = lean_ctor_get(x_393, 0); +lean_inc(x_415); +lean_dec(x_393); +if (lean_obj_tag(x_415) == 0) +{ +lean_object* x_416; +lean_dec(x_415); +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_416 = lean_box(0); +return x_416; +} +else +{ +if (lean_obj_tag(x_392) == 9) +{ +lean_object* x_417; +x_417 = lean_ctor_get(x_392, 0); +lean_inc(x_417); +lean_dec(x_392); +if (lean_obj_tag(x_417) == 0) +{ +lean_object* x_418; +lean_dec(x_417); +lean_dec(x_415); +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_418 = lean_box(0); +return x_418; +} +else +{ +if (lean_obj_tag(x_391) == 9) +{ +lean_object* x_419; +x_419 = lean_ctor_get(x_391, 0); +lean_inc(x_419); +lean_dec(x_391); +if (lean_obj_tag(x_419) == 0) +{ +lean_object* x_420; +lean_dec(x_419); +lean_dec(x_417); +lean_dec(x_415); +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_390); +lean_dec(x_389); +x_420 = lean_box(0); +return x_420; +} +else +{ +if (lean_obj_tag(x_390) == 9) +{ +lean_object* x_421; +x_421 = lean_ctor_get(x_390, 0); +lean_inc(x_421); +lean_dec(x_390); +if (lean_obj_tag(x_421) == 0) +{ +lean_object* x_422; +lean_dec(x_421); +lean_dec(x_419); +lean_dec(x_417); +lean_dec(x_415); +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_389); +x_422 = lean_box(0); +return x_422; +} +else +{ +if (lean_obj_tag(x_389) == 9) +{ +lean_object* x_423; +x_423 = lean_ctor_get(x_389, 0); +lean_inc(x_423); +lean_dec(x_389); +if (lean_obj_tag(x_423) == 0) +{ +lean_object* x_424; +lean_dec(x_423); +lean_dec(x_421); +lean_dec(x_419); +lean_dec(x_417); +lean_dec(x_415); +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +x_424 = lean_box(0); +return x_424; +} +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; lean_object* x_431; uint8_t x_432; +x_425 = lean_ctor_get(x_409, 0); +lean_inc(x_425); +lean_dec(x_409); +x_426 = lean_ctor_get(x_411, 0); +lean_inc(x_426); +lean_dec(x_411); +x_427 = lean_ctor_get(x_413, 0); +lean_inc(x_427); +lean_dec(x_413); +x_428 = lean_ctor_get(x_415, 0); +lean_inc(x_428); +lean_dec(x_415); +x_429 = lean_ctor_get(x_417, 0); +lean_inc(x_429); +lean_dec(x_417); +x_430 = lean_ctor_get(x_419, 0); +lean_inc(x_430); +lean_dec(x_419); +x_431 = lean_ctor_get(x_421, 0); +lean_inc(x_431); +lean_dec(x_421); +x_432 = !lean_is_exclusive(x_423); +if (x_432 == 0) +{ +lean_object* x_433; lean_object* x_434; +x_433 = lean_ctor_get(x_423, 0); +x_434 = l_Lean_Name_mkStr8(x_425, x_426, x_427, x_428, x_429, x_430, x_431, x_433); +lean_ctor_set(x_423, 0, x_434); +return x_423; +} +else +{ +lean_object* x_435; lean_object* x_436; lean_object* x_437; +x_435 = lean_ctor_get(x_423, 0); +lean_inc(x_435); +lean_dec(x_423); +x_436 = l_Lean_Name_mkStr8(x_425, x_426, x_427, x_428, x_429, x_430, x_431, x_435); +x_437 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_437, 0, x_436); +return x_437; +} +} +} +else +{ +lean_object* x_438; +lean_dec(x_421); +lean_dec(x_419); +lean_dec(x_417); +lean_dec(x_415); +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_389); +x_438 = lean_box(0); +return x_438; +} +} +} +else +{ +lean_object* x_439; +lean_dec(x_419); +lean_dec(x_417); +lean_dec(x_415); +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_390); +lean_dec(x_389); +x_439 = lean_box(0); +return x_439; +} +} +} +else +{ +lean_object* x_440; +lean_dec(x_417); +lean_dec(x_415); +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_440 = lean_box(0); +return x_440; +} +} +} +else +{ +lean_object* x_441; +lean_dec(x_415); +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_441 = lean_box(0); +return x_441; +} +} +} +else +{ +lean_object* x_442; +lean_dec(x_413); +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_442 = lean_box(0); +return x_442; +} +} +} +else +{ +lean_object* x_443; +lean_dec(x_411); +lean_dec(x_409); +lean_dec(x_394); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_443 = lean_box(0); +return x_443; +} +} +} +else +{ +lean_object* x_444; +lean_dec(x_409); +lean_dec(x_395); +lean_dec(x_394); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_444 = lean_box(0); +return x_444; +} +} +} +else +{ +lean_object* x_445; +lean_dec(x_396); +lean_dec(x_395); +lean_dec(x_394); +lean_dec(x_393); +lean_dec(x_392); +lean_dec(x_391); +lean_dec(x_390); +lean_dec(x_389); +x_445 = lean_box(0); +return x_445; +} +} +} +} +} +else +{ +lean_object* x_446; +lean_dec(x_388); +lean_dec(x_387); +lean_dec(x_386); +lean_dec(x_385); +lean_dec(x_323); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_446 = lean_box(0); +return x_446; +} +} +else +{ +lean_object* x_447; +lean_dec(x_387); +lean_dec(x_386); +lean_dec(x_385); +lean_dec(x_323); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_447 = lean_box(0); +return x_447; +} +} +else +{ +lean_object* x_448; +lean_dec(x_386); +lean_dec(x_385); +lean_dec(x_323); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_448 = lean_box(0); +return x_448; +} +} +else +{ +lean_object* x_449; +lean_dec(x_385); +lean_dec(x_323); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_449 = lean_box(0); +return x_449; +} +} +else +{ +lean_object* x_450; +lean_dec(x_384); +lean_dec(x_323); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_450 = lean_box(0); +return x_450; +} +} +default: +{ +lean_object* x_451; +lean_dec(x_323); +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_451 = lean_box(0); +return x_451; +} +} +} +default: +{ +lean_object* x_452; +lean_dec(x_267); +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_452 = lean_box(0); +return x_452; +} +} +} +default: +{ +lean_object* x_453; +lean_dec(x_216); +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_453 = lean_box(0); +return x_453; +} +} +} +default: +{ +lean_object* x_454; +lean_dec(x_170); +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_454 = lean_box(0); +return x_454; +} +} +} +default: +{ +lean_object* x_455; +lean_dec(x_129); +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_455 = lean_box(0); +return x_455; +} +} +} +default: +{ +lean_object* x_456; +lean_dec(x_56); +lean_dec(x_23); +lean_dec(x_1); +x_456 = lean_box(0); +return x_456; +} +} +} +default: +{ +lean_object* x_457; +lean_dec(x_23); +lean_dec(x_1); +x_457 = lean_box(0); +return x_457; +} +} +} +default: +{ +lean_object* x_458; +lean_dec(x_1); +x_458 = lean_box(0); +return x_458; +} +} +} +} lean_object* initialize_Lean_Environment(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Util_Recognizers(uint8_t builtin, lean_object* w) { @@ -1252,6 +4569,34 @@ l_Lean_Expr_prod_x3f___closed__1 = _init_l_Lean_Expr_prod_x3f___closed__1(); lean_mark_persistent(l_Lean_Expr_prod_x3f___closed__1); l_Lean_Expr_prod_x3f___closed__2 = _init_l_Lean_Expr_prod_x3f___closed__2(); lean_mark_persistent(l_Lean_Expr_prod_x3f___closed__2); +l_Lean_Expr_name_x3f___closed__1 = _init_l_Lean_Expr_name_x3f___closed__1(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__1); +l_Lean_Expr_name_x3f___closed__2 = _init_l_Lean_Expr_name_x3f___closed__2(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__2); +l_Lean_Expr_name_x3f___closed__3 = _init_l_Lean_Expr_name_x3f___closed__3(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__3); +l_Lean_Expr_name_x3f___closed__4 = _init_l_Lean_Expr_name_x3f___closed__4(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__4); +l_Lean_Expr_name_x3f___closed__5 = _init_l_Lean_Expr_name_x3f___closed__5(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__5); +l_Lean_Expr_name_x3f___closed__6 = _init_l_Lean_Expr_name_x3f___closed__6(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__6); +l_Lean_Expr_name_x3f___closed__7 = _init_l_Lean_Expr_name_x3f___closed__7(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__7); +l_Lean_Expr_name_x3f___closed__8 = _init_l_Lean_Expr_name_x3f___closed__8(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__8); +l_Lean_Expr_name_x3f___closed__9 = _init_l_Lean_Expr_name_x3f___closed__9(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__9); +l_Lean_Expr_name_x3f___closed__10 = _init_l_Lean_Expr_name_x3f___closed__10(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__10); +l_Lean_Expr_name_x3f___closed__11 = _init_l_Lean_Expr_name_x3f___closed__11(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__11); +l_Lean_Expr_name_x3f___closed__12 = _init_l_Lean_Expr_name_x3f___closed__12(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__12); +l_Lean_Expr_name_x3f___closed__13 = _init_l_Lean_Expr_name_x3f___closed__13(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__13); +l_Lean_Expr_name_x3f___closed__14 = _init_l_Lean_Expr_name_x3f___closed__14(); +lean_mark_persistent(l_Lean_Expr_name_x3f___closed__14); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Widget/Diff.c b/stage0/stdlib/Lean/Widget/Diff.c index c6b7bb44d7a9..59c0361c0414 100644 --- a/stage0/stdlib/Lean/Widget/Diff.c +++ b/stage0/stdlib/Lean/Widget/Diff.c @@ -96,6 +96,7 @@ lean_object* l_Lean_Name_quickCmp___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_exprDiffCore___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_SavedState_restore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_diffHypothesesBundle___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Widget_exprDiffCore___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_EXPORT lean_object* l_Lean_throwError___at_Lean_Widget_diffInteractiveGoal___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_diffInteractiveGoals___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___private_Lean_Widget_Diff_0__Lean_Widget_ExprDiffTag_noConfusion(lean_object*); @@ -117,7 +118,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_diffHypotheses_ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_diffInteractiveGoals___spec__3(uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_RBNode_insert___at_Lean_MVarIdMap_insert___spec__1___rarg(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_levelZero; -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Widget_exprDiffCore___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_EXPORT lean_object* l_Lean_throwError___at_Lean_Widget_diffHypothesesBundle_withTypeDiff___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_diffInteractiveGoals___spec__3___at_Lean_Widget_diffInteractiveGoals___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_EXPORT lean_object* l_Lean_throwError___at_Lean_Widget_diffInteractiveGoal___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -145,6 +145,7 @@ static lean_object* l_Lean_Widget_initFn____x40_Lean_Widget_Diff___hyg_5____clos LEAN_EXPORT lean_object* l_Lean_RBNode_find___at_Lean_Widget_addDiffTags___spec__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_ExprDiff_insertAfterChange(lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBMap_toList___at_Lean_Widget_instToStringExprDiff___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Widget_exprDiffCore___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_EXPORT lean_object* l_Lean_Widget_ExprDiff_insertBeforeChange(lean_object*, uint8_t, lean_object*); static lean_object* l_Lean_Widget_diffHypothesesBundle_withTypeDiff___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_diffInteractiveGoals___spec__3___lambda__4(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*); @@ -235,7 +236,6 @@ LEAN_EXPORT lean_object* l_Lean_Widget_diffInteractiveGoal___boxed(lean_object*, LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Widget_exprDiffCore___spec__3(lean_object*, size_t, size_t, lean_object*); uint8_t l_Lean_Exception_isRuntime(lean_object*); lean_object* l_List_toString___at_Lean_MetavarContext_MkBinding_instToStringException___spec__2(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Widget_exprDiffCore___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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Widget_exprDiffCore___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_exprDiffCore___lambda__3___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*); @@ -4513,7 +4513,7 @@ return x_10; } } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Widget_exprDiffCore___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_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Widget_exprDiffCore___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: { lean_object* x_15; uint8_t x_16; @@ -4732,7 +4732,7 @@ x_11 = l_Array_zip___rarg(x_1, x_2); x_12 = lean_array_get_size(x_11); x_13 = lean_mk_empty_array_with_capacity(x_12); x_14 = lean_unsigned_to_nat(0u); -x_15 = l_Array_mapIdxM_map___at_Lean_Widget_exprDiffCore___spec__2(x_3, x_4, x_1, x_11, x_11, x_12, x_14, lean_box(0), x_13, x_6, x_7, x_8, x_9, x_10); +x_15 = l_Array_mapFinIdxM_map___at_Lean_Widget_exprDiffCore___spec__2(x_3, x_4, x_1, x_11, x_11, x_12, x_14, lean_box(0), x_13, x_6, x_7, x_8, x_9, x_10); lean_dec(x_11); if (lean_obj_tag(x_15) == 0) { @@ -5765,11 +5765,11 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Widget_exprDiffCore___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, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Lean_Widget_exprDiffCore___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, lean_object* x_14) { _start: { lean_object* x_15; -x_15 = l_Array_mapIdxM_map___at_Lean_Widget_exprDiffCore___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 = l_Array_mapFinIdxM_map___at_Lean_Widget_exprDiffCore___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); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); diff --git a/stage0/stdlib/Lean/Widget/InteractiveCode.c b/stage0/stdlib/Lean/Widget/InteractiveCode.c index e3015469a58b..730fd3b47fa1 100644 --- a/stage0/stdlib/Lean/Widget/InteractiveCode.c +++ b/stage0/stdlib/Lean/Widget/InteractiveCode.c @@ -197,9 +197,9 @@ extern lean_object* l_Lean_Widget_instTypeNameInfoWithCtx; uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Widget_CodeWithInfos_mergePosMap(lean_object*, lean_object*); lean_object* lean_expr_dbg_to_string(lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_CodeWithInfos_mergePosMap___rarg(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_pp_mvars_anonymous; +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveCode___hyg_352____closed__2; LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveCode___hyg_352____lambda__1___boxed(lean_object*); static lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveCode___hyg_352____closed__22; @@ -1472,7 +1472,7 @@ x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_8); lean_ctor_set(x_16, 1, x_15); x_17 = l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonDiffTag____x40_Lean_Widget_InteractiveCode___hyg_67____closed__1; -x_18 = l_List_bindTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(x_16, x_17); +x_18 = l_List_flatMapTR_go___at___private_Lean_Data_Position_0__Lean_toJsonPosition____x40_Lean_Data_Position___hyg_237____spec__1(x_16, x_17); x_19 = l_Lean_Json_mkObj(x_18); return x_19; } diff --git a/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c b/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c index a2d0cbbd5893..cf54a18ef54d 100644 --- a/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c +++ b/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c @@ -187,6 +187,7 @@ static lean_object* l_Lean_Widget_instInhabitedMsgEmbed___closed__2; static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1935____closed__10; static lean_object* l_Lean_Widget_InteractiveDiagnostic_toDiagnostic_prettyTt___lambda__1___closed__1; lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instImpl____x40_Lean_Widget_InteractiveDiagnostic___hyg_547_; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodableDiagnosticWith_dec____x40_Lean_Widget_InteractiveDiagnostic___hyg_1850____spec__4___closed__2; LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_263_; @@ -220,7 +221,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodabl static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_766____lambda__2___closed__4; static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1935____closed__68; LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_766____lambda__3(lean_object*, lean_object*, lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_766____lambda__1___closed__3; static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___closed__7; lean_object* l_Lean_Option_register___at_Lean_initFn____x40_Lean_Util_RecDepth___hyg_5____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -6165,7 +6165,7 @@ x_40 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_40, 0, x_6); lean_ctor_set(x_40, 1, x_39); x_41 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_2476____closed__1; -x_42 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_40, x_41); +x_42 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_40, x_41); x_43 = l_Lean_Json_mkObj(x_42); return x_43; } diff --git a/stage0/stdlib/Lean/Widget/InteractiveGoal.c b/stage0/stdlib/Lean/Widget/InteractiveGoal.c index a63ef645c449..ee8de2e56998 100644 --- a/stage0/stdlib/Lean/Widget/InteractiveGoal.c +++ b/stage0/stdlib/Lean/Widget/InteractiveGoal.c @@ -188,6 +188,7 @@ static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJ static lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoalCore_pretty___spec__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Widget_instAppendInteractiveGoals; static lean_object* l_Lean_Widget_instFromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveGoal___hyg_657____closed__1; +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveGoal___hyg_176____closed__3; static lean_object* l_Lean_Widget_withGoalCtx___rarg___lambda__2___closed__2; LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Widget_instRpcEncodableInteractiveTermGoal_dec____x40_Lean_Widget_InteractiveGoal___hyg_2227____spec__1___boxed(lean_object*, lean_object*); @@ -218,7 +219,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_goalToInterac LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at_Lean_Widget_goalToInteractive___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Server_instRpcEncodableWithRpcRefOfTypeName_rpcEncode___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveGoal___hyg_3369____closed__7; -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodableInteractiveTermGoal_enc____x40_Lean_Widget_InteractiveGoal___hyg_2227_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_withGoalCtx___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveGoal___hyg_1277____closed__23; @@ -1262,7 +1262,7 @@ x_37 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_37, 0, x_13); lean_ctor_set(x_37, 1, x_36); x_38 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveGoal___hyg_660____closed__1; -x_39 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_37, x_38); +x_39 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_37, x_38); x_40 = l_Lean_Json_mkObj(x_39); return x_40; } @@ -7312,7 +7312,7 @@ x_39 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_39, 0, x_13); lean_ctor_set(x_39, 1, x_38); x_40 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveGoal___hyg_660____closed__1; -x_41 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_39, x_40); +x_41 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_39, x_40); x_42 = l_Lean_Json_mkObj(x_41); return x_42; } @@ -10270,7 +10270,7 @@ x_27 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_27, 0, x_10); lean_ctor_set(x_27, 1, x_26); x_28 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveGoal___hyg_660____closed__1; -x_29 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_27, x_28); +x_29 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_27, x_28); x_30 = l_Lean_Json_mkObj(x_29); return x_30; } @@ -12002,7 +12002,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___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveGoal___hyg_660____closed__1; -x_8 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_6, x_7); +x_8 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_6, x_7); x_9 = l_Lean_Json_mkObj(x_8); return x_9; } diff --git a/stage0/stdlib/Lean/Widget/Types.c b/stage0/stdlib/Lean/Widget/Types.c index c65f357d95f8..22a8979d3241 100644 --- a/stage0/stdlib/Lean/Widget/Types.c +++ b/stage0/stdlib/Lean/Widget/Types.c @@ -35,6 +35,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Widget_Types_0__Lean_Widget_fromJsonRp static lean_object* l___private_Lean_Widget_Types_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_Types___hyg_62____closed__3; LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodableWidgetInstance_enc____x40_Lean_Widget_Types___hyg_3_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodableWidgetInstance_dec____x40_Lean_Widget_Types___hyg_3____lambda__1___boxed(lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Widget_instRpcEncodableWidgetInstance___closed__2; uint8_t lean_string_dec_eq(lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_Types_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_Types___hyg_62____closed__7; @@ -72,7 +73,6 @@ LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodableWidgetInstance; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_Types_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_Types___hyg_62____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Widget_instRpcEncodableWidgetInstance_dec____x40_Lean_Widget_Types___hyg_3____spec__3(lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Widget_Types_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_Types___hyg_62____lambda__1(lean_object*); -lean_object* l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Widget_Types_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_Types___hyg_62____lambda__1___boxed(lean_object*); static lean_object* l___private_Lean_Widget_Types_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_Types___hyg_62____closed__35; LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodableWidgetInstance_dec____x40_Lean_Widget_Types___hyg_3_(lean_object*, lean_object*); @@ -583,7 +583,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_Widget_Types_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Widget_Types___hyg_261____closed__1; -x_19 = l_List_bindTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Server_Rpc_Basic_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Server_Rpc_Basic___hyg_173____spec__1(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } diff --git a/stage0/stdlib/Lean/Widget/UserWidget.c b/stage0/stdlib/Lean/Widget/UserWidget.c index ffaa0ddb82fb..2a004760a5a1 100644 --- a/stage0/stdlib/Lean/Widget/UserWidget.c +++ b/stage0/stdlib/Lean/Widget/UserWidget.c @@ -352,6 +352,7 @@ lean_object* l_Lean_ScopedEnvExtension_modifyState___rarg(lean_object*, lean_obj lean_object* l_Lean_Name_append(lean_object*, lean_object*); static lean_object* l_Lean_Widget_addWidgetSpec___closed__7; LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Widget_elabShowPanelWidgetsCmd___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodableGetWidgetsResponse_enc____x40_Lean_Widget_UserWidget___hyg_4791____spec__1(size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_elabShowPanelWidgetsCmd___spec__13___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_throwUnsupportedSyntax___at_Lean_Widget_elabShowPanelWidgetsCmd___spec__1___boxed(lean_object*, lean_object*); @@ -403,7 +404,6 @@ lean_object* l_Lean_bignumFromJson_x3f(lean_object*); static lean_object* l_Lean_Widget_addWidgetSpec___closed__1; static lean_object* l_Lean_Widget_showPanelWidgetsCmd___closed__9; static lean_object* l_Lean_Widget_instRpcEncodablePanelWidgetInstance___closed__3; -lean_object* l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Widget_widgetInstanceSpec___closed__12; static lean_object* l_Lean_Widget_elabWidgetInstanceSpecAux___closed__46; static lean_object* l_Lean_Widget_instToJsonRpcEncodablePacket____x40_Lean_Widget_UserWidget___hyg_4536____closed__1; @@ -8210,7 +8210,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__8; -x_17 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -8545,7 +8545,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__8; -x_9 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -18772,7 +18772,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__8; -x_16 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -18810,7 +18810,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__8; -x_32 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_30, x_31); +x_32 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_30, x_31); x_33 = l_Lean_Json_mkObj(x_32); return x_33; } @@ -19848,7 +19848,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__8; -x_27 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_25, x_26); +x_27 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_25, x_26); x_28 = l_Lean_Json_mkObj(x_27); return x_28; } @@ -21519,7 +21519,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__8; -x_8 = l_List_bindTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_6, x_7); +x_8 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_Basic___hyg_86____spec__1(x_6, x_7); x_9 = l_Lean_Json_mkObj(x_8); return x_9; } diff --git a/stage0/stdlib/Std/Data/DHashMap/Internal/Defs.c b/stage0/stdlib/Std/Data/DHashMap/Internal/Defs.c index e40f94a4f976..00fdd047a3c0 100644 --- a/stage0/stdlib/Std/Data/DHashMap/Internal/Defs.c +++ b/stage0/stdlib/Std/Data/DHashMap/Internal/Defs.c @@ -41,7 +41,6 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_get_x3f___rarg( LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_filterMap(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_insertManyUnit(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_DHashMap_Internal_Raw_u2080_expand_go___spec__1(lean_object*, lean_object*); 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*); @@ -56,6 +55,7 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_get_x21___rarg(lean_o LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Std_DHashMap_Internal_Raw_u2080_filter___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg___boxed(lean_object*, lean_object*); 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*); @@ -81,6 +81,7 @@ lean_object* lean_array_to_list(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_containsThenInsertIfNew(lean_object*, lean_object*); uint8_t l_Std_DHashMap_Internal_AssocList_contains___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_getKey_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_get___rarg(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_Internal_Raw_u2080_Const_getThenInsertIfNew_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -115,7 +116,6 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expandIfNecessary___b 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_get_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg___boxed(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*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Defs_0__Std_DHashMap_Internal_numBucketsForCapacity(lean_object*); @@ -132,7 +132,6 @@ lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_map___rarg(lean_object*, lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Std_DHashMap_Internal_toListModel___spec__1(lean_object*, lean_object*); lean_object* l_List_foldl___at_Array_appendList___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_empty(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_contains___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -151,6 +150,7 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_computeSize___rarg___boxed(lean LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(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_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1(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*); @@ -192,7 +192,7 @@ lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -214,11 +214,11 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Std_DHashMap_Internal_toListModel___spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_List_bindTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg___boxed), 2, 0); +x_3 = lean_alloc_closure((void*)(l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg___boxed), 2, 0); return x_3; } } @@ -237,7 +237,7 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_toListModel___rarg(lean_object* lean_object* x_2; lean_object* x_3; lean_object* x_4; x_2 = lean_array_to_list(x_1); x_3 = l_Std_DHashMap_Internal_toListModel___rarg___closed__1; -x_4 = l_List_bindTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg(x_2, x_3); +x_4 = l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg(x_2, x_3); lean_dec(x_2); return x_4; } @@ -250,11 +250,11 @@ x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_toListModel___rarg), 1, return x_3; } } -LEAN_EXPORT lean_object* l_List_bindTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_List_bindTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg(x_1, x_2); +x_3 = l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1___rarg(x_1, x_2); lean_dec(x_1); return x_3; } diff --git a/stage0/stdlib/Std/Sat/AIG.c b/stage0/stdlib/Std/Sat/AIG.c index 48e8ab51e33d..9af3dfc5dc70 100644 --- a/stage0/stdlib/Std/Sat/AIG.c +++ b/stage0/stdlib/Std/Sat/AIG.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG -// Imports: Init Std.Sat.AIG.Basic Std.Sat.AIG.LawfulOperator Std.Sat.AIG.Lemmas Std.Sat.AIG.Cached Std.Sat.AIG.CachedLemmas Std.Sat.AIG.CachedGates Std.Sat.AIG.CachedGatesLemmas Std.Sat.AIG.CNF Std.Sat.AIG.Relabel Std.Sat.AIG.RelabelNat Std.Sat.AIG.RefVec Std.Sat.AIG.RefVecOperator Std.Sat.AIG.LawfulVecOperator Std.Sat.AIG.If +// Imports: Std.Sat.AIG.Basic Std.Sat.AIG.LawfulOperator Std.Sat.AIG.Lemmas Std.Sat.AIG.Cached Std.Sat.AIG.CachedLemmas Std.Sat.AIG.CachedGates Std.Sat.AIG.CachedGatesLemmas Std.Sat.AIG.CNF Std.Sat.AIG.Relabel Std.Sat.AIG.RelabelNat Std.Sat.AIG.RefVec Std.Sat.AIG.RefVecOperator Std.Sat.AIG.LawfulVecOperator Std.Sat.AIG.If #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -13,7 +13,6 @@ #ifdef __cplusplus extern "C" { #endif -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_LawfulOperator(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Lemmas(uint8_t builtin, lean_object*); @@ -33,9 +32,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG(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(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/Basic.c b/stage0/stdlib/Std/Sat/AIG/Basic.c index 86f640dde9de..72649cf6f263 100644 --- a/stage0/stdlib/Std/Sat/AIG/Basic.c +++ b/stage0/stdlib/Std/Sat/AIG/Basic.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.Basic -// Imports: Init Std.Data.HashMap Std.Data.HashSet +// Imports: Std.Data.HashMap Std.Data.HashSet #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -5655,7 +5655,6 @@ lean_dec(x_1); return x_6; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Data_HashMap(uint8_t builtin, lean_object*); lean_object* initialize_Std_Data_HashSet(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -5663,9 +5662,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_Basic(uint8_t builtin, lean_obje lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -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); diff --git a/stage0/stdlib/Std/Sat/AIG/CNF.c b/stage0/stdlib/Std/Sat/AIG/CNF.c index 63086e18047d..f2d7121e4c44 100644 --- a/stage0/stdlib/Std/Sat/AIG/CNF.c +++ b/stage0/stdlib/Std/Sat/AIG/CNF.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.CNF -// Imports: Init Std.Sat.CNF Std.Sat.AIG.Basic Std.Sat.AIG.Lemmas +// Imports: Std.Sat.CNF Std.Sat.AIG.Basic Std.Sat.AIG.Lemmas #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -1063,7 +1063,6 @@ x_15 = l_Std_Sat_CNF_relabel___rarg(x_14, x_13); return x_15; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_CNF(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Lemmas(uint8_t builtin, lean_object*); @@ -1072,9 +1071,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_CNF(uint8_t builtin, lean_object lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_CNF(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/Cached.c b/stage0/stdlib/Std/Sat/AIG/Cached.c index 69bee4045bfe..13918a403087 100644 --- a/stage0/stdlib/Std/Sat/AIG/Cached.c +++ b/stage0/stdlib/Std/Sat/AIG/Cached.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.Cached -// Imports: Init Std.Sat.AIG.Basic Std.Sat.AIG.Lemmas +// Imports: Std.Sat.AIG.Basic Std.Sat.AIG.Lemmas #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -1467,7 +1467,6 @@ x_2 = lean_alloc_closure((void*)(l_Std_Sat_AIG_mkGateCached___rarg), 4, 0); return x_2; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Lemmas(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -1475,9 +1474,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_Cached(uint8_t builtin, lean_obj lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/CachedGates.c b/stage0/stdlib/Std/Sat/AIG/CachedGates.c index 1ac889fdd5bd..8cc4869a66e8 100644 --- a/stage0/stdlib/Std/Sat/AIG/CachedGates.c +++ b/stage0/stdlib/Std/Sat/AIG/CachedGates.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.CachedGates -// Imports: Init Std.Sat.AIG.Cached Std.Sat.AIG.CachedLemmas +// Imports: Std.Sat.AIG.Cached Std.Sat.AIG.CachedLemmas #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -646,7 +646,6 @@ x_2 = lean_alloc_closure((void*)(l_Std_Sat_AIG_mkImpCached___rarg), 4, 0); return x_2; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Cached(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_CachedLemmas(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -654,9 +653,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_CachedGates(uint8_t builtin, lea lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_Cached(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/CachedGatesLemmas.c b/stage0/stdlib/Std/Sat/AIG/CachedGatesLemmas.c index 460546e61625..f99ec336c349 100644 --- a/stage0/stdlib/Std/Sat/AIG/CachedGatesLemmas.c +++ b/stage0/stdlib/Std/Sat/AIG/CachedGatesLemmas.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.CachedGatesLemmas -// Imports: Init Std.Sat.AIG.CachedGates Std.Sat.AIG.LawfulOperator +// Imports: Std.Sat.AIG.CachedGates Std.Sat.AIG.LawfulOperator #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -13,7 +13,6 @@ #ifdef __cplusplus extern "C" { #endif -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_CachedGates(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_LawfulOperator(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -21,9 +20,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_CachedGatesLemmas(uint8_t builti lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_CachedGates(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/CachedLemmas.c b/stage0/stdlib/Std/Sat/AIG/CachedLemmas.c index b881f69cee64..faf22391fc17 100644 --- a/stage0/stdlib/Std/Sat/AIG/CachedLemmas.c +++ b/stage0/stdlib/Std/Sat/AIG/CachedLemmas.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.CachedLemmas -// Imports: Init Std.Sat.AIG.Cached +// Imports: Std.Sat.AIG.Cached #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -889,16 +889,12 @@ lean_dec(x_2); return x_5; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Cached(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_CachedLemmas(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(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_Cached(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/If.c b/stage0/stdlib/Std/Sat/AIG/If.c index 8be164b60daf..e897651b0000 100644 --- a/stage0/stdlib/Std/Sat/AIG/If.c +++ b/stage0/stdlib/Std/Sat/AIG/If.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.If -// Imports: Init Std.Sat.AIG.CachedGatesLemmas Std.Sat.AIG.LawfulVecOperator +// Imports: Std.Sat.AIG.CachedGatesLemmas Std.Sat.AIG.LawfulVecOperator #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -201,7 +201,6 @@ lean_dec(x_3); return x_6; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_CachedGatesLemmas(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_LawfulVecOperator(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -209,9 +208,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_If(uint8_t builtin, lean_object* lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_CachedGatesLemmas(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/LawfulOperator.c b/stage0/stdlib/Std/Sat/AIG/LawfulOperator.c index d2d551df2813..4aff9ce69d6b 100644 --- a/stage0/stdlib/Std/Sat/AIG/LawfulOperator.c +++ b/stage0/stdlib/Std/Sat/AIG/LawfulOperator.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.LawfulOperator -// Imports: Init Std.Sat.AIG.Basic +// Imports: Std.Sat.AIG.Basic #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -69,16 +69,12 @@ x_3 = lean_alloc_closure((void*)(l___private_Std_Sat_AIG_LawfulOperator_0__Std_S return x_3; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Basic(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_LawfulOperator(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(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/LawfulVecOperator.c b/stage0/stdlib/Std/Sat/AIG/LawfulVecOperator.c index 50228c352eff..2c72608b1ba9 100644 --- a/stage0/stdlib/Std/Sat/AIG/LawfulVecOperator.c +++ b/stage0/stdlib/Std/Sat/AIG/LawfulVecOperator.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.LawfulVecOperator -// Imports: Init Std.Sat.AIG.LawfulOperator Std.Sat.AIG.RefVec +// Imports: Std.Sat.AIG.LawfulOperator Std.Sat.AIG.RefVec #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -13,7 +13,6 @@ #ifdef __cplusplus extern "C" { #endif -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_LawfulOperator(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_RefVec(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -21,9 +20,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_LawfulVecOperator(uint8_t builti lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_LawfulOperator(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/Lemmas.c b/stage0/stdlib/Std/Sat/AIG/Lemmas.c index a06c3e522032..35bf19ddd042 100644 --- a/stage0/stdlib/Std/Sat/AIG/Lemmas.c +++ b/stage0/stdlib/Std/Sat/AIG/Lemmas.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.Lemmas -// Imports: Init Std.Sat.AIG.Basic Std.Sat.AIG.LawfulOperator +// Imports: Std.Sat.AIG.Basic Std.Sat.AIG.LawfulOperator #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -69,7 +69,6 @@ x_3 = lean_alloc_closure((void*)(l___private_Std_Sat_AIG_Lemmas_0__Std_Sat_AIG_t return x_3; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_LawfulOperator(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -77,9 +76,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_Lemmas(uint8_t builtin, lean_obj lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/RefVec.c b/stage0/stdlib/Std/Sat/AIG/RefVec.c index 845de5f3c0c9..c41cb32b11e9 100644 --- a/stage0/stdlib/Std/Sat/AIG/RefVec.c +++ b/stage0/stdlib/Std/Sat/AIG/RefVec.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.RefVec -// Imports: Init Std.Sat.AIG.LawfulOperator Std.Sat.AIG.CachedGatesLemmas +// Imports: Std.Sat.AIG.LawfulOperator Std.Sat.AIG.CachedGatesLemmas #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -591,7 +591,6 @@ lean_dec(x_2); return x_7; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_LawfulOperator(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_CachedGatesLemmas(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -599,9 +598,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_RefVec(uint8_t builtin, lean_obj lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_LawfulOperator(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/RefVecOperator.c b/stage0/stdlib/Std/Sat/AIG/RefVecOperator.c index 61c8d0cba16b..153a72172d92 100644 --- a/stage0/stdlib/Std/Sat/AIG/RefVecOperator.c +++ b/stage0/stdlib/Std/Sat/AIG/RefVecOperator.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.RefVecOperator -// Imports: Init Std.Sat.AIG.RefVecOperator.Map Std.Sat.AIG.RefVecOperator.Zip Std.Sat.AIG.RefVecOperator.Fold +// Imports: Std.Sat.AIG.RefVecOperator.Map Std.Sat.AIG.RefVecOperator.Zip Std.Sat.AIG.RefVecOperator.Fold #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -13,7 +13,6 @@ #ifdef __cplusplus extern "C" { #endif -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_RefVecOperator_Map(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_RefVecOperator_Zip(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_RefVecOperator_Fold(uint8_t builtin, lean_object*); @@ -22,9 +21,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_RefVecOperator(uint8_t builtin, lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_RefVecOperator_Map(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Fold.c b/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Fold.c index 31a1388f8f0e..ecf2d343b603 100644 --- a/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Fold.c +++ b/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Fold.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.RefVecOperator.Fold -// Imports: Init Std.Sat.AIG.RefVec Std.Sat.AIG.LawfulVecOperator +// Imports: Std.Sat.AIG.RefVec Std.Sat.AIG.LawfulVecOperator #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -154,7 +154,6 @@ x_2 = lean_alloc_closure((void*)(l_Std_Sat_AIG_RefVec_fold___rarg), 4, 0); return x_2; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_RefVec(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_LawfulVecOperator(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -162,9 +161,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_RefVecOperator_Fold(uint8_t buil lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_RefVec(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Map.c b/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Map.c index 86eb7cbc0324..72ad864a69be 100644 --- a/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Map.c +++ b/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Map.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.RefVecOperator.Map -// Imports: Init Std.Sat.AIG.RefVec Std.Sat.AIG.LawfulVecOperator +// Imports: Std.Sat.AIG.RefVec Std.Sat.AIG.LawfulVecOperator #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -119,7 +119,6 @@ lean_dec(x_1); return x_6; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_RefVec(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_LawfulVecOperator(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -127,9 +126,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_RefVecOperator_Map(uint8_t built lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_RefVec(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Zip.c b/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Zip.c index 7325781cbe0f..370cc8eec26c 100644 --- a/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Zip.c +++ b/stage0/stdlib/Std/Sat/AIG/RefVecOperator/Zip.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.RefVecOperator.Zip -// Imports: Init Std.Sat.AIG.RefVec Std.Sat.AIG.LawfulVecOperator +// Imports: Std.Sat.AIG.RefVec Std.Sat.AIG.LawfulVecOperator #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -130,7 +130,6 @@ lean_dec(x_1); return x_6; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_RefVec(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_LawfulVecOperator(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -138,9 +137,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_RefVecOperator_Zip(uint8_t built lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_RefVec(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/Relabel.c b/stage0/stdlib/Std/Sat/AIG/Relabel.c index c80b596fb6f9..e8df5069f458 100644 --- a/stage0/stdlib/Std/Sat/AIG/Relabel.c +++ b/stage0/stdlib/Std/Sat/AIG/Relabel.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.Relabel -// Imports: Init Std.Sat.AIG.Basic Std.Sat.AIG.Lemmas +// Imports: Std.Sat.AIG.Basic Std.Sat.AIG.Lemmas #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -322,7 +322,6 @@ lean_dec(x_2); return x_5; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Lemmas(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -330,9 +329,6 @@ LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_Relabel(uint8_t builtin, lean_ob lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Init(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Sat/AIG/RelabelNat.c b/stage0/stdlib/Std/Sat/AIG/RelabelNat.c index 69c74ae44184..9ccfa74c6d26 100644 --- a/stage0/stdlib/Std/Sat/AIG/RelabelNat.c +++ b/stage0/stdlib/Std/Sat/AIG/RelabelNat.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Sat.AIG.RelabelNat -// Imports: Init Std.Sat.AIG.Relabel +// Imports: Std.Sat.AIG.Relabel #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -1377,16 +1377,12 @@ x_2 = lean_alloc_closure((void*)(l_Std_Sat_AIG_Entrypoint_relabelNat___rarg), 3, return x_2; } } -lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Std_Sat_AIG_Relabel(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Std_Sat_AIG_RelabelNat(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(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Std_Sat_AIG_Relabel(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Expr.c b/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Expr.c index ec8728ccd3d9..d4815fa0a854 100644 --- a/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Expr.c +++ b/stage0/stdlib/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Impl/Expr.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Expr -// Imports: Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Var Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Const Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Not Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.ShiftLeft Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.ShiftRight Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Add Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.ZeroExtend Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Append Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Replicate Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Extract Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.RotateLeft Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.RotateRight Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.SignExtend Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Mul Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Udiv Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Umod +// Imports: Init.Data.AC Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Var Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Const Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Not Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.ShiftLeft Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.ShiftRight Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Add Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.ZeroExtend Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Append Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Replicate Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Extract Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.RotateLeft Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.RotateRight Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.SignExtend Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Mul Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Udiv Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Umod #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -3615,6 +3615,7 @@ x_4 = l_Std_Tactic_BVDecide_BVExpr_bitblast_go(x_1, x_2, x_3); return x_4; } } +lean_object* initialize_Init_Data_AC(uint8_t builtin, lean_object*); lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Var(uint8_t builtin, lean_object*); lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Const(uint8_t builtin, lean_object*); lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Operations_Not(uint8_t builtin, lean_object*); @@ -3636,6 +3637,9 @@ LEAN_EXPORT lean_object* initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_ lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; +res = initialize_Init_Data_AC(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); res = initialize_Std_Tactic_BVDecide_Bitblast_BVExpr_Circuit_Impl_Var(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Std/Tactic/BVDecide/LRAT/Internal/Clause.c b/stage0/stdlib/Std/Tactic/BVDecide/LRAT/Internal/Clause.c index 4535d5388005..207eba069d5a 100644 --- a/stage0/stdlib/Std/Tactic/BVDecide/LRAT/Internal/Clause.c +++ b/stage0/stdlib/Std/Tactic/BVDecide/LRAT/Internal/Clause.c @@ -44,7 +44,6 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Std_Tactic_BVDecide_LRAT LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_ofArray___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_reduce__fold__fn___boxed(lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_unit___rarg(lean_object*); -LEAN_EXPORT lean_object* l___private_Std_Tactic_BVDecide_LRAT_Internal_Clause_0__List_getLast_x3f_match__1_splitter(lean_object*, lean_object*); uint8_t l_List_any___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_eraseTR_go___at_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_delete___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_isUnit___rarg(lean_object*); @@ -63,7 +62,6 @@ LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_empty LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_toList(lean_object*); LEAN_EXPORT lean_object* l_List_toString___at_Std_Tactic_BVDecide_LRAT_Internal_instToStringDefaultClause___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_insert___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Std_Tactic_BVDecide_LRAT_Internal_Clause_0__List_getLast_x3f_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_reduce___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_Clause_instDecidableEvalLiteral___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Std_Tactic_BVDecide_LRAT_Internal_instToStringDefaultClause___spec__3___boxed(lean_object*, lean_object*, lean_object*); @@ -72,7 +70,6 @@ LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_unit_ LEAN_EXPORT uint8_t l_List_elem___at_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_insert___spec__2(lean_object*, lean_object*, lean_object*); lean_object* l_outOfBounds___rarg(lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_instClausePosFin(lean_object*); -LEAN_EXPORT lean_object* l___private_Std_Tactic_BVDecide_LRAT_Internal_Clause_0__List_getLast_x3f_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_empty(lean_object*); LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_toList___boxed(lean_object*); LEAN_EXPORT lean_object* l_List_toString___at_Std_Tactic_BVDecide_LRAT_Internal_instToStringDefaultClause___spec__1___boxed(lean_object*, lean_object*); @@ -816,45 +813,6 @@ lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Std_Tactic_BVDecide_LRAT_Internal_Clause_0__List_getLast_x3f_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_Std_Tactic_BVDecide_LRAT_Internal_Clause_0__List_getLast_x3f_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_Tactic_BVDecide_LRAT_Internal_Clause_0__List_getLast_x3f_match__1_splitter___rarg___boxed), 3, 0); -return x_3; -} -} -LEAN_EXPORT lean_object* l___private_Std_Tactic_BVDecide_LRAT_Internal_Clause_0__List_getLast_x3f_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_Tactic_BVDecide_LRAT_Internal_Clause_0__List_getLast_x3f_match__1_splitter___rarg(x_1, x_2, x_3); -lean_dec(x_2); -return x_4; -} -} LEAN_EXPORT lean_object* l_Std_Tactic_BVDecide_LRAT_Internal_DefaultClause_empty(lean_object* x_1) { _start: { From 810f0ec6d1a0d75e472064f8514a46db410b83ba Mon Sep 17 00:00:00 2001 From: Kim Morrison Date: Tue, 22 Oct 2024 10:30:18 +1100 Subject: [PATCH 3/3] chore: deprecate Array.modifyOp --- src/Init/Data/Array/Basic.lean | 4 +--- 1 file changed, 1 insertion(+), 3 deletions(-) diff --git a/src/Init/Data/Array/Basic.lean b/src/Init/Data/Array/Basic.lean index d057e5e87df6..d8cf2a659252 100644 --- a/src/Init/Data/Array/Basic.lean +++ b/src/Init/Data/Array/Basic.lean @@ -275,9 +275,7 @@ def modifyM [Monad m] (a : Array α) (i : Nat) (f : α → m α) : m (Array α) def modify (a : Array α) (i : Nat) (f : α → α) : Array α := Id.run <| modifyM a i f -@[inline] -def modifyOp (self : Array α) (idx : Nat) (f : α → α) : Array α := - self.modify idx f +@[deprecated modify (since := "2024-10-22")] abbrev modifyOp := @modify /-- We claim this unsafe implementation is correct because an array cannot have more than `usizeSz` elements in our runtime.